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

Bump Iris.

parent bb4669b4
No related branches found
No related tags found
No related merge requests found
Pipeline #26548 passed
...@@ -9,6 +9,6 @@ build: [make "-j%{jobs}%"] ...@@ -9,6 +9,6 @@ build: [make "-j%{jobs}%"]
install: [make "install"] install: [make "install"]
remove: ["rm" "-rf" "%{lib}%/coq/user-contrib/reloc"] remove: ["rm" "-rf" "%{lib}%/coq/user-contrib/reloc"]
depends: [ depends: [
"coq-iris" { (= "dev.2020-04-04.3.9b2ad256") | (= "dev") } "coq-iris" { (= "dev.2020-04-07.7.64bed0ca") | (= "dev") }
"coq-autosubst" { = "dev.coq86" } "coq-autosubst" { = "dev.coq86" }
] ]
...@@ -127,7 +127,7 @@ Section mapsto. ...@@ -127,7 +127,7 @@ Section mapsto.
Global Instance mapsto_fractional l v : Fractional (λ q, l {q} v)%I. Global Instance mapsto_fractional l v : Fractional (λ q, l {q} v)%I.
Proof. Proof.
intros p q. rewrite heapS_mapsto_eq -own_op -auth_frag_op. intros p q. rewrite heapS_mapsto_eq -own_op -auth_frag_op.
by rewrite -pair_op op_singleton -pair_op agree_idemp right_id. by rewrite -pair_op singleton_op -pair_op agree_idemp right_id.
Qed. Qed.
Global Instance mapsto_as_fractional l q v : Global Instance mapsto_as_fractional l q v :
AsFractional (l {q} v) (λ q, l {q} v)%I q. AsFractional (l {q} v) (λ q, l {q} v)%I q.
...@@ -138,7 +138,7 @@ Section mapsto. ...@@ -138,7 +138,7 @@ Section mapsto.
apply bi.wand_intro_r. apply bi.wand_intro_r.
rewrite heapS_mapsto_eq -own_op -auth_frag_op own_valid uPred.discrete_valid. rewrite heapS_mapsto_eq -own_op -auth_frag_op own_valid uPred.discrete_valid.
f_equiv=> /=. f_equiv=> /=.
rewrite -pair_op op_singleton right_id -pair_op. rewrite -pair_op singleton_op right_id -pair_op.
move=> [_ Hv]. move:Hv => /=. move=> [_ Hv]. move:Hv => /=.
rewrite singleton_valid. rewrite singleton_valid.
by intros [_ ?%agree_op_invL']. by intros [_ ?%agree_op_invL'].
......
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