return to top
source
Boolean exclusive or
De Morgan's law for boolean and
De Morgan's law for boolean or
These two rules follow trivially by simp, but are needed to avoid non-termination in false_eq and true_eq.
convert a Bool to a Nat, false -> 0, true -> 1
Bool
Nat
false -> 0
true -> 1
If the return values are propositions, there is no harm in simplifying a bif to an if.
bif
if
This should not be turned on globally as an instance because it degrades performance in Mathlib, but may be used locally.