src/HOL/Probability/Complete_Measure.thy
changeset 41705 1100512e16d8
parent 41689 3e39b0e730d6
child 41959 b460124855b8
equal deleted inserted replaced
41704:8c539202f854 41705:1100512e16d8
   264     AE: "\<forall>i. AE x. f i x = f' i x" by auto
   264     AE: "\<forall>i. AE x. f i x = f' i x" by auto
   265   show ?thesis
   265   show ?thesis
   266   proof (intro bexI)
   266   proof (intro bexI)
   267     from AE[unfolded all_AE_countable]
   267     from AE[unfolded all_AE_countable]
   268     show "AE x. g x = (SUP i. f' i x)" (is "AE x. g x = ?f x")
   268     show "AE x. g x = (SUP i. f' i x)" (is "AE x. g x = ?f x")
   269     proof (rule AE_mp, safe intro!: AE_cong)
   269     proof (elim AE_mp, safe intro!: AE_I2)
   270       fix x assume eq: "\<forall>i. f i x = f' i x"
   270       fix x assume eq: "\<forall>i. f i x = f' i x"
   271       moreover have "g = SUPR UNIV f" using `f \<up> g` unfolding isoton_def by simp
   271       moreover have "g = SUPR UNIV f" using `f \<up> g` unfolding isoton_def by simp
   272       ultimately show "g x = ?f x" by (simp add: SUPR_apply)
   272       ultimately show "g x = ?f x" by (simp add: SUPR_apply)
   273     qed
   273     qed
   274     show "?f \<in> borel_measurable M"
   274     show "?f \<in> borel_measurable M"