doc-src/Intro/bool.thy
author nipkow
Sun, 26 Aug 2007 21:28:08 +0200
changeset 24431 02d29baa42ff
parent 105 216d6ed87399
child 32960 69916a850301
permissions -rw-r--r--
tuned linear arith (once again) with ring_distribs

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