Bound variable preservation in Collect_cong
authorpaulson
Wed, 11 Sep 2002 16:53:59 +0200
changeset 13565 40e4755e57f7
parent 13564 1500a2e48d44
child 13566 52a419210d5c
Bound variable preservation in Collect_cong
src/ZF/ZF.ML
--- a/src/ZF/ZF.ML	Tue Sep 10 16:51:31 2002 +0200
+++ b/src/ZF/ZF.ML	Wed Sep 11 16:53:59 2002 +0200
@@ -321,7 +321,8 @@
 qed "CollectD2";
 
 val prems= Goalw [Collect_def]  
-    "[| A=B;  !!x. x:B ==> P(x) <-> Q(x) |] ==> Collect(A,P) = Collect(B,Q)";
+    "[| A=B;  !!x. x:B ==> P(x) <-> Q(x) |] \
+\    ==> Collect(A, %x. P(x)) = Collect(B, %x. Q(x))";
 by (simp_tac (simpset() addsimps prems) 1) ;
 qed "Collect_cong";