diff -r 4898bae6ef23 -r 0a54cfc9add3 src/HOL/Probability/Lebesgue_Integration.thy --- 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 @@ (\(x,y). f -` {x} \ g -` {y} \ space M) ` (f`space M \ g`space M)" by auto hence "finite (?p ` (A \ 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 \ space M"