diff --git a/theories/tests/proofmode.v b/theories/tests/proofmode.v
index b6b108929ce96f76b6b2e82eb7e0e30b49554f14..7c58ce313a6f4ebf537464acf7f9920948bb7394 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.