diff -r f32fa5f5bdd1 -r 4d51ddd6aa5c src/HOL/Divides.thy --- a/src/HOL/Divides.thy Thu Apr 24 16:53:04 2008 +0200 +++ b/src/HOL/Divides.thy Fri Apr 25 15:30:33 2008 +0200 @@ -7,7 +7,7 @@ header {* The division operators div, mod and the divides relation dvd *} theory Divides -imports Nat Power Product_Type Wellfounded_Recursion +imports Nat Power Product_Type uses "~~/src/Provers/Arith/cancel_div_mod.ML" begin