src/ZF/ex/PropLog.thy
changeset 1478 2b8c2a7547ab
parent 1401 0c439768f45c
child 3840 e0baea4d485a
--- a/src/ZF/ex/PropLog.thy	Mon Feb 05 21:33:14 1996 +0100
+++ b/src/ZF/ex/PropLog.thy	Tue Feb 06 12:27:17 1996 +0100
@@ -1,6 +1,6 @@
-(*  Title: 	ZF/ex/PropLog.thy
+(*  Title:      ZF/ex/PropLog.thy
     ID:         $Id$
-    Author: 	Tobias Nipkow & Lawrence C Paulson
+    Author:     Tobias Nipkow & Lawrence C Paulson
     Copyright   1993  University of Cambridge
 
 Datatype definition of propositional logic formulae and inductive definition
@@ -15,13 +15,13 @@
 
 datatype
   "prop" = Fls
-         | Var ("n: nat")	                ("#_" [100] 100)
-         | "=>" ("p: prop", "q: prop")		(infixr 90)
+         | Var ("n: nat")                       ("#_" [100] 100)
+         | "=>" ("p: prop", "q: prop")          (infixr 90)
 
 (** The proof system **)
 consts
   thms     :: i => i
-  "|-"     :: [i,i] => o    			(infixl 50)
+  "|-"     :: [i,i] => o                        (infixl 50)
 
 translations
   "H |- p" == "p : thms(H)"
@@ -41,7 +41,7 @@
 consts
   prop_rec :: [i, i, i=>i, [i,i,i,i]=>i] => i
   is_true  :: [i,i] => o
-  "|="     :: [i,i] => o    			(infixl 50)
+  "|="     :: [i,i] => o                        (infixl 50)
   hyps     :: [i,i] => i
 
 defs