src/ZF/Nat.thy
changeset 435 ca5356bd315a
parent 124 858ab9a9b047
child 753 ec86863e87c8
equal deleted inserted replaced
434:89d45187f04d 435:ca5356bd315a
     1 (*  Title: 	ZF/nat.thy
     1 (*  Title: 	ZF/Nat.thy
     2     ID:         $Id$
     2     ID:         $Id$
     3     Author: 	Lawrence C Paulson, Cambridge University Computer Laboratory
     3     Author: 	Lawrence C Paulson, Cambridge University Computer Laboratory
     4     Copyright   1992  University of Cambridge
     4     Copyright   1994  University of Cambridge
     5 
     5 
     6 Natural numbers in Zermelo-Fraenkel Set Theory 
     6 Natural numbers in Zermelo-Fraenkel Set Theory 
     7 *)
     7 *)
     8 
     8 
     9 Nat = Ord + Bool + "mono" +
     9 Nat = Ordinal + Bool + "mono" +
    10 consts
    10 consts
    11     nat 	::      "i"
    11     nat 	::      "i"
    12     nat_case    ::      "[i, i=>i, i]=>i"
    12     nat_case    ::      "[i, i=>i, i]=>i"
    13     nat_rec     ::      "[i, i, [i,i]=>i]=>i"
    13     nat_rec     ::      "[i, i, [i,i]=>i]=>i"
    14 
    14