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 and . Then there is a unique such that .
Proof
Let . Then is nonempty (since ) and bounded above since is an upper bound for . Therefore
exists by the Completeness Axiom. We claim that .
Since is the least upper bound of , this means that for all , is not an upper bound, i.e.\ there is such that
Now (by Example) and the rules for
limits), and the constant sequence converges to too, so
by the squeeze theorem, .
By Proposition power-lim, . But
, so for all , so
Proposition~\ref{p:x_n<y_n} gives
Now we will show the reverse inequality, i.e.\ that , and this will imply . Since , is an upper bound for , and so for all , . By the definition of , this means
Again, Propositions~\ref{p:power-lim} and~\ref{p:x_n<y_n}, together with the fact that , imply that
Thus, .
Finally, if then (see Proposition 4.3) and so there is a {\em unique} such that .
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