src/HOL/Hyperreal/Lim.thy
changeset 28562 4e74209f113e
parent 27435 b3f8e9bdf9a7
--- a/src/HOL/Hyperreal/Lim.thy	Fri Oct 10 06:45:50 2008 +0200
+++ b/src/HOL/Hyperreal/Lim.thy	Fri Oct 10 06:45:53 2008 +0200
@@ -16,7 +16,7 @@
 definition
   LIM :: "['a::real_normed_vector => 'b::real_normed_vector, 'a, 'b] => bool"
         ("((_)/ -- (_)/ --> (_))" [60, 0, 60] 60) where
-  [code func del]: "f -- a --> L =
+  [code del]: "f -- a --> L =
      (\<forall>r > 0. \<exists>s > 0. \<forall>x. x \<noteq> a & norm (x - a) < s
         --> norm (f x - L) < r)"
 
@@ -26,7 +26,7 @@
 
 definition
   isUCont :: "['a::real_normed_vector => 'b::real_normed_vector] => bool" where
-  [code func del]: "isUCont f = (\<forall>r>0. \<exists>s>0. \<forall>x y. norm (x - y) < s \<longrightarrow> norm (f x - f y) < r)"
+  [code del]: "isUCont f = (\<forall>r>0. \<exists>s>0. \<forall>x y. norm (x - y) < s \<longrightarrow> norm (f x - f y) < r)"
 
 
 subsection {* Limits of Functions *}