Before proceeding to the main proof, some lemmas :
Lemma 1 : The number of strictly increasing sequences of m elements of $[\![1, n]\!]$ is $ \binom{n}{m} $ with n,m two integers such that $ m \leq n $ (otherwise the answer would be 0) :
Proof of lemma 1 : To choose a strictly increasing sequence it suffices to choose a subset of m distinct elements of $[\![1, n]\!]$, and then order them so that the sequence is strictly increasing ( $ x_1 = Min(A)$, $ x_2 = Min(A-\{x_1\}) $, ...etc), and inversely, any sequence of m strictly increasing elements of $[\![1, n]\!]$ can be associated with a subset of m elements. We have thus established a bijection, and so the number of strictly increasing sequences of m elements is the same as that of subsets of m elements, which is $ \binom{n}{m}$
Lemma 2 : The number of strictly increasing sequences of m elements of $[\![1, n]\!]$ is $ \binom{n+m - 1}{m} $ with n,m two integers such that $ m \leq n $ (otherwise the answer would be 0) :
Proof of lemma 2 : This follows from the first lemma, in short, to each increasing sequence of m elements of $[\![1, n]\!]$ $ (x_1, ..., x_m) $ we associate a strictly increasing sequence of elements : $ (y_1, ..., y_m) $ defined by : $ y_1 = x_1 $, $ y_k = x_k + (k-1) $ for all other k, this is clearly a strictly increasing sequence of m elements of $[\![1, n + m - 1]\!]$, in the same manner, any such strictly increasing sequence of elements of $[\![1, n + m - 1]\!]$ can be associated to an increasing sequence of $[\![1, n]\!]$
Because we'll be dealing with integers that can be null (i.e. elements of $[\![0, n]\!]$ ), we offset the result of lemma 2 (there is a clear bijection between $[\![0, n]\!]$ and $[\![1, n + 1]\!]$ ), So for elements of $[\![0, n]\!]$ , the count is : $ \binom{n+m}{m} $
We can count the number of solutions in a more general setting.
Consider m integers $ 0 \leq x_1, \dots, x_m \leq n $ and $ n \in N^{*} $ such that :
$$ x_1 + \dots + x_m \leq n $$
and let $ 0 \leq y_1, \dots, y_m \leq n $ such that : $ \forall k \in [\![1, m]\!] : y_k = x_1 + \dots + x_k $. It is evident that $(y_k)_{ 1 \leq k \leq m }$ is an increasing sequence of integers of [0,n]. Inversely , given an increasing sequence of integers : $(y_k)_{ 1 \leq k \leq m }$, we consider $(x_k)_{ 1 \leq k \leq m }$ such that $x_1 = y_1$ and $ x_k = y_{k} - y_{k-1} $ for all other k. It is easy to check that $ x_1 + \dots + x_m \leq n $. We have thus established a bijection between two sets, the solution set of the equation and the set of increasing sequences of m elements of $[\![0, n]\!]$. Of which there are : $ \binom{n+m}{m}
$, Thus the number of solutions is also : $ \binom{n+m}{m}$ by taking n = 20 and m = 3, we get the same answer that you've gotten.