declare atomize/defn for Ball;
authorwenzelm
Sun, 29 Jan 2006 19:23:52 +0100
changeset 18845 6cbcfac5b72e
parent 18844 9dd789841018
child 18846 89b0fbbc4d8e
declare atomize/defn for Ball;
src/ZF/ZF.thy
--- a/src/ZF/ZF.thy	Sun Jan 29 19:23:51 2006 +0100
+++ b/src/ZF/ZF.thy	Sun Jan 29 19:23:52 2006 +0100
@@ -336,6 +336,13 @@
     "[| A=A';  !!x. x\<in>A' ==> P(x) <-> P'(x) |] ==> (\<forall>x\<in>A. P(x)) <-> (\<forall>x\<in>A'. P'(x))"
 by (simp add: Ball_def)
 
+lemma atomize_ball:
+    "(!!x. x \<in> A ==> P(x)) == Trueprop (\<forall>x\<in>A. P(x))"
+  by (simp only: Ball_def atomize_all atomize_imp)
+
+lemmas [symmetric, rulify] = atomize_ball
+  and [symmetric, defn] = atomize_ball
+
 
 subsection{*Bounded existential quantifier*}