src/HOL/Divides.thy
changeset 26072 f65a7fa2da6c
parent 26062 16f334d7156a
child 26100 fbc60cd02ae2
--- a/src/HOL/Divides.thy	Fri Feb 15 16:09:10 2008 +0100
+++ b/src/HOL/Divides.thy	Fri Feb 15 16:09:12 2008 +0100
@@ -7,7 +7,7 @@
 header {* The division operators div, mod and the divides relation "dvd" *}
 
 theory Divides
-imports Power
+imports Power Wellfounded_Recursion
 uses "~~/src/Provers/Arith/cancel_div_mod.ML"
 begin