Skip to content
Snippets Groups Projects
Verified Commit 461c9fdd authored by Paolo G. Giarrusso's avatar Paolo G. Giarrusso
Browse files

bupd_forall -> bupd_plain_forall

parent cfe2139e
No related branches found
No related tags found
No related merge requests found
......@@ -40,6 +40,7 @@ Coq 8.11 is no longer supported in this version of Iris.
* Add lemmas for swapping nested big-ops: `big_sep{L,M,S,MS}_sep{L,M,S,MS}`.
* Rename `big_sep{L,L2,M,M2,S}_intuitionistically_forall`
`big_sep{L,L2,M,M2,S}_intro`, and `big_orL_lookup``big_orL_intro`.
* Rename `bupd_forall` to `bupd_plain_forall`.
**Changes in `proofmode`:**
......@@ -102,6 +103,7 @@ s/\bbig_sepM2_lookup_2\b/big_sepM2_lookup_r/g
# big_*_intro
s/\bbig_sep(L|L2|M|M2|S)_intuitionistically_forall\b/big_sep\1_intro/g
s/\bbig_orL_lookup\b/big_orL_intro/g
s/\bbupd_forall\b/bupd_plain_forall/g
EOF
```
......
......@@ -230,7 +230,7 @@ Section bupd_derived.
Lemma bupd_plain P `{!Plain P} : (|==> P) P.
Proof. by rewrite {1}(plain P) bupd_plainly. Qed.
Lemma bupd_forall {A} (Φ : A PROP) `{ x, Plain (Φ x)} :
Lemma bupd_plain_forall {A} (Φ : A PROP) `{ x, Plain (Φ x)} :
(|==> x, Φ x) ⊣⊢ ( x, |==> Φ x).
Proof.
apply (anti_symm _).
......
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