src/HOL/Hyperreal/SEQ.thy
changeset 11701 3d51fbf81c17
parent 10751 a81ea5d3dd41
child 12018 ec054019c910
--- a/src/HOL/Hyperreal/SEQ.thy	Fri Oct 05 21:50:37 2001 +0200
+++ b/src/HOL/Hyperreal/SEQ.thy	Fri Oct 05 21:52:39 2001 +0200
@@ -10,7 +10,7 @@
 
   (* Standard definition of convergence of sequence *)           
   LIMSEQ :: [nat=>real,real] => bool    ("((_)/ ----> (_))" [60, 60] 60)
-  "X ----> L == (ALL r. #0 < r --> (EX no. ALL n. no <= n --> abs (X n + -L) < r))"
+  "X ----> L == (ALL r. Numeral0 < r --> (EX no. ALL n. no <= n --> abs (X n + -L) < r))"
   
   (* Nonstandard definition of convergence of sequence *)
   NSLIMSEQ :: [nat=>real,real] => bool    ("((_)/ ----NS> (_))" [60, 60] 60)
@@ -33,7 +33,7 @@
 
   (* Standard definition for bounded sequence *)
   Bseq :: (nat => real) => bool
-  "Bseq X == (EX K. (#0 < K & (ALL n. abs(X n) <= K)))"
+  "Bseq X == (EX K. (Numeral0 < K & (ALL n. abs(X n) <= K)))"
  
   (* Nonstandard definition for bounded sequence *)
   NSBseq :: (nat=>real) => bool
@@ -52,7 +52,7 @@
 
   (* Standard definition *)
   Cauchy :: (nat => real) => bool
-  "Cauchy X == (ALL e. (#0 < e -->
+  "Cauchy X == (ALL e. (Numeral0 < e -->
                        (EX M. (ALL m n. M <= m & M <= n 
                              --> abs((X m) + -(X n)) < e))))"