src/HOL/Integ/IntDiv.thy
changeset 21409 6aa28caa96c5
parent 20485 3078fd2eec7b
child 22026 cc60e54aa7cb
--- a/src/HOL/Integ/IntDiv.thy	Sat Nov 18 00:20:15 2006 +0100
+++ b/src/HOL/Integ/IntDiv.thy	Sat Nov 18 00:20:16 2006 +0100
@@ -9,7 +9,7 @@
 header{*The Division Operators div and mod; the Divides Relation dvd*}
 
 theory IntDiv
-imports "../SetInterval" "../Recdef"
+imports "../Divides" "../SetInterval" "../Recdef"
 uses ("IntDiv_setup.ML")
 begin