aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
authorGravatar pboutill <pboutill@85f007b7-540e-0410-9357-904b9bb8a0f7>2012-05-25 12:50:13 +0000
committerGravatar pboutill <pboutill@85f007b7-540e-0410-9357-904b9bb8a0f7>2012-05-25 12:50:13 +0000
commitbdeccec95e1d018ffb18af9209060a9806d0235a (patch)
treefcc156e3b6ed411cbae70f06e082f07b0b55f4fe
parent83e8538118c0b060cb6f231726cda9178f4146bc (diff)
Bugs revealed by playing with contribs
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@15364 85f007b7-540e-0410-9357-904b9bb8a0f7
-rw-r--r--ide/project_file.ml42
-rw-r--r--theories/Vectors/VectorDef.v2
-rw-r--r--tools/coq_makefile.ml2
3 files changed, 3 insertions, 3 deletions
diff --git a/ide/project_file.ml4 b/ide/project_file.ml4
index 87ddee081..6ae5e08be 100644
--- a/ide/project_file.ml4
+++ b/ide/project_file.ml4
@@ -54,7 +54,7 @@ let rec process_cmd_line orig_dir ((project_file,makefile,install,opt) as opts)
process_cmd_line orig_dir (project_file,makefile,install,true) l r
| "-impredicative-set" :: r ->
Minilib.log "Please now use \"-arg -impredicative-set\" instead of \"-impredicative-set\" alone to be more uniform.";
- process_cmd_line orig_dir opts (Arg "-impredicative_set" :: l) r
+ process_cmd_line orig_dir opts (Arg "-impredicative-set" :: l) r
| "-no-install" :: r ->
Minilib.log "Option -no-install is deprecated. Use \"-install none\" instead";
process_cmd_line orig_dir (project_file,makefile,NoInstall,opt) l r
diff --git a/theories/Vectors/VectorDef.v b/theories/Vectors/VectorDef.v
index 23427eb86..30a8c5699 100644
--- a/theories/Vectors/VectorDef.v
+++ b/theories/Vectors/VectorDef.v
@@ -19,7 +19,7 @@ have to be the same. complain if you see mistakes ... *)
Require Import Arith_base.
Require Vectors.Fin.
Import EqNotations.
-Open Local Scope nat_scope.
+Local Open Scope nat_scope.
(**
A vector is a list of size n whose elements belong to a set A. *)
diff --git a/tools/coq_makefile.ml b/tools/coq_makefile.ml
index b9113c08e..5105ac6c9 100644
--- a/tools/coq_makefile.ml
+++ b/tools/coq_makefile.ml
@@ -201,7 +201,7 @@ let install_doc some_vfiles some_mlifiles (_,inc_r) =
if some_mlifiles then install_one_kind "mlihtml" rt;
end else begin
prerr_string "Warning: -R options don't have a correct common prefix,
- install-doc will put anything in $INSTALLDEFAULTROOT";
+ install-doc will put anything in $INSTALLDEFAULTROOT\n";
if some_vfiles then install_one_kind "html" "$(INSTALLDEFAULTROOT)";
if some_mlifiles then install_one_kind "mlihtml" "$(INSTALLDEFAULTROOT)";
end in