( ext{Fibonacci Sequence})
(quad quad ext{If we record sequence} {F_n} ext{as Fibonacci Sequence, then }{F_n} ext{ will have these properties:})
(quad quad ext{So we can see that } {F_n} ext{ is like “1,1,2,3,5,8,13,21...”.})
( ext{GCD})
(quad quad ext{“GCD” is the abbreviation of “Greatest Common Divisor”.})
(quad quad ext{And we often record } (a, b) ext{ as the GCD of } a ext{ and } b.)
(quad quad ext{For example, } (12, 15) = 3, (48, 36) = 12.)
( ext{Two Theorems about GCD})
( ext{Euclidean theorem})
( ext{The proof: })
- ( ext{If } a = b, (a, b) = a = b, ext{we can surely tell that the theorem is established.})
- ( ext{If } a < b, (b, a mod b) = (b, a) = (a, b), ext{the theorem is established.})
- ( ext{If } a > b, ext{we can assume that } a = k imes b + r, (k in N_{+}, 0 le r < b), ext{ so } a mod b = r. \ ext{As for } forall d, ext{meeting that } d|a land d|b, d|(a - k imes b), ext{ actually it means } d | r. \ ext{So we can tell that } (a, b) = (b, r), ext{ that is, } (a, b) = (b, a mod b).)
( ext{Stein's Algorithm})
( ext{The proof:})
( ext{Actually, the proof of it is similar to that of Euclidean theorem, you can finish it yourselves.})
( ext{One Lemma})
( ext{The Proof}):
- ( ext{In the case of } n = 1 ext{ and } n = 2, ext{ the lemma is established obviously.})
- ( ext{In the case of } n ge 2 :)
( ext{Obviously:})
(quad ext{According to Euclidean theorem and the lemma above:})
( ext{Fibonacci GCD})
(quad quad ext{Here is the expression of the Fibonacci GCD:})
( ext{The Proof of Fibonacci GCD})
( ext{We assume that } n<m.)
( ext{Then we use } F_n ext{ and }F_{n+1} ext{ to express } F_{n + 2},F_{n + 3},F_{n + 4},F_{n + 5}cdots)
( ext{We can see that in the expressions above, the coefficients of } F_n ext{ and } F_{n + 1} ext{ meet the properties of the Fibonacci Sequence.})
( ext{And obviously we can see that :})
( ext{According to the lemma above:})
( ext{All in all:})
( ext{We can see that }, ext{the change rule of } n ext{ and } m ext{ meet Stein's Algorithm,so we finally discovered that })