src/HOL/Library/Lub_Glb.thy
changeset 68356 46d5a9f428e1
parent 67613 ce654b0e6d69
child 69593 3dda49e08b9d
--- a/src/HOL/Library/Lub_Glb.thy	Sat Jun 02 22:11:09 2018 +0200
+++ b/src/HOL/Library/Lub_Glb.thy	Sat Jun 02 22:14:35 2018 +0200
@@ -221,7 +221,7 @@
 
 lemma isLub_mono_imp_LIMSEQ:
   fixes X :: "nat \<Rightarrow> real"
-  assumes u: "isLub UNIV {x. \<exists>n. X n = x} u" (* FIXME: use 'range X' *)
+  assumes u: "isLub UNIV {x. \<exists>n. X n = x} u" (* FIXME: use \<open>range X\<close> *)
   assumes X: "\<forall>m n. m \<le> n \<longrightarrow> X m \<le> X n"
   shows "X \<longlonglongrightarrow> u"
 proof -