aboutsummaryrefslogtreecommitdiffhomepage
path: root/tactics/auto.mli
diff options
context:
space:
mode:
authorGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2016-03-20 23:00:46 +0100
committerGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2016-03-20 23:22:18 +0100
commitbc1d2825b7f7d0fc828b4ed99cee8ce62c646148 (patch)
tree65646f324fcca3905867941c3d6e0593e29fde4d /tactics/auto.mli
parentdc7b77f09fe5e59e6e48486d9a8c0bdc6acf83b7 (diff)
Relying on generic arguments to represent Extern hints.
Diffstat (limited to 'tactics/auto.mli')
-rw-r--r--tactics/auto.mli5
1 files changed, 1 insertions, 4 deletions
diff --git a/tactics/auto.mli b/tactics/auto.mli
index cd2de99be..8c4f35904 100644
--- a/tactics/auto.mli
+++ b/tactics/auto.mli
@@ -13,9 +13,6 @@ open Pattern
open Decl_kinds
open Hints
-val extern_interp :
- (patvar_map -> Tacexpr.glob_tactic_expr -> unit Proofview.tactic) Hook.t
-
(** Auto and related automation tactics *)
val priority : ('a * full_hint) list -> ('a * full_hint) list
@@ -35,7 +32,7 @@ val unify_resolve : polymorphic -> Unification.unify_flags -> (raw_hint * clause
[Pattern.somatches], then replace [?1] [?2] metavars in tacast by the
right values to build a tactic *)
-val conclPattern : constr -> constr_pattern option -> Tacexpr.glob_tactic_expr -> unit Proofview.tactic
+val conclPattern : constr -> constr_pattern option -> Genarg.glob_generic_argument -> unit Proofview.tactic
(** The Auto tactic *)