src/ZF/AC/DC.thy
author lcp
Tue, 25 Jul 1995 17:31:53 +0200
changeset 1196 d43c1f7a53fe
child 1203 a39bec971684
permissions -rw-r--r--
Numerous small improvements by KG and LCP

(*  Title: 	ZF/AC/DC.thy
    ID:         $Id$
    Author: 	Krzysztof Gr`abczewski

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

DC  =  AC_Equiv + Hartog + first + 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