author | nipkow |
Mon, 20 Jun 1994 12:03:16 +0200 | |
changeset 430 | 89e1986125fe |
parent 124 | 858ab9a9b047 |
child 753 | ec86863e87c8 |
permissions | -rw-r--r-- |
(* Title: ZF/epsilon.thy ID: $Id$ Author: Lawrence C Paulson, Cambridge University Computer Laboratory Copyright 1993 University of Cambridge Epsilon induction and recursion *) Epsilon = Nat + "mono" + consts eclose,rank :: "i=>i" transrec :: "[i, [i,i]=>i] =>i" rules eclose_def "eclose(A) == UN n:nat. nat_rec(n, A, %m r. Union(r))" transrec_def "transrec(a,H) == wfrec(Memrel(eclose({a})), a, H)" rank_def "rank(a) == transrec(a, %x f. UN y:x. succ(f`y))" end