aboutsummaryrefslogtreecommitdiffhomepage
path: root/tactics/eauto.mli
diff options
context:
space:
mode:
authorGravatar msozeau <msozeau@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-02-06 14:47:11 +0000
committerGravatar msozeau <msozeau@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-02-06 14:47:11 +0000
commit37a966bdcf072b2919c46fb19a233aac37ea09a7 (patch)
tree33f963e5edea7feb8c375ce5c4d59c342bee00cb /tactics/eauto.mli
parent619a9aad46a82e9db859e9a7378c8f62e5e927a6 (diff)
Work-in-progress to make eauto accept a list of goals as input and
return a solution for the whole set of goals at once only. Add "debug eauto" and "dfs eauto" syntaxes to get better control on the algorithm from the surface interface. git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@10514 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'tactics/eauto.mli')
-rw-r--r--tactics/eauto.mli7
1 files changed, 7 insertions, 0 deletions
diff --git a/tactics/eauto.mli b/tactics/eauto.mli
index 8fac813a6..34c4cab78 100644
--- a/tactics/eauto.mli
+++ b/tactics/eauto.mli
@@ -12,6 +12,8 @@ open Proof_type
open Tacexpr
open Auto
open Topconstr
+open Evd
+open Environ
(*i*)
val rawwit_hintbases : hint_db_name list option raw_abstract_argument_type
@@ -24,5 +26,10 @@ val registered_e_assumption : tactic
val e_give_exact_constr : constr -> tactic
+val full_eauto_gls : bool -> bool * int -> constr list -> goal list sigma * validation ->
+ goal list sigma * validation
+
+val resolve_all_evars : env -> (constr -> bool) -> evar_defs -> evar_defs
+
val gen_eauto : bool -> bool * int -> constr list ->
hint_db_name list option -> tactic