src/ZF/pair.thy
changeset 14864 419b45cdb400
parent 13544 895994073bdf
child 16417 9bc16273c2d4
--- a/src/ZF/pair.thy	Tue Jun 01 18:52:38 2004 +0200
+++ b/src/ZF/pair.thy	Wed Jun 02 17:35:08 2004 +0200
@@ -149,6 +149,18 @@
 lemma splitD: "split(R,<a,b>) ==> R(a,b)"
 by (simp add: split_def)
 
+text {*
+  \bigskip Complex rules for Sigma.
+*}
+
+lemma split_paired_Bex_Sigma [simp]:
+     "(\<exists>z \<in> Sigma(A,B). P(z)) <-> (\<exists>x \<in> A. \<exists>y \<in> B(x). P(<x,y>))"
+by blast
+
+lemma split_paired_Ball_Sigma [simp]:
+     "(\<forall>z \<in> Sigma(A,B). P(z)) <-> (\<forall>x \<in> A. \<forall>y \<in> B(x). P(<x,y>))"
+by blast
+
 ML
 {*
 val singleton_eq_iff = thm "singleton_eq_iff";