From 0f5eca6768ce158983e2d86096cf99436c157472 Mon Sep 17 00:00:00 2001
From: "Paolo G. Giarrusso" <p.giarrusso@gmail.com>
Date: Fri, 8 Nov 2019 15:57:50 +0100
Subject: [PATCH] Test new hint for `bi_wand` (from !331)

---
 tests/proofmode.v | 6 ++++++
 1 file changed, 6 insertions(+)

diff --git a/tests/proofmode.v b/tests/proofmode.v
index 85903527a..4a962019c 100644
--- a/tests/proofmode.v
+++ b/tests/proofmode.v
@@ -6,6 +6,12 @@ Section tests.
 Context {PROP : sbi}.
 Implicit Types P Q R : PROP.
 
+Lemma test_eauto_emp_isplit_biwand P : emp ⊢ P ∗-∗ P.
+Proof. eauto 6. Qed.
+
+Lemma test_eauto_isplit_biwand P : (P ∗-∗ P)%I.
+Proof. iStartProof. eauto. Qed.
+
 Check "demo_0".
 Lemma demo_0 P Q : □ (P ∨ Q) -∗ (∀ x, ⌜x = 0⌝ ∨ ⌜x = 1⌝) → (Q ∨ P).
 Proof.
-- 
GitLab