src/HOL/Integ/NatBin.thy
changeset 15131 c69542757a4d
parent 15129 fbf90acc5bf4
child 15140 322485b816ac
equal deleted inserted replaced
15130:dc6be28d7f4e 15131:c69542757a4d
     4     Copyright   1999  University of Cambridge
     4     Copyright   1999  University of Cambridge
     5 *)
     5 *)
     6 
     6 
     7 header {* Binary arithmetic for the natural numbers *}
     7 header {* Binary arithmetic for the natural numbers *}
     8 
     8 
     9 theory NatBin = IntDiv:
     9 theory NatBin
       
    10 import IntDiv
       
    11 begin
    10 
    12 
    11 text {*
    13 text {*
    12   Arithmetic for naturals is reduced to that for the non-negative integers.
    14   Arithmetic for naturals is reduced to that for the non-negative integers.
    13 *}
    15 *}
    14 
    16