src/HOL/Library/Lub_Glb.thy
changeset 61969 e01015e49041
parent 61585 a9599d3d7610
child 62343 24106dc44def
--- a/src/HOL/Library/Lub_Glb.thy	Tue Dec 29 22:41:22 2015 +0100
+++ b/src/HOL/Library/Lub_Glb.thy	Tue Dec 29 23:04:53 2015 +0100
@@ -223,9 +223,9 @@
   fixes X :: "nat \<Rightarrow> real"
   assumes u: "isLub UNIV {x. \<exists>n. X n = x} u" (* FIXME: use 'range X' *)
   assumes X: "\<forall>m n. m \<le> n \<longrightarrow> X m \<le> X n"
-  shows "X ----> u"
+  shows "X \<longlonglongrightarrow> u"
 proof -
-  have "X ----> (SUP i. X i)"
+  have "X \<longlonglongrightarrow> (SUP i. X i)"
     using u[THEN isLubD1] X
     by (intro LIMSEQ_incseq_SUP) (auto simp: incseq_def image_def eq_commute bdd_above_setle)
   also have "(SUP i. X i) = u"