--- a/src/ZF/Univ.thy Mon Nov 28 19:48:30 1994 +0100
+++ b/src/ZF/Univ.thy Tue Nov 29 00:31:31 1994 +0100
@@ -21,7 +21,7 @@
translations
"Vset(x)" == "Vfrom(0,x)"
-rules
+defs
Vfrom_def "Vfrom(A,i) == transrec(i, %x f. A Un (UN y:x. Pow(f`y)))"
Vrec_def