aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/bugs
diff options
context:
space:
mode:
authorGravatar xclerc <xclerc@85f007b7-540e-0410-9357-904b9bb8a0f7>2013-09-20 11:21:41 +0000
committerGravatar xclerc <xclerc@85f007b7-540e-0410-9357-904b9bb8a0f7>2013-09-20 11:21:41 +0000
commitb4bcf9b74588b4974bdc680bcad73669e68fc1be (patch)
treef438bb699f0defcd640e2873fbc026d0c0485b15 /test-suite/bugs
parent56b3ad583852438a1378280e9b269f8020a9524c (diff)
Update test for bug 2846 in order to use "Fail".
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@16793 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'test-suite/bugs')
-rw-r--r--test-suite/bugs/closed/shouldfail/2846.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/test-suite/bugs/closed/shouldfail/2846.v b/test-suite/bugs/closed/shouldfail/2846.v
index 2769b4d31..8d6d348a2 100644
--- a/test-suite/bugs/closed/shouldfail/2846.v
+++ b/test-suite/bugs/closed/shouldfail/2846.v
@@ -1,3 +1,3 @@
Variable R : Type.
-Inductive I : R := c : R.
+Fail Inductive I : R := c : R.