aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/success/apply.v
diff options
context:
space:
mode:
Diffstat (limited to 'test-suite/success/apply.v')
-rw-r--r--test-suite/success/apply.v11
1 files changed, 11 insertions, 0 deletions
diff --git a/test-suite/success/apply.v b/test-suite/success/apply.v
index 014f6ffcd..3b4e8af21 100644
--- a/test-suite/success/apply.v
+++ b/test-suite/success/apply.v
@@ -163,3 +163,14 @@ apply H.
try apply H.
unfold ID; apply H0.
Qed.
+
+(* Test coercion below product and on non meta-free terms in with bindings *)
+(* Cf wishes #1408 from E. Makarov *)
+
+Parameter bool_Prop :> bool -> Prop.
+Parameter r : bool -> bool -> bool.
+Axiom ax : forall (A : Set) (R : A -> A -> Prop) (x y : A), R x y.
+
+Theorem t : r true false.
+apply ax with (R := r).
+Qed.