equal
deleted
inserted
replaced
144 \<Longrightarrow> P \<turnstile> (i - size P',s,stk) \<rightarrow>* (j,s',stk') |
144 \<Longrightarrow> P \<turnstile> (i - size P',s,stk) \<rightarrow>* (j,s',stk') |
145 \<Longrightarrow> i' = size P' + j |
145 \<Longrightarrow> i' = size P' + j |
146 \<Longrightarrow> P' @ P \<turnstile> (i,s,stk) \<rightarrow>* (i',s',stk')" |
146 \<Longrightarrow> P' @ P \<turnstile> (i,s,stk) \<rightarrow>* (i',s',stk')" |
147 by (drule exec_appendL[where P'=P']) simp |
147 by (drule exec_appendL[where P'=P']) simp |
148 |
148 |
149 text{* Split the execution of a compound program up into the excution of its |
149 text{* Split the execution of a compound program up into the execution of its |
150 parts: *} |
150 parts: *} |
151 |
151 |
152 lemma exec_append_trans[intro]: |
152 lemma exec_append_trans[intro]: |
153 fixes i' i'' j'' :: int |
153 fixes i' i'' j'' :: int |
154 shows |
154 shows |