Skip to content

Commit

Permalink
arm-hyp crefine: reduce diff to arm crefine
Browse files Browse the repository at this point in the history
Use the same proof text for both architectures to increase likelihood
that patches will apply to both.

Signed-off-by: Gerwin Klein <[email protected]>
  • Loading branch information
lsf37 committed Jul 11, 2024
1 parent 858dd86 commit a30419f
Showing 1 changed file with 3 additions and 3 deletions.
6 changes: 3 additions & 3 deletions proof/crefine/ARM_HYP/Refine_C.thy
Original file line number Diff line number Diff line change
Expand Up @@ -274,7 +274,7 @@ lemma handleSyscall_ccorres:
apply (subst ccorres_seq_skip'[symmetric])
apply (rule ccorres_split_nothrow_novcg)
apply (rule_tac R=\<top> and xf=xfdc in ccorres_when)
apply (case_tac rv; clarsimp simp: irq_type_never_invalid)
apply (auto simp: irq_type_never_invalid split: option.splits)[1]
apply (ctac (no_vcg) add: handleInterrupt_ccorres)
apply ceqv
apply (rule_tac r=dc and xf=xfdc in ccorres_returnOk_skip[unfolded returnOk_def,simplified])
Expand Down Expand Up @@ -303,7 +303,7 @@ lemma handleSyscall_ccorres:
apply (rule ccorres_split_nothrow_novcg)
apply (rule ccorres_Guard)?
apply (rule_tac R=\<top> and xf=xfdc in ccorres_when)
apply (case_tac rv; clarsimp simp: irq_type_never_invalid)
apply (auto simp: irq_type_never_invalid split: option.splits)[1]
apply (ctac (no_vcg) add: handleInterrupt_ccorres)
apply ceqv
apply (rule_tac ccorres_returnOk_skip[unfolded returnOk_def,simplified])
Expand Down Expand Up @@ -331,7 +331,7 @@ lemma handleSyscall_ccorres:
apply (rule ccorres_split_nothrow_novcg)
apply (rule ccorres_Guard)?
apply (rule_tac R=\<top> and xf=xfdc in ccorres_when)
apply (case_tac rv; clarsimp simp: irq_type_never_invalid)
apply (auto simp: irq_type_never_invalid split: option.splits)[1]
apply (ctac (no_vcg) add: handleInterrupt_ccorres)
apply ceqv
apply (rule_tac ccorres_returnOk_skip[unfolded returnOk_def,simplified])
Expand Down

0 comments on commit a30419f

Please sign in to comment.