diff -r e1bd8a54c40f -r d7728f65b353 src/HOL/Probability/Borel.thy --- a/src/HOL/Probability/Borel.thy Mon Sep 13 08:43:48 2010 +0200 +++ b/src/HOL/Probability/Borel.thy Mon Sep 13 11:13:15 2010 +0200 @@ -1031,7 +1031,7 @@ have "f -` {\} \ space M = {x\space M. f x = \}" by auto with * have **: "{x\space M. f x = \} \ sets M" by simp have f: "f = (\x. if f x = \ then \ else Real (real (f x)))" - by (simp add: ext_iff Real_real) + by (simp add: fun_eq_iff Real_real) show "f \ borel_measurable M" apply (subst f) apply (rule measurable_If) @@ -1264,7 +1264,7 @@ proof - have *: "(\x. f x + g x) = (\x. if f x = \ then \ else if g x = \ then \ else Real (real (f x) + real (g x)))" - by (auto simp: ext_iff pinfreal_noteq_omega_Ex) + by (auto simp: fun_eq_iff pinfreal_noteq_omega_Ex) show ?thesis using assms unfolding * by (auto intro!: measurable_If) qed @@ -1276,7 +1276,7 @@ have *: "(\x. f x * g x) = (\x. if f x = 0 then 0 else if g x = 0 then 0 else if f x = \ then \ else if g x = \ then \ else Real (real (f x) * real (g x)))" - by (auto simp: ext_iff pinfreal_noteq_omega_Ex) + by (auto simp: fun_eq_iff pinfreal_noteq_omega_Ex) show ?thesis using assms unfolding * by (auto intro!: measurable_If) qed