src/ZF/AC/WO_AC.ML
author wenzelm
Sat, 24 Nov 2001 16:54:32 +0100
changeset 12282 f98beaaa7c4f
parent 11317 7f9e4c389318
permissions -rw-r--r--
generic_merge;

(*  Title:      ZF/AC/WO_AC.ML
    ID:         $Id$
    Author:     Krzysztof Grabczewski

Lemmas used in the proofs like WO? ==> AC?
*)

Goal "[| well_ord(Union(A),r); 0\\<notin>A; B \\<in> A |]  \
\               ==> (THE b. first(b,B,r)) \\<in> B";
by (fast_tac (claset() addSEs [well_ord_imp_ex1_first RS theI RS
                (first_def RS def_imp_iff RS iffD1 RS conjunct1)]) 1);
qed "first_in_B";

Goal "[| well_ord(Union(A), R); 0\\<notin>A |] ==> \\<exists>f. f:(\\<Pi>X \\<in> A. X)";
by (fast_tac (claset() addSEs [first_in_B] addSIs [lam_type]) 1);
qed "ex_choice_fun";

Goal "well_ord(A, R) ==> \\<exists>f. f:(\\<Pi>X \\<in> Pow(A)-{0}. X)";
by (fast_tac (claset() addSEs [well_ord_subset RS ex_choice_fun]) 1);
qed "ex_choice_fun_Pow";