Skip to content

Commit

Permalink
Bugs revealed by playing with contribs
Browse files Browse the repository at this point in the history
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@15364 85f007b7-540e-0410-9357-904b9bb8a0f7
  • Loading branch information
pirbo committed May 25, 2012
1 parent 83e8538 commit bdeccec
Show file tree
Hide file tree
Showing 3 changed files with 3 additions and 3 deletions.
2 changes: 1 addition & 1 deletion ide/project_file.ml4
Expand Up @@ -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
Expand Down
2 changes: 1 addition & 1 deletion theories/Vectors/VectorDef.v
Expand Up @@ -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. *)
Expand Down
2 changes: 1 addition & 1 deletion tools/coq_makefile.ml
Expand Up @@ -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
Expand Down

0 comments on commit bdeccec

Please sign in to comment.