diff -r 60bc63b13857 -r b37764a46b16 src/ZF/AC/DC.thy --- a/src/ZF/AC/DC.thy Tue Jul 16 18:46:13 2002 +0200 +++ b/src/ZF/AC/DC.thy Tue Jul 16 18:46:59 2002 +0200 @@ -94,7 +94,7 @@ transrec(b, %c r. THE x. first(x, {x \ X. \ R}, Q))" -locale DC0_imp = +locale (open) DC0_imp = fixes XX and RR and X and R assumes all_ex: "\Y \ Pow(X). Y \ nat --> (\x \ X. \ R)" @@ -292,7 +292,7 @@ done -locale imp_DC0 = +locale (open) imp_DC0 = fixes XX and RR and x and R and f and allRR defines XX_def: "XX == (\n \ nat. {f \ succ(n)->domain(R). \k \ n. \ R})"