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

Apply 1 suggestion(s) to 1 file(s)

parent eeefffca
No related branches found
No related tags found
No related merge requests found
......@@ -346,7 +346,7 @@ Section big_op_instances.
Lemma big_opL_own_1 {B} γ (f : nat B A) (l : list B) :
own γ ([^op list] kx l, f k x) [ list] kx l, own γ (f k x).
Proof. apply (big_opL_commute _). Qed.
Lemma big_opM_own_1 {B} `{Countable K} γ (g : K B A) (m : gmap K B) :
Lemma big_opM_own_1 `{Countable K} {B} γ (g : K B A) (m : gmap K B) :
own γ ([^op map] kx m, g k x) [ map] kx m, own γ (g k x).
Proof. apply (big_opM_commute _). Qed.
Lemma big_opS_own_1 `{Countable B} γ (g : B A) (X : gset 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