aboutsummaryrefslogtreecommitdiffhomepage
path: root/printing
diff options
context:
space:
mode:
authorGravatar Pierre Letouzey <pierre.letouzey@inria.fr>2013-12-16 17:08:46 +0100
committerGravatar Pierre Letouzey <pierre.letouzey@inria.fr>2013-12-16 17:24:55 +0100
commit4759f60b04a278ecd46c8a120340ba55b185c6d1 (patch)
treef5e24b08d23bd5efc9d0f80b86cde32ad548220f /printing
parent9f005304183ca9c46f6516c08c3c0cc2f1efc05f (diff)
A few fixes to the build system (mostly for ocamlbuild)
* vars.mli was mentionning Term instead of Constr, leading to a dep cycle * Having a file named toplevel/toplevel.ml isn't a good idea when we also have a toplevel/toplevel.mllib that ought to produce a toplevel.cma. We rename toplevel.ml into Coqloop.ml * Extra cleanup of toplevel.mllib : - Ppextra isn't anywhere around (?!) - Ppvernac was mentionned twice, and rather belongs to printing.mllib anyway - Vernacexpr is a .mli and shouldn't appear in an .mllib * During the link, printing.cma now comes after parsing.cma (Ppvernac uses Egramml) * A few extra -threads in ocamlbuild files (btw, it's a bit sad to need -thread for coqchk).
Diffstat (limited to 'printing')
-rw-r--r--printing/ppvernac.ml1
-rw-r--r--printing/ppvernac.mli18
-rw-r--r--printing/printing.mllib1
3 files changed, 3 insertions, 17 deletions
diff --git a/printing/ppvernac.ml b/printing/ppvernac.ml
index ba640863d..4ece6cb24 100644
--- a/printing/ppvernac.ml
+++ b/printing/ppvernac.ml
@@ -9,7 +9,6 @@
open Pp
open Names
-(* open Compat *)
open Errors
open Util
open Extend
diff --git a/printing/ppvernac.mli b/printing/ppvernac.mli
index 0e6eba267..a3d0465a6 100644
--- a/printing/ppvernac.mli
+++ b/printing/ppvernac.mli
@@ -6,22 +6,8 @@
(* * GNU Lesser General Public License Version 2.1 *)
(************************************************************************)
-open Pp
-open Genarg
-open Vernacexpr
-open Names
-open Nameops
-open Nametab
-open Ppconstr
-open Pptactic
-open Glob_term
-open Pcoq
-open Libnames
-open Ppextend
-open Topconstr
-
(** Prints a vernac expression *)
-val pr_vernac_body : vernac_expr -> std_ppcmds
+val pr_vernac_body : Vernacexpr.vernac_expr -> Pp.std_ppcmds
(** Prints a vernac expression and closes it with a dot. *)
-val pr_vernac : vernac_expr -> std_ppcmds
+val pr_vernac : Vernacexpr.vernac_expr -> Pp.std_ppcmds
diff --git a/printing/printing.mllib b/printing/printing.mllib
index 9b3bffc8d..2a8f1030f 100644
--- a/printing/printing.mllib
+++ b/printing/printing.mllib
@@ -5,3 +5,4 @@ Printer
Pptactic
Printmod
Prettyp
+Ppvernac