diff -r 1255ba99ed1e -r 74fb4f03bb51 src/HOL/Nominal/Examples/CK_Machine.thy --- a/src/HOL/Nominal/Examples/CK_Machine.thy Mon Jun 07 13:20:05 2010 +0200 +++ b/src/HOL/Nominal/Examples/CK_Machine.thy Mon Jun 07 16:00:35 2010 +0200 @@ -492,7 +492,7 @@ shows "(\@\) \ e[x::=e'] : T" using a b proof (nominal_induct \'\"\@[(x,T')]@\" e T avoiding: x e' \ rule: typing.strong_induct) - case (t_VAR \' y T x e' \) + case (t_VAR y T x e' \) then have a1: "valid (\@[(x,T')]@\)" and a2: "(y,T) \ set (\@[(x,T')]@\)" and a3: "\ \ e' : T'" by simp_all