src/HOL/Archimedean_Field.thy
changeset 43704 47b0be18ccbe
parent 41959 b460124855b8
child 43732 6b2bdc57155b
--- a/src/HOL/Archimedean_Field.thy	Wed Jul 06 23:11:59 2011 +0200
+++ b/src/HOL/Archimedean_Field.thy	Thu Jul 07 23:33:14 2011 +0200
@@ -143,7 +143,7 @@
 
 definition
   floor :: "'a::archimedean_field \<Rightarrow> int" where
-  "floor x = (THE z. of_int z \<le> x \<and> x < of_int (z + 1))"
+  [code del]: "floor x = (THE z. of_int z \<le> x \<and> x < of_int (z + 1))"
 
 notation (xsymbols)
   floor  ("\<lfloor>_\<rfloor>")
@@ -274,7 +274,7 @@
 
 definition
   ceiling :: "'a::archimedean_field \<Rightarrow> int" where
-  "ceiling x = - floor (- x)"
+  [code del]: "ceiling x = - floor (- x)"
 
 notation (xsymbols)
   ceiling  ("\<lceil>_\<rceil>")