aboutsummaryrefslogtreecommitdiffhomepage
path: root/myocamlbuild.ml
diff options
context:
space:
mode:
authorGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2009-12-08 15:01:19 +0000
committerGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2009-12-08 15:01:19 +0000
commitc046b33aa98537a157becad80dafd1ebf4e01534 (patch)
tree37c848f8ff6749ba77f77ce188af2e6915e90328 /myocamlbuild.ml
parentb92217497f9642c17191b6212f5977ce43c992e3 (diff)
Fix the build of coq via ocamlbuild
- no more plugins/interface - a few missing files in theories.itarget - a few things required Unix now git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@12572 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'myocamlbuild.ml')
-rw-r--r--myocamlbuild.ml12
1 files changed, 7 insertions, 5 deletions
diff --git a/myocamlbuild.ml b/myocamlbuild.ml
index 963adcc7c..f7c014aba 100644
--- a/myocamlbuild.ml
+++ b/myocamlbuild.ml
@@ -124,18 +124,18 @@ let theoriesv =
let vo = string_list_of_file "theories/theories.itarget" in
List.map (fun s -> "theories/"^(Filename.chop_suffix s "o")) vo
-let contribv =
+let pluginsv =
let vo = string_list_of_file "plugins/pluginsvo.itarget" in
List.map (fun s -> "plugins/"^(Filename.chop_suffix s "o")) vo
-let contribmllib =
+let pluginsmllib =
let cma = string_list_of_file "plugins/pluginsbyte.itarget" in
List.map (fun s -> "plugins/"^(Filename.chop_suffix s ".cma")^".mllib") cma
(** for correct execution of coqdep_boot, source files should have
been imported in _build (and NMake.v should have been created). *)
-let coqdepdeps = theoriesv @ contribv @ contribmllib
+let coqdepdeps = theoriesv @ pluginsv @ pluginsmllib
let coqtop = "toplevel/coqtop"
let coqide = "ide/coqide"
@@ -209,9 +209,11 @@ let incl f = Ocaml_utils.ocaml_include_flags f
let cmd cl = (fun _ _ -> (Cmd (S cl)))
let initial_actions () = begin
- make_bin_links all_binaries;
- (** We "pre-create" a few subdirs in _build to please coqtop *)
+ (** We "pre-create" a few subdirs in _build *)
Shell.mkdir_p (!_build^"/dev");
+ Shell.mkdir_p (!_build^"/bin");
+ Shell.mkdir_p (!_build^"/plugins/micromega");
+ make_bin_links all_binaries;
end
let extra_rules () = begin