aboutsummaryrefslogtreecommitdiffhomepage
path: root/interp
diff options
context:
space:
mode:
Diffstat (limited to 'interp')
-rw-r--r--interp/constrarg.ml3
-rw-r--r--interp/constrarg.mli5
2 files changed, 8 insertions, 0 deletions
diff --git a/interp/constrarg.ml b/interp/constrarg.ml
index 011b31d9a..ca828102b 100644
--- a/interp/constrarg.ml
+++ b/interp/constrarg.ml
@@ -61,6 +61,9 @@ let wit_red_expr = make0 "redexpr"
let wit_clause_dft_concl =
make0 "clause_dft_concl"
+let wit_destruction_arg =
+ make0 "destruction_arg"
+
(** Aliases *)
let wit_reference = wit_ref
diff --git a/interp/constrarg.mli b/interp/constrarg.mli
index 70c9c0de2..6ccd944d4 100644
--- a/interp/constrarg.mli
+++ b/interp/constrarg.mli
@@ -69,6 +69,11 @@ val wit_ltac : (raw_tactic_expr, glob_tactic_expr, unit) genarg_type
val wit_clause_dft_concl : (Names.Id.t Loc.located Locus.clause_expr,Names.Id.t Loc.located Locus.clause_expr,Names.Id.t Locus.clause_expr) genarg_type
+val wit_destruction_arg :
+ (constr_expr with_bindings destruction_arg,
+ glob_constr_and_expr with_bindings destruction_arg,
+ delayed_open_constr_with_bindings destruction_arg) genarg_type
+
(** Aliases for compatibility *)
val wit_reference : (reference, global_reference located or_var, global_reference) genarg_type