src/HOL/Probability/Complete_Measure.thy
changeset 41097 a1abfa4e2b44
parent 41023 9118eb4eb8dc
child 41689 3e39b0e730d6
--- a/src/HOL/Probability/Complete_Measure.thy	Wed Dec 08 16:15:14 2010 +0100
+++ b/src/HOL/Probability/Complete_Measure.thy	Wed Dec 08 19:32:11 2010 +0100
@@ -257,17 +257,14 @@
   show ?thesis
   proof (intro bexI)
     from AE[unfolded all_AE_countable]
-    show "AE x. g x = (SUP i. f' i) x" (is "AE x. g x = ?f x")
+    show "AE x. g x = (SUP i. f' i x)" (is "AE x. g x = ?f x")
     proof (rule AE_mp, safe intro!: AE_cong)
       fix x assume eq: "\<forall>i. f i x = f' i x"
-      have "g x = (SUP i. f i x)"
-        using `f \<up> g` unfolding isoton_def SUPR_fun_expand by auto
-      then show "g x = ?f x"
-        using eq unfolding SUPR_fun_expand by auto
+      moreover have "g = SUPR UNIV f" using `f \<up> g` unfolding isoton_def by simp
+      ultimately show "g x = ?f x" by (simp add: SUPR_apply)
     qed
     show "?f \<in> borel_measurable M"
-      using sf by (auto intro!: borel_measurable_SUP
-        intro: borel_measurable_simple_function)
+      using sf by (auto intro: borel_measurable_simple_function)
   qed
 qed