aboutsummaryrefslogtreecommitdiffhomepage
path: root/doc/stdlib
diff options
context:
space:
mode:
authorGravatar msozeau <msozeau@85f007b7-540e-0410-9357-904b9bb8a0f7>2007-08-08 13:14:05 +0000
committerGravatar msozeau <msozeau@85f007b7-540e-0410-9357-904b9bb8a0f7>2007-08-08 13:14:05 +0000
commitea3763f3bc406dd3257e1d8ec4d489a0790ae713 (patch)
treefa5424106a5387155dbdab2b2ed6814e6bf79291 /doc/stdlib
parent2de683db51b44b8051ead6d89be67f0185e7e87d (diff)
A better Program documentation. Include it in the generated stdlib doc.
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@10061 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'doc/stdlib')
-rwxr-xr-xdoc/stdlib/Library.tex2
-rw-r--r--doc/stdlib/index-list.html.template12
-rwxr-xr-xdoc/stdlib/make-library-files2
-rwxr-xr-xdoc/stdlib/make-library-index2
4 files changed, 16 insertions, 2 deletions
diff --git a/doc/stdlib/Library.tex b/doc/stdlib/Library.tex
index fffcddc85..81fdd2a6e 100755
--- a/doc/stdlib/Library.tex
+++ b/doc/stdlib/Library.tex
@@ -45,6 +45,8 @@ The standard library is composed of the following subdirectories:
\item[Wellfounded] Well-founded relations (basic results).
\item[IntMap] Representation of finite sets by an efficient
structure of map (trees indexed by binary integers).
+ \item[Program] Tactcis to deal with dependently-typed programs and
+ their proofs.
\end{description}
diff --git a/doc/stdlib/index-list.html.template b/doc/stdlib/index-list.html.template
index 2a8693438..65d69a1d8 100644
--- a/doc/stdlib/index-list.html.template
+++ b/doc/stdlib/index-list.html.template
@@ -402,5 +402,17 @@ through the <tt>Require Import</tt> command.</p>
theories/Ints/num/ZnZ.v
</dd>
+
+ <dt> <b>Program</b>:
+ Support for dependently-typed programming.
+ </dt>
+ <dd>
+ theories/Program/Wf.v
+ theories/Program/Equality.v
+ theories/Program/Tactics.v
+ theories/Program/Utils.v
+ theories/Program/Program.v
+ theories/Program/FunctionalExtensionality.v
+ </dd>
</dl>
diff --git a/doc/stdlib/make-library-files b/doc/stdlib/make-library-files
index 91e3cc3f4..6eb1333a5 100755
--- a/doc/stdlib/make-library-files
+++ b/doc/stdlib/make-library-files
@@ -10,7 +10,7 @@
# En supposant que make fait son boulot, ca fait un tri topologique du
# graphe des dépendances
-LIBDIRS="Arith NArith ZArith Reals Logic Bool Lists IntMap Relations Sets Sorting Wellfounded Setoids"
+LIBDIRS="Arith NArith ZArith Reals Logic Bool Lists IntMap Relations Sets Sorting Wellfounded Setoids Program"
rm -f library.files.ls.tmp
(cd $COQTOP/theories; find $LIBDIR -name "*.v" -ls) > library.files.ls.tmp
diff --git a/doc/stdlib/make-library-index b/doc/stdlib/make-library-index
index cbcd15ef3..27dfc434f 100755
--- a/doc/stdlib/make-library-index
+++ b/doc/stdlib/make-library-index
@@ -7,7 +7,7 @@ FILE=$1
cp -f $FILE.template tmp
echo -n Building file index-list.prehtml ...
-LIBDIRS="Init Logic Bool Arith NArith ZArith QArith Relations Sets Setoids Lists Sorting Wellfounded IntMap FSets Reals Ints Ints/num"
+LIBDIRS="Init Logic Bool Arith NArith ZArith QArith Relations Sets Setoids Lists Sorting Wellfounded IntMap FSets Reals Ints Ints/num Program"
for k in $LIBDIRS; do
i=../theories/$k