Zulip Chat Archive

Stream: new members

Topic: Uniqueness of roots


Sammy Webb (Mar 10 2024 at 11:29):

Hello, I am wondering if anyone can tell me if I have misstated a theorem I am trying to prove.

The theorem is as follows:

Let x>0x>0 and kNk\in\mathbb{N}. Then there is a unique y>0y>0 such that yk=xy^{k}=x.

Proof

Let S={s0    sk<x}S=\{s \geq 0 \; | \; s^{k}<x\}. Then SS is nonempty (since 0S0 \in S) and bounded above since max{x,1}\max \{x, 1\} is an upper bound for SS. Therefore

y=LUB(S)=LUB({s0    sk<x})y=\text{LUB}(S)=\text{LUB}(\{s \geq0 \; | \; s^{k}<x\})

exists by the Completeness Axiom. We claim that yk=xy^{k}=x.

Since yy is the least upper bound of SS, this means that for all nNn\in\mathbb{N}, y1ny-\frac{1}{n} is not an upper bound, i.e.\ there is ynSy_{n}\in S such that

y1n<yny.y-\frac{1}{n}<y_{n}\leq y.

Now y1nyy - \frac{1}{n} \to y (by Example) and the rules for
limits), and the constant sequence y,y,y, y, \ldots converges to yy too, so
by the squeeze theorem, ynyy_n \to y.

By Proposition power-lim, ynkyky_n^k \to y^k. But
ynSy_n\in S, so ynk<xy_{n}^{k}<x for all nn, so
Proposition~\ref{p:x_n<y_n} gives

ykx.y^{k} \leq x.

Now we will show the reverse inequality, i.e.\ that xykx\leq y^{k}, and this will imply yk=xy^k=x. Since y=LUB(S)y=\text{LUB}(S), yy is an upper bound for SS, and so for all nn, y+1n∉Sy+\frac{1}{n}\not\in S. By the definition of SS, this means

(y+1n)kx.\left(y+\frac{1}{n}\right)^{k}\geq x.

Again, Propositions~\ref{p:power-lim} and~\ref{p:x_n<y_n}, together with the fact that y+1nyy + \frac{1}{n}\rightarrow y, imply that

ykx.y^{k} \geq x.

Thus, yk=xy^k=x.

Finally, if 0<w<z0 < w < z then wk<zkw^k < z^k (see Proposition 4.3) and so there is a {\em unique} y>0y >0 such that yk=xy^k = x.

I have stated it as follows:

theorem theorem_6_6 {x:} (k:) (hx: 0 < x) (hk:1  k): ∃! y, 0 < y  y^k = x := by

Should this implication be an and statement?

However, while I am able to prove the existence I am struggling with the uniqueness.

Kevin Buzzard (Mar 10 2024 at 11:39):

Uniqueness isn't true the way you've written it, because any y which isn't >0 will also work. Yes it should be an "and" statement in the conclusion

Sammy Webb (Mar 10 2024 at 11:48):

Thank you I will try that.

Kevin Buzzard (Mar 10 2024 at 11:52):

I made the same error of logic in my initial definition of a scheme, and Commelin pointed it out to me.


Last updated: May 02 2025 at 03:31 UTC