Skip to content

Commit

Permalink
ainvs: remove hoare_seq_ext[wp] declaration
Browse files Browse the repository at this point in the history
This is no longer necessary now that the nondet monad setup already
makes it a wp rule.

Signed-off-by: Corey Lewis <[email protected]>
  • Loading branch information
corlewis committed Apr 22, 2024
1 parent fe1bbae commit 3ce8811
Showing 1 changed file with 0 additions and 2 deletions.
2 changes: 0 additions & 2 deletions proof/invariant-abstract/Syscall_AI.thy
Original file line number Diff line number Diff line change
Expand Up @@ -1146,8 +1146,6 @@ lemma hy_inv: "(\<And>s f. P (trans_state f s) = P s) \<Longrightarrow> \<lbrace
apply (wp | simp)+
done

declare hoare_seq_ext[wp]

lemma ct_active_simple [elim!]:
"ct_active s \<Longrightarrow> st_tcb_at simple (cur_thread s) s"
by (fastforce simp: ct_in_state_def elim!: pred_tcb_weakenE)
Expand Down

0 comments on commit 3ce8811

Please sign in to comment.