login
Search: a005993 -id:a005993
     Sort: relevance | references | number | modified | created      Format: long | short | data
Rows of Losanitsch's triangle T(n, k), n >= 0, 0 <= k <= n.
+10
68
1, 1, 1, 1, 1, 1, 1, 2, 2, 1, 1, 2, 4, 2, 1, 1, 3, 6, 6, 3, 1, 1, 3, 9, 10, 9, 3, 1, 1, 4, 12, 19, 19, 12, 4, 1, 1, 4, 16, 28, 38, 28, 16, 4, 1, 1, 5, 20, 44, 66, 66, 44, 20, 5, 1, 1, 5, 25, 60, 110, 126, 110, 60, 25, 5, 1, 1, 6, 30, 85, 170, 236, 236, 170, 85, 30, 6, 1, 1, 6, 36, 110, 255
OFFSET
0,8
COMMENTS
Sometimes erroneously called "Lossnitsch's triangle". But the author's name is Losanitsch (I have seen the original paper in Chem. Ber.). This is a German version of the Serbian name Lozanic. - N. J. A. Sloane, Jun 29 2008
For n >= 3, a(n-3,k) is the number of series-reduced (or homeomorphically irreducible) trees which become a path P(k+1) on k+1 nodes, k >= 0, when all leaves are omitted (see illustration). Proof by Pólya's enumeration theorem. - Wolfdieter Lang, Jun 08 2001
The number of ways to put beads of two colors in a line, but take symmetry into consideration, so that 011 and 110 are considered the same. - Yong Kong (ykong(AT)nus.edu.sg), Jan 04 2005
Alternating row sums are 1,0,1,0,2,0,4,0,8,0,16,0,... - Gerald McGarvey, Oct 20 2008
The triangle sums, see A180662 for their definitions, link Losanitsch's triangle A034851 with several sequences, see the crossrefs. We observe that the Ze3 and Ze4 sums link Losanitsch's triangle with A005683, i.e., R. K. Guy's Twopins game. - Johannes W. Meijer, Jul 14 2011
T(n-(L-1)k, k) is the number of ways to cover an n-length line by exactly k L-length segments excluding symmetric covers. For L=2 it is corresponds to A102541, for L=3 to A228570 and for L=4 to A228572. - Philipp O. Tsvetkov, Nov 08 2013
Also the number of equivalence classes of ways of placing k 1 X 1 tiles in an n X 1 rectangle under all symmetry operations of the rectangle. - Christopher Hunt Gribble, Feb 16 2014
T(n, k) is the number of non-isomorphic outer planar graphs of order n+3, size n+3+k, and maximum degree k+2. - Christian Barrientos, Oct 18 2018
From Álvar Ibeas, Jun 01 2020: (Start)
T(n, k) is the sum of even-degree coefficients of the Gaussian polynomial [n, k]_q. The area below a NE lattice path between (0,0) and (k, n-k) is even for T(n, k) paths and odd for A034852(n, k) of them.
For a (non-reversible) string of k black and n-k white beads, consider the minimum number of bead transpositions needed to place the black ones to the left and the white ones to the right (in other words, the number of inversions of the permutation obtained by labeling the black beads by integers 1,...,k and the white ones by k+1,...,n, in the same order they take on the string). It is even for T(n, k) strings and odd for A034852(n, k) cases.
(End)
Named after the Serbian chemist, politician and diplomat Simeon Milivoje "Sima" Lozanić (1847-1935). - Amiram Eldar, Jun 10 2021
T(n, k) is the number of caterpillars with a perfect matching, with 2n+2 vertices and diameter 2n-1-k. - Christian Barrientos, Sep 12 2023
LINKS
F. Al-Kharousi, R. Kehinde, and A. Umar, Combinatorial results for certain semigroups of partial isometries of a finite chain, The Australasian Journal of Combinatorics, Vol. 58, No. 3 (2014), pp. 363-375.
Tewodros Amdeberhan, Mahir Bilen Can and Victor H. Moll, Broken bracelets, Molien series, paraffin wax and the elliptic curve of conductor 48, SIAM Journal of Discrete Math., Vol. 25, No. 4 (2011), p. 1843-1859; arXiv preprint, arXiv:1106.4693 [math.CO], 2011. See Theorem 2.8.
Johann Cigler, Some remarks on Rogers-Szegö polynomials and Losanitsch's triangle, arXiv:1711.03340 [math.CO], 2017.
Sahir Gill, Bounds for Region Containing All Zeros of a Complex Polynomial, International Journal of Mathematical Analysis Vol. 12, No. 7 (2018), pp. 325-333.
Stephen G. Hartke and A. J. Radcliffe, Signatures of Strings, Annals of Combinatorics, Vol. 17, No. 1 (March, 2013), pp. 131-150.
Rethinasamy K. Kittappa, Combinatorial enumeration of rectangular kolam designs of the Tamil land, Abstracts Amer. Math. Soc., Vol. 29, No. 1 (2008), p. 24 (Abstract 1035-05-543).
S. M. Losanitsch, Die Isomerie-Arten bei den Homologen der Paraffin-Reihe, Chem. Ber. Vol. 30 (1897), pp. 1917-1926.
S. M. Losanitsch, Die Isomerie-Arten bei den Homologen der Paraffin-Reihe, Chem. Ber., Vol. 30 (1897), pp. 1917-1926. (Annotated scanned copy)
Jesse Pajwani, Herman Rohrbach, and Anna M. Viergever, Compactly supported A^1-Euler characteristics of symmetric powers of cellular varieties, arXiv:2404.08486 [math.AG], 2024. See p. 15.
N. J. A. Sloane, Classic Sequences.
Eric Weisstein's World of Mathematics, Losanitsch's Triangle.
Wikipedia, Sima Lozanic.
FORMULA
T(n, k) = (1/2) * (A007318(n, k) + A051159(n, k)).
G.f. for k-th column (if formatted as lower triangular matrix a(n, k)): x^k*Pe(floor((k+1)/2), x^2)/(((1-x)^(k+1))*(1+x)^(floor((k+1)/2))), where Pe(n, x^2) := Sum_{m=0..floor(n/2)} A034839(n, m)*x^(2*m) (row polynomials of Pascal array even numbered columns). - Wolfdieter Lang, May 08 2001
a(n, k) = a(n-1, k-1) + a(n-1, k) - C(n/2-1, (k-1)/2), where the last term is present only if n is even and k is odd (see Sloane link).
T(n, k) = T(n-2, k-2) + T(n-2, k) + C(n-2, k-1), n > 1.
Let P(n, x, y) = Sum_{m=0..n} a(n, m)*x^m*y^(n-m), then for x > 0, y > 0 we have P(n, x, y) = (x+y)*P(n-1, x, y) for n odd and P(n, x, y) = (x+y)*P(n-1, x, y) - x*y*(x^2+y^2)^((n-2)/2) for n even. - Gerald McGarvey, Feb 15 2005
T(n, k) = T(n-1, k-1) + T(n-1, k) - A204293(n-2, k-1), 0 < k <= n and n > 1. - Reinhard Zumkeller, Jan 14 2012
From Christopher Hunt Gribble, Feb 25 2014: (Start)
It appears that:
T(n,k) = C(n,k)/2, n even, k odd;
T(n,k) = (C(n,k) + C(n/2,k/2))/2, n even, k even;
T(n,k) = (C(n,k) + C((n-1)/2,(k-1)/2))/2, n odd, k odd;
T(n,k) = (C(n,k) + C((n-1)/2,k/2))/2, n odd, k even.
(End)
EXAMPLE
Triangle begins
1;
1, 1;
1, 1, 1;
1, 2, 2, 1;
1, 2, 4, 2, 1;
1, 3, 6, 6, 3, 1;
1, 3, 9, 10, 9, 3, 1;
1, 4, 12, 19, 19, 12, 4, 1;
1, 4, 16, 28, 38, 28, 16, 4, 1;
1, 5, 20, 44, 66, 66, 44, 20, 5, 1;
MAPLE
A034851 := proc(n, k) option remember; local t; if k = 0 or k = n then return(1) fi; if n mod 2 = 0 and k mod 2 = 1 then t := binomial(n/2-1, (k-1)/2) else t := 0; fi; A034851(n-1, k-1)+A034851(n-1, k)-t; end: seq(seq(A034851(n, k), k=0..n), n=0..11);
MATHEMATICA
t[n_?EvenQ, k_?OddQ] := Binomial[n, k]/2; t[n_, k_] := (Binomial[n, k] + Binomial[Quotient[n, 2], Quotient[k, 2]])/2; Flatten[Table[t[n, k], {n, 0, 12}, {k, 0, n}]](* Jean-François Alcover, Feb 07 2012, after PARI *)
PROG
(PARI) {T(n, k) = (1/2) *(binomial(n, k) + binomial(n%2, k%2) * binomial(n\2, k\2))}; /* Michael Somos, Oct 20 1999 */
(Haskell)
a034851 n k = a034851_row n !! k
a034851_row 0 = [1]
a034851_row 1 = [1, 1]
a034851_row n = zipWith (-) (zipWith (+) ([0] ++ losa) (losa ++ [0]))
([0] ++ a204293_row (n-2) ++ [0])
where losa = a034851_row (n-1)
a034851_tabl = map a034851_row [0..]
-- Reinhard Zumkeller, Jan 14 2012
CROSSREFS
Triangle sums (see the comments): A005418 (Row), A011782 (Related to Row2), A102526 (Related to Kn11, Kn12, Kn13, Kn21, Kn22, Kn23), A005207 (Kn3, Kn4), A005418 (Fi1, Fi2), A102543 (Ca1, Ca2), A192928 (Gi1, Gi2), A005683 (Ze3, Ze4).
Sums of squares of terms in rows equal A211208.
KEYWORD
nonn,tabl,easy,nice
EXTENSIONS
More terms from James A. Sellers, May 04 2000
Name edited by Johannes W. Meijer, Aug 26 2013
STATUS
approved
Triangle read by rows giving coefficient T(i,j) of x^i y^j in 1/(1-y-x*y-x^2) = 1/((1+x)(1-x-y)) for (i,j) = (0,0), (1,0), (0,1), (2,0), (1,1), (0,2), ...
+10
26
1, 0, 1, 1, 1, 1, 0, 2, 2, 1, 1, 2, 4, 3, 1, 0, 3, 6, 7, 4, 1, 1, 3, 9, 13, 11, 5, 1, 0, 4, 12, 22, 24, 16, 6, 1, 1, 4, 16, 34, 46, 40, 22, 7, 1, 0, 5, 20, 50, 80, 86, 62, 29, 8, 1, 1, 5, 25, 70, 130, 166, 148, 91, 37, 9, 1, 0, 6, 30, 95, 200, 296, 314, 239, 128, 46, 10, 1
OFFSET
0,8
COMMENTS
Coefficients of the (left, normalized) shifted cyclotomic polynomial. Or, coefficients of the basic n-th q-series for q=-2. Indeed, let Y_n(x) = Sum_{k=0..n} x^k, having as roots all the n-th roots of unity except for 0; then coefficients in x of (-1)^n Y_n(-x-1) give exactly the n-th row of A059260 and a practical way to compute it. - Olivier Gérard, Jul 30 2002
The maximum in the (2n)-th row is T(n,n), which is A026641; also T(n,n) ~ (2/3)*binomial(2n,n). The maximum in the (2n-1)-th row is T(n-1,n), which is A014300 (but T does not have the same definition as in A026637); also T(n-1,n) ~ (1/3)*binomial(2n,n). Here is a generalization of the formula given in A026641: T(i,j) = Sum_{k=0..j} binomial(i+k-x,j-k)*binomial(j-k+x,k) for all x real (the proof is easy by induction on i+j using T(i,j) = T(i-1,j) + T(i,j-1)). - Claude Morin, May 21 2002
The second greatest term in the (2n)-th row is T(n-1,n+1), which is A014301; the second greatest term in the (2n+1)-th row is T(n+1,n) = 2*T(n-1,n+1), which is 2*A014301. - Claude Morin
Diagonal sums give A008346. - Paul Barry, Sep 23 2004
Riordan array (1/(1-x^2), x/(1-x)). As a product of Riordan arrays, factors into the product of (1/(1+x),x) and (1/(1-x),1/(1-x)) (binomial matrix). - Paul Barry, Oct 25 2004
Signed version is A239473 with relations to partial sums of sequences. - Tom Copeland, Mar 24 2014
From Robert Coquereaux, Oct 01 2014: (Start)
Columns of the triangle (cf. Example below) give alternate partial sums along nw-se diagonals of the Pascal triangle, i.e., sequences A000035, A004526, A002620 (or A087811), A002623 (or A173196), A001752, A001753, A001769, A001779, A001780, A001781, A001786, A001808, etc.
The dimension of the space of closed currents (distributional forms) of degree p on Gr(n), the Grassmann algebra with n generators, equivalently, the dimension of the space of Gr(n)-valued symmetric multilinear forms with vanishing graded divergence, is V(n,p) = 2^n T(p,n-1) - (-1)^p.
If p is odd V(n,p) is also the dimension of the cyclic cohomology group of order p of the Z2 graded algebra Gr(n).
If p is even the dimension of this cohomology group is V(n,p)+1.
Cf. A193844. (End)
From Peter Bala, Feb 07 2024: (Start)
The following remarks assume the row indexing starts at n = 1.
The sequence of row polynomials R(n,x), beginning R(1,x) = 1, R(2,x) = x, R(3,x) = 1 + x + x^2 , ..., is a strong divisibility sequence of polynomials in the ring Z[x]; that is, for all positive integers n and m, poly_gcd( R(n,x), R(m,x)) = R(gcd(n, m), x) - apply Norfleet (2005), Theorem 3. Consequently, the polynomial sequence {R(n,x): n >= 1} is a divisibility sequence; that is, if n divides m then R(n,x) divides R(m,x) in Z[x]. (End)
From Miquel A. Fiol, Oct 04 2024 (Start):
For j>=1, T(i,j) is the independence number of the (i-j)-supertoken graph FF_(i-j)(S_j) of the star graph S_j with j points.
(Given a graph G on n vertices and an integer k>=1, the k-supertoken (or reduced k-th power) FF_k(G) of G has vertices representing configurations of k indistinguishable tokens in the (not necessarily different) vertices of G, with two configurations being adjacent if one can be obtained from the other by moving one token along an edge. See an example below.)
Following the suggestion of Peter Munn, the k-supertoken graph FF_k(S_j) can also be defined as follows: Consider the Lattice graph L(k,j), whose vertices are the k^j j-vectors with elements in the set {0,..,k-1}, two being adjacent if they differ in just one coordinate by one unity. Then, FF_k(S_j) is the subgraph of L(k+1,j) induced by the vertices at distance at most k from (0,..,0).
End
LINKS
Roland Bacher, Chebyshev polynomials, quadratic surds and a variation of Pascal's triangle, arXiv:1509.09054 [math.CO], 2015.
Joseph Briggs, Alex Parker, Coy Schwieder, and Chris Wells, Frogs, hats and common subsequences, arXiv:2404.07285 [math.CO], 2024. See p. 28.
Robert Coquereaux and Éric Ragoucy, Currents on Grassmann algebras, J. of Geometry and Physics, 1995, Vol 15, pp 333-352.
Robert Coquereaux and Éric Ragoucy, Currents on Grassmann algebras, arXiv:hep-th/9310147, 1993.
Robert Coquereaux and Jean-Bernard Zuber, Counting partitions by genus. II. A compendium of results, arXiv:2305.01100 [math.CO], 2023. See p. 8.
R. H. Hammack and G. D. Smith, Cycle bases of reduced powers of graphs, Ars Math. Contemp. 12 (2017) 183-203.
Christian Kassel, A Künneth formula for the cyclic cohomology of Z2-graded algebras, Math. Ann. 275 (1986) 683.
Ana Filipa Loureiro and Pascal Maroni, Polynomial sequences associated with the classical linear functionals, Numerical Algorithms, June 2012, Volume 60, Issue 2, pp 297-314. - From N. J. A. Sloane, Oct 12 2012
Ana Filipa Loureiro and Pascal Maroni, Polynomial sequences associated with the classical linear functionals, preprint, Centro de Matemática da Universidade do Porto.
Mark Norfleet, Characterization of second-order strong divisibility sequences of polynomials, The Fibonacci Quarterly, 43(2) (2005), 166-169.
FORMULA
G.f.: 1/(1-y-x*y-x^2) = 1 + y + x^2 + xy + y^2 + 2x^2y + 2xy^2 + y^3 + ...
E.g.f: (exp(-t)+(x+1)*exp((x+1)*t))/(x+2). - Tom Copeland, Mar 19 2014
O.g.f. (n-th row): ((-1)^n+(x+1)^(n+1))/(x+2). - Tom Copeland, Mar 19 2014
T(i, 0) = 1 if i is even or 0 if i is odd, T(0, i) = 1 and otherwise T(i, j) = T(i-1, j) + T(i, j-1); also T(i, j) = Sum_{m=j..i+j} (-1)^(i+j+m)*binomial(m, j). - Robert FERREOL, May 17 2002
T(i, j) ~ (i+j)/(2*i+j)*binomial(i+j, j); more precisely, abs(T(i, j)/binomial(i+j, j) - (i+j)/(2*i+j) )<=1/(4*(i+j)-2); the proof is by induction on i+j using the formula 2*T(i, j) = binomial(i+j, j)+T(i, j-1). - Claude Morin, May 21 2002
T(n, k) = Sum_{j=0..n} (-1)^(n-j)binomial(j, k). - Paul Barry, Aug 25 2004
T(n, k) = Sum_{j=0..n-k} binomial(n-j, j)*binomial(j, n-k-j). - Paul Barry, Jul 25 2005
Equals A097807 * A007318. - Gary W. Adamson, Feb 21 2007
Equals A128173 * A007318 as infinite lower triangular matrices. - Gary W. Adamson, Feb 17 2007
Equals A130595*A097805*A007318 = (inverse Pascal matrix)*(padded Pascal matrix)*(Pascal matrix) = A130595*A200139. Inverse is A097808 = A130595*(padded A130595)*A007318. - Tom Copeland, Nov 14 2016
T(i, j) = binomial(i+j, j)-T(i-1, j). - Laszlo Major, Apr 11 2017
Recurrence for row polynomials (with row indexing starting at n = 1): R(n,x) = x*R(n-1,x) + (x + 1)*R(n-2,x) with R(1,x) = 1 and R(2,x) = x. - Peter Bala, Feb 07 2024
From Miquel A. Fiol, Sep 30 2024 (Start):
The triangle can be seen as a slice of a 3-dimensional table that links it to well-known sequences as follows.
The j-th column of the triangle, T(i,j) for i >= j, equals A(n,c1,c2) = Sum_{k=0..floor(n/2)} binomial(c1+2*k-1,2*k)*binomial(c2+n-2*k-1,n-2*k) when c1=1, c2=j, and n=i-j.
This gives T(i,j) = Sum_{k=0..floor((i-j)/2)} binomial(i-2*k-1, j-1). For other values of (c1,c2), see the example below.
(End)
EXAMPLE
Triangle begins
1;
0, 1;
1, 1, 1;
0, 2, 2, 1;
1, 2, 4, 3, 1;
0, 3, 6, 7, 4, 1;
1, 3, 9, 13, 11, 5, 1;
0, 4, 12, 22, 24, 16, 6, 1;
1, 4, 16, 34, 46, 40, 22, 7, 1;
0, 5, 20, 50, 80, 86, 62, 29, 8, 1;
Sequences obtained with Miquel A. Fiol's Sep 30 2024 formula of A(n,c1,c2) for other values of (c1,c2). (In the table, rows are indexed by c1=0..6 and columns by c2=0..6):
A193356 A008794* A005993 A005994 ------- ------- -------
------- ------- ------- A005995 A018210 ------- A052267
------- ------- ------- ------- A018211 A018212 -------
------- ------- ------- ------- ------- A018213 A018214
------- ------- ------- ------- ------- ------- A062136
*requires offset adjustment.
The 2-supertoken FF_2(S_3) of the star graph S_3 with central vertex 1 and peripheral vertices 2,3,4. (The vertex `ij' of FF_2(S_3) represents the configuration of one token in `ì' and the other token in `j'). The T(5,3)=7 independent vertices are 22, 24, 44, 23, 11, 34, and 33.
22--12---24---14---44
| \ / |
23 11 34
\ | /
13
|
33
MAPLE
read transforms; 1/(1-y-x*y-x^2); SERIES2(%, x, y, 12); SERIES2TOLIST(%, x, y, 12);
MATHEMATICA
t[n_, k_] := Sum[ (-1)^(n-j)*Binomial[j, k], {j, 0, n}]; Flatten[ Table[t[n, k], {n, 0, 12}, {k, 0, n}]] (* Jean-François Alcover, Oct 20 2011, after Paul Barry *)
PROG
(Sage)
def A059260_row(n):
@cached_function
def prec(n, k):
if k==n: return 1
if k==0: return 0
return -prec(n-1, k-1)-sum(prec(n, k+i-1) for i in (2..n-k+1))
return [(-1)^(n-k+1)*prec(n+1, n-k+1) for k in (1..n)]
for n in (1..9): print(A059260_row(n)) # Peter Luschny, Mar 16 2016
(PARI) T(n, k) = sum(j=0, n, (-1)^(n - j)*binomial(j, k));
for(n=0, 12, for(k=0, n, print1(T(n, k), ", "); ); print(); ) \\ Indranil Ghosh, Apr 11 2017
(Python)
from sympy import binomial
def T(n, k): return sum((-1)**(n - j)*binomial(j, k) for j in range(n + 1))
for n in range(13): print([T(n, k) for k in range(n + 1)]) # Indranil Ghosh, Apr 11 2017
CROSSREFS
Cf. A059259. Row sums give A001045.
Seen as a square array read by antidiagonals this is the coefficient of x^k in expansion of 1/((1-x^2)*(1-x)^n) with rows A002620, A002623, A001752, A001753, A001769, A001779, A001780, A001781, A001786, A001808 etc. (allowing for signs). A058393 would then effectively provide the table for nonpositive n. - Henry Bottomley, Jun 25 2001
KEYWORD
nonn,tabl,nice
AUTHOR
N. J. A. Sloane, Jan 23 2001
EXTENSIONS
Formula corrected by Philippe Deléham, Jan 11 2014
STATUS
approved
Number T(n,k) of k-element subsets of [n] having an even sum; triangle T(n,k), n>=0, 0<=k<=n, read by rows.
+10
20
1, 1, 0, 1, 1, 0, 1, 1, 1, 1, 1, 2, 2, 2, 1, 1, 2, 4, 6, 3, 0, 1, 3, 6, 10, 9, 3, 0, 1, 3, 9, 19, 19, 9, 3, 1, 1, 4, 12, 28, 38, 28, 12, 4, 1, 1, 4, 16, 44, 66, 60, 40, 20, 5, 0, 1, 5, 20, 60, 110, 126, 100, 60, 25, 5, 0, 1, 5, 25, 85, 170, 226, 226, 170, 85, 25, 5, 1, 1, 6, 30, 110, 255, 396, 452, 396, 255, 110, 30, 6, 1
OFFSET
0,12
COMMENTS
Row n is symmetric if and only if n mod 4 in {0,3} (or if T(n,n) = 1).
LINKS
Johann Cigler, Some remarks on Rogers-Szegö polynomials and Losanitsch's triangle, arXiv:1711.03340 [math.CO], 2017.
Johann Cigler, Some Pascal-like triangles, 2018.
FORMULA
T(n,k) = Sum_{j=0..floor((n+1)/4)} C(ceiling(n/2),2*j) * C(floor(n/2),k-2*j).
T(n,k) = A007318(n,k) - A159916(n,k).
Sum_{k=0..n} k * T(n,k) = A057711(n-1) for n>0.
Sum_{k=0..n} (k+1) * T(n,k) = A087447(n) + [n=2].
EXAMPLE
T(5,0) = 1: {}.
T(5,1) = 2: {2}, {4}.
T(5,2) = 4: {1,3}, {1,5}, {2,4}, {3,5}.
T(5,3) = 6: {1,2,3}, {1,2,5}, {1,3,4}, {1,4,5}, {2,3,5}, {3,4,5}.
T(5,4) = 3: {1,2,3,4}, {1,2,4,5}, {2,3,4,5}.
T(5,5) = 0.
T(7,7) = 1: {1,2,3,4,5,6,7}.
Triangle T(n,k) begins:
1;
1, 0;
1, 1, 0;
1, 1, 1, 1;
1, 2, 2, 2, 1;
1, 2, 4, 6, 3, 0;
1, 3, 6, 10, 9, 3, 0;
1, 3, 9, 19, 19, 9, 3, 1;
1, 4, 12, 28, 38, 28, 12, 4, 1;
1, 4, 16, 44, 66, 60, 40, 20, 5, 0;
1, 5, 20, 60, 110, 126, 100, 60, 25, 5, 0;
1, 5, 25, 85, 170, 226, 226, 170, 85, 25, 5, 1;
1, 6, 30, 110, 255, 396, 452, 396, 255, 110, 30, 6, 1;
MAPLE
b:= proc(n, s) option remember; expand(
`if`(n=0, s, b(n-1, s)+x*b(n-1, irem(s+n, 2))))
end:
T:= n-> (p-> seq(coeff(p, x, i), i=0..n))(b(n, 1)):
seq(T(n), n=0..16);
MATHEMATICA
Flatten[Table[Sum[Binomial[Ceiling[n/2], 2j]Binomial[Floor[n/2], k-2j], {j, 0, Floor[(n+1)/4]}], {n, 0, 10}, {k, 0, n}]] (* Indranil Ghosh, Feb 26 2017 *)
PROG
(PARI) a(n, k)=sum(j=0, floor((n+1)/4), binomial(ceil(n/2), 2*j)*binomial(floor(n/2), k-2*j));
tabl(nn)={for(n=0, nn, for(k=0, n, print1(a(n, k), ", "); ); print(); ); } \\ Indranil Ghosh, Feb 26 2017
CROSSREFS
Columns k=0..10 give (offsets may differ): A000012, A004526, A002620, A005993, A005994, A032092, A032093, A018211, A018212, A282077, A282078.
Row sums give A011782.
Main diaginal gives A133872(n+1).
Lower diagonals T(n+j,n) for j=1..10 give: A004525(n+1), A282079, A228705, A282080, A282081, A282082, A282083, A282084, A282085, A282086.
T(2n,n) gives A119358.
KEYWORD
nonn,tabl
AUTHOR
Alois P. Heinz, Feb 04 2017
STATUS
approved
Row sums of A168281.
+10
19
2, 4, 12, 20, 38, 56, 88, 120, 170, 220, 292, 364, 462, 560, 688, 816, 978, 1140, 1340, 1540, 1782, 2024, 2312, 2600, 2938, 3276, 3668, 4060, 4510, 4960, 5472, 5984, 6562, 7140, 7788, 8436, 9158, 9880, 10680, 11480, 12362, 13244, 14212, 15180, 16238, 17296, 18448, 19600, 20850, 22100
OFFSET
1,1
COMMENTS
The atomic numbers of the augmented alkaline earth group in Charles Janet's spiral periodic table are 0 and the first eight terms of this sequence (see Stewart reference). - Alonso del Arte, May 13 2011
Maximum number of 123 patterns in an alternating permutation of length n+3. - Lara Pudwell, Jun 09 2019
LINKS
Robert Dougherty-Bliss, Experimental Methods in Number Theory and Combinatorics, Ph. D. Dissertation, Rutgers Univ. (2024). See p. 4.
Lara Pudwell, From permutation patterns to the periodic table, Notices of the American Mathematical Society. 67.7 (2020), 994-1001.
Philip Stewart, Charles Janet: unrecognized genius of the Periodic System. Foundations of Chemistry (2010), p. 9.
FORMULA
a(n) = 2*A005993(n-1).
a(n) = (n+1)*(3 + 2*n^2 + 4*n - 3*(-1)^n)/12.
a(n+1) - a(n) = A093907(n) = A137583(n+1).
a(2n+1) = A035597(n+1), a(2n) = A002492(n).
a(n) = A099956(n-1), 2 <= n <= 7.
a(n) = 2*a(n-1) + a(n-2) - 4*a(n-3) + a(n-4) + 2*a(n-5) - a(n-6).
G.f.: 2*x*(1 + x^2) / ( (1+x)^2*(x-1)^4 ).
a(n) = A000292(n) + A027656(n-1). - Paul Curtz, Oct 26 2012
E.g.f.: (1/12)*(3*(x - 1) + (3 + 15*x + 12*x^2 + 2*x^3)*exp(2*x))*exp(-x). - G. C. Greubel, Jul 19 2016
EXAMPLE
From Lara Pudwell, Jun 09 2019: (Start)
a(1)=2. The alternating permutation of length 1+3=4 with the maximum number of copies of 123 is 1324. The two copies are 124 and 134.
a(2)=4. The alternating permutation of length 2+3=5 with the maximum number of copies of 123 is 13254. The four copies are 124, 125, 134, and 135.
a(3)=12. The alternating permutation of length 3+3=6 with the maximum number of copies of 123 is 132546. The twelve copies are 124, 125, 126, 134, 135, 136, 146, 156, 246, 256, 346, and 356. (End)
MATHEMATICA
LinearRecurrence[{2, 1, -4, 1, 2, -1}, {2, 4, 12, 20, 38, 56}, 50] (* G. C. Greubel, Jul 19 2016 *)
Table[(n + 1) (3 + 2 n^2 + 4 n - 3 (-1)^n)/12, {n, 50}] (* Michael De Vlieger, Jul 20 2016 *)
PROG
(Magma) [(n+1)*(3+2*n^2+4*n-3*(-1)^n)/12: n in [1..50] ]; // Vincenzo Librandi, Aug 06 2011
(PARI) a(n)=([0, 1, 0, 0, 0, 0; 0, 0, 1, 0, 0, 0; 0, 0, 0, 1, 0, 0; 0, 0, 0, 0, 1, 0; 0, 0, 0, 0, 0, 1; -1, 2, 1, -4, 1, 2]^(n-1)*[2; 4; 12; 20; 38; 56])[1, 1] \\ Charles R Greathouse IV, Jul 21 2016
KEYWORD
nonn,easy
AUTHOR
Paul Curtz, Nov 24 2009
STATUS
approved
Infinite square array: T(n,k) = number of directed multigraphs with loops with n arcs and k vertices; read by falling antidiagonals.
+10
14
1, 1, 0, 1, 1, 0, 1, 2, 1, 0, 1, 2, 6, 1, 0, 1, 2, 10, 10, 1, 0, 1, 2, 11, 31, 19, 1, 0, 1, 2, 11, 47, 90, 28, 1, 0, 1, 2, 11, 51, 198, 222, 44, 1, 0, 1, 2, 11, 52, 269, 713, 520, 60, 1, 0, 1, 2, 11, 52, 291, 1270, 2423, 1090, 85, 1, 0, 1, 2, 11, 52, 295, 1596, 5776, 7388, 2180, 110, 1, 0
OFFSET
0,8
COMMENTS
Partial sums of the rows of A136564.
LINKS
R. J. Mathar, Statistics on Small Graphs, arXiv:1709.09000 [math.CO] (2017) Table 79.
FORMULA
T(n,k) = Sum_{p=0..k} A136564(n,p).
If k >= 2n, T(n,k) = A052171(n).
EXAMPLE
The array begins:
1, 1, 1, 1, 1, 1, 1, 1, 1, ...
0, 1, 2, 2, 2, 2, 2, 2, 2, ...
0, 1, 6, 10, 11, 11, 11, 11, 11, ...
0, 1, 10, 31, 47, 51, 52, 52, 52, ...
0, 1, 19, 90, 198, 269, 291, 295, 296, 296, ...
0, 1, 28, 222, 713, 1270, 1596, 1697, 1719, 1723, ...
0, 1, 44, 520, 2423, 5776, 8838, 10425, 10922, ...
0, 1, 60, 1090, 7388, 24032, 46384, ...
0, 1, 85, 2180, 21003, 93067, ...
0, 1, 110, 4090, ...
...
PROG
(PARI)
permcount(v) = {my(m=1, s=0, k=0, t); for(i=1, #v, t=v[i]; k=if(i>1&&t==v[i-1], k+1, 1); m*=t*k; s+=t); s!/m}
edges(v, t) = {prod(i=2, #v, prod(j=1, i-1, my(g=gcd(v[i], v[j])); t(v[i]*v[j]/g)^(2*g))) * prod(i=1, #v, t(v[i])^v[i])}
G(n, x)={my(s=0); forpart(p=n, s+=permcount(p)/edges(p, i->1-x^i)); s/n!}
T(n)={Mat(vector(n+1, k, Col(O(y*y^n) + G(k-1, y + O(y*y^n)))))}
{my(A=T(10)); for(n=1, #A, print(A[n, ]))} \\ Andrew Howroyd, Oct 22 2019
CROSSREFS
Columns k=0..4 are: A000007, A000012, A005993, A050927, A050929.
Main diagonal is A362387.
KEYWORD
nonn,tabl
AUTHOR
Benoit Jubin, May 03 2008
EXTENSIONS
More terms from Vladeta Jovovic and Benoit Jubin, Sep 10 2008
STATUS
approved
Alkane (or paraffin) numbers l(7,n).
(Formerly M2774)
+10
9
1, 3, 9, 19, 38, 66, 110, 170, 255, 365, 511, 693, 924, 1204, 1548, 1956, 2445, 3015, 3685, 4455, 5346, 6358, 7514, 8814, 10283, 11921, 13755, 15785, 18040, 20520, 23256, 26248, 29529, 33099, 36993, 41211, 45790, 50730, 56070, 61810, 67991
OFFSET
0,2
COMMENTS
Equals A000217 (1, 3, 6, 10, 15, ...) convolved with A193356 (1, 0, 3, 0, 5, ...). - Gary W. Adamson, Feb 16 2009
F(1,4,n) is the number of bracelets with 1 blue, 4 red and n black beads. If F(1,4,1)=3 and F(1,4,2)=9 taken as a base;
F(1,4,n) = n(n+1)(n+2)/6+F(1,2,n) + F(1,4,n-2). [F(1,2,n) is the number of bracelets with 1 blue, 2 red and n black beads. If F(1,2,1)=2 and F(1,2,2)=4 taken as a base F(1,2,n)=n+1+F(1,2,n-2)]. - Ata Aydin Uslu and Hamdi G. Ozmenekse, Jan 11 2012
a(A254338(n)) = 6 for n > 0. - Reinhard Zumkeller, Feb 27 2015
REFERENCES
S. M. Losanitsch, Die Isomerie-Arten bei den Homologen der Paraffin-Reihe, Chem. Ber. 30 (1897), 1917-1926.
N. J. A. Sloane and Simon Plouffe, The Encyclopedia of Integer Sequences, Academic Press, 1995 (includes this sequence).
LINKS
Johann Cigler, Some remarks on Rogers-Szegö polynomials and Losanitsch's triangle, arXiv:1711.03340 [math.CO], 2017.
S. M. Losanitsch, Die Isomerie-Arten bei den Homologen der Paraffin-Reihe, Chem. Ber. 30 (1897), 1917-1926. (Annotated scanned copy)
N. J. A. Sloane, Classic Sequences
FORMULA
G.f.: (1+x^2)/((1-x)^3*(1-x^2)^2) = (1+x^2)/((1-x)^5*(1+x)^2).
l(c, r) = 1/2 C(c+r-3, r) + 1/2 d(c, r), where d(c, r) is C((c + r - 3)/2, r/2) if c is odd and r is even, 0 if c is even and r is odd, C((c + r - 4)/2, r/2) if c is even and r is even, C((c + r - 4)/2, (r - 1)/2) if c is odd and r is odd.
a(-5-n)=a(n). - Michael Somos, Mar 08 2007
Euler transform of length 4 sequence [3, 3, 0, -1]. - Michael Somos, Mar 08 2007
a(n) = 3a(n-1) - a(n-2) - 5a(n-3) + 5a(n-4) + a(n-5) - 3a(n-6) + a(n-7), with a(0)=1, a(1)=3, a(2)=9, a(4)=19, a(5)=38, a(6)=66, a(7)=110. - Harvey P. Dale, May 02 2011
a(n) = A006009(n)/2 - A000332(n+4) = ((1/2)*Sum_{i=1..n+1} (i+1)*floor((i+1)^2/2)) - binomial(n+4,4). - Enrique Pérez Herrero, May 11 2012
a(n) = (1/48)*(n+1)*(n+3)*((n+2)*(n+4)+3)+1/32*(2*n+5)*(1+(-1)^n). - Yosu Yurramendi, Jun 20 2013
Conjecture: a(n)+a(n+1) = A203286(n+1). - R. J. Mathar, Mar 08 2025
MAPLE
a:= n -> (Matrix([[1, 0$4, 1, 3]]). Matrix(7, (i, j)-> if (i=j-1) then 1 elif j=1 then [3, -1, -5, 5, 1, -3, 1][i] else 0 fi)^n)[1, 1]: seq (a(n), n=0..40); # Alois P. Heinz, Jul 31 2008
MATHEMATICA
LinearRecurrence[{3, -1, -5, 5, 1, -3, 1}, {1, 3, 9, 19, 38, 66, 110}, 50] (* or *) CoefficientList[Series[(1+x^2)/((1-x)^3(1-x^2)^2), {x, 0, 50}], x] (* Harvey P. Dale, May 02 2011 *)
nn=45; With[{a=Accumulate[Range[nn]], b=Riffle[Range[1, nn, 2], 0]}, Flatten[ Table[ListConvolve[Take[a, n], Take[b, n]], {n, nn}]]] (* Harvey P. Dale, Nov 11 2011 *)
PROG
(PARI) {a(n)=if(n<-4, n=-5-n); polcoeff( (1+x^2)/((1-x)^3*(1-x^2)^2)+x*O(x^n), n)} /* Michael Somos, Mar 08 2007 */
(Haskell) -- Following Gary W. Adamson.
import Data.List (inits, intersperse)
a005994 n = a005994_list !! n
a005994_list = map (sum . zipWith (*) (intersperse 0 [1, 3 ..]) . reverse) $
tail $ inits $ tail a000217_list
-- Reinhard Zumkeller, Feb 27 2015
CROSSREFS
Cf. A006009, A005997, A005993 (first differences).
KEYWORD
nonn,easy,nice,changed
AUTHOR
N. J. A. Sloane, Winston C. Yang (yang(AT)math.wisc.edu)
STATUS
approved
Number of directed multigraphs with loops on an infinite set of nodes containing a total of n arcs.
+10
9
1, 2, 11, 52, 296, 1724, 11060, 74527, 533046, 3999187, 31412182, 257150093, 2188063401, 19299062896, 176059781439, 1657961491087, 16089088019098, 160643776819423, 1648068916722737, 17351137043998280, 187255329043638437, 2069426416836401375, 23397468305569068113, 270406562951254606048, 3191908298072118225550, 38454691427657997701136
OFFSET
0,2
COMMENTS
Row sums of A136564, limiting values of A138107. - Benoit Jubin, May 13 2008
Euler transform of A137975. - M. F. Hasler, Jul 31 2017
LINKS
Banglei Guan, Ji Zhao, and Laurent Kneip, Six-Point Method for Multi-Camera Systems with Reduced Solution Space, arXiv:2402.18066 [cs.CV], 2024. See p. 10.
J.-C. Novelli, J.-Y. Thibon and N. M. Thiery, Algèbres de Hopf de graphes, C.R. Acad. Sci. Paris (Comptes Rendus Mathématique), 339 (2004), 607-610.
Sanjaye Ramgoolam, Permutation Invariant Gaussian Matrix Models, arXiv:1809.07559 [hep-th], 2018.
FORMULA
a(n) = A138107(2*n,n). - Max Alekseyev, Oct 17 2017
CROSSREFS
Cf. A104209. Cf. A137975 (connected).
KEYWORD
nonn
AUTHOR
Vladeta Jovovic, Jan 26 2000
EXTENSIONS
a(16)-a(25) from Max Alekseyev, Jun 21 2011
STATUS
approved
Initial digits of A254143 in decimal representation.
+10
8
1, 4, 7, 1, 2, 3, 3, 4, 6, 1, 1, 2, 2, 2, 3, 3, 3, 4, 6, 1, 1, 1, 1, 1, 1, 2, 2, 2, 2, 2, 2, 3, 3, 3, 3, 4, 4, 6, 1, 1, 1, 1, 1, 1, 1, 1, 1, 1, 2, 2, 2, 2, 2, 2, 2, 2, 2, 2, 3, 3, 3, 3, 3, 4, 4, 6, 1, 1, 1, 1, 1, 1, 1, 1, 1, 1, 1, 1, 1, 1, 1, 1, 1, 1, 1, 2
OFFSET
1,2
COMMENTS
a(n) = A000030(A254143(n));
also initial digits of A254323: a(n) = A000030(A254323(n)).
all terms are of the form u*v mod 10, where u <= v and belonging to {1,3,4,6,7}, the distinct elements of A254397:
length of k-th run of consecutive 1s = A005993(k-2), k > 1;
length of k-th run of consecutive 2s = k*(k+1)/2 = A000217(k), k >= 1;
length of k-th run of consecutive 3s = k+1, k >= 1;
length of k-th run of consecutive 4s = A065033(k-1);
n with a(n) = 4: A237424(n) = (10^a+10^b+1)/3 with b = 0, see also A093137, A133384;
n with a(n) = 6: A237424(n) = (10^a+10^b+1)/3 with a = b; A005994(a(n)) = 6 for n > 1; see also A199682;
LINKS
PROG
(Haskell)
a254338 = a000030 . a254143
(PARI) listA237424(lim)=my(v=List(), a, t); while(1, for(b=0, a, t=(10^a+10^b+1)/3; if(t>lim, return(Set(v))); listput(v, t)); a++)
do(lim)=my(v=List(), u=listA237424(lim), t); for(i=1, #u, for(j=1, i, t=u[i]*u[j]; if(t>lim, break); listput(v, t))); apply(n->digits(n)[1], Set(v)) \\ Charles R Greathouse IV, May 13 2015
KEYWORD
nonn,base
AUTHOR
Reinhard Zumkeller, Feb 27 2015
STATUS
approved
Triangle read by rows T(n,k) in which column k lists the partial sums of the k-th column of triangle A236104.
+10
8
1, 5, 14, 1, 30, 2, 55, 6, 91, 10, 1, 140, 19, 2, 204, 28, 3, 285, 44, 7, 385, 60, 11, 1, 506, 85, 15, 2, 650, 110, 24, 3, 819, 146, 33, 4, 1015, 182, 42, 8, 1240, 231, 58, 12, 1, 1496, 280, 74, 16, 2, 1785, 344, 90, 20, 3, 2109, 408, 115, 29, 4, 2470, 489, 140, 38, 5, 2870, 570, 165, 47, 9, 3311, 670, 201, 56, 13, 1
OFFSET
1,2
COMMENTS
Alternating sum of row n equals A175254(n), i.e., Sum_{k=1..A003056(n)} (-1)^(k-1)*T(n,k) = A175254(n), which is also the volume (or the total number of units cubes) in the first n levels of the stepped pyramid described in A245092.
Row n has length A003056(n) hence the first element of column k is in row A000217(k).
EXAMPLE
Triangle begins:
1;
5;
14, 1;
30, 2;
55, 6;
91, 10, 1;
140, 19, 2;
204, 28, 3;
285, 44, 7;
385, 60, 11, 1;
506, 85, 15, 2;
650, 110, 24, 3;
819, 146, 33, 4;
1015, 182, 42, 8;
1240, 231, 58, 12, 1;
1496, 280, 74, 16, 2;
1785, 344, 90, 20, 3;
2109, 408, 115, 29, 4;
2470, 489, 140, 38, 5;
2870, 570, 165, 47, 9;
3311, 670, 201, 56, 13, 1;
3795, 770, 237, 72, 17, 2;
4324, 891, 273, 88, 21, 3;
4900, 1012, 322, 104, 25, 4;
...
For n = 6 we have that A175254(6) = [1] + [1 + 3] + [1 + 3 + 4] + [1 + 3 + 4 + 7] + [1 + 3 + 4 + 7 + 6] + [1 + 3 + 4 + 7 + 6 + 12] = 1 + 4 + 8 + 15 + 21 + 33 = 82. On the other hand the alternating sum of the 6th row of the triangle is 91 - 10 + 1 = 82, equaling A175254(6).
CROSSREFS
Column 1 gives A000330, n >= 1. Column 2 is A005993. It appears that column 3 is A092353.
KEYWORD
nonn,tabf
AUTHOR
Omar E. Pol, Nov 03 2015
STATUS
approved
Triangle read by rows: T(n,m) = number of planar partitions of n with trace m.
+10
7
1, 2, 1, 3, 2, 1, 4, 6, 2, 1, 5, 10, 6, 2, 1, 6, 19, 14, 6, 2, 1, 7, 28, 28, 14, 6, 2, 1, 8, 44, 52, 33, 14, 6, 2, 1, 9, 60, 93, 64, 33, 14, 6, 2, 1, 10, 85, 152, 127, 70, 33, 14, 6, 2, 1, 11, 110, 242, 228, 142, 70, 33, 14, 6, 2, 1, 12, 146, 370, 404, 272, 149, 70, 33, 14, 6, 2, 1, 13
OFFSET
1,2
COMMENTS
Also number of partitions of n objects of 2 colors into k parts, each part containing at least one black object.
T(n+m, m) = A005380(n), n >= 1, for all m >= n. T(m, m) = 1 for m >= 1. See the Stanley reference Exercise 7.99. With offset n=0 a column for m=0 with the only non-vanishing entry T(0, 0) = 1 could be added. - Wolfdieter Lang, Mar 09 2015
REFERENCES
G. E. Andrews, The Theory of Partitions, Addison-Wesley, 1976 (Ch. 11, Example 5 and Ch. 12, Example 5).
R. P. Stanley, Enumerative Combinatorics, Cambridge University Press, Vol. 2, 1999; p. 365 and Exercise 7.99, p. 484 and pp. 548-549.
LINKS
FORMULA
G.f.: Product_{k>=1} 1/(1-q*x^k)^k (with offset n=0 in x powers).
EXAMPLE
The triangle T(n,m) begins:
n\m 1 2 3 4 5 6 7 8 9 10 11 12 ...
1: 1
2: 2 1
3: 3 2 1
4: 4 6 2 1
5: 5 10 6 2 1
6: 6 19 14 6 2 1
7: 7 28 28 14 6 2 1
8: 8 44 52 33 14 6 2 1
9: 9 60 93 64 33 14 6 2 1
10: 10 85 152 127 70 33 14 6 2 1
11: 11 110 242 228 142 70 33 14 6 2 1
12: 12 146 370 404 272 149 70 33 14 6 2 1
... reformatted, Wolfdieter Lang, Mar 09 2015
MAPLE
b:= proc(n, i) option remember; expand(`if`(n=0, 1,
`if`(i<1, 0, add(b(n-i*j, i-1)*x^j*
binomial(i+j-1, j), j=0..n/i))))
end:
T:= n-> (p-> seq(coeff(p, x, i), i=1..degree(p)))(b(n$2)):
seq(T(n), n=1..12); # Alois P. Heinz, Apr 13 2017
MATHEMATICA
b[n_, i_] := b[n, i] = Expand[If[n == 0, 1, If[i < 1, 0, Sum[b[n - i*j, i - 1]*x^j*Binomial[i + j - 1, j], {j, 0, n/i}]]]];
T[n_] := Table[Coefficient[#, x, i], {i, 1, Exponent[#, x]}]]& @ b[n, n];
Table[T[n], {n, 1, 12}] // Flatten (* Jean-François Alcover, May 19 2018, after Alois P. Heinz *)
CROSSREFS
Cf. A000219 (row sums), A005380, A005993 (trace 2), A050531 (trace 3), A089351 (trace 4).
KEYWORD
nonn,tabl
AUTHOR
EXTENSIONS
Edited by Christian G. Bower, Jan 08 2004
STATUS
approved

Search completed in 0.026 seconds