aboutsummaryrefslogtreecommitdiffhomepage
path: root/parsing
diff options
context:
space:
mode:
authorGravatar Gaetan Gilbert <gaetan.gilbert@ens-lyon.fr>2017-04-21 20:11:47 +0200
committerGravatar Gaetan Gilbert <gaetan.gilbert@ens-lyon.fr>2017-04-27 21:42:01 +0200
commit4e84e83911c1cf7613a35b921b1e68e097f84b5a (patch)
tree86caa28a08dde1e771c365350550ffdd633ba1f8 /parsing
parente1d2a898feacbe4bd363818f259bce5fd74c2ee7 (diff)
Remove unused [open] statements
Diffstat (limited to 'parsing')
-rw-r--r--parsing/egramcoq.ml1
-rw-r--r--parsing/egramcoq.mli8
-rw-r--r--parsing/g_prim.ml41
-rw-r--r--parsing/g_proofs.ml41
4 files changed, 0 insertions, 11 deletions
diff --git a/parsing/egramcoq.ml b/parsing/egramcoq.ml
index 65e99d1b9..86c66ec5f 100644
--- a/parsing/egramcoq.ml
+++ b/parsing/egramcoq.ml
@@ -10,7 +10,6 @@ open CErrors
open Util
open Pcoq
open Constrexpr
-open Notation
open Notation_term
open Extend
open Libnames
diff --git a/parsing/egramcoq.mli b/parsing/egramcoq.mli
index 6dda3817a..0a0430ba6 100644
--- a/parsing/egramcoq.mli
+++ b/parsing/egramcoq.mli
@@ -6,14 +6,6 @@
(* * GNU Lesser General Public License Version 2.1 *)
(************************************************************************)
-open Names
-open Constrexpr
-open Notation_term
-open Pcoq
-open Extend
-open Genarg
-open Egramml
-
(** Mapping of grammar productions to camlp4 actions *)
(** This is the part specific to Coq-level Notation and Tactic Notation.
diff --git a/parsing/g_prim.ml4 b/parsing/g_prim.ml4
index 2af4ed533..abb463f82 100644
--- a/parsing/g_prim.ml4
+++ b/parsing/g_prim.ml4
@@ -8,7 +8,6 @@
open Names
open Libnames
-open Tok (* necessary for camlp4 *)
open Pcoq
open Pcoq.Prim
diff --git a/parsing/g_proofs.ml4 b/parsing/g_proofs.ml4
index 7ca2e4a4f..68b8be6b8 100644
--- a/parsing/g_proofs.ml4
+++ b/parsing/g_proofs.ml4
@@ -9,7 +9,6 @@
open Constrexpr
open Vernacexpr
open Misctypes
-open Tok
open Pcoq
open Pcoq.Prim