diff -r af72dfc4b9f9 -r ca1ac9e81bc8 src/HOL/Nominal/Examples/Lam_substs.thy --- a/src/HOL/Nominal/Examples/Lam_substs.thy Wed Nov 30 15:24:32 2005 +0100 +++ b/src/HOL/Nominal/Examples/Lam_substs.thy Wed Nov 30 15:27:30 2005 +0100 @@ -1348,6 +1348,14 @@ apply(simp add: fresh_prod a b fresh_atm) done +lemma subst_Lam'': + assumes a: "a\b" + and b: "a\t" + shows "subst_lam b t (Lam [a].t1) = Lam [a].(subst_lam b t t1)" +apply(rule subst_Lam) +apply(simp add: fresh_prod a b) +done + consts subst_syn :: "lam \ name \ lam \ lam" ("_[_::=_]" [100,100,100] 900) translations @@ -1357,6 +1365,7 @@ declare subst_App[simp] declare subst_Lam[simp] declare subst_Lam'[simp] +declare subst_Lam''[simp] lemma subst_eqvt[simp]: fixes pi:: "name prm"