summaryrefslogtreecommitdiff
path: root/theories/Numbers/NaryFunctions.v
diff options
context:
space:
mode:
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 6fdf0a2a..376620dd 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