doc-src/Intro/bool.thy
changeset 32960 69916a850301
parent 105 216d6ed87399
--- a/doc-src/Intro/bool.thy	Sat Oct 17 01:05:59 2009 +0200
+++ b/doc-src/Intro/bool.thy	Sat Oct 17 14:43:18 2009 +0200
@@ -1,5 +1,5 @@
 Bool = FOL +
-types 	bool 0
-arities bool 	:: term
-consts tt,ff	:: "bool"
+types   bool 0
+arities bool    :: term
+consts tt,ff    :: "bool"
 end