src/HOL/NSA/HLim.thy
changeset 28562 4e74209f113e
parent 27468 0783dd1dc13d
child 31338 d41a8ba25b67
--- a/src/HOL/NSA/HLim.thy	Fri Oct 10 06:45:50 2008 +0200
+++ b/src/HOL/NSA/HLim.thy	Fri Oct 10 06:45:53 2008 +0200
@@ -16,18 +16,18 @@
 definition
   NSLIM :: "['a::real_normed_vector => 'b::real_normed_vector, 'a, 'b] => bool"
             ("((_)/ -- (_)/ --NS> (_))" [60, 0, 60] 60) where
-  [code func del]: "f -- a --NS> L =
+  [code del]: "f -- a --NS> L =
     (\<forall>x. (x \<noteq> star_of a & x @= star_of a --> ( *f* f) x @= star_of L))"
 
 definition
   isNSCont :: "['a::real_normed_vector => 'b::real_normed_vector, 'a] => bool" where
     --{*NS definition dispenses with limit notions*}
-  [code func del]: "isNSCont f a = (\<forall>y. y @= star_of a -->
+  [code del]: "isNSCont f a = (\<forall>y. y @= star_of a -->
          ( *f* f) y @= star_of (f a))"
 
 definition
   isNSUCont :: "['a::real_normed_vector => 'b::real_normed_vector] => bool" where
-  [code func del]: "isNSUCont f = (\<forall>x y. x @= y --> ( *f* f) x @= ( *f* f) y)"
+  [code del]: "isNSUCont f = (\<forall>x y. x @= y --> ( *f* f) x @= ( *f* f) y)"
 
 
 subsection {* Limits of Functions *}