src/HOL/IntDiv.thy
changeset 25571 c9e39eafc7a0
parent 25134 3d4953e88449
child 25919 8b1c0d434824
--- a/src/HOL/IntDiv.thy	Fri Dec 07 15:07:56 2007 +0100
+++ b/src/HOL/IntDiv.thy	Fri Dec 07 15:07:59 2007 +0100
@@ -62,9 +62,18 @@
                   if 0<b then negDivAlg a b
                   else negateSnd (posDivAlg (-a) (-b))))"
 
-instance int :: Divides.div
-  div_def: "a div b == fst (divAlg (a, b))"
-  mod_def: "a mod b == snd (divAlg (a, b))" ..
+instantiation int :: Divides.div
+begin
+
+definition
+  div_def: "a div b = fst (divAlg (a, b))"
+
+definition
+  mod_def: "a mod b = snd (divAlg (a, b))"
+
+instance ..
+
+end
 
 lemma divAlg_mod_div:
   "divAlg (p, q) = (p div q, p mod q)"