# HG changeset patch # User paulson # Date 1022252128 -7200 # Node ID bc54319f687594d14c413fd2648336ab026bdf9f # Parent ba734cc2887d998b12b40be40b66e11670878369 new quantifier lemmas diff -r ba734cc2887d -r bc54319f6875 src/ZF/equalities.thy --- a/src/ZF/equalities.thy Fri May 24 15:24:29 2002 +0200 +++ b/src/ZF/equalities.thy Fri May 24 16:55:28 2002 +0200 @@ -26,6 +26,23 @@ lemma the_eq_0 [simp]: "(THE x. False) = 0" by (blast intro: the_0) +text {* \medskip Bounded quantifiers. + + The following are not added to the default simpset because + (a) they duplicate the body and (b) there are no similar rules for @{text Int}. *} + +lemma ball_Un: "(\x \ A\B. P(x)) <-> (\x \ A. P(x)) & (\x \ B. P(x))"; + by blast + +lemma bex_Un: "(\x \ A\B. P(x)) <-> (\x \ A. P(x)) | (\x \ B. P(x))"; + by blast + +lemma ball_UN: "(\z \ (UN x:A. B(x)). P(z)) <-> (\x\A. \z \ B(x). P(z))" + by blast + +lemma bex_UN: "(\z \ (UN x:A. B(x)). P(z)) <-> (\x\A. \z\B(x). P(z))" + by blast + (*** converse ***) lemma converse_iff [iff]: ": converse(r) <-> :r"