src/HOL/IntDiv.thy
changeset 28562 4e74209f113e
parent 28262 aa7ca36d67fd
child 29045 3c8f48333731
--- a/src/HOL/IntDiv.thy	Fri Oct 10 06:45:50 2008 +0200
+++ b/src/HOL/IntDiv.thy	Fri Oct 10 06:45:53 2008 +0200
@@ -14,13 +14,13 @@
 constdefs
   quorem :: "(int*int) * (int*int) => bool"
     --{*definition of quotient and remainder*}
-    [code func]: "quorem == %((a,b), (q,r)).
+    [code]: "quorem == %((a,b), (q,r)).
                       a = b*q + r &
                       (if 0 < b then 0\<le>r & r<b else b<r & r \<le> 0)"
 
   adjust :: "[int, int*int] => int*int"
     --{*for the division algorithm*}
-    [code func]: "adjust b == %(q,r). if 0 \<le> r-b then (2*q + 1, r-b)
+    [code]: "adjust b == %(q,r). if 0 \<le> r-b then (2*q + 1, r-b)
                          else (2*q, r)"
 
 text{*algorithm for the case @{text "a\<ge>0, b>0"}*}
@@ -46,7 +46,7 @@
 text{*algorithm for the general case @{term "b\<noteq>0"}*}
 constdefs
   negateSnd :: "int*int => int*int"
-    [code func]: "negateSnd == %(q,r). (q,-r)"
+    [code]: "negateSnd == %(q,r). (q,-r)"
 
 definition
   divAlg :: "int \<times> int \<Rightarrow> int \<times> int"
@@ -1477,7 +1477,7 @@
 context ring_1
 begin
 
-lemma of_int_num [code func]:
+lemma of_int_num [code]:
   "of_int k = (if k = 0 then 0 else if k < 0 then
      - of_int (- k) else let
        (l, m) = divAlg (k, 2);