src/HOL/Probability/Probability_Mass_Function.thy
changeset 59092 d469103c0737
parent 59053 43e07797269b
child 59093 2b106e58a177
--- a/src/HOL/Probability/Probability_Mass_Function.thy	Thu Dec 04 21:28:35 2014 +0100
+++ b/src/HOL/Probability/Probability_Mass_Function.thy	Fri Dec 05 12:06:18 2014 +0100
@@ -385,7 +385,7 @@
     by (simp split: split_indicator)
   show "AE x in density (count_space UNIV) (ereal \<circ> f).
     measure (density (count_space UNIV) (ereal \<circ> f)) {x} \<noteq> 0"
-    by (simp add: AE_density nonneg emeasure_density measure_def nn_integral_cmult_indicator)
+    by (simp add: AE_density nonneg measure_def emeasure_density max_def)
   show "prob_space (density (count_space UNIV) (ereal \<circ> f))"
     by default (simp add: emeasure_density prob)
 qed simp
@@ -395,7 +395,7 @@
   have *[simp]: "\<And>x y. ereal (f y) * indicator {x} y = ereal (f x) * indicator {x} y"
     by (simp split: split_indicator)
   fix x show "measure (density (count_space UNIV) (ereal \<circ> f)) {x} = f x"
-    by transfer (simp add: measure_def emeasure_density nn_integral_cmult_indicator nonneg)
+    by transfer (simp add: measure_def emeasure_density nonneg max_def)
 qed
 
 end