aboutsummaryrefslogtreecommitdiff
diff options
context:
space:
mode:
-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 57945e47ea..57945e47ea 100644
--- a/dev/doc/header
+++ b/dev/header
diff --git a/doc/refman/RefMan-oth.tex b/doc/refman/RefMan-oth.tex
index 63e43dd7d4..d5935ed345 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 717abaa66a..8c570b0fdc 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 a693ebdb5c..ae860d978d 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 5e86abe7bf..014f6ffcd5 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.