src/HOL/Probability/Lebesgue_Integration.thy
changeset 50021 d96a3f468203
parent 50003 8c213922ed49
child 50027 7747a9f4c358
--- a/src/HOL/Probability/Lebesgue_Integration.thy	Tue Nov 06 15:15:33 2012 +0100
+++ b/src/HOL/Probability/Lebesgue_Integration.thy	Tue Nov 06 19:18:35 2012 +0100
@@ -270,7 +270,7 @@
     have "simple_function M (\<lambda>x. real (f x i))"
     proof (intro simple_function_borel_measurable)
       show "(\<lambda>x. real (f x i)) \<in> borel_measurable M"
-        using u by (auto intro!: measurable_If simp: real_f)
+        using u by (auto simp: real_f)
       have "(\<lambda>x. real (f x i))`space M \<subseteq> real`{..i*2^i}"
         using f_upper[of _ i] by auto
       then show "finite ((\<lambda>x. real (f x i))`space M)"