aboutsummaryrefslogtreecommitdiff
path: root/test-suite/ltac2
diff options
context:
space:
mode:
authorGaëtan Gilbert2019-09-24 10:23:06 +0200
committerGaëtan Gilbert2019-09-24 10:23:06 +0200
commitf92b5e4a91e8edb7ccac2ebe64d68c8d89e2e0db (patch)
tree3f72fbbe405333b16fafcad5f9e30d95fd337de4 /test-suite/ltac2
parentdc690e7067aa91a05472b5d573cb463223ef4dec (diff)
Fix #10783: use binder_annot in Ltac2.Constr.Unsafe.kind
Diffstat (limited to 'test-suite/ltac2')
-rw-r--r--test-suite/ltac2/constr.v12
1 files changed, 12 insertions, 0 deletions
diff --git a/test-suite/ltac2/constr.v b/test-suite/ltac2/constr.v
new file mode 100644
index 0000000000..39601d99a8
--- /dev/null
+++ b/test-suite/ltac2/constr.v
@@ -0,0 +1,12 @@
+Require Import Ltac2.Constr Ltac2.Init Ltac2.Control.
+Import Unsafe.
+
+Ltac2 Eval match (kind '(nat -> bool)) with
+ | Prod a b c => a
+ | _ => throw Match_failure end.
+
+Set Allow StrictProp.
+Axiom something : SProp.
+Ltac2 Eval match (kind '(forall x : something, bool)) with
+ | Prod a b c => a
+ | _ => throw Match_failure end.