diff -r 56544d061e1d -r e0baea4d485a src/ZF/ZF.thy --- a/src/ZF/ZF.thy Fri Oct 10 18:17:17 1997 +0200 +++ b/src/ZF/ZF.thy Fri Oct 10 18:23:31 1997 +0200 @@ -129,7 +129,7 @@ "" == ">" "" == "Pair(x, y)" "%.b" == "split(%x .b)" - "%.b" == "split(%x y.b)" + "%.b" == "split(%x y. b)" syntax (symbols) @@ -190,7 +190,7 @@ The resulting set (for functional P) is the same as with PrimReplace, but the rules are simpler. *) - Replace_def "Replace(A,P) == PrimReplace(A, %x y. (EX!z.P(x,z)) & P(x,y))" + Replace_def "Replace(A,P) == PrimReplace(A, %x y. (EX!z. P(x,z)) & P(x,y))" (* Functional form of replacement -- analgous to ML's map functional *) @@ -246,7 +246,7 @@ Pi_def "Pi(A,B) == {f: Pow(Sigma(A,B)). A<=domain(f) & function(f)}" (* Restrict the function f to the domain A *) - restrict_def "restrict(f,A) == lam x:A.f`x" + restrict_def "restrict(f,A) == lam x:A. f`x" end