doc-src/Intro/bool.thy
author blanchet
Thu, 24 Mar 2011 17:56:59 +0100
changeset 42108 f55562e77d5c
parent 32960 69916a850301
permissions -rw-r--r--
add "-?" to "nitrox" tool

Bool = FOL +
types   bool 0
arities bool    :: term
consts tt,ff    :: "bool"
end