src/ZF/AC/DC.thy
changeset 1478 2b8c2a7547ab
parent 1401 0c439768f45c
child 2469 b50b8c0eec01
equal deleted inserted replaced
1477:4c51ab632cda 1478:2b8c2a7547ab
     1 (*  Title: 	ZF/AC/DC.thy
     1 (*  Title:      ZF/AC/DC.thy
     2     ID:         $Id$
     2     ID:         $Id$
     3     Author: 	Krzysztof Grabczewski
     3     Author:     Krzysztof Grabczewski
     4 
     4 
     5 Theory file for the proofs concernind the Axiom of Dependent Choice
     5 Theory file for the proofs concernind the Axiom of Dependent Choice
     6 *)
     6 *)
     7 
     7 
     8 DC  =  AC_Equiv + Hartog + first + Cardinal_aux + "DC_lemmas" + 
     8 DC  =  AC_Equiv + Hartog + first + Cardinal_aux + "DC_lemmas" + 
    14   ff  :: [i, i, i, i] => i
    14   ff  :: [i, i, i, i] => i
    15 
    15 
    16 rules
    16 rules
    17 
    17 
    18   DC_def  "DC(a) == ALL X R. R<=Pow(X)*X &
    18   DC_def  "DC(a) == ALL X R. R<=Pow(X)*X &
    19 	   (ALL Y:Pow(X). Y lesspoll a --> (EX x:X. <Y,x> : R)) 
    19            (ALL Y:Pow(X). Y lesspoll a --> (EX x:X. <Y,x> : R)) 
    20 	   --> (EX f:a->X. ALL b<a. <f``b,f`b> : R)"
    20            --> (EX f:a->X. ALL b<a. <f``b,f`b> : R)"
    21 
    21 
    22   DC0_def "DC0 == ALL A B R. R <= A*B & R~=0 & range(R) <= domain(R) 
    22   DC0_def "DC0 == ALL A B R. R <= A*B & R~=0 & range(R) <= domain(R) 
    23 	   --> (EX f:nat->domain(R). ALL n:nat. <f`n,f`succ(n)>:R)"
    23            --> (EX f:nat->domain(R). ALL n:nat. <f`n,f`succ(n)>:R)"
    24 
    24 
    25   ff_def  "ff(b, X, Q, R) == transrec(b, %c r. 
    25   ff_def  "ff(b, X, Q, R) == transrec(b, %c r. 
    26 	                     THE x. first(x, {x:X. <r``c, x> : R}, Q))"
    26                              THE x. first(x, {x:X. <r``c, x> : R}, Q))"
    27   
    27   
    28 end
    28 end