Skip to content
Snippets Groups Projects
Commit f49a7f18 authored by Jacques-Henri Jourdan's avatar Jacques-Henri Jourdan
Browse files

Merge branch 'master' of gitlab.mpi-sws.org:FP/iris-coq

parents 9ae19ed5 38d61951
No related branches found
No related tags found
No related merge requests found
...@@ -526,6 +526,17 @@ Section gset. ...@@ -526,6 +526,17 @@ Section gset.
by rewrite !big_sepS_insert // IH pure_False // False_impl left_id. by rewrite !big_sepS_insert // IH pure_False // False_impl left_id.
Qed. Qed.
Lemma big_sepS_filter_acc (P : A Prop) `{ y, Decision (P y)} Φ X Y :
( y, y Y P y y X)
([ set] y X, Φ y) -∗
([ set] y Y, P y Φ y)
(([ set] y Y, P y Φ y) -∗ [ set] y X, Φ y).
Proof.
intros ?. destruct (proj1 (subseteq_disjoint_union_L (filter P Y) X))
as (Z&->&?); first set_solver.
rewrite big_sepS_union // big_sepS_filter. by apply sep_mono_r, wand_intro_l.
Qed.
Lemma big_sepS_sepS Φ Ψ X : Lemma big_sepS_sepS Φ Ψ X :
([ set] y X, Φ y Ψ y) ⊣⊢ ([ set] y X, Φ y) ([ set] y X, Ψ y). ([ set] y X, Φ y Ψ y) ⊣⊢ ([ set] y X, Φ y) ([ set] y X, Ψ y).
Proof. apply: big_opS_opS. Qed. Proof. apply: big_opS_opS. Qed.
......
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