src/ZF/AC/recfunAC16.thy
author paulson
Wed, 09 Oct 1996 13:32:33 +0200
changeset 2073 fb0655539d05
parent 1478 2b8c2a7547ab
child 2469 b50b8c0eec01
permissions -rw-r--r--
New unified treatment of sequent calculi by Sara Kalvala combines the old LK and Modal with the new ILL (Int. Linear Logic)

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

A recursive definition used in the proof of WO2 ==> AC16
*)

recfunAC16 = Transrec2 + Cardinal +

consts

  recfunAC16              :: [i, i, i, i] => i

defs

  recfunAC16_def
    "recfunAC16(f,fa,i,a) == 
         transrec2(i, 0, 
              %g r. if(EX y:r. fa`g <= y, r, 
                       r Un {f`(LEAST i. fa`g <= f`i & 
                       (ALL b<a. (fa`b <= f`i --> (ALL t:r. ~ fa`b <= t))))}))"

end