aboutsummaryrefslogtreecommitdiffhomepage
path: root/tactics
diff options
context:
space:
mode:
authorGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2016-03-06 03:56:11 +0100
committerGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2016-03-06 03:57:10 +0100
commitb18bc8d5fe64d395197b172b5574f03d50d8157d (patch)
tree99f34c73a44a895c85becbb4fd7fa24c9a075f9a /tactics
parent8f6d74c1e771966e3dd44704805a1e848af4802a (diff)
Removing useless grammar.cma dependencies.
Diffstat (limited to 'tactics')
-rw-r--r--tactics/eauto.ml2
-rw-r--r--tactics/eqdecide.ml2
-rw-r--r--tactics/rewrite.ml2
-rw-r--r--tactics/tauto.ml2
4 files changed, 0 insertions, 8 deletions
diff --git a/tactics/eauto.ml b/tactics/eauto.ml
index a118f2642..044946759 100644
--- a/tactics/eauto.ml
+++ b/tactics/eauto.ml
@@ -6,8 +6,6 @@
(* * GNU Lesser General Public License Version 2.1 *)
(************************************************************************)
-(*i camlp4deps: "grammar/grammar.cma" i*)
-
open Pp
open Errors
open Util
diff --git a/tactics/eqdecide.ml b/tactics/eqdecide.ml
index 7c821ddcb..7d0df2f52 100644
--- a/tactics/eqdecide.ml
+++ b/tactics/eqdecide.ml
@@ -12,8 +12,6 @@
(* by Eduardo Gimenez *)
(************************************************************************)
-(*i camlp4deps: "grammar/grammar.cma" i*)
-
open Errors
open Util
open Names
diff --git a/tactics/rewrite.ml b/tactics/rewrite.ml
index 953235463..1be78c2ad 100644
--- a/tactics/rewrite.ml
+++ b/tactics/rewrite.ml
@@ -6,8 +6,6 @@
(* * GNU Lesser General Public License Version 2.1 *)
(************************************************************************)
-(*i camlp4deps: "grammar/grammar.cma" i*)
-
open Names
open Pp
open Errors
diff --git a/tactics/tauto.ml b/tactics/tauto.ml
index 67ef25d49..d3e0b1f44 100644
--- a/tactics/tauto.ml
+++ b/tactics/tauto.ml
@@ -6,8 +6,6 @@
(* * GNU Lesser General Public License Version 2.1 *)
(************************************************************************)
-(*i camlp4deps: "grammar/grammar.cma" i*)
-
open Term
open Hipattern
open Names