diff -r 6536fb8c9fc6 -r 8b84ee2cc79c src/ZF/Resid/Substitution.thy --- a/src/ZF/Resid/Substitution.thy Mon May 21 14:46:30 2001 +0200 +++ b/src/ZF/Resid/Substitution.thy Mon May 21 14:51:46 2001 +0200 @@ -29,23 +29,23 @@ in the recursive calls ***) primrec - "lift_aux(Var(i)) = (lam k:nat. if ik \\ nat. if ik \\ nat. Fun(lift_aux(t) ` succ(k)))" - "lift_aux(App(b,f,a)) = (lam k:nat. App(b, lift_aux(f)`k, lift_aux(a)`k))" + "lift_aux(App(b,f,a)) = (\\k \\ nat. App(b, lift_aux(f)`k, lift_aux(a)`k))" primrec "subst_aux(Var(i)) = - (lam r:redexes. lam k:nat. if kr \\ redexes. \\k \\ nat. if kr \\ redexes. \\k \\ nat. Fun(subst_aux(t) ` lift(r) ` succ(k)))" "subst_aux(App(b,f,a)) = - (lam r:redexes. lam k:nat. App(b, subst_aux(f)`r`k, subst_aux(a)`r`k))" + (\\r \\ redexes. \\k \\ nat. App(b, subst_aux(f)`r`k, subst_aux(a)`r`k))" end