aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Numbers/NaryFunctions.v
diff options
context:
space:
mode:
authorGravatar Guillaume Melquiond <guillaume.melquiond@inria.fr>2015-10-13 18:30:47 +0200
committerGravatar Guillaume Melquiond <guillaume.melquiond@inria.fr>2015-10-13 18:30:47 +0200
commited95f122f3c68becc09c653471dc2982b346d343 (patch)
tree87e323b2d382c285e1eae864338ea397fda0923d /theories/Numbers/NaryFunctions.v
parent26974a4a2301cc7b1188a3f2f29f3d3368eccc0b (diff)
Fix some typos.
Diffstat (limited to 'theories/Numbers/NaryFunctions.v')
-rw-r--r--theories/Numbers/NaryFunctions.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/Numbers/NaryFunctions.v b/theories/Numbers/NaryFunctions.v
index 6fdf0a2a5..376620ddc 100644
--- a/theories/Numbers/NaryFunctions.v
+++ b/theories/Numbers/NaryFunctions.v
@@ -15,7 +15,7 @@ Require Import List.
(** * Generic dependently-typed operators about [n]-ary functions *)
(** The type of [n]-ary function: [nfun A n B] is
- [A -> ... -> A -> B] with [n] occurences of [A] in this type. *)
+ [A -> ... -> A -> B] with [n] occurrences of [A] in this type. *)
Fixpoint nfun A n B :=
match n with