aboutsummaryrefslogtreecommitdiffhomepage
path: root/tactics/eauto.mli
diff options
context:
space:
mode:
Diffstat (limited to 'tactics/eauto.mli')
-rw-r--r--tactics/eauto.mli6
1 files changed, 5 insertions, 1 deletions
diff --git a/tactics/eauto.mli b/tactics/eauto.mli
index 57f6a4171..4621088e2 100644
--- a/tactics/eauto.mli
+++ b/tactics/eauto.mli
@@ -11,10 +11,13 @@ open Term
open Proof_type
open Tacexpr
open Auto
+open Topconstr
(*i*)
val rawwit_hintbases : hint_db_name list option raw_abstract_argument_type
+val rawwit_auto_using : constr_expr list raw_abstract_argument_type
+
val e_assumption : tactic
val registered_e_assumption : tactic
@@ -25,5 +28,6 @@ val vernac_e_resolve_constr : constr -> tactic
val e_give_exact_constr : constr -> tactic
-val gen_eauto : bool -> bool * int -> hint_db_name list option -> tactic
+val gen_eauto : bool -> bool * int -> constr list ->
+ hint_db_name list option -> tactic