This is in response to @joriki's observation that the constraint of the weekly total studying hours could be loosen while the conclusion of minimum $20$ days would still hold. I am not sure if it's appropriate to post this as an answer, but it turns out to be too long to fit in the comment section.
We shall prove the following, by using a slightly different pigeonhole construction than what's in the nice answer by @NP-hard:
(apologies for the slight notation change)
Suppose $m,n$ are positive integers and
$$0=S_0<S_1<\ldots<S_n$$ is a sequence of integers that satisfy:
$$\tag{1}S_{i+7}\le S_i+m\label{1},$$
for all $0\le i\le n-7$, then there exists $0\le j<k\le n$ so that $S_k-S_j=20$ if
$(1)~m\le 13$ and $n\ge 20$; or
$(2)~m=14$ and $n\ge 26$.
We prove the following lemma first:
If
$$\tag{2}S_{i+20}<S_i+40\label{2}$$
for any $0\le i\le n-20$, then $S_k-S_j=20$ for some $0\le j<k\le i+20$.
Proof of the lemma:
Note if any $S_l=S_i+20$ for $i+1\le l\le i+20$, we can take $(j,k)=(i,l)$; otherwise consider the following $19$ integer subsets:
$$\{S_i+1,S_i+21\}, \{S_i+2,S_i+22\}, \ldots, \{S_i+19,S_i+39\}$$
and $20$ distinctive values of $S_{i+1}, S_{i+2}, \ldots, S_{i+20}$, by the pigeonhole principle, we conclude that there exists $i+1\le j<k\le i+20$ with $S_k$ and $S_j$ residing in the same subset, i.e., $S_k-S_j=20$.
Note we have not yet used the constraint \eqref{1}.
added: as @Shagnik pointed out, the proof above can be simplified by considering instead $20$ subsets $\{S_i,S_i+20\}, \{S_i+1,S_i+21\}, \ldots, \{S_i+19,S_i+39\}$ along with $21$ values $S_i, S_{i+1}, \ldots, S_{i+20}$.
Proof of the original propositions:
$(1)~m\le 13$, then
$$S_{20}\le S_{13}+m\le S_6+2m<S_7+2m\le S_0+3m<S_0+40,$$
by repeatedly applying \eqref{1}. We are done by taking $i=0$ in \eqref{2} and applying the lemma.
As @NP-hard pointed out, $n=19$ does not suffice as $S_i=i$ is a counterexample.
$(2)~m=14$, by the lemma, we only need to consider the case when
$$\tag{3}S_{i+20}\ge S_i+40\label{3}$$
for all $0\le i\le 6$. We have on the one hand
$$S_{10}\stackrel{\eqref{1}}\le S_3+14\stackrel{\eqref{3}}\le S_{23}-26\stackrel{\eqref{1}}\le S_2+16\stackrel{\eqref{3}}\le S_{22}-24\stackrel{\eqref{1}}\le S_1+18\stackrel{\eqref{3}}\le S_{21}-22\stackrel{\eqref{1}}\le 20$$
and on the other hand
$$S_{10}\stackrel{\eqref{1}}\ge S_{24}-28\stackrel{\eqref{3}}\ge S_4+12\stackrel{\eqref{1}}\ge S_{25}-30\stackrel{\eqref{3}}\ge S_5+10\stackrel{\eqref{1}}\ge S_{26}-32\stackrel{\eqref{3}}\ge S_6+8\stackrel{\eqref{1}}\ge S_{20}-20\stackrel{\eqref{3}}\ge 20,$$
therefore $S_{10}=20$, i.e., we can take $(k,j)=(0,10)$ in this case.
For $n=25$, one counterexample is
$$\left\{S_i\right\}=\left\{1,2,3,4,5,13,14,15,16,17,18,19,26,27,28,29,30,31,32,40,41,42,43,44,45\right\}$$
or in terms of daily studying hours:
$$\left\{1,1,1,1,1,8,1,1,1,1,1,1,7,1,1,1,1,1,1,8,1,1,1,1,1\right\}.$$
added: regarding @Joffan's counterexamples for $n=25$, the way we came up with the case above is by similarly applying \eqref{1} and \eqref{3} to prove that $S_i\le 2i$ for all $i\le 25$ except $i\in\{6,13,20\}$ when $S_i\ge 2i$ (as the inequality chain above now breaks into two at $S_{26}$). In addition, the set $\{S_0+20,S_1+20,\ldots,S_i+20,S_{10},S_{11},\ldots,S_{10+i}\}$ is precisely $\{10,11,\ldots,20+2i\}$ when $i\notin\{3,6,10,13\}$. These constraints above allow us to check handful cases and would be useful in general cases (e.g., when $20$ is replaced by some larger number and computer search could be infeasible).