aboutsummaryrefslogtreecommitdiff
path: root/toplevel/ccompile.mli
diff options
context:
space:
mode:
authorEmilio Jesus Gallego Arias2018-10-09 23:02:28 +0200
committerEmilio Jesus Gallego Arias2019-02-01 15:37:36 +0100
commit103f59ed6b8174ed9359cb11c909f1b2219390c9 (patch)
treed168a704d3ae43128e28c43b8f0cfab5826b8a26 /toplevel/ccompile.mli
parentaa2394d4ee6525b811db1e1eb58573c2f7aa749c (diff)
[toplevel] Split interactive toplevel and compiler binaries.
We make `coqc` a truly standalone binary, whereas `coqtop` is restricted to interactive use. Thus, `coqtop -compile` will emit a warning and call `coqc`. We have also refactored `Coqargs` into a common `Coqargs` module and a compilation-specific module `Coqcargs`. This solves problems related to `coqc` having its own argument parsing, and reduces the number of strange argument combinations a lot.
Diffstat (limited to 'toplevel/ccompile.mli')
-rw-r--r--toplevel/ccompile.mli6
1 files changed, 3 insertions, 3 deletions
diff --git a/toplevel/ccompile.mli b/toplevel/ccompile.mli
index 757c91c408..29a76eb966 100644
--- a/toplevel/ccompile.mli
+++ b/toplevel/ccompile.mli
@@ -10,10 +10,10 @@
(** [load_init_vernaculars opts ~state] Load vernaculars from
the init (rc) file *)
-val load_init_vernaculars : Coqargs.coq_cmdopts -> state:Vernac.State.t-> Vernac.State.t
+val load_init_vernaculars : Coqargs.t -> state:Vernac.State.t-> Vernac.State.t
(** [compile_files opts] compile files specified in [opts] *)
-val compile_files : Coqargs.coq_cmdopts -> unit
+val compile_files : Coqargs.t -> Coqcargs.t -> unit
(** [do_vio opts] process [.vio] files in [opts] *)
-val do_vio : Coqargs.coq_cmdopts -> unit
+val do_vio : Coqargs.t -> Coqcargs.t -> unit