From 7a1be53efa73c19d3c8497a090394901bef0ae6c Mon Sep 17 00:00:00 2001
From: Ralf Jung <jung@mpi-sws.org>
Date: Wed, 7 Mar 2018 19:43:40 +0100
Subject: [PATCH] more unicode

---
 theories/tests/proofmode.v | 2 +-
 1 file changed, 1 insertion(+), 1 deletion(-)

diff --git a/theories/tests/proofmode.v b/theories/tests/proofmode.v
index b6b108929..7c58ce313 100644
--- a/theories/tests/proofmode.v
+++ b/theories/tests/proofmode.v
@@ -408,7 +408,7 @@ Proof.
   eexists. split. iIntros "#? ? ? ?". iAccu. done.
 Qed.
 
-Lemma test_iAssumption_evar P : ∃ R, (R ⊢ P) /\ R = P.
+Lemma test_iAssumption_evar P : ∃ R, (R ⊢ P) ∧ R = P.
 Proof.
   eexists. split.
   - iIntros "H". iAssumption.
-- 
GitLab