caml-list - the Caml user's mailing list
 help / color / mirror / Atom feed
* [Caml-list] Build Cycle
@ 2003-10-12  1:39 HFX
  0 siblings, 0 replies; only message in thread
From: HFX @ 2003-10-12  1:39 UTC (permalink / raw)
  To: caml-list

As the Readme.win32 file states I build it using the Unix directions 
from the INSTALL file.


I build as follows.

mkdir logs
./configure -verbose > logs/configure.log 2>&1
make world > logs/world.log 2>&1'
tail logs/world.log

seems fine

make bootstrap > logs/bootstrap.log 2>&1
tail logs/bootstrap.log

Error message is as follows:
sh ./runocamldoc false -man -d stdlib_man -I ../parsing -I ../utils -I 
../typing
  -I ../driver -I ../bytecomp -I ../tools -I ../toplevel/ -I ../stdlib 
-I ../othe
rlibs/str -I ../otherlibs/dynlink -I ../otherlibs/unix -I 
../otherlibs/num -I ..
/otherlibs/graph \
-t "OCaml library" -man-mini -man-suffix 3o \
../stdlib/*.mli ../otherlibs/unix/unix.mli ../otherlibs/str/str.mli 
../otherlibs
/bigarray/bigarray.mli ../otherlibs/num/num.mli
make[2]: Leaving directory 
`/home/Administrator/downloads/ocaml-3.07/ocamldoc'
make[1]: Leaving directory `/home/Administrator/downloads/ocaml-3.07'
make compare
make[1]: Entering directory `/home/Administrator/downloads/ocaml-3.07'
boot/ocamlc ocamlc differ: char 137, line 2
Fixpoint not reached, try one more bootstrapping cycle.
make[1]: Leaving directory `/home/Administrator/downloads/ocaml-3.07'



Next I try to do the optimized compiler

make opt > logs/opt.log 2>&1
tail logs/opt.log

Seems fine.

make opt.opt > logs/opt.opt.log 2>&1
tail logs/opt.opt.log

Seems fine also

So the only problem I seem to have found is with trying to bootstrap the 
bytecode compiler.

System is as follows:

Athlon 2000 XP on an Asus A7V333
512 Megs of RAM
Geforce 2 MX 400 64 Meg
Windows 2000 w SP4 and all other patches
Cygwin D/L and install as of September 20, 2003

I hope this helps.

HFX













-------------------
To unsubscribe, mail caml-list-request@inria.fr Archives: http://caml.inria.fr
Bug reports: http://caml.inria.fr/bin/caml-bugs FAQ: http://caml.inria.fr/FAQ/
Beginner's list: http://groups.yahoo.com/group/ocaml_beginners


^ permalink raw reply	[flat|nested] only message in thread

only message in thread, other threads:[~2003-10-12  1:38 UTC | newest]

Thread overview: (only message) (download: mbox.gz / follow: Atom feed)
-- links below jump to the message on this page --
2003-10-12  1:39 [Caml-list] Build Cycle HFX

This is a public inbox, see mirroring instructions
for how to clone and mirror all data and code used for this inbox;
as well as URLs for NNTP newsgroup(s).