doc-src/Intro/gate.thy
author wenzelm
Sun, 13 Mar 2011 19:16:19 +0100
changeset 41952 c7297638599b
parent 105 216d6ed87399
permissions -rw-r--r--
cleanup of former settings GHC_PATH, EXEC_GHC, EXEC_OCAML, EXEC_SWIPL, EXEC_YAP -- discontinued implicit detection; determine swipl_version at runtime;

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