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

Local update on product.

parent 8d4fa046
No related branches found
No related tags found
No related merge requests found
...@@ -590,7 +590,18 @@ Section prod. ...@@ -590,7 +590,18 @@ Section prod.
Lemma prod_updateP' P1 P2 x : Lemma prod_updateP' P1 P2 x :
x.1 ~~>: P1 x.2 ~~>: P2 x ~~>: λ y, P1 (y.1) P2 (y.2). x.1 ~~>: P1 x.2 ~~>: P2 x ~~>: λ y, P1 (y.1) P2 (y.2).
Proof. eauto using prod_updateP. Qed. Proof. eauto using prod_updateP. Qed.
Global Instance prod_local_update
(LA : A A) `{!LocalUpdate LvA LA} (LB : B B) `{!LocalUpdate LvB LB} :
LocalUpdate (λ x, LvA (x.1) LvB (x.2)) (prod_map LA LB).
Proof.
constructor.
- intros n x y [??]; constructor; simpl; by apply local_update_ne.
- intros n ?? [??] [??];
constructor; simpl in *; eapply local_updateN; eauto.
Qed.
End prod. End prod.
Arguments prodR : clear implicits. Arguments prodR : clear implicits.
Instance prod_map_cmra_monotone {A A' B B' : cmraT} (f : A A') (g : B B') : Instance prod_map_cmra_monotone {A A' B B' : cmraT} (f : A A') (g : B B') :
......
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