aboutsummaryrefslogtreecommitdiff
path: root/plugins
diff options
context:
space:
mode:
Diffstat (limited to 'plugins')
-rw-r--r--plugins/btauto/refl_btauto.ml1
-rw-r--r--plugins/cc/cctac.ml2
-rw-r--r--plugins/decl_mode/decl_expr.mli1
-rw-r--r--plugins/decl_mode/decl_interp.ml1
-rw-r--r--plugins/decl_mode/decl_interp.mli1
-rw-r--r--plugins/decl_mode/decl_mode.mli1
-rw-r--r--plugins/decl_mode/decl_proof_instr.ml1
-rw-r--r--plugins/decl_mode/decl_proof_instr.mli1
-rw-r--r--plugins/decl_mode/g_decl_mode.ml42
-rw-r--r--plugins/extraction/common.mli1
-rw-r--r--plugins/extraction/extraction.mli1
-rw-r--r--plugins/extraction/mlutil.ml1
-rw-r--r--plugins/extraction/mlutil.mli1
-rw-r--r--plugins/extraction/modutil.mli3
-rw-r--r--plugins/firstorder/ground.ml1
-rw-r--r--plugins/firstorder/instances.mli3
-rw-r--r--plugins/firstorder/sequent.mli1
-rw-r--r--plugins/fourier/fourierR.ml1
-rw-r--r--plugins/funind/functional_principles_types.ml1
-rw-r--r--plugins/funind/g_indfun.ml41
-rw-r--r--plugins/funind/indfun.mli7
-rw-r--r--plugins/funind/recdef.ml2
-rw-r--r--plugins/omega/coq_omega.ml1
-rw-r--r--plugins/omega/g_omega.ml41
-rw-r--r--plugins/quote/quote.ml1
-rw-r--r--plugins/romega/g_romega.ml41
-rw-r--r--plugins/setoid_ring/newring.ml43
27 files changed, 1 insertions, 41 deletions
diff --git a/plugins/btauto/refl_btauto.ml b/plugins/btauto/refl_btauto.ml
index 8232604f78..b81821a2e5 100644
--- a/plugins/btauto/refl_btauto.ml
+++ b/plugins/btauto/refl_btauto.ml
@@ -1,4 +1,3 @@
-open Proofview.Notations
let contrib_name = "btauto"
diff --git a/plugins/cc/cctac.ml b/plugins/cc/cctac.ml
index b086190f4e..f4f62cb852 100644
--- a/plugins/cc/cctac.ml
+++ b/plugins/cc/cctac.ml
@@ -16,14 +16,12 @@ open Term
open Vars
open Tacmach
open Tactics
-open Tacticals
open Typing
open Ccalgo
open Ccproof
open Pp
open Errors
open Util
-open Proofview.Notations
let constant dir s = lazy (Coqlib.gen_constant "CC" dir s)
diff --git a/plugins/decl_mode/decl_expr.mli b/plugins/decl_mode/decl_expr.mli
index 7548c338a0..982fb47ad2 100644
--- a/plugins/decl_mode/decl_expr.mli
+++ b/plugins/decl_mode/decl_expr.mli
@@ -7,7 +7,6 @@
(************************************************************************)
open Names
-open Pp
open Tacexpr
type 'it statement =
diff --git a/plugins/decl_mode/decl_interp.ml b/plugins/decl_mode/decl_interp.ml
index a722daca52..505d7dba5c 100644
--- a/plugins/decl_mode/decl_interp.ml
+++ b/plugins/decl_mode/decl_interp.ml
@@ -11,7 +11,6 @@ open Util
open Names
open Constrexpr
open Tacintern
-open Tacinterp
open Decl_expr
open Decl_mode
open Pretyping
diff --git a/plugins/decl_mode/decl_interp.mli b/plugins/decl_mode/decl_interp.mli
index 88fb9653ae..6fbf5d25c9 100644
--- a/plugins/decl_mode/decl_interp.mli
+++ b/plugins/decl_mode/decl_interp.mli
@@ -8,7 +8,6 @@
open Tacintern
open Decl_expr
-open Mod_subst
val intern_proof_instr : glob_sign -> raw_proof_instr -> glob_proof_instr
diff --git a/plugins/decl_mode/decl_mode.mli b/plugins/decl_mode/decl_mode.mli
index 8e691f508f..1ed1abaf75 100644
--- a/plugins/decl_mode/decl_mode.mli
+++ b/plugins/decl_mode/decl_mode.mli
@@ -9,7 +9,6 @@
open Names
open Term
open Evd
-open Tacmach
val set_daimon_flag : unit -> unit
val clear_daimon_flag : unit -> unit
diff --git a/plugins/decl_mode/decl_proof_instr.ml b/plugins/decl_mode/decl_proof_instr.ml
index 45ffb450f6..de57330ecf 100644
--- a/plugins/decl_mode/decl_proof_instr.ml
+++ b/plugins/decl_mode/decl_proof_instr.ml
@@ -13,7 +13,6 @@ open Evd
open Tacmach
open Tacintern
-open Tacinterp
open Decl_expr
open Decl_mode
open Decl_interp
diff --git a/plugins/decl_mode/decl_proof_instr.mli b/plugins/decl_mode/decl_proof_instr.mli
index d78ca84d12..458318264e 100644
--- a/plugins/decl_mode/decl_proof_instr.mli
+++ b/plugins/decl_mode/decl_proof_instr.mli
@@ -6,7 +6,6 @@
(* * GNU Lesser General Public License Version 2.1 *)
(************************************************************************)
-open Refiner
open Names
open Term
open Tacmach
diff --git a/plugins/decl_mode/g_decl_mode.ml4 b/plugins/decl_mode/g_decl_mode.ml4
index fe75d17f6a..7c9ef3c2a8 100644
--- a/plugins/decl_mode/g_decl_mode.ml4
+++ b/plugins/decl_mode/g_decl_mode.ml4
@@ -11,11 +11,11 @@
open Util
open Compat
open Pp
-open Tok
open Decl_expr
open Names
open Pcoq
open Vernacexpr
+open Tok (* necessary for camlp4 *)
open Pcoq.Constr
open Pcoq.Tactic
diff --git a/plugins/extraction/common.mli b/plugins/extraction/common.mli
index 0fd3e7bb7b..3058b91b66 100644
--- a/plugins/extraction/common.mli
+++ b/plugins/extraction/common.mli
@@ -9,7 +9,6 @@
open Names
open Globnames
open Miniml
-open Mlutil
open Pp
(** By default, in module Format, you can do horizontal placing of blocks
diff --git a/plugins/extraction/extraction.mli b/plugins/extraction/extraction.mli
index 89db50e630..8d3cf76fdd 100644
--- a/plugins/extraction/extraction.mli
+++ b/plugins/extraction/extraction.mli
@@ -12,7 +12,6 @@ open Names
open Term
open Declarations
open Environ
-open Libnames
open Miniml
val extract_constant : env -> constant -> constant_body -> ml_decl
diff --git a/plugins/extraction/mlutil.ml b/plugins/extraction/mlutil.ml
index 1a4cfb45fa..9b72c3e9fd 100644
--- a/plugins/extraction/mlutil.ml
+++ b/plugins/extraction/mlutil.ml
@@ -1363,7 +1363,6 @@ let is_not_strict t =
restriction for the moment.
*)
-open Declarations
open Declareops
let inline_test r t =
diff --git a/plugins/extraction/mlutil.mli b/plugins/extraction/mlutil.mli
index f25f0bb89d..ff5dee31f8 100644
--- a/plugins/extraction/mlutil.mli
+++ b/plugins/extraction/mlutil.mli
@@ -7,7 +7,6 @@
(************************************************************************)
open Names
-open Term
open Globnames
open Miniml
open Table
diff --git a/plugins/extraction/modutil.mli b/plugins/extraction/modutil.mli
index 52805bc87f..42c8b11f3f 100644
--- a/plugins/extraction/modutil.mli
+++ b/plugins/extraction/modutil.mli
@@ -7,11 +7,8 @@
(************************************************************************)
open Names
-open Declarations
-open Environ
open Globnames
open Miniml
-open Mod_subst
(*s Functions upon ML modules. *)
diff --git a/plugins/firstorder/ground.ml b/plugins/firstorder/ground.ml
index 5133801ee7..6c1709140b 100644
--- a/plugins/firstorder/ground.ml
+++ b/plugins/firstorder/ground.ml
@@ -11,7 +11,6 @@ open Sequent
open Rules
open Instances
open Term
-open Vars
open Tacmach
open Tacticals
diff --git a/plugins/firstorder/instances.mli b/plugins/firstorder/instances.mli
index 753f2d76e1..66c42e1e64 100644
--- a/plugins/firstorder/instances.mli
+++ b/plugins/firstorder/instances.mli
@@ -6,9 +6,6 @@
(* * GNU Lesser General Public License Version 2.1 *)
(************************************************************************)
-open Term
-open Tacmach
-open Names
open Globnames
open Rules
diff --git a/plugins/firstorder/sequent.mli b/plugins/firstorder/sequent.mli
index 0e5223d6bd..536ee7cc34 100644
--- a/plugins/firstorder/sequent.mli
+++ b/plugins/firstorder/sequent.mli
@@ -9,7 +9,6 @@
open Term
open Formula
open Tacmach
-open Names
open Globnames
module OrderedConstr: Set.OrderedType with type t=constr
diff --git a/plugins/fourier/fourierR.ml b/plugins/fourier/fourierR.ml
index 2a5e81ec0d..aeb07fc3a2 100644
--- a/plugins/fourier/fourierR.ml
+++ b/plugins/fourier/fourierR.ml
@@ -15,7 +15,6 @@ des inéquations et équations sont entiers. En attendant la tactique Field.
open Term
open Tactics
open Names
-open Libnames
open Globnames
open Tacticals
open Tacmach
diff --git a/plugins/funind/functional_principles_types.ml b/plugins/funind/functional_principles_types.ml
index 56b1a3f1cb..d6f21fb86b 100644
--- a/plugins/funind/functional_principles_types.ml
+++ b/plugins/funind/functional_principles_types.ml
@@ -6,7 +6,6 @@ open Vars
open Context
open Namegen
open Names
-open Declarations
open Declareops
open Pp
open Entries
diff --git a/plugins/funind/g_indfun.ml4 b/plugins/funind/g_indfun.ml4
index cc9ae912dc..2dd78d8908 100644
--- a/plugins/funind/g_indfun.ml4
+++ b/plugins/funind/g_indfun.ml4
@@ -18,7 +18,6 @@ open Indfun
open Genarg
open Tacticals
open Misctypes
-open Miscops
let pr_binding prc = function
| loc, NamedHyp id, c -> hov 1 (Ppconstr.pr_id id ++ str " := " ++ cut () ++ prc c)
diff --git a/plugins/funind/indfun.mli b/plugins/funind/indfun.mli
index 56fc9bd2cd..91a5ddf826 100644
--- a/plugins/funind/indfun.mli
+++ b/plugins/funind/indfun.mli
@@ -1,10 +1,3 @@
-open Names
-open Term
-open Pp
-open Indfun_common
-open Libnames
-open Glob_term
-open Declarations
open Misctypes
val do_generate_principle :
diff --git a/plugins/funind/recdef.ml b/plugins/funind/recdef.ml
index f951debfde..ca0a432d6a 100644
--- a/plugins/funind/recdef.ml
+++ b/plugins/funind/recdef.ml
@@ -10,7 +10,6 @@ open Term
open Vars
open Namegen
open Environ
-open Declarations
open Declareops
open Entries
open Pp
@@ -24,7 +23,6 @@ open Tacticals
open Tacmach
open Tactics
open Nametab
-open Decls
open Declare
open Decl_kinds
open Tacred
diff --git a/plugins/omega/coq_omega.ml b/plugins/omega/coq_omega.ml
index 74f1ba713f..de20756b3c 100644
--- a/plugins/omega/coq_omega.ml
+++ b/plugins/omega/coq_omega.ml
@@ -27,7 +27,6 @@ open Globnames
open Nametab
open Contradiction
open Misctypes
-open Proofview.Notations
module OmegaSolver = Omega.MakeOmegaSolver (Bigint)
open OmegaSolver
diff --git a/plugins/omega/g_omega.ml4 b/plugins/omega/g_omega.ml4
index 0aad364c16..b384478ae2 100644
--- a/plugins/omega/g_omega.ml4
+++ b/plugins/omega/g_omega.ml4
@@ -16,7 +16,6 @@
(*i camlp4deps: "grammar/grammar.cma" i*)
open Coq_omega
-open Refiner
let omega_tactic l =
let tacs = List.map
diff --git a/plugins/quote/quote.ml b/plugins/quote/quote.ml
index affe31d790..9ee16a5827 100644
--- a/plugins/quote/quote.ml
+++ b/plugins/quote/quote.ml
@@ -109,7 +109,6 @@ open Pattern
open Patternops
open ConstrMatching
open Tacmach
-open Proofview.Notations
(*i*)
(*s First, we need to access some Coq constants
diff --git a/plugins/romega/g_romega.ml4 b/plugins/romega/g_romega.ml4
index efe11b99cb..c07825f8cd 100644
--- a/plugins/romega/g_romega.ml4
+++ b/plugins/romega/g_romega.ml4
@@ -9,7 +9,6 @@
(*i camlp4deps: "grammar/grammar.cma" i*)
open Refl_omega
-open Refiner
let romega_tactic l =
let tacs = List.map
diff --git a/plugins/setoid_ring/newring.ml4 b/plugins/setoid_ring/newring.ml4
index b8507041f3..0cb9d4460f 100644
--- a/plugins/setoid_ring/newring.ml4
+++ b/plugins/setoid_ring/newring.ml4
@@ -22,7 +22,6 @@ open Glob_term
open Tacticals
open Tacexpr
open Coqlib
-open Tacmach
open Mod_subst
open Tacinterp
open Libobject
@@ -797,8 +796,6 @@ let ltac_ring_structure e =
[req;sth;ext;morph;th;cst_tac;pow_tac;
lemma1;lemma2;pretac;posttac]
-open Proofview.Notations
-
let ring_lookup (f:glob_tactic_expr) lH rl t =
Proofview.Goal.enter begin fun gl ->
let sigma = Proofview.Goal.sigma gl in