aboutsummaryrefslogtreecommitdiff
path: root/plugins/decl_mode
diff options
context:
space:
mode:
authorregisgia2012-09-14 15:59:23 +0000
committerregisgia2012-09-14 15:59:23 +0000
commit6dae53d279afe2b8dcfc43dd2aded9431944c5c8 (patch)
tree716cb069d32317bdc620dc997ba6b0eb085ffbdd /plugins/decl_mode
parent0affc36749655cd0a906af0c0aad64fd350d4fec (diff)
This patch removes unused "open" (automatically generated from
compiler warnings). I was afraid that such a brutal refactoring breaks some obscure invariant about linking order and side-effects but the standard library still compiles. git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@15800 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'plugins/decl_mode')
-rw-r--r--plugins/decl_mode/decl_interp.ml1
-rw-r--r--plugins/decl_mode/decl_proof_instr.ml1
-rw-r--r--plugins/decl_mode/ppdecl_proof.ml1
3 files changed, 0 insertions, 3 deletions
diff --git a/plugins/decl_mode/decl_interp.ml b/plugins/decl_mode/decl_interp.ml
index e387b31a58..5e128bc423 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 Tacinterp
-open Tacmach
open Decl_expr
open Decl_mode
open Pretyping
diff --git a/plugins/decl_mode/decl_proof_instr.ml b/plugins/decl_mode/decl_proof_instr.ml
index 4fc5862c14..31e15081b2 100644
--- a/plugins/decl_mode/decl_proof_instr.ml
+++ b/plugins/decl_mode/decl_proof_instr.ml
@@ -11,7 +11,6 @@ open Util
open Pp
open Evd
-open Refiner
open Proof_type
open Tacmach
open Tacinterp
diff --git a/plugins/decl_mode/ppdecl_proof.ml b/plugins/decl_mode/ppdecl_proof.ml
index b72476a756..01f32e4a32 100644
--- a/plugins/decl_mode/ppdecl_proof.ml
+++ b/plugins/decl_mode/ppdecl_proof.ml
@@ -7,7 +7,6 @@
(************************************************************************)
open Errors
-open Util
open Pp
open Decl_expr
open Names