src/ZF/AC/Transrec2.thy
author lcp
Tue, 25 Apr 1995 11:14:03 +0200
changeset 1072 0140ff702b23
parent 992 4ef4f7ff2aeb
child 1155 928a16e02f9f
permissions -rw-r--r--
updated version

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

Transfinite recursion introduced to handle definitions based on the three
cases of ordinals.
*)

Transrec2 = OrdQuant + Epsilon +

consts
  
  transrec2               :: "[i, i, [i,i]=>i] =>i"

defs

  transrec2_def  "transrec2(alpha, a, b) ==   			\
\		         transrec(alpha, %i r. if(i=0,   	\
\		                  a, if(EX j. i=succ(j),   	\
\		                  b(THE j. i=succ(j), r`(THE j. i=succ(j))),   \
\		                  UN j<i. r`j)))"

end