src/ZF/AC/Transrec2.thy
author clasohm
Tue, 06 Feb 1996 12:27:17 +0100
changeset 1478 2b8c2a7547ab
parent 1401 0c439768f45c
permissions -rw-r--r--
expanded tabs

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

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