diff -r a3f37b3d303a -r cf26dd7395e4 src/HOL/Library/ContNotDenum.thy --- a/src/HOL/Library/ContNotDenum.thy Wed Nov 24 10:52:02 2010 +0100 +++ b/src/HOL/Library/ContNotDenum.thy Mon Nov 22 10:34:33 2010 +0100 @@ -565,8 +565,7 @@ shows "\ (\f::nat\real. surj f)" proof -- "by contradiction" assume "\f::nat\real. surj f" - then obtain f::"nat\real" where "surj f" by auto - hence rangeF: "range f = UNIV" by (rule surj_range) + then obtain f::"nat\real" where rangeF: "surj f" by auto -- "We now produce a real number x that is not in the range of f, using the properties of newInt. " have "\x. x \ (\n. newInt n f)" using newInt_notempty by blast moreover have "\n. f n \ (\n. newInt n f)" by (rule newInt_inter)