diff -r 08c3ef07cef7 -r 5ebd327ffb96 Nominal/Ex/LetInv.thy --- 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 \ trm \ trm \ trm" where "subst s t (Var x) = (if (s = x) then t else (Var x))"