aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/bugs/opened
diff options
context:
space:
mode:
authorGravatar Matthieu Sozeau <matthieu.sozeau@inria.fr>2015-03-03 23:32:44 +0100
committerGravatar Matthieu Sozeau <matthieu.sozeau@inria.fr>2015-03-03 23:32:44 +0100
commitc35c97e7c904f2109110c64f2ba9e45e945de381 (patch)
tree80c6272e987d27e78550ed021075a9f48c7dbf1b /test-suite/bugs/opened
parent1b7e788a2bc6c7beb5d2e6971574e3349fd2a1cf (diff)
Fix test-suite file, this is open.
Diffstat (limited to 'test-suite/bugs/opened')
-rw-r--r--test-suite/bugs/opened/3794.v4
1 files changed, 2 insertions, 2 deletions
diff --git a/test-suite/bugs/opened/3794.v b/test-suite/bugs/opened/3794.v
index 511a92b2a..99ca6cb39 100644
--- a/test-suite/bugs/opened/3794.v
+++ b/test-suite/bugs/opened/3794.v
@@ -3,5 +3,5 @@ Hint Unfold not : core.
Goal true<>false.
Set Typeclasses Debug.
-typeclasses eauto with core.
-Qed. \ No newline at end of file
+Fail typeclasses eauto with core.
+Abort. \ No newline at end of file