aboutsummaryrefslogtreecommitdiffhomepage
path: root/tactics/eauto.mli
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-10-31 21:19:29 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-10-31 21:19:29 +0000
commit841bc4617470a30d4025fc279c5a3e72edbb6e13 (patch)
tree07d18ac3c7a4ae7908b3545590248c841232b348 /tactics/eauto.mli
parent30f6fd59780f57201e93ef4986422b6c89077ab4 (diff)
An experimental support for open constrs in hints and in "using"
option of "auto". Works for not too complicated hints (e.g. "@pair _ _ 0"). Would be simpler if make_apply_entry supported lemmas containing evars. git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@13598 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'tactics/eauto.mli')
-rw-r--r--tactics/eauto.mli7
1 files changed, 3 insertions, 4 deletions
diff --git a/tactics/eauto.mli b/tactics/eauto.mli
index 093cd56e1..68ec42f4e 100644
--- a/tactics/eauto.mli
+++ b/tactics/eauto.mli
@@ -19,7 +19,7 @@ val hintbases : hint_db_name list option Pcoq.Gram.entry
val wit_hintbases : hint_db_name list option typed_abstract_argument_type
val rawwit_hintbases : hint_db_name list option raw_abstract_argument_type
-val rawwit_auto_using : constr_expr list raw_abstract_argument_type
+val rawwit_auto_using : Genarg.open_constr_expr list raw_abstract_argument_type
val e_assumption : tactic
@@ -27,13 +27,12 @@ val registered_e_assumption : tactic
val e_give_exact : ?flags:Unification.unify_flags -> constr -> tactic
-val gen_eauto : bool -> bool * int -> constr list ->
+val gen_eauto : bool -> bool * int -> open_constr list ->
hint_db_name list option -> tactic
-
val eauto_with_bases :
bool ->
bool * int ->
- Term.constr list -> Auto.hint_db list -> Proof_type.tactic
+ open_constr list -> Auto.hint_db list -> Proof_type.tactic
val autounfold : hint_db_name list -> Tacticals.clause -> tactic