doc-src/Intro/bool.thy
author wenzelm
Fri, 28 Jan 2011 14:59:48 +0100
changeset 41645 0e6e253ac82c
parent 32960 69916a850301
permissions -rw-r--r--
some adhoc patches for ProofGeneral-4.1pre110112;

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