src/ZF/AC/DC.thy
author wenzelm
Wed, 06 Aug 1997 14:42:44 +0200
changeset 3631 88a279998f90
parent 2469 b50b8c0eec01
child 3892 1d184682ac9f
permissions -rw-r--r--
renamed use_string to use_strings;

(*  Title:      ZF/AC/DC.thy
    ID:         $Id$
    Author:     Krzysztof Grabczewski

Theory file for the proofs concernind the Axiom of Dependent Choice
*)

DC  =  AC_Equiv + Hartog + Cardinal_aux + "DC_lemmas" + 

consts

  DC  :: i => o
  DC0 :: o
  ff  :: [i, i, i, i] => i

rules

  DC_def  "DC(a) == ALL X R. R<=Pow(X)*X &
           (ALL Y:Pow(X). Y lesspoll a --> (EX x:X. <Y,x> : R)) 
           --> (EX f:a->X. ALL b<a. <f``b,f`b> : R)"

  DC0_def "DC0 == ALL A B R. R <= A*B & R~=0 & range(R) <= domain(R) 
           --> (EX f:nat->domain(R). ALL n:nat. <f`n,f`succ(n)>:R)"

  ff_def  "ff(b, X, Q, R) == transrec(b, %c r. 
                             THE x. first(x, {x:X. <r``c, x> : R}, Q))"
  
end