diff --git a/tests/tactics.v b/tests/tactics.v
index 11d0a3c581c2d06f6a9225ee94e2bcb8aca6d745..e5eef5152e57a9b006397c9bd4337aa08c60c93f 100644
--- a/tests/tactics.v
+++ b/tests/tactics.v
@@ -1,4 +1,4 @@
-From stdpp Require Import tactics.
+From stdpp Require Import tactics option.
 
 Goal ∀ P1 P2 P3 P4 (P: Prop),
   P1 ∨ (Is_true (P2 || P3)) ∨ P4 →
@@ -69,3 +69,8 @@ universe, like [Is_true : bool → Prop]. *)
 Goal True.
 let x := mk_evar true in idtac.
 Abort.
+
+(** Make sure that [done] is not called recursively when solving [is_Some],
+which might leave an unresolved evar before performing ex falso. *)
+Goal False → is_Some (@None nat).
+Proof. done. Qed.