src/HOL/Library/ContNotDenum.thy
changeset 61585 a9599d3d7610
parent 60500 903bb1495239
child 61880 ff4d33058566
--- a/src/HOL/Library/ContNotDenum.thy	Thu Nov 05 10:35:37 2015 +0100
+++ b/src/HOL/Library/ContNotDenum.thy	Thu Nov 05 10:39:49 2015 +0100
@@ -15,8 +15,8 @@
 uncountable. It is formalised in the Isabelle/Isar theorem proving
 system.
 
-{\em Theorem:} The Continuum @{text "\<real>"} is not denumerable. In other
-words, there does not exist a function @{text "f: \<nat> \<Rightarrow> \<real>"} such that f is
+{\em Theorem:} The Continuum \<open>\<real>\<close> is not denumerable. In other
+words, there does not exist a function \<open>f: \<nat> \<Rightarrow> \<real>\<close> such that f is
 surjective.
 
 {\em Outline:} An elegant informal proof of this result uses Cantor's
@@ -26,8 +26,7 @@
 completeness of the Real numbers and is the foundation for our
 argument. Informally it states that an intersection of countable
 closed intervals (where each successive interval is a subset of the
-last) is non-empty. We then assume a surjective function @{text
-"f: \<nat> \<Rightarrow> \<real>"} exists and find a real x such that x is not in the range of f
+last) is non-empty. We then assume a surjective function \<open>f: \<nat> \<Rightarrow> \<real>\<close> exists and find a real x such that x is not in the range of f
 by generating a sequence of closed intervals then using the NIP.\<close>
 
 theorem real_non_denum: "\<not> (\<exists>f :: nat \<Rightarrow> real. surj f)"