aboutsummaryrefslogtreecommitdiffhomepage
path: root/interp/constrarg.mli
diff options
context:
space:
mode:
authorGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2016-04-09 16:39:07 +0200
committerGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2016-04-27 21:55:46 +0200
commitc4ce1baa9f66210ebc1909988b3dd8baa1b8ef27 (patch)
tree7e32910be8528987dcb29e4606672cdebead9732 /interp/constrarg.mli
parent9e038688af8f7f054c1c2acdb2fe65d78cccdd81 (diff)
Honor parsing and printing levels for tactic entry in TACTIC EXTEND and
VERNAC EXTEND.
Diffstat (limited to 'interp/constrarg.mli')
-rw-r--r--interp/constrarg.mli12
1 files changed, 12 insertions, 0 deletions
diff --git a/interp/constrarg.mli b/interp/constrarg.mli
index d38b1183c..b4029758a 100644
--- a/interp/constrarg.mli
+++ b/interp/constrarg.mli
@@ -71,6 +71,18 @@ val wit_red_expr :
val wit_tactic : (raw_tactic_expr, glob_tactic_expr, Val.t) genarg_type
+val wit_tactic0 : (raw_tactic_expr, glob_tactic_expr, Val.t) genarg_type
+
+val wit_tactic1 : (raw_tactic_expr, glob_tactic_expr, Val.t) genarg_type
+
+val wit_tactic2 : (raw_tactic_expr, glob_tactic_expr, Val.t) genarg_type
+
+val wit_tactic3 : (raw_tactic_expr, glob_tactic_expr, Val.t) genarg_type
+
+val wit_tactic4 : (raw_tactic_expr, glob_tactic_expr, Val.t) genarg_type
+
+val wit_tactic5 : (raw_tactic_expr, glob_tactic_expr, Val.t) genarg_type
+
(** [wit_ltac] is subtly different from [wit_tactic]: they only change for their
toplevel interpretation. The one of [wit_ltac] forces the tactic and
discards the result. *)