src/HOL/Quotient_Examples/Quotient_Int.thy
changeset 37767 a2b7a20d6ea3
parent 37594 32ad67684ee7
child 39198 f967a16dfcdd
--- a/src/HOL/Quotient_Examples/Quotient_Int.thy	Mon Jul 12 08:58:27 2010 +0200
+++ b/src/HOL/Quotient_Examples/Quotient_Int.thy	Mon Jul 12 10:48:37 2010 +0200
@@ -42,7 +42,7 @@
   "(uminus \<Colon> (int \<Rightarrow> int))" is "uminus_int_raw"
 
 definition
-  minus_int_def [code del]:  "z - w = z + (-w\<Colon>int)"
+  minus_int_def:  "z - w = z + (-w\<Colon>int)"
 
 fun
   times_int_raw :: "(nat \<times> nat) \<Rightarrow> (nat \<times> nat) \<Rightarrow> (nat \<times> nat)"
@@ -61,7 +61,7 @@
   le_int_def: "(op \<le>) :: int \<Rightarrow> int \<Rightarrow> bool" is "le_int_raw"
 
 definition
-  less_int_def [code del]: "(z\<Colon>int) < w = (z \<le> w \<and> z \<noteq> w)"
+  less_int_def: "(z\<Colon>int) < w = (z \<le> w \<and> z \<noteq> w)"
 
 definition
   zabs_def: "\<bar>i\<Colon>int\<bar> = (if i < 0 then - i else i)"