doc-src/Intro/bool.thy
author wenzelm
Tue, 23 Aug 2011 16:53:05 +0200
changeset 44389 a3b5fdfb04a3
parent 32960 69916a850301
permissions -rw-r--r--
tuned signature -- contrast physical output primitives versus Output.raw_message;

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