aboutsummaryrefslogtreecommitdiffhomepage
path: root/tactics/eauto.mli
diff options
context:
space:
mode:
authorGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2016-03-06 03:02:01 +0100
committerGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2016-03-06 03:25:30 +0100
commit8d828a124d66a79b6e35c02097b05df252d1e1d4 (patch)
treea86a185c64e9e998eb871e37f50ec3030250d1d6 /tactics/eauto.mli
parentf8b624f7bec0406258eee4e08b0cec8d756da6ff (diff)
Moving Eauto to a simple ML file.
Diffstat (limited to 'tactics/eauto.mli')
-rw-r--r--tactics/eauto.mli14
1 files changed, 8 insertions, 6 deletions
diff --git a/tactics/eauto.mli b/tactics/eauto.mli
index 0a490c65d..8812093d5 100644
--- a/tactics/eauto.mli
+++ b/tactics/eauto.mli
@@ -10,22 +10,24 @@ open Term
open Proof_type
open Hints
-val hintbases : hint_db_name list option Pcoq.Gram.entry
-
-val wit_hintbases : hint_db_name list option Genarg.uniform_genarg_type
-
val e_assumption : unit Proofview.tactic
val registered_e_assumption : unit Proofview.tactic
val e_give_exact : ?flags:Unification.unify_flags -> constr -> unit Proofview.tactic
+val prolog_tac : Tacexpr.delayed_open_constr list -> int -> unit Proofview.tactic
+
val gen_eauto : ?debug:Tacexpr.debug -> bool * int -> Tacexpr.delayed_open_constr list ->
- hint_db_name list option -> tactic
+ hint_db_name list option -> unit Proofview.tactic
val eauto_with_bases :
?debug:Tacexpr.debug ->
bool * int ->
Tacexpr.delayed_open_constr list -> hint_db list -> Proof_type.tactic
-val autounfold : hint_db_name list -> Locus.clause -> tactic
+val autounfold : hint_db_name list -> Locus.clause -> unit Proofview.tactic
+val autounfold_tac : hint_db_name list option -> Locus.clause -> unit Proofview.tactic
+val autounfold_one : hint_db_name list -> Locus.hyp_location option -> unit Proofview.tactic
+
+val make_dimension : int option -> int option -> bool * int