changeset 3235 | 5ebd327ffb96 |
parent 2956 | 7e1c309bf820 |
--- a/Nominal/Ex/LetInv.thy Mon May 19 11:19:48 2014 +0100 +++ b/Nominal/Ex/LetInv.thy Mon May 19 12:45:26 2014 +0100 @@ -223,7 +223,7 @@ apply (simp add: Abs_eq_iff alphas supp_atom fresh_star_def neq) done -nominal_primrec +nominal_function subst :: "name \<Rightarrow> trm \<Rightarrow> trm \<Rightarrow> trm" where "subst s t (Var x) = (if (s = x) then t else (Var x))"