src/HOL/Nominal/Examples/SOS.thy
changeset 34915 7894c7dab132
parent 29300 e841a9de5445
child 41893 dde7df1176b7
--- a/src/HOL/Nominal/Examples/SOS.thy	Sun Jan 10 18:41:07 2010 +0100
+++ b/src/HOL/Nominal/Examples/SOS.thy	Sun Jan 10 18:43:45 2010 +0100
@@ -220,10 +220,10 @@
   shows "(\<Delta>@\<Gamma>) \<turnstile> e[x::=e'] : T" 
 using a b 
 proof (nominal_induct \<Gamma>\<equiv>"\<Delta>@[(x,T')]@\<Gamma>" e T avoiding: e' \<Delta> rule: typing.strong_induct)
-  case (t_Var \<Gamma>' y T e' \<Delta>)
+  case (t_Var y T 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
+       and  a3: "\<Gamma> \<turnstile> e' : T'" .
   from a1 have a4: "valid (\<Delta>@\<Gamma>)" by (rule valid_insert)
   { assume eq: "x=y"
     from a1 a2 have "T=T'" using eq by (auto intro: context_unique)