aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/bugs/closed/3625.v
diff options
context:
space:
mode:
authorGravatar Matthieu Sozeau <matthieu.sozeau@inria.fr>2014-10-15 10:43:03 +0200
committerGravatar Matthieu Sozeau <matthieu.sozeau@inria.fr>2014-10-15 11:49:00 +0200
commit04ee4f9160dec2d854bd45fcff4dac08ada39b61 (patch)
tree360bf2853a7ab56a386faa207bf88881a3345eb7 /test-suite/bugs/closed/3625.v
parent6bcb0ebf3552e544db8b3ac8f7d00beaec81059d (diff)
Implement a different strategy to expand primitive projections only when
required, i.e. in first-order unification cases where the head of the other side is a hole or the eta-expanded constant.
Diffstat (limited to 'test-suite/bugs/closed/3625.v')
-rw-r--r--test-suite/bugs/closed/3625.v2
1 files changed, 2 insertions, 0 deletions
diff --git a/test-suite/bugs/closed/3625.v b/test-suite/bugs/closed/3625.v
index a0f977eea..3d30b62f8 100644
--- a/test-suite/bugs/closed/3625.v
+++ b/test-suite/bugs/closed/3625.v
@@ -4,6 +4,8 @@ Record prod A B := pair { fst : A ; snd : B }.
Goal forall x y : prod Set Set, x.(@fst _ _) = y.(@fst _ _).
intros.
+ refine (f_equal _ _).
+ Undo.
apply f_equal.
admit.
Qed.