1 Defs = Types +
2 consts nand, exor :: gate
3 defs nand_def "nand A B == ~(A & B)"
4 exor_def "exor A B == A & ~B | ~A & B"
5 end