diff -r 0c18df79b1c8 -r a642599ffdea src/ZF/Bool.thy --- a/src/ZF/Bool.thy Tue Sep 27 17:03:23 2022 +0100 +++ b/src/ZF/Bool.thy Tue Sep 27 17:46:52 2022 +0100 @@ -24,15 +24,15 @@ definition "not(b) \ cond(b,0,1)" definition - "and" :: "[i,i]=>i" (infixl \and\ 70) where + "and" :: "[i,i]\i" (infixl \and\ 70) where "a and b \ cond(a,b,0)" definition - or :: "[i,i]=>i" (infixl \or\ 65) where + or :: "[i,i]\i" (infixl \or\ 65) where "a or b \ cond(a,1,b)" definition - xor :: "[i,i]=>i" (infixl \xor\ 65) where + xor :: "[i,i]\i" (infixl \xor\ 65) where "a xor b \ cond(a,not(b),b)" @@ -152,7 +152,7 @@ definition - bool_of_o :: "o=>i" where + bool_of_o :: "o\i" where "bool_of_o(P) \ (if P then 1 else 0)" lemma [simp]: "bool_of_o(True) = 1"