aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/bugs/closed/3484.v
diff options
context:
space:
mode:
authorGravatar Matthieu Sozeau <matthieu.sozeau@inria.fr>2014-10-15 13:31:46 +0200
committerGravatar Matthieu Sozeau <matthieu.sozeau@inria.fr>2014-10-15 13:34:02 +0200
commit6bca54599ab2b8ab928bfc92b8ddfb0aeba4345f (patch)
tree9730a7ee84044a8ee5062cc6340cc982b31f7722 /test-suite/bugs/closed/3484.v
parent5e1713d8fe9032a3f5c783cce288b409b6fdf816 (diff)
Reenable FO unification of primitive projections and their eta-expanded
forms in evarconv and unification, as well as fallback to first-order unification when eta for constructors fail. Update test-suite file 3484 to test for the FO case in evarconv as well.
Diffstat (limited to 'test-suite/bugs/closed/3484.v')
-rw-r--r--test-suite/bugs/closed/3484.v5
1 files changed, 4 insertions, 1 deletions
diff --git a/test-suite/bugs/closed/3484.v b/test-suite/bugs/closed/3484.v
index 3070a4128..6c40a4266 100644
--- a/test-suite/bugs/closed/3484.v
+++ b/test-suite/bugs/closed/3484.v
@@ -14,7 +14,10 @@ Proof.
apply (@ap _ _ pr1 _ y).
Undo.
Unset Printing Notations.
- apply (ap pr1). admit.
+ apply (ap pr1).
+ Undo.
+ refine (ap pr1 _).
+admit.
Defined.
(* Toplevel input, characters 22-28: