New rewrites for bounded quantifiers
authorpaulson
Fri, 17 Jan 1997 16:17:31 +0100
changeset 2519 761e3094e32f
parent 2518 bee082efaa46
child 2520 aecaa76e7eff
New rewrites for bounded quantifiers
src/HOL/equalities.ML
--- a/src/HOL/equalities.ML	Fri Jan 17 13:21:54 1997 +0100
+++ b/src/HOL/equalities.ML	Fri Jan 17 16:17:31 1997 +0100
@@ -458,13 +458,16 @@
 
 section"Bounded quantifiers";
 
-goal Set.thy "(!x:insert a A.P x) = (P a & (!x:A.P x))";
-by (Fast_tac 1);
-qed "Ball_insert";
+(** These are not added to the default simpset because (a) they duplicate the
+    body and (b) there are no similar rules for Int. **)
 
-goal Set.thy "(!x:A Un B.P x) = ((!x:A.P x) & (!x:B.P x))";
+goal Set.thy "(ALL x:A Un B.P x) = ((ALL x:A.P x) & (ALL x:B.P x))";
 by (Fast_tac 1);
-qed "Ball_Un";
+qed "ball_Un";
+
+goal Set.thy "(EX x:A Un B.P x) = ((EX x:A.P x) | (EX x:B.P x))";
+by (Fast_tac 1);
+qed "bex_Un";
 
 
 section "-";