diff -r 9d5013661ac6 -r 9c66f7c541fb src/HOL/Probability/Nonnegative_Lebesgue_Integration.thy --- a/src/HOL/Probability/Nonnegative_Lebesgue_Integration.thy Mon Oct 06 21:21:46 2014 +0200 +++ b/src/HOL/Probability/Nonnegative_Lebesgue_Integration.thy Tue Oct 07 10:34:24 2014 +0200 @@ -748,6 +748,9 @@ lemma nn_integral_nonneg: "0 \ integral\<^sup>N M f" by (auto intro!: SUP_upper2[of "\x. 0"] simp: nn_integral_def le_fun_def) +lemma nn_integral_le_0[simp]: "integral\<^sup>N M f \ 0 \ integral\<^sup>N M f = 0" + using nn_integral_nonneg[of M f] by auto + lemma nn_integral_not_MInfty[simp]: "integral\<^sup>N M f \ -\" using nn_integral_nonneg[of M f] by auto @@ -2187,6 +2190,10 @@ using emeasure_uniform_measure[OF emeasure_neq_0_sets[OF A(1)] B] A by (cases "emeasure M A" "emeasure M (A \ B)" rule: ereal2_cases) (simp_all add: measure_def) +lemma AE_uniform_measureI: + "A \ sets M \ (AE x in M. x \ A \ P x) \ (AE x in uniform_measure M A. P x)" + unfolding uniform_measure_def by (auto simp: AE_density) + subsubsection {* Uniform count measure *} definition "uniform_count_measure A = point_measure A (\x. 1 / card A)"