Limits, yes another limits thread.

  • Thread starter Thread starter MathematicalPhysicist
  • Start date Start date
  • Tags Tags
    Limits Thread
AI Thread Summary
The discussion revolves around computing limits, specifically lim (a^n - b^n)^(1/n) for a > b > 0 and lim ((3n)!/((2^3n)n!(2n!)))^(1/n). Participants suggest using the lemma that relates limits of sequences and provide algebraic identities to simplify the expressions. A geometrical argument involving the unit circle is also proposed to demonstrate that x ≥ sin(x) for 0 < x < 2π. The conversation highlights the importance of finding suitable bounds and applying the sandwich lemma to prove convergence in limit calculations. Overall, the thread emphasizes the complexity of limit evaluation and the various strategies to approach these mathematical problems.
MathematicalPhysicist
Science Advisor
Gold Member
Messages
4,662
Reaction score
372
i need to compute lim (a^n-b^n)^(1/n) when a>b>0.
lim ((3n)!/((2^3n)n!(2n!)))^(1/n) where i need to use the lemma that:
if an>0 for every n, and lim(x_n+1/x_n)=L then lim x_n^(1/n)=L, how to use it here?

for the first i used practically everything i know, the formual for a^n-b^n, and the fact that 0<a^n-b^n<a^n and lots more algebraic techniques, apparently not everything.

your help is appreciated.
 
Mathematics news on Phys.org
another thing, seemingly unrealted.
i need to show that for 0<x<2pi x>=sinx.
i tried to dissect it into parts, i.e:
x>1 and for x<1, for x>1 it's obvious, my problem is with x<1, then how to solve it?
 
It is relatively simple to show that there IS a limit, and that it lies between a and b, however any more precise than that, I don't know.

Use the following identity in a clever manner:
a^{n}-b^{n}=(a-b)\sum_{i=0}^{n-1}a^{n-1-i}b^{i}
 
Last edited:
The last one, to show that x\ge sin x for all 0\le x\le 2\pi is easy. What is the derivative of f(x)= x- sin(x)? For what values of x is that positive? Since sin(0)= 0, what does that tell you?
 
oh, come on halls, you don't know a proof which doesn't employ derivatives, sure it's easy with derivative but i want to show it without.
 
Well, what's wrong with a geometrical argument on the unit circle, then?
 
arildno said:
It is relatively simple to show that there IS a limit, and that it lies between a and b, however any more precise than that, I don't know.

Use the following identity in a clever manner:
a^{n}-b^{n}=(a-b)\sum_{i=0}^{n-1}a^{n-1-i}b^{i}

as i said i tried this equality, i got something like this: (a-b)a^n>=(a-b)(a^(n-1)+a^(n-2)b+...+b^n-2a+b^(n-1))>=(a-b)(b^(n-1)+...+b^(n-1))=(a-b)b^n but as you said that's easy to show, the problem is to what does it converge?
any other tips?

btw, i also need some help in the other limit.

