src/ZF/Zorn.thy
changeset 1478 2b8c2a7547ab
parent 1401 0c439768f45c
child 6053 8a1059aa01f0
--- a/src/ZF/Zorn.thy	Mon Feb 05 21:33:14 1996 +0100
+++ b/src/ZF/Zorn.thy	Tue Feb 06 12:27:17 1996 +0100
@@ -1,6 +1,6 @@
-(*  Title: 	ZF/Zorn.thy
+(*  Title:      ZF/Zorn.thy
     ID:         $Id$
-    Author: 	Lawrence C Paulson, Cambridge University Computer Laboratory
+    Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
     Copyright   1994  University of Cambridge
 
 Based upon the article
@@ -39,10 +39,10 @@
 inductive
   domains       "TFin(S,next)" <= "Pow(S)"
   intrs
-    nextI	"[| x : TFin(S,next);  next: increasing(S) 
+    nextI       "[| x : TFin(S,next);  next: increasing(S) 
                 |] ==> next`x : TFin(S,next)"
 
-    Pow_UnionI	"Y : Pow(TFin(S,next)) ==> Union(Y) : TFin(S,next)"
+    Pow_UnionI  "Y : Pow(TFin(S,next)) ==> Union(Y) : TFin(S,next)"
 
   monos         "[Pow_mono]"
   con_defs      "[increasing_def]"