diff options
| author | Matthieu Sozeau | 2013-11-30 13:41:39 +0100 |
|---|---|---|
| committer | Matthieu Sozeau | 2014-05-06 09:58:56 +0200 |
| commit | 12fd678c3cf163f76110b3b5edeb8a8bcfa82787 (patch) | |
| tree | 6b3609126c16260c6222510f741185161e8c79ff /doc/stdlib | |
| parent | cd11c5d2ff5d91603a6043a667e5918e99ef303a (diff) | |
- Fix index-list to show computational relations for rewriting files.
- Fix hasheq which didn't have a case for Proj making hashconsing exponentially slower.
Conflicts:
kernel/constr.ml
kernel/univ.ml
proofs/proof_global.ml
Diffstat (limited to 'doc/stdlib')
| -rw-r--r-- | doc/stdlib/index-list.html.template | 3 |
1 files changed, 3 insertions, 0 deletions
diff --git a/doc/stdlib/index-list.html.template b/doc/stdlib/index-list.html.template index 1f8ff94e1b..d774ed5974 100644 --- a/doc/stdlib/index-list.html.template +++ b/doc/stdlib/index-list.html.template @@ -393,6 +393,9 @@ through the <tt>Require Import</tt> command.</p> theories/Classes/Morphisms_Prop.v theories/Classes/Morphisms_Relations.v theories/Classes/Equivalence.v + theories/Classes/CRelationClasses.v + theories/Classes/CMorphisms.v + theories/Classes/CEquivalence.v theories/Classes/EquivDec.v theories/Classes/SetoidTactics.v theories/Classes/SetoidClass.v |
