aboutsummaryrefslogtreecommitdiffhomepage
path: root/doc/stdlib
diff options
context:
space:
mode:
authorGravatar Guillaume Melquiond <guillaume.melquiond@inria.fr>2015-10-02 21:32:25 +0200
committerGravatar Guillaume Melquiond <guillaume.melquiond@inria.fr>2015-10-02 21:32:35 +0200
commitf41de34bcd48f008cf7d3fae4c7fce925048e606 (patch)
treeb546003de4dfdd99dbe0865f2cd77e41096cc429 /doc/stdlib
parentbeedccef9ddc8633c705d7c5ee2f1bbbb3ec8a47 (diff)
Mark the Coq.Compat files for documentation. (Fix bug #4353)
Diffstat (limited to 'doc/stdlib')
-rw-r--r--doc/stdlib/index-list.html.template10
1 files changed, 9 insertions, 1 deletions
diff --git a/doc/stdlib/index-list.html.template b/doc/stdlib/index-list.html.template
index 024e13413..866193ffb 100644
--- a/doc/stdlib/index-list.html.template
+++ b/doc/stdlib/index-list.html.template
@@ -591,7 +591,7 @@ through the <tt>Require Import</tt> command.</p>
</dd>
<dt> <b>Program</b>:
- Support for dependently-typed programming.
+ Support for dependently-typed programming
</dt>
<dd>
theories/Program/Basics.v
@@ -612,4 +612,12 @@ through the <tt>Require Import</tt> command.</p>
theories/Unicode/Utf8_core.v
theories/Unicode/Utf8.v
</dd>
+
+ <dt> <b>Compat</b>:
+ Compatibility wrappers for previous versions of Coq
+ </dt>
+ <dd>
+ theories/Compat/Coq84.v
+ theories/Compat/Coq85.v
+ </dd>
</dl>