aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-04-03 14:09:56 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-04-03 14:09:56 +0000
commitff94dcd516111978dfd7b782cbda2d9eae837a60 (patch)
treeca47bc958cd8318fc14feef0debd950adf0eabb4
parent987b1ff5edb3fd0a694163ca46521d35466c7ea8 (diff)
Chgts mineurs:
- correction commit incorrect d'une modif de test-suite/success/apply.v - réorganisation dev/ - renommage Print Modules en Print Libraries - $Id:$ dans g_vernac.ml4 git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@10744 85f007b7-540e-0410-9357-904b9bb8a0f7
-rw-r--r--dev/header (renamed from dev/doc/header)0
-rw-r--r--doc/refman/RefMan-oth.tex6
-rw-r--r--parsing/g_ascii_syntax.ml2
-rw-r--r--parsing/g_vernac.ml44
-rw-r--r--test-suite/success/apply.v2
5 files changed, 9 insertions, 5 deletions
diff --git a/dev/doc/header b/dev/header
index 57945e47e..57945e47e 100644
--- a/dev/doc/header
+++ b/dev/header
diff --git a/doc/refman/RefMan-oth.tex b/doc/refman/RefMan-oth.tex
index 63e43dd7d..d5935ed34 100644
--- a/doc/refman/RefMan-oth.tex
+++ b/doc/refman/RefMan-oth.tex
@@ -584,9 +584,9 @@ These different variants can be combined.
\SeeAlso Chapter~\ref{Addoc-coqc}
-\subsection[\tt Print Modules.]{\tt Print Modules.\comindex{Print Modules}}
-This command shows the currently loaded and currently opened
-(imported) modules.
+\subsection[\tt Print Libraries.]{\tt Print Libraries.\comindex{Print Libraries}}
+This command shows the currently loaded (required) and currently
+imported libraries.
\subsection[\tt Declare ML Module {\str$_1$} .. {\str$_n$}.]{\tt Declare ML Module {\str$_1$} .. {\str$_n$}.\comindex{Declare ML Module}}
This commands loads the Objective Caml compiled files {\str$_1$} \dots
diff --git a/parsing/g_ascii_syntax.ml b/parsing/g_ascii_syntax.ml
index 717abaa66..8c570b0fd 100644
--- a/parsing/g_ascii_syntax.ml
+++ b/parsing/g_ascii_syntax.ml
@@ -6,6 +6,8 @@
(* * GNU Lesser General Public License Version 2.1 *)
(***********************************************************************)
+(*i $Id:$ i*)
+
open Pp
open Util
open Names
diff --git a/parsing/g_vernac.ml4 b/parsing/g_vernac.ml4
index a693ebdb5..ae860d978 100644
--- a/parsing/g_vernac.ml4
+++ b/parsing/g_vernac.ml4
@@ -668,7 +668,9 @@ GEXTEND Gram
(* This should be in "syntax" section but is here for factorization*)
PrintGrammar ent
| IDENT "LoadPath" -> PrintLoadPath
- | IDENT "Modules" -> PrintModules
+ | IDENT "Modules" ->
+ error "Print Modules is obsolete; use Print Libraries instead"
+ | IDENT "Libraries" -> PrintModules
| IDENT "ML"; IDENT "Path" -> PrintMLLoadPath
| IDENT "ML"; IDENT "Modules" -> PrintMLModules
diff --git a/test-suite/success/apply.v b/test-suite/success/apply.v
index 5e86abe7b..014f6ffcd 100644
--- a/test-suite/success/apply.v
+++ b/test-suite/success/apply.v
@@ -51,7 +51,7 @@ Abort.
(* Check insertion of coercions in bindings *)
-(*Coercion eq_true : bool >-> Sortclass.*)
+Coercion eq_true : bool >-> Sortclass.
Goal exists A:Prop, A = A.
exists true.
trivial.