src/ZF/Univ.thy
changeset 1478 2b8c2a7547ab
parent 1401 0c439768f45c
child 2469 b50b8c0eec01
--- a/src/ZF/Univ.thy	Mon Feb 05 21:33:14 1996 +0100
+++ b/src/ZF/Univ.thy	Tue Feb 06 12:27:17 1996 +0100
@@ -1,6 +1,6 @@
-(*  Title: 	ZF/univ.thy
+(*  Title:      ZF/univ.thy
     ID:         $Id$
-    Author: 	Lawrence C Paulson, Cambridge University Computer Laboratory
+    Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
     Copyright   1992  University of Cambridge
 
 The cumulative hierarchy and a small universe for recursive types
@@ -19,13 +19,13 @@
     univ        :: i=>i
 
 translations
-    "Vset(x)"   == 	"Vfrom(0,x)"
+    "Vset(x)"   ==      "Vfrom(0,x)"
 
 defs
     Vfrom_def   "Vfrom(A,i) == transrec(i, %x f. A Un (UN y:x. Pow(f`y)))"
 
     Vrec_def
-   	"Vrec(a,H) == transrec(rank(a), %x g. lam z: Vset(succ(x)).      
+        "Vrec(a,H) == transrec(rank(a), %x g. lam z: Vset(succ(x)).      
                              H(z, lam w:Vset(x). g`rank(w)`w)) ` a"
 
     univ_def    "univ(A) == Vfrom(A,nat)"