I am reading the book by Kleene "Introduction to Metamathematics". In Chapter 2 Paragraph 7 on "Mathematical Induction" there is a problem to prove the following lemma.
Lemma 1: A proper pairing of $2n$ parentheses ($n>0$ and $n$ is a natural number) contains an innermost pair, i.e. a pair which includes no other of the parentheses between them.
Following definitions are used:
Proper pairing - one-to-one pairing between $n$ left parentheses "$($" and $n$ right parentheses "$)$" such that for each pair left parenthesis is on the left from the right parenthesis and if no two pairs separate each other.
Pairs of parentheses that separate each other - two pairs separate each other if they occur in the order $(_i (_j )_i )_j$ (ignoring everything else).
To prove this lemma Kleene suggests to use the principle of course-of-values induction, which I assume is known to you.
I wanted to try to prove this lemma using "ordinary" induction. What I would like to ask is whether my proof is correct, and, if it is not, where is the mistake? Also, any comments are appreciated.
Consider the basis step, i.e. when $n=1$. Then, there are only two possible arrangements of parenthesis, namely, $()$ and $)($. The latter is not proper, therefore, there is only one proper pairing. This pair satisfies the definition of an innermost pair, so the lemma is true in this case.
Assume that if $n = m$ then the lemma holds. Consider $n = m+1$, which means that there is given a proper pairing of $2m+2$ parentheses. Consider one (arbitrary) pair. Either it is innermost or it is not (here, I am using law of excluded middle, but since this theorem is supposed to be in metamathematics where there is no axioms a priori, and, thus, I feel that theorems in metamathematics should be just some statements with some justifiable reason to be assumed, this is okay. In other words, there is no law of excluded middle in metamathematics and the argument is considered valid due to the construction of parentheses and our intuition). If it is innermost then the lemma is true. If it is not, then consider remaining $2m$ parentheses. By induction principle, we have that pairing between these parentheses has an innermost pair. Now, it could be that for these $2m$ parentheses it is an innermost pair, but adding the additional pair, it is not innermost anymore. If it still is the innermost pair, then the lemma is true. Otherwise, it should be the case that at least one of two additional parentheses is in this pair. It couldn't be one of the parentheses because then the pairing would not be proper. So, then, there must be both of the parentheses inside this pair. That would imply that the additional pair is innermost pair. But that is a contradiction as we assumed the pair that is removed and added is not innermost. It must be then that the innermost pair of remaining $2m$ parentheses is indeed innermost also for $2m+2$ parentheses. In any case, there is an innermost pair.
Therefore, by the principle of induction, the lemma is true for all natural numbers.