aboutsummaryrefslogtreecommitdiffhomepage
path: root/tactics/extraargs.mli
diff options
context:
space:
mode:
authorGravatar jforest <jforest@85f007b7-540e-0410-9357-904b9bb8a0f7>2006-08-22 09:06:33 +0000
committerGravatar jforest <jforest@85f007b7-540e-0410-9357-904b9bb8a0f7>2006-08-22 09:06:33 +0000
commit24f9e6fad117fc9e0aca42beb60c45763b0d0903 (patch)
tree6dd2120b9f94e68be7e390478743e401e1df5212 /tactics/extraargs.mli
parent1e0b3352390e4bbc3be4206e9c49e7c7fba3df45 (diff)
Forgot a file in previous commit
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@9074 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'tactics/extraargs.mli')
-rw-r--r--tactics/extraargs.mli17
1 files changed, 17 insertions, 0 deletions
diff --git a/tactics/extraargs.mli b/tactics/extraargs.mli
index cc1db7eb3..81acf8548 100644
--- a/tactics/extraargs.mli
+++ b/tactics/extraargs.mli
@@ -39,3 +39,20 @@ val rawwit_hloc : loc_place raw_abstract_argument_type
val wit_hloc : place closed_abstract_argument_type
val hloc : loc_place Pcoq.Gram.Entry.e
+
+val in_arg_hyp: (Names.identifier Util.located list option * bool) Pcoq.Gram.Entry.e
+val rawwit_in_arg_hyp : (Names.identifier Util.located list option * bool) raw_abstract_argument_type
+val wit_in_arg_hyp : (Names.identifier list option * bool) closed_abstract_argument_type
+val raw_in_arg_hyp_to_clause : (Names.identifier Util.located list option * bool) -> Tacticals.clause
+val glob_in_arg_hyp_to_clause : (Names.identifier list option * bool) -> Tacticals.clause
+
+
+val by_arg_tac : Tacexpr.raw_tactic_expr option Pcoq.Gram.Entry.e
+val rawwit_by_arg_tac : raw_tactic_expr option raw_abstract_argument_type
+val wit_by_arg_tac : glob_tactic_expr option closed_abstract_argument_type
+
+
+
+val replace_term_dir : bool Pcoq.Gram.Entry.e
+val rawwit_replace_term_dir : bool raw_abstract_argument_type
+val wit_replace_term_dir : bool closed_abstract_argument_type