merged
authornipkow
Sun, 02 Mar 2014 18:41:41 +0100
changeset 55835 eb8e231a335f
parent 55833 6fe16c8a6474 (current diff)
parent 55834 459b5561ba4e (diff)
child 55836 8093590e49e4
child 55837 154855d9a564
merged
--- a/src/HOL/IMP/Small_Step.thy	Sun Mar 02 18:20:08 2014 +0100
+++ b/src/HOL/IMP/Small_Step.thy	Sun Mar 02 18:41:41 2014 +0100
@@ -157,15 +157,12 @@
 apply auto
 done
 
-lemma small_big_continue:
-  "cs \<rightarrow>* cs' \<Longrightarrow> cs' \<Rightarrow> t \<Longrightarrow> cs \<Rightarrow> t"
-apply (induction rule: star.induct)
+lemma small_to_big:
+  "cs \<rightarrow>* (SKIP,t) \<Longrightarrow> cs \<Rightarrow> t"
+apply (induction cs "(SKIP,t)" arbitrary: t rule: star.induct)
 apply (auto intro: small1_big_continue)
 done
 
-lemma small_to_big: "cs \<rightarrow>* (SKIP,t) \<Longrightarrow> cs \<Rightarrow> t"
-by (metis small_big_continue Skip)
-
 text {*
   Finally, the equivalence theorem:
 *}