Skip to content

Commit c4aafb6

Browse files
committed
add comment
1 parent e59cb6c commit c4aafb6

File tree

1 file changed

+1
-1
lines changed

1 file changed

+1
-1
lines changed

BoogieLang/Ast_Cfg_Transformation.thy

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -462,7 +462,7 @@ lemma guard_fails_push_through_assumption:
462462
lemma guard_fails_push_through_assumption2:
463463
assumes block_correctness: "reached_state \<noteq> Failure \<and> (\<forall> ns1'. reached_state = Normal ns1' \<longrightarrow> (red_cmd_list A M \<Lambda> \<Gamma> \<Omega> (c#cs2) (Normal ns1) (Normal ns1')))"
464464
and assume_cmd: "c = Assume not_guard"
465-
and "UnOp Not guard \<sim> not_guard"
465+
and "UnOp Not guard \<sim> not_guard" \<comment>\<open>not required for lemma, but makes lemma in sync with analogous lemma above\<close>
466466
and guard_fails: "A,\<Lambda>,\<Gamma>,\<Omega> \<turnstile> \<langle>guard, ns1\<rangle> \<Down> LitV (LBool False)"
467467
shows "reached_state \<noteq> Failure \<and> (\<forall> ns1'. reached_state = Normal ns1' \<longrightarrow> (red_cmd_list A M \<Lambda> \<Gamma> \<Omega> (cs2) (Normal ns1) (Normal ns1')))"
468468
using assume_cmd assume_true_cmds block_correctness by blast

0 commit comments

Comments
 (0)