src/HOL/Probability/Binary_Product_Measure.thy
changeset 62083 7582b39f51ed
parent 61808 fc1556774cfe
child 62390 842917225d56
--- a/src/HOL/Probability/Binary_Product_Measure.thy	Wed Jan 06 13:04:31 2016 +0100
+++ b/src/HOL/Probability/Binary_Product_Measure.thy	Wed Jan 06 12:18:53 2016 +0100
@@ -1012,7 +1012,7 @@
     also have "\<dots> = (\<integral>\<^sup>+ y. ereal (1 / Suc n) * indicator C' (x, y) \<partial>count_space UNIV)"
       by(rule nn_integral_cong)(force split: split_indicator intro: rev_image_eqI simp add: C')
     also have "\<dots> = (\<integral>\<^sup>+ x'. (\<integral>\<^sup>+ y. ereal (1 / Suc n) * indicator C' (x, y) \<partial>count_space UNIV) * indicator {x} x' \<partial>count_space UNIV)"
-      by(simp add: one_ereal_def[symmetric] nn_integral_nonneg nn_integral_cmult_indicator)
+      by(simp add: one_ereal_def[symmetric] nn_integral_nonneg max_def)
     also have "\<dots> \<le> (\<integral>\<^sup>+ x. \<integral>\<^sup>+ y. ereal (1 / Suc n) * indicator C' (x, y) \<partial>count_space UNIV \<partial>count_space UNIV)"
       by(rule nn_integral_mono)(simp split: split_indicator add: nn_integral_nonneg)
     also have "\<dots> \<le> ?lhs" using **
@@ -1024,7 +1024,7 @@
     have "\<infinity> = \<integral>\<^sup>+ x. ereal (1 / Suc n) * indicator C' x \<partial>count_space UNIV"
       using C'_def False by(simp add: nn_integral_cmult)
     also have "\<dots> = \<integral>\<^sup>+ x. \<integral>\<^sup>+ y. ereal (1 / Suc n) * indicator C' x * indicator {SOME y. (x, y) \<in> C} y \<partial>count_space UNIV \<partial>count_space UNIV"
-      by(auto simp add: one_ereal_def[symmetric] nn_integral_cmult_indicator intro: nn_integral_cong)
+      by(auto simp add: one_ereal_def[symmetric] max_def intro: nn_integral_cong)
     also have "\<dots> \<le> \<integral>\<^sup>+ x. \<integral>\<^sup>+ y. ereal (1 / Suc n) * indicator C (x, y) \<partial>count_space UNIV \<partial>count_space UNIV"
       by(intro nn_integral_mono)(auto simp add: C'_def split: split_indicator intro: someI)
     also have "\<dots> \<le> ?lhs" using C
@@ -1121,4 +1121,4 @@
     by (auto simp: space_pair_measure M.emeasure_pair_measure_Times)
 qed
 
-end
\ No newline at end of file
+end