src/HOL/Hyperreal/SEQ.thy
changeset 20693 f763367e332f
parent 20691 53cbea20e4d9
child 20695 1cc6fefbff1a
--- a/src/HOL/Hyperreal/SEQ.thy	Sun Sep 24 05:49:50 2006 +0200
+++ b/src/HOL/Hyperreal/SEQ.thy	Sun Sep 24 06:54:39 2006 +0200
@@ -24,11 +24,11 @@
     --{*Nonstandard definition of convergence of sequence*}
   "X ----NS> L = (\<forall>N \<in> HNatInfinite. ( *f* X) N \<approx> star_of L)"
 
-  lim :: "(nat => real) => real"
+  lim :: "(nat => 'a::real_normed_vector) => 'a"
     --{*Standard definition of limit using choice operator*}
   "lim X = (THE L. X ----> L)"
 
-  nslim :: "(nat => real) => real"
+  nslim :: "(nat => 'a::real_normed_vector) => 'a"
     --{*Nonstandard definition of limit using choice operator*}
   "nslim X = (THE L. X ----NS> L)"