Skip to content

Commit

Permalink
remove find_theorems squash
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 6133838 commit ad270c3
Show file tree
Hide file tree
Showing 5 changed files with 0 additions and 5 deletions.
1 change: 0 additions & 1 deletion proof/crefine/AARCH64/Finalise_C.thy
Original file line number Diff line number Diff line change
Expand Up @@ -316,7 +316,6 @@ lemma cancel_all_ccorres_helper:
Guard C_Guard \<lbrace>hrs_htd \<acute>t_hrs \<Turnstile>\<^sub>t \<acute>thread\<rbrace>
(\<acute>thread :== h_val (hrs_mem \<acute>t_hrs) (Ptr &(\<acute>thread\<rightarrow>[''tcbEPNext_C'']) :: tcb_C ptr ptr))
OD)"
find_theorems ccorres_underlying name: cross
unfolding whileAnno_def
proof (induct ts)
case Nil
Expand Down
1 change: 0 additions & 1 deletion proof/crefine/ARM/Finalise_C.thy
Original file line number Diff line number Diff line change
Expand Up @@ -314,7 +314,6 @@ lemma cancel_all_ccorres_helper:
Guard C_Guard \<lbrace>hrs_htd \<acute>t_hrs \<Turnstile>\<^sub>t \<acute>thread\<rbrace>
(\<acute>thread :== h_val (hrs_mem \<acute>t_hrs) (Ptr &(\<acute>thread\<rightarrow>[''tcbEPNext_C'']) :: tcb_C ptr ptr))
OD)"
find_theorems ccorres_underlying name: cross
unfolding whileAnno_def
proof (induct ts)
case Nil
Expand Down
1 change: 0 additions & 1 deletion proof/crefine/ARM_HYP/Finalise_C.thy
Original file line number Diff line number Diff line change
Expand Up @@ -314,7 +314,6 @@ lemma cancel_all_ccorres_helper:
Guard C_Guard \<lbrace>hrs_htd \<acute>t_hrs \<Turnstile>\<^sub>t \<acute>thread\<rbrace>
(\<acute>thread :== h_val (hrs_mem \<acute>t_hrs) (Ptr &(\<acute>thread\<rightarrow>[''tcbEPNext_C'']) :: tcb_C ptr ptr))
OD)"
find_theorems ccorres_underlying name: cross
unfolding whileAnno_def
proof (induct ts)
case Nil
Expand Down
1 change: 0 additions & 1 deletion proof/crefine/RISCV64/Finalise_C.thy
Original file line number Diff line number Diff line change
Expand Up @@ -333,7 +333,6 @@ lemma cancel_all_ccorres_helper:
Guard C_Guard \<lbrace>hrs_htd \<acute>t_hrs \<Turnstile>\<^sub>t \<acute>thread\<rbrace>
(\<acute>thread :== h_val (hrs_mem \<acute>t_hrs) (Ptr &(\<acute>thread\<rightarrow>[''tcbEPNext_C'']) :: tcb_C ptr ptr))
OD)"
find_theorems ccorres_underlying name: cross
unfolding whileAnno_def
proof (induct ts)
case Nil
Expand Down
1 change: 0 additions & 1 deletion proof/crefine/X64/Finalise_C.thy
Original file line number Diff line number Diff line change
Expand Up @@ -315,7 +315,6 @@ lemma cancel_all_ccorres_helper:
Guard C_Guard \<lbrace>hrs_htd \<acute>t_hrs \<Turnstile>\<^sub>t \<acute>thread\<rbrace>
(\<acute>thread :== h_val (hrs_mem \<acute>t_hrs) (Ptr &(\<acute>thread\<rightarrow>[''tcbEPNext_C'']) :: tcb_C ptr ptr))
OD)"
find_theorems ccorres_underlying name: cross
unfolding whileAnno_def
proof (induct ts)
case Nil
Expand Down

0 comments on commit ad270c3

Please sign in to comment.