doc-src/Intro/bool.thy
author huffman
Wed, 10 Aug 2011 16:35:50 -0700
changeset 44140 2c10c35dd4be
parent 32960 69916a850301
permissions -rw-r--r--
remove several redundant and unused theorems about derivatives

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