src/HOL/Nominal/Examples/SN.thy
changeset 23393 31781b2de73d
parent 23142 cb1dbe64a4d5
child 23760 aca2c7f80e2f
--- a/src/HOL/Nominal/Examples/SN.thy	Thu Jun 14 22:59:42 2007 +0200
+++ b/src/HOL/Nominal/Examples/SN.thy	Thu Jun 14 23:04:36 2007 +0200
@@ -374,7 +374,7 @@
   proof (induct a rule: acc.induct)
     case (accI x)
     note accI' = accI
-    have "acc r b" .
+    have "acc r b" by fact
     thus ?case
     proof (induct b rule: acc.induct)
       case (accI y)
@@ -501,7 +501,7 @@
   case (t3 a \<Gamma> \<sigma> t \<tau> \<theta>) --"lambda case"
   have ih: "\<And>\<theta>. \<theta> closes ((a,\<sigma>)#\<Gamma>) \<Longrightarrow> \<theta><t> \<in> RED \<tau>" by fact
   have \<theta>_cond: "\<theta> closes \<Gamma>" by fact
-  have fresh: "a\<sharp>\<Gamma>" "a\<sharp>\<theta>" by fact
+  have fresh: "a\<sharp>\<Gamma>" "a\<sharp>\<theta>" by fact+
   from ih have "\<forall>s\<in>RED \<sigma>. ((a,s)#\<theta>)<t> \<in> RED \<tau>" 
     using fresh \<theta>_cond fresh_context by simp
   then have "\<forall>s\<in>RED \<sigma>. \<theta><t>[a::=s] \<in> RED \<tau>"