aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/success/evars.v
diff options
context:
space:
mode:
authorGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2015-01-01 09:32:02 +0100
committerGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2015-01-01 09:35:58 +0100
commit3bd9cb26be01d0791fdf2dc56d3aacaa1379e50c (patch)
tree6771bc930f8ec5eb67f7eb388f7b16c6a74faa8f /test-suite/success/evars.v
parent47b8109321446ebf153807fe8a26151c7c0b003a (diff)
An optimization in the use of unification candidates so as to get the
following working: Definition test {A B:Type} {H:A=B} (a:A) : B := rew H in a.
Diffstat (limited to 'test-suite/success/evars.v')
-rw-r--r--test-suite/success/evars.v7
1 files changed, 7 insertions, 0 deletions
diff --git a/test-suite/success/evars.v b/test-suite/success/evars.v
index f42c6a036..4e2bf4511 100644
--- a/test-suite/success/evars.v
+++ b/test-suite/success/evars.v
@@ -408,3 +408,10 @@ Check match Some _ with None => _ | _ => _ end.
(* Used to fail for a couple of days in Nov 2014 *)
Axiom test : forall P1 P2, P1 = P2 -> P1 -> P2.
+
+(* Check use of candidates *)
+
+Import EqNotations.
+Definition test2 {A B:Type} {H:A=B} (a:A) : B := rew H in a.
+
+