as always your help is appreciated.
(my custom mantra (-: ).
 
arildno said:
Well, what's wrong with a geometrical argument on the unit circle, then?
i don't follow you, how to use the unit circle here?
i mean the identity which seems to be good here is sin^2x+cos^2x=1
sin^2x=1-cos^2x
sinx/x=sqrt(1-cos^2x)/x<=1 when 0<sinx<=1
cause 1-x^2<=cos^2x<=1
is this correct?
 
Remember that in general, we have NO infallible technique that enables us to "calculate" a limit.
For practical purposes (say when solving a non-linear system numerically), we use the Cauchy criterion to say we have "essentially" reached the limit.
But formally, of course, this is bogus.


What we DO have, is first and foremost a PROPERTY that the limit must have. It is by no means guaranteed by this that we actually manage to FIND that number.
 
  • #10
so to sum up, you don't know how to calculate the limit, correct?
if it's any good, i got a hint to use the sandwich lemma.
 
  • #11
loop quantum gravity said:
so to sum up, you don't know how to calculate the limit, correct?
i

Correct! :smile:
I already said that in my first post.
 
  • #12
loop quantum gravity said:
i don't follow you, how to use the unit circle here?
i mean the identity which seems to be good here is sin^2x+cos^2x=1
sin^2x=1-cos^2x
sinx/x=sqrt(1-cos^2x)/x<=1 when 0<sinx<=1
cause 1-x^2<=cos^2x<=1
is this correct?

No. What length does "sin(x)" represent on the unit circle, and where can you find the length "x" on the same circle?
Compare those lengths!
 
  • #13
ah, i see your point. x is the length of the arc and sinx is the length of the y coordinate on the coordiantion system.
 
  • #14
Of course, the geometrical argument rests also upon the assumption that the straight line is the shortest distance between two points..
 
  • #15
about the limit with a and b, i think it converges to a, the problem is how to prove it, obviously (a^n-b^n)^{\frac{1}{n}}&lt;a
one way to show that it converges to a is by the sandwich lemma, the problem is to find the suitable lower bound, i thought perhaps a^n/n can be a good candidate, but I am not sure this is correct, can someone help?
 
  • #16
It's always easier to get rid of two things that depend on n, and replace it with one.

What can you say about the convergence, or otherwise, of

(1-r^n)^{1/n} where 0<r<1?

It is quite straight forward just using the most naive bounds there are for (1-r^n) (assuming we don't think 0 is a naive lower bound, I mean).
 
Last edited:
  • #17
it converges to 1, is it not?
anyway, i need to find a suitable lower bound for the limit.
 
  • #18
matt grime said:
It's always easier to get rid of two things that depend on n, and replace it with one.

What can you say about the convergence, or otherwise, of

(1-r^n)^{1/n} where 0<r<1?

It is quite straight forward just using the most naive bounds there are for (1-r^n) (assuming we don't think 0 is a naive lower bound, I mean).
obviously it's smaller than 1, but from what it's bigger?
it's bigger than 1-r^n cause (1-r^n)^n<=1-r^n and 1-r^n<1.
will this also work fro number besides 1 and r<1, i mean:
0<b<a (a^n-b^n)^(1/n)<a, but is it: a^n-b^n<(a^n-b^n)^(1/n)
in order for to be true, a^n-b^n should be smaller than 1.
 
  • #19
Think about it a little bit longer, please... For instance, have you figured out what relation I might intend r to have with a and b? How did I get from 0<b<a to 0<r<1?Why have you not used the fact that r^n<r , for instance? You don't appear to have thought the suggestion through at all.
 
  • #20
well you replaced r with b and 1 with, and i did you use the fact that r^n<r when i said that (1-r^n)^n<1-r^n obviously r^n<r<1 and thus also what i wrote is correct.
anyway, i think i understand.
r^n<r
then 1-r^n>1-r so we have a lower bound and an upper.
but my question still stands, how can i use it here?
i mean a>b>0 so a^n>a^n-b^n but i cannot say anything from lower besides 0, cause I am not given that b<1.

perhaps you want to dissect this problem into situations where 0<b<a<1
0<b<1<a 1<b<a, i thought about this and obviously this is the way to go, but i thought perhaps there's a starightforward approahc which doesn't employ splitting into three situations.
 
  • #21
No, I do not want to restrict a and b at all. My answer proves the general case for all a and b - you really can't see what to do to (a^n-b^n)^{1/n} to get something like (1-r^n)^{1/n}? I don't believe that.
 
  • #22
geez louis, ok tell me if this is correct (sorry for not seeing it earlier):
(a^n-b^n)^(1/n)=a(1-(b/a)^n)^(1/n) b/a<1.

****,****
bloody ****. how the bloody hell this little simple thing has alluded me?!

thanks matt.
 
  • #23
i have a tendency to make a simple problem harder than it is.
 
  • #24
quick question:
lim
x--> -1 f(x) x + 3/|x - 2|
my answers were 2/3, and -2/3, so as there is no unique value the limit does not exist. am i right or wrong? please help:)
 
  • #25
J-Girl said:
quick question:
lim
x--> -1 f(x) x + 3/|x - 2|
my answers were 2/3, and -2/3, so as there is no unique value the limit does not exist. am i right or wrong? please help:)

Wrong.

Limx→-1|x - 2 | = 3, for both cases: x approaches -1 from the right and x approaches -1 from the left. In either case, x approaches -1.
 
  • #26
I deleted my reply because I noticed that this thread has been around since 2006
 

Similar threads

Back
Top