Skip to content

Commit 91cded0

Browse files
committed
add helper lemma for proof generation of CFG optimizations
This helper lemma is used in cases when the loop head set representation is different in a proof goal and in a lemma. Previously, the simplifier was used on the proof goal, but the result does not always match the representation of the lemma that is then applied. Now, the helper lemma is applied instead.
1 parent b005c01 commit 91cded0

File tree

1 file changed

+6
-0
lines changed

1 file changed

+6
-0
lines changed

BoogieLang/CFGOptimizationsLoop.thy

Lines changed: 6 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -308,6 +308,12 @@ next
308308
by simp
309309
qed
310310

311+
lemma hybrid_block_lemma_loop_eq_loop_heads:
312+
assumes "hybrid_block_lemma_loop A M \<Lambda> \<Gamma> \<Omega> G G' succ tgt_block tgt_cmds_0 lsLoopHeads1 posts"
313+
and "lsLoopHeads1 = lsLoopHeads2"
314+
shows "hybrid_block_lemma_loop A M \<Lambda> \<Gamma> \<Omega> G G' succ tgt_block tgt_cmds_0 lsLoopHeads2 posts"
315+
using assms
316+
by simp
311317

312318
subsection \<open>Main Lemmas for Loops\<close>
313319

0 commit comments

Comments
 (0)