src/HOL/Nominal/Examples/Type_Preservation.thy
changeset 37358 74fb4f03bb51
parent 29097 68245155eb58
child 37362 017146b7d139
--- a/src/HOL/Nominal/Examples/Type_Preservation.thy	Mon Jun 07 13:20:05 2010 +0200
+++ b/src/HOL/Nominal/Examples/Type_Preservation.thy	Mon Jun 07 16:00:35 2010 +0200
@@ -142,7 +142,7 @@
   shows "(\<Delta>@\<Gamma>) \<turnstile> e[x::=e'] : T" 
 using a b 
 proof (nominal_induct \<Gamma>'\<equiv>"\<Delta>@[(x,T')]@\<Gamma>" e T avoiding: x e' \<Delta> rule: typing.strong_induct)
-  case (t_Var \<Gamma>' y T x e' \<Delta>)
+  case (t_Var y T x e' \<Delta>)
   then have a1: "valid (\<Delta>@[(x,T')]@\<Gamma>)" 
        and  a2: "(y,T) \<in> set (\<Delta>@[(x,T')]@\<Gamma>)" 
        and  a3: "\<Gamma> \<turnstile> e' : T'" by simp_all