aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/bugs/closed/4198.v
diff options
context:
space:
mode:
authorGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2015-04-21 17:12:29 +0200
committerGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2015-04-22 18:49:36 +0200
commit3d2cf9fea0aec4ae839f70acd896958772b4caaf (patch)
treead3a5c758b05c19761643b9cc07ec99c3777e8cd /test-suite/bugs/closed/4198.v
parent8e5ecc6a3e334620ff6149706008fe4432567870 (diff)
Test for #4198 (appcontext in return clause of match).
Diffstat (limited to 'test-suite/bugs/closed/4198.v')
-rw-r--r--test-suite/bugs/closed/4198.v13
1 files changed, 13 insertions, 0 deletions
diff --git a/test-suite/bugs/closed/4198.v b/test-suite/bugs/closed/4198.v
new file mode 100644
index 000000000..ef991365d
--- /dev/null
+++ b/test-suite/bugs/closed/4198.v
@@ -0,0 +1,13 @@
+Require Import List.
+Open Scope list_scope.
+Goal forall A (x x' : A) (xs xs' : list A) (H : x::xs = x'::xs'),
+ let k :=
+ (match H in (_ = y) return x = hd x y with
+ | eq_refl => eq_refl
+ end : x = x')
+ in k = k.
+ simpl.
+ intros.
+ match goal with
+ | [ |- appcontext G[@hd] ] => idtac
+ end.