aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/bugs/opened/3848.v
diff options
context:
space:
mode:
Diffstat (limited to 'test-suite/bugs/opened/3848.v')
-rw-r--r--test-suite/bugs/opened/3848.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/test-suite/bugs/opened/3848.v b/test-suite/bugs/opened/3848.v
index b66aeccaf..9413daa04 100644
--- a/test-suite/bugs/opened/3848.v
+++ b/test-suite/bugs/opened/3848.v
@@ -18,4 +18,4 @@ Proof.
refine (functor_forall
(f^-1)
(fun (x:A) (y:Q (f^-1 x)) => eisretr f x # (g (f^-1 x))^-1 y)).
-Defined. (* Error: Attempt to save an incomplete proof *)
+Fail Defined. (* Error: Attempt to save an incomplete proof *)