src/HOL/Divides.thy
changeset 15140 322485b816ac
parent 15131 c69542757a4d
child 15251 bb6f072c8d10
--- a/src/HOL/Divides.thy	Tue Aug 17 11:00:24 2004 +0200
+++ b/src/HOL/Divides.thy	Wed Aug 18 11:09:40 2004 +0200
@@ -7,7 +7,7 @@
 *)
 
 theory Divides
-import NatArith
+imports NatArith
 begin
 
 (*We use the same class for div and mod;