aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/bugs/closed/4467.v
diff options
context:
space:
mode:
authorGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2016-01-12 22:12:40 +0100
committerGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2016-01-12 22:17:45 +0100
commit9f8ae1aa2678944888d80ce0867bfb2bba0c8c71 (patch)
treefc01eae01222a4cc45d5d6892a72cfb437c8bd0f /test-suite/bugs/closed/4467.v
parentbe4bfc78c493464cb0af40d7fae08ba86295a6f9 (diff)
Fixing #4467 (missing shadowing of variables in cases pattern).
This fixes a TODO in map_constr_expr_with_binders, a bug in is_constructor, as well as a bug and TODOS in ids_of_cases_indtype.
Diffstat (limited to 'test-suite/bugs/closed/4467.v')
-rw-r--r--test-suite/bugs/closed/4467.v15
1 files changed, 15 insertions, 0 deletions
diff --git a/test-suite/bugs/closed/4467.v b/test-suite/bugs/closed/4467.v
new file mode 100644
index 000000000..6f8631d45
--- /dev/null
+++ b/test-suite/bugs/closed/4467.v
@@ -0,0 +1,15 @@
+(* Fixing missing test for variable shadowing *)
+
+Definition test (x y:bool*bool) :=
+ match x with
+ | (e as e1, (true) as e2)
+ | ((true) as e1, e as e2) =>
+ let '(e, b) := y in
+ e
+ | _ => true
+ end.
+
+Goal test (true,false) (true,true) = true.
+(* used to evaluate to "false = true" in 8.4 *)
+reflexivity.
+Qed.