src/HOL/Complex.thy
changeset 31419 74fc28c5d68c
parent 31417 c12b25b7f015
child 31492 5400beeddb55
--- a/src/HOL/Complex.thy	Wed Jun 03 10:02:59 2009 -0700
+++ b/src/HOL/Complex.thy	Wed Jun 03 10:29:11 2009 -0700
@@ -281,7 +281,7 @@
 definition dist_complex_def:
   "dist x y = cmod (x - y)"
 
-definition topo_complex_def:
+definition topo_complex_def [code del]:
   "topo = {S::complex set. \<forall>x\<in>S. \<exists>e>0. \<forall>y. dist y x < e \<longrightarrow> y \<in> S}"
 
 lemmas cmod_def = complex_norm_def