aboutsummaryrefslogtreecommitdiffhomepage
path: root/doc/stdlib
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2013-06-02 21:42:14 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2013-06-02 21:42:14 +0000
commitfe008055f8adc7acd6af1483a8e7fef98d27e267 (patch)
treed484eb859c9210babdd9408fa46c21ca671ebd2d /doc/stdlib
parentd51d98682fcff981a1e6b95574c25fc7edf97b3f (diff)
A constructive proof of Fan theorem where paths are represented by predicates.
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@16557 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'doc/stdlib')
-rw-r--r--doc/stdlib/index-list.html.template3
1 files changed, 2 insertions, 1 deletions
diff --git a/doc/stdlib/index-list.html.template b/doc/stdlib/index-list.html.template
index b7a76b94f..9382a0890 100644
--- a/doc/stdlib/index-list.html.template
+++ b/doc/stdlib/index-list.html.template
@@ -37,7 +37,7 @@ through the <tt>Require Import</tt> command.</p>
</dd>
<dt> <b>Logic</b>:
- Classical logic and dependent equality
+ Classical logic, dependent equality, extensionality, choice axioms
</dt>
<dd>
theories/Logic/SetIsType.v
@@ -69,6 +69,7 @@ through the <tt>Require Import</tt> command.</p>
theories/Logic/IndefiniteDescription.v
theories/Logic/FunctionalExtensionality.v
theories/Logic/ExtensionalityFacts.v
+ theories/Logic/Fan.v
</dd>
<dt> <b>Structures</b>: