Skip to content
Snippets Groups Projects
Commit 9af5ee4f authored by Ralf Jung's avatar Ralf Jung
Browse files

cleanup

parent 2e1f67ac
No related branches found
No related tags found
No related merge requests found
Pipeline #
coq-iris https://gitlab.mpi-sws.org/FP/iris-coq e2b843075894275afd52c19c83e4f5f812afdbab coq-iris https://gitlab.mpi-sws.org/FP/iris-coq adfa07525e071b2a47aed37dac276aa38c10099d
...@@ -98,36 +98,6 @@ Section type. ...@@ -98,36 +98,6 @@ Section type.
rewrite shr_locsE_shift na_own_union //. apply shr_locsE_disj. rewrite shr_locsE_shift na_own_union //. apply shr_locsE_disj.
Qed. Qed.
Lemma na_own_acc F2 F1 tid :
F2 F1
na_own tid F1 -∗ na_own tid F2
(na_own tid F2 -∗ na_own tid F1).
Proof.
intros HF. assert (F1 = F2 (F1 F2)) as -> by exact: union_difference_L.
rewrite na_own_union; last by set_solver+.
iIntros "[$ $]". auto.
Qed.
(* Lemma shr_locsE_get_tok l n F tid :
shr_locsE l n ⊆ F →
na_own tid F -∗ na_own tid (shr_locsE l n) ∗
(na_own tid (shr_locsE l n) -∗ na_own tid F).
Proof.
intros HF.
assert (F = shr_locsE l n ∪ (F ∖ shr_locsE l n)) as -> by exact: union_difference_L.
rewrite na_own_union; last by set_solver+.
iIntros "[$ $]". by iIntros "?".
Qed.
Lemma shr_locsE_get_tokS l n F tid :
shr_locsE l (n + 1) ⊆ F →
na_own tid F -∗ na_own tid (shr_locsE l n) ∗
(na_own tid (shr_locsE l n) -∗ na_own tid F).
Proof.
intros HF. apply shr_locsE_get_tok. rewrite <-HF.
apply shr_locsE_subseteq. omega.
Qed.
*)
(** Copy types *) (** Copy types *)
Class Copy (t : type) := { Class Copy (t : type) := {
copy_persistent tid vl : PersistentP (t.(ty_own) tid vl); copy_persistent tid vl : PersistentP (t.(ty_own) tid vl);
......
0% Loading or .
You are about to add 0 people to the discussion. Proceed with caution.
Finish editing this message first!
Please register or to comment