doc-src/Intro/bool.thy
author huffman
Thu, 08 Sep 2011 07:16:47 -0700
changeset 44842 282eef2c0f77
parent 32960 69916a850301
permissions -rw-r--r--
remove obsolete intermediate lemma complex_inverse_complex_split

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