aboutsummaryrefslogtreecommitdiffhomepage
path: root/tactics/tactics.mli
diff options
context:
space:
mode:
authorGravatar filliatr <filliatr@85f007b7-540e-0410-9357-904b9bb8a0f7>1999-12-02 16:43:08 +0000
committerGravatar filliatr <filliatr@85f007b7-540e-0410-9357-904b9bb8a0f7>1999-12-02 16:43:08 +0000
commit162fc39bcc36953402d668b5d7ac7b88c9966461 (patch)
tree764403e3752e1c183ecf6831ba71e430a4b3799b /tactics/tactics.mli
parent33019e47a55caf3923d08acd66077f0a52947b47 (diff)
modifs pour premiere edition de liens
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@189 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'tactics/tactics.mli')
-rw-r--r--tactics/tactics.mli9
1 files changed, 6 insertions, 3 deletions
diff --git a/tactics/tactics.mli b/tactics/tactics.mli
index db60df966..1c4287169 100644
--- a/tactics/tactics.mli
+++ b/tactics/tactics.mli
@@ -4,6 +4,7 @@
(*i*)
open Names
open Term
+open Environ
open Tacmach
open Proof_trees
open Reduction
@@ -84,9 +85,11 @@ val dyn_exact : tactic_arg list -> tactic
(*s Reduction tactics. *)
-val reduct_in_hyp : 'a reduction_function -> identifier -> tactic
-val reduct_option : 'a reduction_function -> identifier option -> tactic
-val reduct_in_concl : 'a reduction_function -> tactic
+type 'a tactic_reduction = env -> evar_declarations -> constr -> constr
+
+val reduct_in_hyp : 'a tactic_reduction -> identifier -> tactic
+val reduct_option : 'a tactic_reduction -> identifier option -> tactic
+val reduct_in_concl : 'a tactic_reduction -> tactic
val change_in_concl : constr -> tactic
val change_in_hyp : constr -> identifier -> tactic