diff --git a/tests/proofmode.v b/tests/proofmode.v
index 331ea7d5b781d72b6591e316c4837ece76657b7b..ef03c12c62b126ee37d59b23a0af8adf99c3c67b 100644
--- a/tests/proofmode.v
+++ b/tests/proofmode.v
@@ -410,15 +410,13 @@ Proof.
 Qed.
 
 (* Test for issue #288 *)
-(* FIXME: Restore once we drop support for Coq 8.8 and Coq 8.9.
-Lemma test_iExists_unused : (∃ P : PROP, ∃ x : nat, P)%I.
+Lemma test_iExists_unused : ⊢ ∃ P : PROP, ∃ x : nat, P.
 Proof.
   iExists _.
   iExists 10.
   iAssert emp%I as "H"; first done.
   iExact "H".
 Qed.
-*)
 
 (* Check coercions *)
 Lemma test_iExist_coercion (P : Z → PROP) : (∀ x, P x) -∗ ∃ x, P x.