# HG changeset patch # User wenzelm # Date 1466436308 -7200 # Node ID 814541a57d89fd856fbaf96188105f556a822637 # Parent bc1f17d45e9127ca66c704fda4e8531d752df135 tuned proof; diff -r bc1f17d45e91 -r 814541a57d89 src/HOL/Fun.thy --- a/src/HOL/Fun.thy Mon Jun 20 17:03:50 2016 +0200 +++ b/src/HOL/Fun.thy Mon Jun 20 17:25:08 2016 +0200 @@ -793,15 +793,15 @@ subsection \Cantor's Paradox\ -lemma Cantors_paradox: "\ (\f. f ` A = Pow A)" -proof clarify - fix f - assume "f ` A = Pow A" - then have *: "Pow A \ f ` A" by blast +theorem Cantors_paradox: "\f. f ` A = Pow A" +proof + assume "\f. f ` A = Pow A" + then obtain f where f: "f ` A = Pow A" .. let ?X = "{a \ A. a \ f a}" - have "?X \ Pow A" unfolding Pow_def by auto - with * obtain x where "x \ A \ f x = ?X" by blast - then show False by best + have "?X \ Pow A" by blast + then have "?X \ f ` A" by (simp only: f) + then obtain x where "x \ A" and "f x = ?X" by blast + then show False by blast qed