aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/bugs
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-09-20 17:10:55 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-09-20 17:10:55 +0000
commite22907304afd393f527b70c2a11d00c6abd2efb0 (patch)
treedbba9c3ccbdf8a0162962f2f4a9e638ffffcf34b /test-suite/bugs
parent4102fedccf34dc3f759685cda7018c605be1c22c (diff)
Fixed test of bug #2360 (use of Fail to check a regular error instead
of an anomaly). git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@13442 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'test-suite/bugs')
-rw-r--r--test-suite/bugs/closed/shouldsucceed/2360.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/test-suite/bugs/closed/shouldsucceed/2360.v b/test-suite/bugs/closed/shouldsucceed/2360.v
index b0974a3fd..4ae97c97b 100644
--- a/test-suite/bugs/closed/shouldsucceed/2360.v
+++ b/test-suite/bugs/closed/shouldsucceed/2360.v
@@ -9,5 +9,5 @@ Record Value (etyp : nat -> Type) := Mk {
Definition some_value (etyp : nat -> Type) : (Value etyp).
Proof.
intros.
- apply Mk.
+ Fail apply Mk. (* Check that it does not raise an anomaly *)