1 Exor = Main +
2 constdefs
3 exor :: bool => bool => bool
4 "exor A B == (A & ~B) | (~A & B)"
5 end