# HG changeset patch # User berghofe # Date 1275925982 -7200 # Node ID 017146b7d139952ab1c51a3fecb8a4ccc9a1add2 # Parent 250f487b3034698152f515393a01c8b971d763d5 Tuned. diff -r 250f487b3034 -r 017146b7d139 src/HOL/Nominal/Examples/CK_Machine.thy --- a/src/HOL/Nominal/Examples/CK_Machine.thy Mon Jun 07 17:52:30 2010 +0200 +++ b/src/HOL/Nominal/Examples/CK_Machine.thy Mon Jun 07 17:53:02 2010 +0200 @@ -491,11 +491,11 @@ and b: "\ \ e' : T'" shows "(\@\) \ e[x::=e'] : T" using a b -proof (nominal_induct \'\"\@[(x,T')]@\" e T avoiding: x e' \ rule: typing.strong_induct) +proof (nominal_induct "\@[(x,T')]@\" e T avoiding: x e' \ rule: typing.strong_induct) 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 + and a3: "\ \ e' : T'" . from a1 have a4: "valid (\@\)" by (rule valid_insert) { assume eq: "x=y" from a1 a2 have "T=T'" using eq by (auto intro: context_unique) diff -r 250f487b3034 -r 017146b7d139 src/HOL/Nominal/Examples/Type_Preservation.thy --- a/src/HOL/Nominal/Examples/Type_Preservation.thy Mon Jun 07 17:52:30 2010 +0200 +++ b/src/HOL/Nominal/Examples/Type_Preservation.thy Mon Jun 07 17:53:02 2010 +0200 @@ -141,11 +141,11 @@ and b: "\ \ e' : T'" shows "(\@\) \ e[x::=e'] : T" using a b -proof (nominal_induct \'\"\@[(x,T')]@\" e T avoiding: x e' \ rule: typing.strong_induct) +proof (nominal_induct "\@[(x,T')]@\" e T avoiding: x e' \ rule: typing.strong_induct) 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 + and a3: "\ \ e' : T'" . from a1 have a4: "valid (\@\)" by (rule valid_insert) { assume eq: "x=y" from a1 a2 have "T=T'" using eq by (auto intro: context_unique)