src/HOL/Hyperreal/HSeries.thy
changeset 21404 eb85850d3eb7
parent 20898 113c9516a2d7
child 21841 1701f05aa1b0
--- a/src/HOL/Hyperreal/HSeries.thy	Fri Nov 17 02:19:55 2006 +0100
+++ b/src/HOL/Hyperreal/HSeries.thy	Fri Nov 17 02:20:03 2006 +0100
@@ -12,17 +12,20 @@
 begin
 
 definition
-  sumhr :: "(hypnat * hypnat * (nat=>real)) => hypreal"
+  sumhr :: "(hypnat * hypnat * (nat=>real)) => hypreal" where
   "sumhr = 
       (%(M,N,f). starfun2 (%m n. setsum f {m..<n}) M N)"
 
-  NSsums  :: "[nat=>real,real] => bool"     (infixr "NSsums" 80)
+definition
+  NSsums  :: "[nat=>real,real] => bool"     (infixr "NSsums" 80) where
   "f NSsums s = (%n. setsum f {0..<n}) ----NS> s"
 
-  NSsummable :: "(nat=>real) => bool"
+definition
+  NSsummable :: "(nat=>real) => bool" where
   "NSsummable f = (\<exists>s. f NSsums s)"
 
-  NSsuminf   :: "(nat=>real) => real"
+definition
+  NSsuminf   :: "(nat=>real) => real" where
   "NSsuminf f = (THE s. f NSsums s)"