aboutsummaryrefslogtreecommitdiff
path: root/plugins
diff options
context:
space:
mode:
authorPierre-Marie Pédrot2018-10-11 19:17:47 +0200
committerPierre-Marie Pédrot2018-10-15 22:55:18 +0200
commitdba567555fed9c88887b463a975c3d7e0852ebd3 (patch)
treead13dbed713a64ddbd53137881eab0ffdfc96d99 /plugins
parent7f39d17e7c1d7655be595ccbe741a15ba780b785 (diff)
Plug ARGUMENT EXTEND into the argument extension API.
Diffstat (limited to 'plugins')
-rw-r--r--plugins/extraction/g_extraction.ml41
-rw-r--r--plugins/firstorder/g_ground.ml41
-rw-r--r--plugins/funind/g_indfun.ml41
-rw-r--r--plugins/ltac/extraargs.ml41
-rw-r--r--plugins/ltac/g_auto.ml41
-rw-r--r--plugins/ltac/g_class.ml42
-rw-r--r--plugins/ssr/ssrparser.ml41
-rw-r--r--plugins/ssr/ssrvernac.ml41
-rw-r--r--plugins/ssrmatching/g_ssrmatching.ml41
9 files changed, 0 insertions, 10 deletions
diff --git a/plugins/extraction/g_extraction.ml4 b/plugins/extraction/g_extraction.ml4
index 93909f3e64..370d3c248f 100644
--- a/plugins/extraction/g_extraction.ml4
+++ b/plugins/extraction/g_extraction.ml4
@@ -15,7 +15,6 @@ DECLARE PLUGIN "extraction_plugin"
(* ML names *)
open Ltac_plugin
-open Genarg
open Stdarg
open Pp
open Names
diff --git a/plugins/firstorder/g_ground.ml4 b/plugins/firstorder/g_ground.ml4
index ff106404c8..db753fc672 100644
--- a/plugins/firstorder/g_ground.ml4
+++ b/plugins/firstorder/g_ground.ml4
@@ -123,7 +123,6 @@ let normalize_evaluables=
unfold_in_hyp (Lazy.force defined_connectives)
(Tacexpr.InHypType id)) *)
-open Genarg
open Ppconstr
open Printer
let pr_firstorder_using_raw _ _ _ = Pptactic.pr_auto_using pr_qualid
diff --git a/plugins/funind/g_indfun.ml4 b/plugins/funind/g_indfun.ml4
index 272852d47a..c7555c44eb 100644
--- a/plugins/funind/g_indfun.ml4
+++ b/plugins/funind/g_indfun.ml4
@@ -13,7 +13,6 @@ open Pp
open Constrexpr
open Indfun_common
open Indfun
-open Genarg
open Stdarg
open Tacarg
open Tactypes
diff --git a/plugins/ltac/extraargs.ml4 b/plugins/ltac/extraargs.ml4
index 0c6d10bf8c..4de27e8138 100644
--- a/plugins/ltac/extraargs.ml4
+++ b/plugins/ltac/extraargs.ml4
@@ -9,7 +9,6 @@
(************************************************************************)
open Pp
-open Genarg
open Stdarg
open Tacarg
open Pcoq.Prim
diff --git a/plugins/ltac/g_auto.ml4 b/plugins/ltac/g_auto.ml4
index 8eadb66edc..6913543c9a 100644
--- a/plugins/ltac/g_auto.ml4
+++ b/plugins/ltac/g_auto.ml4
@@ -10,7 +10,6 @@
open Pp
open Constr
-open Genarg
open Stdarg
open Pcoq.Prim
open Pcoq.Constr
diff --git a/plugins/ltac/g_class.ml4 b/plugins/ltac/g_class.ml4
index 1c2f90b670..265368833b 100644
--- a/plugins/ltac/g_class.ml4
+++ b/plugins/ltac/g_class.ml4
@@ -32,8 +32,6 @@ VERNAC COMMAND EXTEND Typeclasses_Rigid_Settings CLASSIFIED AS SIDEFF
set_transparency cl false ]
END
-open Genarg
-
let pr_debug _prc _prlc _prt b =
if b then Pp.str "debug" else Pp.mt()
diff --git a/plugins/ssr/ssrparser.ml4 b/plugins/ssr/ssrparser.ml4
index e4a0910673..319f58931a 100644
--- a/plugins/ssr/ssrparser.ml4
+++ b/plugins/ssr/ssrparser.ml4
@@ -15,7 +15,6 @@ open Names
open Pp
open Pcoq
open Ltac_plugin
-open Genarg
open Stdarg
open Tacarg
open Libnames
diff --git a/plugins/ssr/ssrvernac.ml4 b/plugins/ssr/ssrvernac.ml4
index d62656f95f..02a5d08507 100644
--- a/plugins/ssr/ssrvernac.ml4
+++ b/plugins/ssr/ssrvernac.ml4
@@ -25,7 +25,6 @@ open Notation_ops
open Notation_term
open Glob_term
open Stdarg
-open Genarg
open Decl_kinds
open Pp
open Ppconstr
diff --git a/plugins/ssrmatching/g_ssrmatching.ml4 b/plugins/ssrmatching/g_ssrmatching.ml4
index 746c368aa9..9e1f992f38 100644
--- a/plugins/ssrmatching/g_ssrmatching.ml4
+++ b/plugins/ssrmatching/g_ssrmatching.ml4
@@ -9,7 +9,6 @@
(************************************************************************)
open Ltac_plugin
-open Genarg
open Pcoq
open Pcoq.Constr
open Ssrmatching