changeset 3923 | c257b82a1200 |
parent 2469 | b50b8c0eec01 |
child 3940 | 1d5bee4d047f |
--- a/src/ZF/Univ.thy Fri Oct 17 17:39:04 1997 +0200 +++ b/src/ZF/Univ.thy Fri Oct 17 17:40:02 1997 +0200 @@ -12,6 +12,9 @@ *) Univ = Arith + Sum + Finite + mono + + +global + consts Vfrom :: [i,i]=>i Vset :: i=>i @@ -21,6 +24,8 @@ translations "Vset(x)" == "Vfrom(0,x)" +path Univ + defs Vfrom_def "Vfrom(A,i) == transrec(i, %x f. A Un (UN y:x. Pow(f`y)))"