aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Lists
diff options
context:
space:
mode:
authorGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2015-10-15 09:47:43 +0200
committerGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2015-10-15 09:47:43 +0200
commitcbd28511526dfb561017c3d27a73598f6ce5f68d (patch)
treea8786b32433caa850e24f67ab5a3aa85f29a683a /theories/Lists
parent10e5883fed21f9631e1aa65adb7a7e62a529987f (diff)
parent7402a7788b6a73bd5c0cb9078823d48e6f01a357 (diff)
Merge branch 'v8.5'
Diffstat (limited to 'theories/Lists')
-rw-r--r--theories/Lists/List.v8
1 files changed, 4 insertions, 4 deletions
diff --git a/theories/Lists/List.v b/theories/Lists/List.v
index 2437184a9..45306caf0 100644
--- a/theories/Lists/List.v
+++ b/theories/Lists/List.v
@@ -69,7 +69,7 @@ Section Facts.
Variable A : Type.
- (** *** Genereric facts *)
+ (** *** Generic facts *)
(** Discrimination *)
Theorem nil_cons : forall (x:A) (l:list A), [] <> x :: l.
@@ -622,9 +622,9 @@ Section Elts.
Qed.
- (****************************************)
- (** ** Counting occurences of a element *)
- (****************************************)
+ (******************************************)
+ (** ** Counting occurrences of an element *)
+ (******************************************)
Fixpoint count_occ (l : list A) (x : A) : nat :=
match l with