src/ZF/ex/Comb.thy
changeset 1478 2b8c2a7547ab
parent 1401 0c439768f45c
child 1702 4aa538e82f76
--- a/src/ZF/ex/Comb.thy	Mon Feb 05 21:33:14 1996 +0100
+++ b/src/ZF/ex/Comb.thy	Tue Feb 06 12:27:17 1996 +0100
@@ -1,6 +1,6 @@
-(*  Title: 	ZF/ex/Comb.thy
+(*  Title:      ZF/ex/Comb.thy
     ID:         $Id$
-    Author: 	Lawrence C Paulson
+    Author:     Lawrence C Paulson
     Copyright   1994  University of Cambridge
 
 Combinatory Logic example: the Church-Rosser Theorem
@@ -27,8 +27,8 @@
 **)
 consts
   contract  :: i
-  "-1->"    :: [i,i] => o    			(infixl 50)
-  "--->"    :: [i,i] => o    			(infixl 50)
+  "-1->"    :: [i,i] => o                       (infixl 50)
+  "--->"    :: [i,i] => o                       (infixl 50)
 
 translations
   "p -1-> q" == "<p,q> : contract"
@@ -49,8 +49,8 @@
 **)
 consts
   parcontract :: i
-  "=1=>"    :: [i,i] => o    			(infixl 50)
-  "===>"    :: [i,i] => o    			(infixl 50)
+  "=1=>"    :: [i,i] => o                       (infixl 50)
+  "===>"    :: [i,i] => o                       (infixl 50)
 
 translations
   "p =1=> q" == "<p,q> : parcontract"