Zulip Chat Archive

Stream: Is there code for X?

Topic: Real.cos N cannot be 1


Christian K (Mar 03 2024 at 17:35):

How can i prove that there is no Natural Number n, so that Real.cos n = 1.

I have this set A

def A : Set r_3 := {w : r_3 |  n : , w = ![Real.cos n, Real.sin n, 0]}

and i want to prove that ![1,0,0] is not in this set

lemma origin_not_in_A : ![1,0,0]  A := by

btw, r_3 is defined as

abbrev r_3 := Fin 3 -> 

And, while were at it, is there a smarter way to define A ?

David Renshaw (Mar 03 2024 at 17:43):

this could help: docs#Real.cos_eq_one_iff

Edward van de Meent (Mar 03 2024 at 17:47):

isn't this just not true because of n=0?

Christian K (Mar 03 2024 at 17:49):

Ohh, right, i forgot, n cannot be 0

Edward van de Meent (Mar 03 2024 at 17:56):

i think your proof will hinge on pi being irrational, and i'm not sure we have that... a quick search didn't reveal any such lemmas...

Christian K (Mar 03 2024 at 17:58):

Yeah, i found some stuff with irrational numbers. But there is nothing about Pi being irrational? And this also doesn't sound like something that would be very easy?

Christian K (Mar 03 2024 at 18:00):

Ok it seems like there is a github issue about this but it is still open...

Edward van de Meent (Mar 03 2024 at 18:01):

out of curiosity, what do you need this result for?

Christian K (Mar 03 2024 at 18:02):

The big project is formalizing the Banach Tarski Paradox, i need this specific lemma for Proving that a Circle is equidecomposable

Edward van de Meent (Mar 03 2024 at 18:05):

it might be the case that we do have the tools for proving pi is irrational...
maybe have a look at https://en.wikipedia.org/wiki/Proof_that_%CF%80_is_irrational and see if one of those is viable?

Eric Wieser (Mar 03 2024 at 18:09):

@loogle Irrational, Real.pi

loogle (Mar 03 2024 at 18:09):

:shrug: nothing found

Ruben Van de Velde (Mar 03 2024 at 18:09):

#6718 includes it

Christian K (Mar 03 2024 at 18:10):

OK, this look intersting, I'll look if i can contribute something helpfull.

Kevin Buzzard (Mar 03 2024 at 18:16):

Why don't you use another irrational number and rescale?

Christian K (Mar 03 2024 at 18:17):

How would i do that?

Kevin Buzzard (Mar 03 2024 at 18:22):

If you want to prove some geometric fact about the circle then my guess is that irrationality of pi is irrelevant (I'm working on some distant memory of having worked through Banach-Tarski years ago) so I'm suggesting that if you understand the proof and believe me then just modify it so that it relies on some other number like 2\sqrt{2} being irrational instead. I might be wrong but if I'm right then this might well be the simplest solution. Don't you just need some dense infinite set which is sent to a proper subset of itself after a rotation, or something? This has nothing to do with irrationality of pi.

Christian K (Mar 03 2024 at 18:27):

Ohhh, yeah i see, this could work, thank you very much for this idea. I'll try it and let you know if it works


Last updated: May 02 2025 at 03:31 UTC