Skip to content

Commit

Permalink
fix naming conflict causing errors in InfoFlowC
Browse files Browse the repository at this point in the history
Signed-off-by: Michael McInerney <[email protected]>
  • Loading branch information
michaelmcinerney committed May 8, 2024
1 parent 1c54809 commit b914ce2
Show file tree
Hide file tree
Showing 2 changed files with 5 additions and 5 deletions.
2 changes: 1 addition & 1 deletion proof/infoflow/refine/ADT_IF_Refine.thy
Original file line number Diff line number Diff line change
Expand Up @@ -509,7 +509,7 @@ lemma scheduler'_if_ex_abs[wp]:
apply wp
apply (clarsimp simp: ex_abs_def)
apply (rule exI, rule conjI, assumption)
apply (frule state_relation_schact)
apply (frule state_relation_sched_act_relation)
apply (auto simp: domain_list_rel_eq domain_time_rel_eq)
done

Expand Down
8 changes: 4 additions & 4 deletions proof/refine/ARM/StateRelation.thy
Original file line number Diff line number Diff line change
Expand Up @@ -654,14 +654,14 @@ lemma state_relation_pspace_relation[elim!]:
"(s,s') \<in> state_relation \<Longrightarrow> pspace_relation (kheap s) (ksPSpace s')"
by (simp add: state_relation_def)

lemma state_relation_schact[elim!]:
"(s,s') \<in> state_relation \<Longrightarrow> sched_act_relation (scheduler_action s) (ksSchedulerAction s')"
by (simp add: state_relation_def)

lemma state_relation_ekheap_relation[elim!]:
"(s,s') \<in> state_relation \<Longrightarrow> ekheap_relation (ekheap s) (ksPSpace s')"
by (simp add: state_relation_def)

lemma state_relation_sched_act_relation[elim!]:
"(s,s') \<in> state_relation \<Longrightarrow> sched_act_relation (scheduler_action s) (ksSchedulerAction s')"
by (clarsimp simp: state_relation_def)

lemma state_relation_ready_queues_relation[elim!]:
"(s, s') \<in> state_relation \<Longrightarrow> ready_queues_relation s s'"
by (simp add: state_relation_def)
Expand Down

0 comments on commit b914ce2

Please sign in to comment.