Skip to content

Commit

Permalink
fixup crunch squash
Browse files Browse the repository at this point in the history
Signed-off-by: Michael McInerney <[email protected]>
  • Loading branch information
michaelmcinerney committed Aug 8, 2024
1 parent 099f263 commit 447f34a
Show file tree
Hide file tree
Showing 2 changed files with 7 additions and 2 deletions.
3 changes: 1 addition & 2 deletions proof/refine/RISCV64/IpcCancel_R.thy
Original file line number Diff line number Diff line change
Expand Up @@ -1051,8 +1051,7 @@ lemma scReplies_of_scTCB_update[simp]:
crunch schedContextDonate
for replies_of': "\<lambda>s. P (replies_of' s)" (* this interfers with list_refs_of_replies' *)
and scReplies_of[wp]: "\<lambda>s. P' (scReplies_of s)"
(simp: crunch_simps wp: crunch_wps
rule: schedContextDonate_def[simplified updateSchedContext_def])
(simp: crunch_simps wp: crunch_wps updateSchedContext_scReplies_of)

lemma updateReply_replyNext_update_None:
"\<lbrace> \<top> \<rbrace>
Expand Down
6 changes: 6 additions & 0 deletions proof/refine/RISCV64/KHeap_R.thy
Original file line number Diff line number Diff line change
Expand Up @@ -4900,6 +4900,12 @@ lemma setSchedContext_scReplies_of:
apply (erule back_subst[where P=P], rule ext)
by (clarsimp simp: opt_map_def)

lemma updateSchedContext_scReplies_of:
"(\<And>sc. scReply (f sc) = scReply sc) \<Longrightarrow> updateSchedContext scPtr f \<lbrace>\<lambda>s. P' (scReplies_of s)\<rbrace>"
apply (wpsimp simp: updateSchedContext_def wp: setSchedContext_scReplies_of)
apply (auto elim!: rsubst[where P=P'] simp: opt_map_def obj_at'_def)
done

lemma getObject_tcb_wp:
"\<lbrace>\<lambda>s. tcb_at' p s \<longrightarrow> (\<exists>t::tcb. ko_at' t p s \<and> Q t s)\<rbrace> getObject p \<lbrace>Q\<rbrace>"
by (clarsimp simp: getObject_def valid_def in_monad
Expand Down

0 comments on commit 447f34a

Please sign in to comment.