diff -r 88a69da5d3fa -r eff000cab70f src/HOL/Probability/Regularity.thy --- a/src/HOL/Probability/Regularity.thy Sat May 25 15:44:08 2013 +0200 +++ b/src/HOL/Probability/Regularity.thy Sat May 25 15:44:29 2013 +0200 @@ -209,8 +209,8 @@ from nat_approx_posE[OF this] guess n . note n = this let ?k = "from_nat_into X ` {0..k e (Suc n)}" have "finite ?k" by simp - moreover have "K \ \(\x. ball x e') ` ?k" unfolding K_def B_def using n by force - ultimately show "\k. finite k \ K \ \(\x. ball x e') ` k" by blast + moreover have "K \ \((\x. ball x e') ` ?k)" unfolding K_def B_def using n by force + ultimately show "\k. finite k \ K \ \((\x. ball x e') ` k)" by blast qed ultimately show "?thesis e " by (auto simp: sU)