From 484a0c35662d3bb78aa1f2cd83ffcc1b1f761968 Mon Sep 17 00:00:00 2001 From: Pierre Letouzey Date: Fri, 5 Dec 2014 16:28:15 +0100 Subject: doc/stdlib: fix the xhtml validity of the index-list template --- doc/stdlib/index-list.html.template | 87 ++++++++++++++++++++----------------- 1 file changed, 47 insertions(+), 40 deletions(-) (limited to 'doc/stdlib') diff --git a/doc/stdlib/index-list.html.template b/doc/stdlib/index-list.html.template index 9873dd071..854c786c1 100644 --- a/doc/stdlib/index-list.html.template +++ b/doc/stdlib/index-list.html.template @@ -3,7 +3,7 @@

Here is a short description of the Coq standard library, which is distributed with the system. -It provides a set of modules directly available +It provides a set of modules directly available through the Require Import command.

The standard library is composed of the following subdirectories:

@@ -12,7 +12,7 @@ through the Require Import command.

Init: The core library (automatically loaded when starting Coq)
-
+
theories/Init/Notations.v theories/Init/Datatypes.v theories/Init/Logic.v @@ -24,7 +24,7 @@ through the Require Import command.

theories/Init/Wf.v (theories/Init/Prelude.v)
- +
Logic: Classical logic, dependent equality, extensionality, choice axioms
@@ -60,7 +60,7 @@ through the Require Import command.

theories/Logic/WKL.v theories/Logic/FinFun.v - +
Structures: Algebraic structures (types with equality, with order, ...). DecidableType* and OrderedType* are there only for compatibility. @@ -85,7 +85,7 @@ through the Require Import command.

Bool: Booleans (basic functions and results)
-
+
theories/Bool/Bool.v theories/Bool/BoolEq.v theories/Bool/DecBool.v @@ -94,7 +94,7 @@ through the Require Import command.

theories/Bool/Zerob.v theories/Bool/Bvector.v
- +
Arith: Basic Peano arithmetic
@@ -207,10 +207,13 @@ through the Require Import command.

theories/QArith/Qminmax.v -
Numbers: +
Numbers: An experimental modular architecture for arithmetic
-
  Prelude: +
+
+
  Prelude: +
theories/Numbers/BinNums.v theories/Numbers/NumPrelude.v @@ -220,6 +223,7 @@ through the Require Import command.

  NatInt: Abstract mixed natural/integer/cyclic arithmetic +
theories/Numbers/NatInt/NZAdd.v theories/Numbers/NatInt/NZAddOrder.v @@ -238,10 +242,10 @@ through the Require Import command.

theories/Numbers/NatInt/NZGcd.v theories/Numbers/NatInt/NZBits.v
- -
  Cyclic: +
  Cyclic: Abstract and 31-bits-based cyclic arithmetic +
theories/Numbers/Cyclic/Abstract/CyclicAxioms.v theories/Numbers/Cyclic/Abstract/NZCyclic.v @@ -260,10 +264,10 @@ through the Require Import command.

theories/Numbers/Cyclic/Int31/Int31.v theories/Numbers/Cyclic/ZModulo/ZModulo.v
- -
  Natural: +
  Natural: Abstract and 31-bits-words-based natural arithmetic +
theories/Numbers/Natural/Abstract/NAdd.v theories/Numbers/Natural/Abstract/NAddOrder.v @@ -294,10 +298,11 @@ through the Require Import command.

theories/Numbers/Natural/BigN/NMake.v theories/Numbers/Natural/BigN/NMake_gen.v
- -
  Integer: - Abstract and concrete (especially 31-bits-words-based) integer arithmetic +
  Integer: + Abstract and concrete (especially 31-bits-words-based) integer + arithmetic +
theories/Numbers/Integer/Abstract/ZAdd.v theories/Numbers/Integer/Abstract/ZAddOrder.v @@ -324,32 +329,32 @@ through the Require Import command.

theories/Numbers/Integer/BigZ/BigZ.v theories/Numbers/Integer/BigZ/ZMake.v
-
  Rational: Abstract and 31-bits-words-based rational arithmetic +
theories/Numbers/Rational/SpecViaQ/QSig.v theories/Numbers/Rational/BigQ/BigQ.v theories/Numbers/Rational/BigQ/QMake.v
- - - +
+
+
Relations: Relations (definitions and basic results)
-
+
theories/Relations/Relation_Definitions.v theories/Relations/Relation_Operators.v theories/Relations/Relations.v theories/Relations/Operators_Properties.v
- +
Sets: Sets (classical, constructive, finite, infinite, powerset, etc.)
-
+
theories/Sets/Classical_sets.v theories/Sets/Constructive_sets.v theories/Sets/Cpo.v @@ -373,9 +378,10 @@ through the Require Import command.

theories/Sets/Relations_3.v theories/Sets/Uniset.v
- +
Classes: -
+ +
theories/Classes/Init.v theories/Classes/RelationClasses.v theories/Classes/Morphisms.v @@ -394,14 +400,15 @@ through the Require Import command.

Setoids: -
+ +
theories/Setoids/Setoid.v
- +
Lists: Polymorphic lists, Streams (infinite sequences)
-
+
theories/Lists/List.v theories/Lists/ListDec.v theories/Lists/ListSet.v @@ -415,18 +422,18 @@ through the Require Import command.

Vectors: Dependent datastructures storing their length
-
- theories/Vectors/Fin.v - theories/Vectors/VectorDef.v - theories/Vectors/VectorSpec.v - theories/Vectors/VectorEq.v - (theories/Vectors/Vector.v) -
+
+ theories/Vectors/Fin.v + theories/Vectors/VectorDef.v + theories/Vectors/VectorSpec.v + theories/Vectors/VectorEq.v + (theories/Vectors/Vector.v) +
Sorting: Axiomatizations of sorts
-
+
theories/Sorting/Heap.v theories/Sorting/Permutation.v theories/Sorting/Sorting.v @@ -439,7 +446,7 @@ through the Require Import command.

Wellfounded: Well-founded Relations
-
+
theories/Wellfounded/Disjoint_Union.v theories/Wellfounded/Inclusion.v theories/Wellfounded/Inverse_Image.v @@ -507,11 +514,11 @@ through the Require Import command.

theories/Strings/Ascii.v theories/Strings/String.v
- +
Reals: Formalization of real numbers
-
+
theories/Reals/Rdefinitions.v theories/Reals/Raxioms.v theories/Reals/RIneq.v @@ -575,11 +582,11 @@ through the Require Import command.

theories/Reals/Rlogic.v (theories/Reals/Reals.v)
- +
Program: Support for dependently-typed programming.
-
+
theories/Program/Basics.v theories/Program/Wf.v theories/Program/Subset.v -- cgit v1.2.3