aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/bugs/closed/4318.v
diff options
context:
space:
mode:
authorGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2015-08-21 19:45:39 +0200
committerGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2015-08-21 20:20:01 +0200
commit081a649157d2460c924404cd51b4ba50c23b1956 (patch)
tree0a07d1cd8f6deff1061786654eb7c2225036fd82 /test-suite/bugs/closed/4318.v
parent15e6e2d666252cad3c1e0de4622ef51c2830b6b8 (diff)
Fixing #4318 (anomaly when applying args to a recursive notation in patterns).
I don't know what was the intent of Pierre B here. In 8.4, it was not supported, raising with an error at parsing time. I changed the anomaly into an error at interpretation time, so it is still not supported but we could support it if some legitimate use of it eventually appears.
Diffstat (limited to 'test-suite/bugs/closed/4318.v')
-rw-r--r--test-suite/bugs/closed/4318.v2
1 files changed, 2 insertions, 0 deletions
diff --git a/test-suite/bugs/closed/4318.v b/test-suite/bugs/closed/4318.v
new file mode 100644
index 000000000..e3140ed5a
--- /dev/null
+++ b/test-suite/bugs/closed/4318.v
@@ -0,0 +1,2 @@
+(* Check no anomaly is raised *)
+Fail Definition foo p := match p with (x, y) z => tt end.