aboutsummaryrefslogtreecommitdiff
path: root/mathcomp/ssreflect/binomial.v
diff options
context:
space:
mode:
authorAntonio Nikishaev2020-04-05 02:54:23 +0400
committerAntonio Nikishaev2020-04-08 01:13:13 +0400
commit815d3cbfa2bf98b4b8f2bcd14819a20eca843e78 (patch)
treed3564d7ccb62b38493fde1a0fc23ff94410074ec /mathcomp/ssreflect/binomial.v
parent14e28e78155e3e6cfbe78aee0964569283f04d7d (diff)
fix typos in documentation: text
Diffstat (limited to 'mathcomp/ssreflect/binomial.v')
-rw-r--r--mathcomp/ssreflect/binomial.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/mathcomp/ssreflect/binomial.v b/mathcomp/ssreflect/binomial.v
index 3a484a1..2af7953 100644
--- a/mathcomp/ssreflect/binomial.v
+++ b/mathcomp/ssreflect/binomial.v
@@ -5,7 +5,7 @@ From mathcomp Require Import div fintype tuple finfun bigop prime finset.
(******************************************************************************)
(* This files contains the definition of: *)
-(* 'C(n, m) == the binomial coeficient n choose m. *)
+(* 'C(n, m) == the binomial coefficient n choose m. *)
(* n ^_ m == the falling (or lower) factorial of n with m terms, i.e., *)
(* the product n * (n - 1) * ... * (n - m + 1). *)
(* Note that n ^_ m = 0 if m > n, and 'C(n, m) = n ^_ m %/ m/!. *)