doc-src/Intro/bool.thy
author wenzelm
Fri, 07 Jan 2011 14:36:41 +0100
changeset 41442 4cfb51a5a444
parent 32960 69916a850301
permissions -rw-r--r--
updated for 2011; emphasize "contributors" in the header as well, which are already mentioned in the body text;

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