diff options
| author | Antonio Nikishaev | 2020-04-08 00:32:35 +0400 |
|---|---|---|
| committer | Antonio Nikishaev | 2020-04-08 01:34:03 +0400 |
| commit | bfd4b28b835e6918d7f4dea848c8b94f4c1c6f7f (patch) | |
| tree | 5eda6b55c8907856c311c798b8ff5dc8fb7ca82c /mathcomp/ssreflect/binomial.v | |
| parent | 815d3cbfa2bf98b4b8f2bcd14819a20eca843e78 (diff) | |
fix typos in documentation: formulae
Diffstat (limited to 'mathcomp/ssreflect/binomial.v')
| -rw-r--r-- | mathcomp/ssreflect/binomial.v | 2 |
1 files changed, 1 insertions, 1 deletions
diff --git a/mathcomp/ssreflect/binomial.v b/mathcomp/ssreflect/binomial.v index 2af7953..aef8e27 100644 --- a/mathcomp/ssreflect/binomial.v +++ b/mathcomp/ssreflect/binomial.v @@ -8,7 +8,7 @@ From mathcomp Require Import div fintype tuple finfun bigop prime finset. (* '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/!. *) +(* Note that n ^_ m = 0 if m > n, and 'C(n, m) = n ^_ m %/ m`!. *) (* *) (* In additions to the properties of these functions, we prove a few seminal *) (* results such as triangular_sum, Wilson and Pascal; their proofs are good *) |
