src/ZF/AC.thy
changeset 13134 bf37a3049251
parent 6053 8a1059aa01f0
child 13149 773657d466cb
--- a/src/ZF/AC.thy	Fri May 10 18:00:48 2002 +0200
+++ b/src/ZF/AC.thy	Fri May 10 22:50:08 2002 +0200
@@ -8,13 +8,59 @@
 This definition comes from Halmos (1960), page 59.
 *)
 
-AC = func +
+theory AC = Main:
+
+axioms AC: "[| a: A;  !!x. x:A ==> (EX y. y:B(x)) |] ==> EX z. z : Pi(A,B)"
+
+(*The same as AC, but no premise a \<in> A*)
+lemma AC_Pi: "[| !!x. x \<in> A ==> (\<exists>y. y \<in> B(x)) |] ==> \<exists>z. z \<in> Pi(A,B)"
+apply (case_tac "A=0")
+apply (simp add: Pi_empty1, blast)
+(*The non-trivial case*)
+apply (blast intro: AC)
+done
+
+(*Using dtac, this has the advantage of DELETING the universal quantifier*)
+lemma AC_ball_Pi: "\<forall>x \<in> A. \<exists>y. y \<in> B(x) ==> \<exists>y. y \<in> Pi(A,B)"
+apply (rule AC_Pi)
+apply (erule bspec)
+apply assumption
+done
+
+lemma AC_Pi_Pow: "\<exists>f. f \<in> (\<Pi>X \<in> Pow(C)-{0}. X)"
+apply (rule_tac B1 = "%x. x" in AC_Pi [THEN exE])
+apply (erule_tac [2] exI)
+apply blast
+done
 
-constdefs
-  (*Needs to be visible for Zorn.thy*)
-  increasing :: i=>i
-    "increasing(A) == {f: Pow(A)->Pow(A). ALL x. x<=A --> x<=f`x}"
+lemma AC_func:
+     "[| !!x. x \<in> A ==> (\<exists>y. y \<in> x) |] ==> \<exists>f \<in> A->Union(A). \<forall>x \<in> A. f`x \<in> x"
+apply (rule_tac B1 = "%x. x" in AC_Pi [THEN exE])
+prefer 2 apply (blast dest: apply_type intro: Pi_type)
+apply (blast intro: elim:); 
+done
+
+lemma non_empty_family: "[| 0 \<notin> A;  x \<in> A |] ==> \<exists>y. y \<in> x"
+apply (subgoal_tac "x \<noteq> 0")
+apply blast+
+done
 
-rules
-  AC    "[| a: A;  !!x. x:A ==> (EX y. y:B(x)) |] ==> EX z. z : Pi(A,B)"
+lemma AC_func0: "0 \<notin> A ==> \<exists>f \<in> A->Union(A). \<forall>x \<in> A. f`x \<in> x"
+apply (rule AC_func)
+apply (simp_all add: non_empty_family) 
+done
+
+lemma AC_func_Pow: "\<exists>f \<in> (Pow(C)-{0}) -> C. \<forall>x \<in> Pow(C)-{0}. f`x \<in> x"
+apply (rule AC_func0 [THEN bexE])
+apply (rule_tac [2] bexI)
+prefer 2 apply (assumption)
+apply (erule_tac [2] fun_weaken_type)
+apply blast+
+done
+
+lemma AC_Pi0: "0 \<notin> A ==> \<exists>f. f \<in> (\<Pi>x \<in> A. x)"
+apply (rule AC_Pi)
+apply (simp_all add: non_empty_family) 
+done
+
 end