src/HOL/Divides.thy
changeset 10214 77349ed89f45
parent 10212 33fe2d701ddd
child 10559 d3fd54fc659b
equal deleted inserted replaced
10213:01c2744a3786 10214:77349ed89f45
     4     Copyright   1999  University of Cambridge
     4     Copyright   1999  University of Cambridge
     5 
     5 
     6 The division operators div, mod and the divides relation "dvd"
     6 The division operators div, mod and the divides relation "dvd"
     7 *)
     7 *)
     8 
     8 
     9 Divides = Arithmetic +
     9 Divides = NatArith +
    10 
    10 
    11 (*We use the same class for div and mod;
    11 (*We use the same class for div and mod;
    12   moreover, dvd is defined whenever multiplication is*)
    12   moreover, dvd is defined whenever multiplication is*)
    13 axclass
    13 axclass
    14   div < term
    14   div < term