src/ZF/Constructible/Relative.thy
changeset 13339 0f89104dd377
parent 13323 2c287f50c9f3
child 13348 374d05460db4
--- a/src/ZF/Constructible/Relative.thy	Wed Jul 10 16:07:52 2002 +0200
+++ b/src/ZF/Constructible/Relative.thy	Wed Jul 10 16:54:07 2002 +0200
@@ -227,18 +227,20 @@
 
 text{*Congruence rule for separation: can assume the variable is in @{text M}*}
 lemma separation_cong [cong]:
-     "(!!x. M(x) ==> P(x) <-> P'(x)) ==> separation(M,P) <-> separation(M,P')"
+     "(!!x. M(x) ==> P(x) <-> P'(x)) 
+      ==> separation(M, %x. P(x)) <-> separation(M, %x. P'(x))"
 by (simp add: separation_def) 
 
 text{*Congruence rules for replacement*}
 lemma univalent_cong [cong]:
      "[| A=A'; !!x y. [| x\<in>A; M(x); M(y) |] ==> P(x,y) <-> P'(x,y) |] 
-      ==> univalent(M,A,P) <-> univalent(M,A',P')"
+      ==> univalent(M, A, %x y. P(x,y)) <-> univalent(M, A', %x y. P'(x,y))"
 by (simp add: univalent_def) 
 
 lemma strong_replacement_cong [cong]:
      "[| !!x y. [| M(x); M(y) |] ==> P(x,y) <-> P'(x,y) |] 
-      ==> strong_replacement(M,P) <-> strong_replacement(M,P')" 
+      ==> strong_replacement(M, %x y. P(x,y)) <-> 
+          strong_replacement(M, %x y. P'(x,y))" 
 by (simp add: strong_replacement_def) 
 
 text{*The extensionality axiom*}
@@ -268,7 +270,7 @@
 
 lemma "separation(\<lambda>x. x \<in> univ(0), P)"
 apply (simp add: separation_def, clarify) 
-apply (rule_tac x = "Collect(x,P)" in bexI) 
+apply (rule_tac x = "Collect(z,P)" in bexI) 
 apply (blast intro: Collect_in_univ Transset_0)+
 done