doc-src/Intro/bool.thy
author huffman
Fri, 12 Jun 2009 16:23:07 -0700
changeset 31590 776d6a4c1327
parent 105 216d6ed87399
child 32960 69916a850301
permissions -rw-r--r--
declare inner_add, inner_diff [algebra_simps]; declare inner_scaleR [simp]

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