src/ZF/Univ.thy
changeset 6093 87bf8c03b169
parent 6053 8a1059aa01f0
child 9395 1c9851cdfe9f
--- a/src/ZF/Univ.thy	Tue Jan 12 13:54:51 1999 +0100
+++ b/src/ZF/Univ.thy	Tue Jan 12 15:17:37 1999 +0100
@@ -8,13 +8,11 @@
 Standard notation for Vset(i) is V(i), but users might want V for a variable
 
 NOTE: univ(A) could be a translation; would simplify many proofs!
-  But Ind_Syntax.univ refers to the constant "univ"
+  But Ind_Syntax.univ refers to the constant "Univ.univ"
 *)
 
 Univ = Arith + Sum + Finite + mono +
 
-global
-
 consts
     Vfrom       :: [i,i]=>i
     Vset        :: i=>i
@@ -25,7 +23,6 @@
 translations
     "Vset(x)"   ==      "Vfrom(0,x)"
 
-local
 
 defs
     Vfrom_def   "Vfrom(A,i) == transrec(i, %x f. A Un (UN y:x. Pow(f`y)))"