doc-src/Intro/bool.thy
author wenzelm
Wed, 25 Jan 2012 15:39:08 +0100
changeset 46256 bc874d2ee55a
parent 32960 69916a850301
permissions -rw-r--r--
updated RSN, RL, RLN, MRS; discontinued obscure MRL;

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