aboutsummaryrefslogtreecommitdiffhomepage
path: root/doc/stdlib
diff options
context:
space:
mode:
authorGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2011-05-06 09:28:40 +0000
committerGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2011-05-06 09:28:40 +0000
commit071c47c40c7818f6871a9883a48a59754d015cca (patch)
treef0ddb010d9d5b788f973b92e6c7d55820f03564b /doc/stdlib
parent4958a463c54694ca1dca6bb9f793e994dbc10856 (diff)
update of the file list in doc/stdlib
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@14112 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'doc/stdlib')
-rw-r--r--doc/stdlib/index-list.html.template11
1 files changed, 6 insertions, 5 deletions
diff --git a/doc/stdlib/index-list.html.template b/doc/stdlib/index-list.html.template
index 712681856..2c46ba047 100644
--- a/doc/stdlib/index-list.html.template
+++ b/doc/stdlib/index-list.html.template
@@ -135,19 +135,18 @@ through the <tt>Require Import</tt> command.</p>
Binary positive integers
</dt>
<dd>
+ theories/PArith/BinPosDef.v
theories/PArith/BinPos.v
theories/PArith/Pnat.v
theories/PArith/POrderedType.v
- theories/PArith/Pminmax.v
- theories/PArith/Psqrt.v
- theories/PArith/Pgcd.v
(theories/PArith/PArith.v)
</dd>
<dt> <b>NArith</b>:
Binary natural numbers
</dt>
- <dd>
+ <dd>
+ theories/NArith/BinNatDef.v
theories/NArith/BinNat.v
theories/NArith/Nnat.v
theories/NArith/Ndigits.v
@@ -162,7 +161,8 @@ through the <tt>Require Import</tt> command.</p>
<dt> <b>ZArith</b>:
Binary integers
</dt>
- <dd>
+ <dd>
+ theories/ZArith/BinIntDef.v
theories/ZArith/BinInt.v
theories/ZArith/Zorder.v
theories/ZArith/Zcompare.v
@@ -224,6 +224,7 @@ through the <tt>Require Import</tt> command.</p>
</dt>
<dt> <b>&nbsp;&nbsp;Prelude</b>:
<dd>
+ theories/Numbers/BinNums.v
theories/Numbers/NumPrelude.v
theories/Numbers/BigNumPrelude.v
theories/Numbers/NaryFunctions.v