doc-src/Intro/bool.thy
changeset 32960 69916a850301
parent 105 216d6ed87399
equal deleted inserted replaced
32959:23a8c5ac35f8 32960:69916a850301
     1 Bool = FOL +
     1 Bool = FOL +
     2 types 	bool 0
     2 types   bool 0
     3 arities bool 	:: term
     3 arities bool    :: term
     4 consts tt,ff	:: "bool"
     4 consts tt,ff    :: "bool"
     5 end
     5 end