src/HOL/NSA/HSeries.thy
changeset 28562 4e74209f113e
parent 27468 0783dd1dc13d
child 30273 ecd6f0ca62ea
--- a/src/HOL/NSA/HSeries.thy	Fri Oct 10 06:45:50 2008 +0200
+++ b/src/HOL/NSA/HSeries.thy	Fri Oct 10 06:45:53 2008 +0200
@@ -13,7 +13,7 @@
 
 definition
   sumhr :: "(hypnat * hypnat * (nat=>real)) => hypreal" where
-  [code func del]: "sumhr = 
+  [code del]: "sumhr = 
       (%(M,N,f). starfun2 (%m n. setsum f {m..<n}) M N)"
 
 definition
@@ -22,7 +22,7 @@
 
 definition
   NSsummable :: "(nat=>real) => bool" where
-  [code func del]: "NSsummable f = (\<exists>s. f NSsums s)"
+  [code del]: "NSsummable f = (\<exists>s. f NSsums s)"
 
 definition
   NSsuminf   :: "(nat=>real) => real" where