doc-src/Intro/bool.thy
author blanchet
Wed, 08 Sep 2010 15:57:50 +0200
changeset 39222 decf607a5a67
parent 32960 69916a850301
permissions -rw-r--r--
remove "safe" (as suggested by Tobias) and added "arith" to "try"

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