src/ZF/AC/Transrec2.thy
author clasohm
Sat, 09 Dec 1995 13:36:11 +0100
changeset 1401 0c439768f45c
parent 1203 a39bec971684
child 1478 2b8c2a7547ab
permissions -rw-r--r--
removed quotes from consts and syntax sections

(*  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