src/HOL/Probability/Lebesgue_Integration.thy
changeset 40786 0a54cfc9add3
parent 39910 10097e0a9dbd
child 40859 de0b30e6c2d2
--- a/src/HOL/Probability/Lebesgue_Integration.thy	Sat Nov 27 17:44:36 2010 -0800
+++ b/src/HOL/Probability/Lebesgue_Integration.thy	Sun Nov 28 15:20:51 2010 +0100
@@ -511,7 +511,7 @@
       (\<lambda>(x,y). f -` {x} \<inter> g -` {y} \<inter> space M) ` (f`space M \<times> g`space M)"
       by auto
     hence "finite (?p ` (A \<inter> space M))"
-      by (rule finite_subset) (auto intro: finite_SigmaI finite_imageI) }
+      by (rule finite_subset) auto }
   note this[intro, simp]
 
   { fix x assume "x \<in> space M"