src/HOL/Integ/IntDiv.thy
changeset 7706 da41066983e5
parent 6993 efb605156ca3
child 8902 a705822f4e2a
--- a/src/HOL/Integ/IntDiv.thy	Mon Oct 04 21:46:49 1999 +0200
+++ b/src/HOL/Integ/IntDiv.thy	Mon Oct 04 21:47:16 1999 +0200
@@ -6,7 +6,7 @@
 The division operators div, mod and the divides relation "dvd"
 *)
 
-IntDiv = Bin + Recdef + 
+IntDiv = IntArith + Recdef + 
 
 constdefs
   quorem :: "(int*int) * (int*int) => bool"