Let $a$ and $b$ be integers. Then $(ca,cb)=c(a,b)$ for any positive integer $c > 0$.
I have proved this using Bezout's lemma. However, I am trying to prove this again by following the sketch of the proof from The Theory of Numbers: A Text and Source Book of Problems which states:
Note that the smallest positive integer which is a linear combination of $ca$ and $cb$ is simply $c$ times the least positive integer which is a linear combination of $a$ and $b$. Now apply (1.5)
Theorem 1.5 in this case is:
Suppose $a$ and $b$ are not both $0$, and let $d=(a,b)$. Then $d$ is the smallest positive integer that can be expressed as a linear combination of $a$ and $b$.
This is the proof I came up with, but the argument feels like it is missing something.
Proof. Let $a,b,c \in \mathbb{Z}$ such that $c > 0$ and $a$ and $b$ are not both zero. Let $S = \{cak + cbm : k,m \in \mathbb{Z}\}$. Now, consider the subset $S' = \{x \in S: x > 0\}$. $S'$ has a smallest element by the Well Ordering Principle, and by definition this element is $d=(ca,cb)=c(ak+bm)$. Since $d>0$ and $c>0$, this means that $ak + bm > 0$. Note that multiplication over the integers preserves ordering, and since $d$ is the smallest element of $S'$ this means that $ak + bm$ is the smallest positive linear combination of $a$ and $b$. By definition, this is $(a,b)$. Hence, $(ca,cb)=c(a,b)$. $\blacksquare$