Skip to content
Snippets Groups Projects
Commit 7ae0b644 authored by Robbert Krebbers's avatar Robbert Krebbers
Browse files

Merge branch 'master' into gen_proofmode

parents efd17201 497bd8a8
No related branches found
No related tags found
No related merge requests found
...@@ -11,5 +11,5 @@ install: [make "install"] ...@@ -11,5 +11,5 @@ install: [make "install"]
remove: ["rm" "-rf" "%{lib}%/coq/user-contrib/iris"] remove: ["rm" "-rf" "%{lib}%/coq/user-contrib/iris"]
depends: [ depends: [
"coq" { (>= "8.7.1" & < "8.9~") | (= "dev") } "coq" { (>= "8.7.1" & < "8.9~") | (= "dev") }
"coq-stdpp" { (= "dev.2018-05-14.0.8fdeb77f") | (= "dev") } "coq-stdpp" { (= "dev.2018-05-23.0.a8f65af5") | (= "dev") }
] ]
...@@ -52,6 +52,13 @@ Section updates. ...@@ -52,6 +52,13 @@ Section updates.
apply (cancelableN x); first done. by rewrite -cmra_op_opM_assoc. apply (cancelableN x); first done. by rewrite -cmra_op_opM_assoc.
Qed. Qed.
Lemma replace_local_update x y `{!IdFree x} :
y (x, x) ~l~> (y, y).
Proof.
intros ? n mz ? Heq; simpl in *; split; first by apply cmra_valid_validN.
destruct mz as [z|]; [|done]. by destruct (id_freeN_r n n x z).
Qed.
Lemma local_update_discrete `{!CmraDiscrete A} (x y x' y' : A) : Lemma local_update_discrete `{!CmraDiscrete A} (x y x' y' : A) :
(x,y) ~l~> (x',y') mz, x x y ? mz x' x' y' ? mz. (x,y) ~l~> (x',y') mz, x x y ? mz x' x' y' ? mz.
Proof. Proof.
......
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