src/HOL/Analysis/Continuum_Not_Denumerable.thy
changeset 69597 ff784d5a5bfb
parent 69565 1daf07b65385
child 70136 f03a01a18c6e
--- a/src/HOL/Analysis/Continuum_Not_Denumerable.thy	Sat Jan 05 17:00:43 2019 +0100
+++ b/src/HOL/Analysis/Continuum_Not_Denumerable.thy	Sat Jan 05 17:24:33 2019 +0100
@@ -38,7 +38,7 @@
   assume "\<exists>f::nat \<Rightarrow> real. surj f"
   then obtain f :: "nat \<Rightarrow> real" where "surj f" ..
 
-  txt \<open>First we construct a sequence of nested intervals, ignoring @{term "range f"}.\<close>
+  txt \<open>First we construct a sequence of nested intervals, ignoring \<^term>\<open>range f\<close>.\<close>
 
   have "a < b \<Longrightarrow> \<exists>ka kb. ka < kb \<and> {ka..kb} \<subseteq> {a..b} \<and> c \<notin> {ka..kb}" for a b c :: real
     by (auto simp add: not_le cong: conj_cong)