From e88994afb28d312bc895e1176f9ef05d045f6094 Mon Sep 17 00:00:00 2001
From: Robbert Krebbers <mail@robbertkrebbers.nl>
Date: Sun, 3 Dec 2017 22:21:08 +0100
Subject: [PATCH] =?UTF-8?q?Rename=20`wand=5Fimpl=5Fplainly`=20=E2=86=92=20?=
 =?UTF-8?q?`impl=5Fwand=5Fplainly`=20and=20swap=20direction.?=
MIME-Version: 1.0
Content-Type: text/plain; charset=UTF-8
Content-Transfer-Encoding: 8bit

To be consistent with the lemma for the persistence modality.
---
 theories/base_logic/derived.v | 8 ++++----
 1 file changed, 4 insertions(+), 4 deletions(-)

diff --git a/theories/base_logic/derived.v b/theories/base_logic/derived.v
index 55f213448..5b1521234 100644
--- a/theories/base_logic/derived.v
+++ b/theories/base_logic/derived.v
@@ -566,9 +566,9 @@ Proof.
   apply plainly_intro', impl_intro_r.
   by rewrite plainly_and_sep_l' plainly_elim wand_elim_l.
 Qed.
-Lemma wand_impl_plainly P Q : (■ P -∗ Q) ⊣⊢ (■ P → Q).
+Lemma impl_wand_plainly P Q : (■ P → Q) ⊣⊢ (■ P -∗ Q).
 Proof.
-  apply (anti_symm (⊢)); [|by rewrite -impl_wand_1].
+  apply (anti_symm (⊢)); [by rewrite -impl_wand_1|].
   apply impl_intro_l. by rewrite plainly_and_sep_l' wand_elim_r.
 Qed.
 Lemma plainly_entails_l' P Q : (P ⊢ ■ Q) → P ⊢ ■ Q ∗ P.
@@ -1029,7 +1029,7 @@ Qed.
 Global Instance wand_plain P Q : Plain P → Plain Q → Plain (P -∗ Q)%I.
 Proof.
   rewrite /Plain=> HP HQ.
-  by rewrite {2}HP -{1}(plainly_elim P) !wand_impl_plainly -plainly_impl_plainly -HQ.
+  by rewrite {2}HP -{1}(plainly_elim P) -!impl_wand_plainly -plainly_impl_plainly -HQ.
 Qed.
 Global Instance plainly_plain P : Plain (â–  P).
 Proof. by intros; apply plainly_intro'. Qed.
@@ -1079,7 +1079,7 @@ Global Instance wand_persistent P Q :
   Plain P → Persistent Q → Persistent (P -∗ Q)%I.
 Proof.
   rewrite /Plain /Persistent=> HP HQ.
-  by rewrite {2}HP -{1}(plainly_elim P) !wand_impl_plainly -persistently_impl_plainly -HQ.
+  by rewrite {2}HP -{1}(plainly_elim P) -!impl_wand_plainly -persistently_impl_plainly -HQ.
 Qed.
 Global Instance plainly_persistent P : Persistent (â–  P).
 Proof. by rewrite /Persistent persistently_plainly. Qed.
-- 
GitLab