aboutsummaryrefslogtreecommitdiffhomepage
path: root/tactics/eauto.mli
diff options
context:
space:
mode:
authorGravatar msozeau <msozeau@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-02-14 12:56:21 +0000
committerGravatar msozeau <msozeau@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-02-14 12:56:21 +0000
commitbb3560885d943baef87b7f99a5d646942f0fb288 (patch)
treee5eaa2c4dc00c2a2d0d53a561e3ff910a0139906 /tactics/eauto.mli
parentf3e1ed674ebf3281e65f871d366dce38cf980539 (diff)
Backtrack changes on eauto, move specialized version of eauto in
class_tactics for further customizations. Add Equivalence.v for typeclass definitions on equivalences and clrewrite.v test-suite for clrewrite. Debugging the tactic I found missing morphisms that are now in Morphisms.v and removed some that made proof search fail or take too long, not sure it's complete however. git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@10565 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'tactics/eauto.mli')
-rw-r--r--tactics/eauto.mli45
1 files changed, 0 insertions, 45 deletions
diff --git a/tactics/eauto.mli b/tactics/eauto.mli
index a1ff89905..34655b134 100644
--- a/tactics/eauto.mli
+++ b/tactics/eauto.mli
@@ -27,50 +27,5 @@ val registered_e_assumption : tactic
val e_give_exact_constr : constr -> tactic
-type search_state = {
- depth : int; (*r depth of search before failing *)
- tacres : goal list sigma * validation;
- last_tactic : Pp.std_ppcmds;
- dblist : Auto.Hint_db.t list;
- localdb : Auto.Hint_db.t list }
-
-module SearchProblem : sig
- type state = search_state
-
- val filter_tactics : Proof_type.goal list Tacmach.sigma * (Proof_type.proof_tree list -> 'a) ->
- (Tacmach.tactic * Pp.std_ppcmds) list ->
- ((Proof_type.goal list Tacmach.sigma * (Proof_type.proof_tree list -> 'a)) *
- Pp.std_ppcmds)
- list
-
- val compare : search_state -> search_state -> int
-
- val branching : state -> state list
- val success : state -> bool
- val pp : state -> unit
-end
-
-module Search : sig
- val depth_first : search_state -> search_state
- val debug_depth_first : search_state -> search_state
-
- val breadth_first : search_state -> search_state
- val debug_breadth_first : search_state -> search_state
-end
-
-val full_eauto_gls : bool -> bool * int -> constr list -> goal list sigma * validation ->
- goal list sigma * validation
-
-val resolve_all_evars_once : bool -> bool * int -> env -> (evar -> evar_info -> bool) -> evar_defs ->
- evar_defs
-
-val resolve_all_evars : bool -> bool * int -> env -> (evar -> evar_info -> bool) -> evar_defs ->
- evar_defs
-
-val valid : Evd.evar_map ->
- (Evd.evar -> Evd.evar_info -> bool) ->
- Evd.evar_map ref -> Proof_type.proof_tree list -> 'a
-
-
val gen_eauto : bool -> bool * int -> constr list ->
hint_db_name list option -> tactic