src/HOL/Integ/NatBin.thy
author nipkow
Mon, 06 Aug 2001 13:43:24 +0200
changeset 11464 ddea204de5bc
parent 10574 8f98f0301d67
child 11468 02cd5d5bc497
permissions -rw-r--r--
turned translation for 1::nat into def.
introduced 1' and replaced most occurrences of 1 by 1'.
     1 (*  Title:      HOL/NatBin.thy
     2     ID:         $Id$
     3     Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
     4     Copyright   1999  University of Cambridge
     5 
     6 Binary arithmetic for the natural numbers
     7 
     8 This case is simply reduced to that for the non-negative integers
     9 *)
    10 
    11 theory NatBin = IntPower
    12 files ("nat_bin.ML"):
    13 
    14 instance  nat :: number ..
    15 
    16 defs
    17   nat_number_of_def:
    18     "number_of v == nat (number_of v)"
    19      (*::bin=>nat        ::bin=>int*)
    20 
    21 axioms
    22 neg_number_of_bin_pred_iff_0:
    23   "neg (number_of (bin_pred v)) = (number_of v = (0::nat))"
    24 
    25 use "nat_bin.ML"	setup nat_bin_arith_setup
    26 
    27 end