src/ZF/AC/AC17_AC1.ML
changeset 3731 71366483323b
parent 2496 40efb87985b5
child 4091 771b1f6422a8
equal deleted inserted replaced
3730:6933d20f335f 3731:71366483323b
    17 \       ==> EX r. well_ord(x,r)";
    17 \       ==> EX r. well_ord(x,r)";
    18 by (rtac exI 1);
    18 by (rtac exI 1);
    19 by (eresolve_tac [[bij_Least_HH_x RS bij_converse_bij RS bij_is_inj,
    19 by (eresolve_tac [[bij_Least_HH_x RS bij_converse_bij RS bij_is_inj,
    20                 Ord_Least RS well_ord_Memrel] MRS well_ord_rvimage] 1);
    20                 Ord_Least RS well_ord_Memrel] MRS well_ord_rvimage] 1);
    21 by (assume_tac 1);
    21 by (assume_tac 1);
    22 val UN_eq_imp_well_ord = result();
    22 qed "UN_eq_imp_well_ord";
    23 
    23 
    24 (* *********************************************************************** *)
    24 (* *********************************************************************** *)
    25 (* theorems closer to the proof                                            *)
    25 (* theorems closer to the proof                                            *)
    26 (* *********************************************************************** *)
    26 (* *********************************************************************** *)
    27 
    27 
    33 by (res_inst_tac [("x","Union(A)")] exI 1);
    33 by (res_inst_tac [("x","Union(A)")] exI 1);
    34 by (rtac ballI 1);
    34 by (rtac ballI 1);
    35 by (etac swap 1);
    35 by (etac swap 1);
    36 by (rtac impI 1);
    36 by (rtac impI 1);
    37 by (fast_tac (!claset addSIs [restrict_type]) 1);
    37 by (fast_tac (!claset addSIs [restrict_type]) 1);
    38 val not_AC1_imp_ex = result();
    38 qed "not_AC1_imp_ex";
    39 
    39 
    40 goal thy "!!x. [| ALL f:Pow(x) - {0} -> x. EX u: Pow(x) - {0}. f`u~:u;  \
    40 goal thy "!!x. [| ALL f:Pow(x) - {0} -> x. EX u: Pow(x) - {0}. f`u~:u;  \
    41 \       EX f: Pow(x)-{0}->x. \
    41 \       EX f: Pow(x)-{0}->x. \
    42 \       x - (UN a:(LEAST i. HH(lam X:Pow(x)-{0}. {f`X},x,i)={x}).  \
    42 \       x - (UN a:(LEAST i. HH(lam X:Pow(x)-{0}. {f`X},x,i)={x}).  \
    43 \       HH(lam X:Pow(x)-{0}. {f`X},x,a)) = 0 |] \
    43 \       HH(lam X:Pow(x)-{0}. {f`X},x,a)) = 0 |] \