doc-src/Tutorial/Misc/Defs.thy
author kleing
Mon, 29 Mar 2004 10:17:35 +0200
changeset 14493 216179c782a6
parent 5377 efb799c5ed3c
permissions -rw-r--r--
include exercises again

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