doc-src/Intro/bool.thy
author boehmes
Tue, 27 Oct 2009 18:09:11 +0100
changeset 33249 2b65e9ed2e6e
parent 32960 69916a850301
permissions -rw-r--r--
removed unused file smt_builtin.ML, made negative pattern polymorphic (similar to positve pattern)

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