src/HOL/Nonstandard_Analysis/HSEQ.thy
changeset 67443 3abf6a722518
parent 67006 b1278ed3cd46
child 68614 3cb44b0abc5c
--- a/src/HOL/Nonstandard_Analysis/HSEQ.thy	Tue Jan 16 09:12:16 2018 +0100
+++ b/src/HOL/Nonstandard_Analysis/HSEQ.thy	Tue Jan 16 09:30:00 2018 +0100
@@ -17,7 +17,7 @@
 
 definition NSLIMSEQ :: "(nat \<Rightarrow> 'a::real_normed_vector) \<Rightarrow> 'a \<Rightarrow> bool"
     ("((_)/ \<longlonglongrightarrow>\<^sub>N\<^sub>S (_))" [60, 60] 60) where
-    \<comment>\<open>Nonstandard definition of convergence of sequence\<close>
+    \<comment> \<open>Nonstandard definition of convergence of sequence\<close>
   "X \<longlonglongrightarrow>\<^sub>N\<^sub>S L \<longleftrightarrow> (\<forall>N \<in> HNatInfinite. ( *f* X) N \<approx> star_of L)"
 
 definition nslim :: "(nat \<Rightarrow> 'a::real_normed_vector) \<Rightarrow> 'a"