src/ZF/Resid/Redex.thy
changeset 1155 928a16e02f9f
parent 1048 5ba0314f8214
child 1401 0c439768f45c
equal deleted inserted replaced
1154:bc295e3dc078 1155:928a16e02f9f
    19 consts
    19 consts
    20   redex_rec   	:: "[i, i=>i, [i,i]=>i, [i,i,i,i,i]=>i]=>i"
    20   redex_rec   	:: "[i, i=>i, [i,i]=>i, [i,i,i,i,i]=>i]=>i"
    21  
    21  
    22 defs
    22 defs
    23   redex_rec_def
    23   redex_rec_def
    24    "redex_rec(p,b,c,d) == \
    24    "redex_rec(p,b,c,d) == 
    25 \   Vrec(p, %p g.redexes_case(b, %x.c(x,g`x),   \
    25    Vrec(p, %p g.redexes_case(b, %x.c(x,g`x),   
    26 \                             %n x y.d(n, x, y, g`x, g`y), p))"
    26                              %n x y.d(n, x, y, g`x, g`y), p))"
    27 end
    27 end
    28 
    28