aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite
diff options
context:
space:
mode:
authorGravatar Matthieu Sozeau <matthieu.sozeau@inria.fr>2014-08-29 00:50:08 +0200
committerGravatar Matthieu Sozeau <matthieu.sozeau@inria.fr>2014-08-29 00:50:08 +0200
commite368bcd7e16fda4d011ad2c960c647c7da72bcb6 (patch)
tree352297625b07485c667250b691b20a12cf8663ef /test-suite
parent23f064547758a491bb7cb709797c2b1338a17558 (diff)
Add test-suite file. Compute the name for the record binder in the
eta-expanded version of a projection as before.
Diffstat (limited to 'test-suite')
-rw-r--r--test-suite/bugs/closed/3402.v7
1 files changed, 7 insertions, 0 deletions
diff --git a/test-suite/bugs/closed/3402.v b/test-suite/bugs/closed/3402.v
new file mode 100644
index 000000000..ed47ec825
--- /dev/null
+++ b/test-suite/bugs/closed/3402.v
@@ -0,0 +1,7 @@
+Set Primitive Projections.
+Record prod A B := pair { fst : A ; snd : B }.
+Goal forall A B (p : prod A B), p = let (x, y) := p in pair A B x y.
+Proof.
+ intros A B p.
+ exact eq_refl.
+Qed. \ No newline at end of file