aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Lists
diff options
context:
space:
mode:
authorGravatar pboutill <pboutill@85f007b7-540e-0410-9357-904b9bb8a0f7>2011-09-02 15:59:22 +0000
committerGravatar pboutill <pboutill@85f007b7-540e-0410-9357-904b9bb8a0f7>2011-09-02 15:59:22 +0000
commit041e70dd5f0ed46a01229a2f352e5d2ddecda518 (patch)
treee5a50e91c21183e7ba426a20492eae8c6dbd9d2d /theories/Lists
parent95e60e7769f8fcf25e44774b78a4be17b7e4fb3c (diff)
Bug 2589: Documentation patch of Hendrik Tews
+ s/cbv/lazy of bug 2542 git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@14446 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Lists')
-rw-r--r--theories/Lists/List.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/Lists/List.v b/theories/Lists/List.v
index 84e145271..ecadddbc8 100644
--- a/theories/Lists/List.v
+++ b/theories/Lists/List.v
@@ -259,7 +259,7 @@ Section Facts.
Qed.
- (** Compatibility wtih other operations *)
+ (** Compatibility with other operations *)
Lemma app_length : forall l l' : list A, length (l++l') = length l + length l'.
Proof.