diff -r 19efc2af3e6c -r f967a16dfcdd src/HOL/Probability/Borel.thy --- a/src/HOL/Probability/Borel.thy Mon Sep 06 22:58:06 2010 +0200 +++ b/src/HOL/Probability/Borel.thy Tue Sep 07 10:05:19 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: expand_fun_eq Real_real) + by (simp add: ext_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: expand_fun_eq pinfreal_noteq_omega_Ex) + by (auto simp: ext_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: expand_fun_eq pinfreal_noteq_omega_Ex) + by (auto simp: ext_iff pinfreal_noteq_omega_Ex) show ?thesis using assms unfolding * by (auto intro!: measurable_If) qed