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

Add lemma `map_seq_ne`.

parent b3896878
No related branches found
No related tags found
No related merge requests found
From stdpp Require Export list gmap.
From iris.algebra Require Export cmra.
From iris.algebra Require Export list cmra.
From iris.algebra Require Import updates local_updates proofmode_classes big_op.
From iris.prelude Require Import options.
......@@ -97,6 +97,13 @@ Proof. intros (y'&?&->)%dist_Some_inv_r'. by rewrite insert_id. Qed.
(** Internalized properties *)
End ofe.
Global Instance map_seq_ne {A : ofe} start :
NonExpansive (map_seq (M:=gmap nat A) start).
Proof.
intros n l1 l2 Hl. revert start.
induction Hl; intros; simpl; repeat (done || f_equiv).
Qed.
Global Arguments gmapO _ {_ _} _.
(** Non-expansiveness of higher-order map functions and big-ops *)
......
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