src/HOL/Lim.thy
changeset 31353 14a58e2ca374
parent 31349 2261c8781f73
child 31355 3d18766ddc4b
--- a/src/HOL/Lim.thy	Mon Jun 01 07:45:49 2009 -0700
+++ b/src/HOL/Lim.thy	Mon Jun 01 07:57:37 2009 -0700
@@ -14,7 +14,7 @@
 
 definition
   at :: "'a::metric_space \<Rightarrow> 'a filter" where
-  "at a = Abs_filter (\<lambda>P. \<exists>r>0. \<forall>x. x \<noteq> a \<and> dist x a < r \<longrightarrow> P x)"
+  [code del]: "at a = Abs_filter (\<lambda>P. \<exists>r>0. \<forall>x. x \<noteq> a \<and> dist x a < r \<longrightarrow> P x)"
 
 definition
   LIM :: "['a::metric_space \<Rightarrow> 'b::metric_space, 'a, 'b] \<Rightarrow> bool"