more IMP fragments
authorkleing
Thu, 03 Nov 2011 18:10:47 +1100
changeset 45324 4ef9220b886b
parent 45323 df7554ebe024
child 45325 26b6179b5a45
more IMP fragments
src/HOL/IMP/Big_Step.thy
--- a/src/HOL/IMP/Big_Step.thy	Thu Nov 03 18:10:13 2011 +1100
+++ b/src/HOL/IMP/Big_Step.thy	Thu Nov 03 18:10:47 2011 +1100
@@ -23,12 +23,14 @@
              (WHILE b DO c, s\<^isub>1) \<Rightarrow> s\<^isub>3"
 text_raw{*}\end{isaverbatimwrite}*}
 
+text_raw{*\begin{isaverbatimwrite}\newcommand{\BigStepEx}{% *}
 schematic_lemma ex: "(''x'' ::= N 5; ''y'' ::= V ''x'', s) \<Rightarrow> ?t"
 apply(rule Semi)
 apply(rule Assign)
 apply simp
 apply(rule Assign)
 done
+text_raw{*}\end{isaverbatimwrite}*}
 
 thm ex[simplified]
 
@@ -228,7 +230,7 @@
   This is the proof as you might present it in a lecture. The remaining
   cases are simple enough to be proved automatically:
 *}
-text_raw{*\begin{isaverbatimwrite}\newcommand{\BigStepDet2}{% *}
+text_raw{*\begin{isaverbatimwrite}\newcommand{\BigStepDetLong}{% *}
 theorem
   "(c,s) \<Rightarrow> t  \<Longrightarrow>  (c,s) \<Rightarrow> t'  \<Longrightarrow>  t' = t"
 proof (induction arbitrary: t' rule: big_step.induct)