src/HOL/Divides.thy
changeset 10212 33fe2d701ddd
parent 8961 b547482dd127
child 10214 77349ed89f45
--- a/src/HOL/Divides.thy	Thu Oct 12 18:09:06 2000 +0200
+++ b/src/HOL/Divides.thy	Thu Oct 12 18:38:23 2000 +0200
@@ -6,7 +6,7 @@
 The division operators div, mod and the divides relation "dvd"
 *)
 
-Divides = Arith +
+Divides = Arithmetic +
 
 (*We use the same class for div and mod;
   moreover, dvd is defined whenever multiplication is*)