Skip to content

Commit

Permalink
aarch64 crefine: update to match other arches
Browse files Browse the repository at this point in the history
Signed-off-by: Corey Lewis <[email protected]>
  • Loading branch information
corlewis committed Mar 27, 2024
1 parent e98ecec commit 9d6443a
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion proof/crefine/AARCH64/VSpace_C.thy
Original file line number Diff line number Diff line change
Expand Up @@ -335,7 +335,7 @@ lemma corres_symb_exec_unknown_r:
assumes "\<And>rv. corres_underlying sr nf nf' r P P' a (c rv)"
shows "corres_underlying sr nf nf' r P P' a (unknown >>= c)"
apply (simp add: unknown_def)
apply (rule corres_symb_exec_r[OF assms]; wp select_inv no_fail_select)
apply (rule corres_symb_exec_r[OF assms]; wp select_inv)
done

lemma isPageTablePTE_def2:
Expand Down

0 comments on commit 9d6443a

Please sign in to comment.