recovered some untested theories;
authorwenzelm
Mon, 07 Jun 2010 16:00:35 +0200
changeset 37358 74fb4f03bb51
parent 37355 1255ba99ed1e
child 37359 7b0ccc20cddc
recovered some untested theories;
src/HOL/Nominal/Examples/CK_Machine.thy
src/HOL/Nominal/Examples/Nominal_Examples.thy
src/HOL/Nominal/Examples/Type_Preservation.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 "(\<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
--- a/src/HOL/Nominal/Examples/Nominal_Examples.thy	Mon Jun 07 13:20:05 2010 +0200
+++ b/src/HOL/Nominal/Examples/Nominal_Examples.thy	Mon Jun 07 16:00:35 2010 +0200
@@ -4,23 +4,25 @@
 
 theory Nominal_Examples
 imports
+  CK_Machine
   CR
   CR_Takahashi
   Class3
   Compile
+  Contexts
+  Crary
   Fsub
   Height
   Lambda_mu
+  LocalWeakening
+  Pattern
   SN
-  Weakening
-  Crary
   SOS
-  LocalWeakening
+  Standardization
   Support
-  Contexts
-  Standardization
+  Type_Preservation
   W
-  Pattern
+  Weakening
 begin
 
 end
--- 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