aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/bugs
diff options
context:
space:
mode:
authorGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2015-07-27 14:02:50 +0200
committerGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2015-07-27 14:20:45 +0200
commitc2a67e6f1cdd803b46a3ff4dc259c1cc57ade33f (patch)
treefddd64aff32870b76c5c36e7c27c346fdef8a5a5 /test-suite/bugs
parente46b3b6ab289f73abc240a765e81c2fe6220dce7 (diff)
Fixing #4305 (compatibility wrt 8.4 in not interpreting an
abbreviation not bound to an applied constructor as itself but rather as a binding variable as it was the case for non-applied constructor). This was broken by e5c02503 while fixed #3483 (Not_found uncaught with a notation to a non-constructor).
Diffstat (limited to 'test-suite/bugs')
-rw-r--r--test-suite/bugs/closed/4305.v17
1 files changed, 17 insertions, 0 deletions
diff --git a/test-suite/bugs/closed/4305.v b/test-suite/bugs/closed/4305.v
new file mode 100644
index 000000000..39fc02d22
--- /dev/null
+++ b/test-suite/bugs/closed/4305.v
@@ -0,0 +1,17 @@
+(* Check fallback when an abbreviation is not interpretable as a pattern *)
+
+Notation foo := Type.
+
+Definition t :=
+ match 0 with
+ | S foo => foo
+ | _ => 0
+ end.
+
+Notation bar := (option Type).
+
+Definition u :=
+ match 0 with
+ | S bar => bar
+ | _ => 0
+ end.