aboutsummaryrefslogtreecommitdiffhomepage
path: root/tactics
diff options
context:
space:
mode:
authorGravatar Guillaume Melquiond <guillaume.melquiond@inria.fr>2016-01-02 16:55:03 +0100
committerGravatar Guillaume Melquiond <guillaume.melquiond@inria.fr>2016-01-02 16:55:03 +0100
commit5129c5b02bcab1426636d18583ec7a4a46195f0a (patch)
tree4451c458340f449eaffe2195e01e16d55431370a /tactics
parent82ac0604888679bc2fbdeda9ac264d7cd10f7928 (diff)
Reduce dependencies of interface files.
Diffstat (limited to 'tactics')
-rw-r--r--tactics/auto.mli1
-rw-r--r--tactics/eauto.mli1
-rw-r--r--tactics/tacintern.mli1
3 files changed, 0 insertions, 3 deletions
diff --git a/tactics/auto.mli b/tactics/auto.mli
index eca592ad6..3e05d8821 100644
--- a/tactics/auto.mli
+++ b/tactics/auto.mli
@@ -10,7 +10,6 @@ open Names
open Term
open Clenv
open Pattern
-open Evd
open Decl_kinds
open Hints
diff --git a/tactics/eauto.mli b/tactics/eauto.mli
index 8e20793c4..985c08f93 100644
--- a/tactics/eauto.mli
+++ b/tactics/eauto.mli
@@ -8,7 +8,6 @@
open Term
open Proof_type
-open Evd
open Hints
val hintbases : hint_db_name list option Pcoq.Gram.entry
diff --git a/tactics/tacintern.mli b/tactics/tacintern.mli
index a6e28d568..112475694 100644
--- a/tactics/tacintern.mli
+++ b/tactics/tacintern.mli
@@ -12,7 +12,6 @@ open Tacexpr
open Genarg
open Constrexpr
open Misctypes
-open Nametab
(** Globalization of tactic expressions :
Conversion from [raw_tactic_expr] to [glob_tactic_expr] *)