doc-src/Intro/gate.thy
author lcp
Fri, 12 Aug 1994 10:57:55 +0200
changeset 512 55755ed9fab9
parent 105 216d6ed87399
permissions -rw-r--r--
Pure/library/enclose, Pure/Syntax/pretty/enclose: renamed from parents Pure/library/is_blank: now handles form feeds () too, in accordance with ML definition

Gate = FOL +
consts  nand,xor :: "[o,o] => o"
rules   nand_def "nand(P,Q) == ~(P & Q)"
        xor_def  "xor(P,Q)  == P & ~Q | ~P & Q"
end