src/ZF/Bool.thy
changeset 1401 0c439768f45c
parent 837 778f01546669
child 1478 2b8c2a7547ab
equal deleted inserted replaced
1400:5d909faf0e04 1401:0c439768f45c
     8 2 is equal to bool, but serves a different purpose
     8 2 is equal to bool, but serves a different purpose
     9 *)
     9 *)
    10 
    10 
    11 Bool = ZF + "simpdata" +
    11 Bool = ZF + "simpdata" +
    12 consts
    12 consts
    13     "1"		:: "i"     	   ("1")
    13     "1"		:: i     	   ("1")
    14     "2"         :: "i"             ("2")
    14     "2"         :: i             ("2")
    15     bool        :: "i"
    15     bool        :: i
    16     cond        :: "[i,i,i]=>i"
    16     cond        :: [i,i,i]=>i
    17     not		:: "i=>i"
    17     not		:: i=>i
    18     "and"       :: "[i,i]=>i"      (infixl 70)
    18     "and"       :: [i,i]=>i      (infixl 70)
    19     or		:: "[i,i]=>i"      (infixl 65)
    19     or		:: [i,i]=>i      (infixl 65)
    20     xor		:: "[i,i]=>i"      (infixl 65)
    20     xor		:: [i,i]=>i      (infixl 65)
    21 
    21 
    22 translations
    22 translations
    23    "1"  == "succ(0)"
    23    "1"  == "succ(0)"
    24    "2"  == "succ(1)"
    24    "2"  == "succ(1)"
    25 
    25