Zulip Chat Archive
Stream: new members
Topic: Formalize the limit and check the answer
Nick_adfor (Feb 26 2025 at 01:22):
import Mathlib
open Real
noncomputable def f (x : ℝ) : ℝ :=
limUnder atTop (λ n : ℕ, (cos x ^ n + sin x ^ n) ^ (1 / n))
theorem part_1 : ∀ x ∈ Set.Icc 0 (π / 2), f x = max (cos x) (sin x) := by sorry
I want to formalize the limit of (cos x ^ n + sin x ^ n) ^ (1 / n) and check the answer f(x). (I don't want to calculate the answer in Lean because I think it may be hard for lean to calculate this.) But Lean has an error:
unexpected token ','; expected '↦', '=>'
"," is "λ n : ℕ, " here. Experience tells me that the error in Lean Infoview can't tell me where the grammar is wrong. So I seek help here.
Thank you!
Zhang Qinchuan (Feb 26 2025 at 01:39):
Your code is not #mwe. Seems you are writing random code and hoping it can compile. Just read TPIL to learn the basic grammar.
And read MIL to learn the concept of docs#Filter.Tendsto .
Nick_adfor (Feb 26 2025 at 01:40):
Zhang Qinchuan said:
Your code is not #mwe. Seems you are writing random code and hoping it can compile. Just read TPIL to learn the basic grammar.
And read MIL to learn the concept of docs#Filter.Tendsto .
Oh...Seems that the definition of limit in Lean is a little difficult
Zhang Qinchuan (Feb 26 2025 at 01:52):
Nick_adfor said:
Oh...Seems that he definition of limit is a little difficult
Most people is familiar with , but Mathlib says docs#Filter is more powerful once you get used to.
You can try to the following code:
Aaron Liu (Feb 26 2025 at 02:09):
Here's what I came up with
import Mathlib
open Real Filter Topology
-- This statement simultaneously asserts that the limit exists and is equal to `max (cos x) (sin x)`.
example
-- forall real numbers `0 ≤ x ≤ π / 2`
(x : ℝ) (hx : x ∈ Set.Icc 0 (π / 2)) :
-- in the limit
Tendsto
-- the sequence `fₙ = ⁿ√(cos x ^ n + sin x ^ n)`
(fun (n : Nat) ↦ (cos x ^ n + sin x ^ n) ^ (n⁻¹ : ℝ))
-- as `n → ∞`
atTop
-- approaches `max (cos x) (sin x)`
(𝓝 (max (cos x) (sin x))) := by
sorry
-- The reason we use `Tendsto` is that small variations on the statement do not require a new definition.
example
-- forall real numbers `0 ≤ x ≤ π / 2`
(x : ℝ) (hx : x ∈ Set.Icc 0 (π / 2)) :
-- in the limit
Tendsto
-- the sequence `fₙ = ⁿ√(cos x ^ n + sin x ^ n)`
(fun (n : Nat) ↦ (cos x ^ n + sin x ^ n) ^ (n⁻¹ : ℝ))
-- as `n → ∞`
atTop
-- approaches `max (cos x) (sin x)` from the left
(𝓝[≤] (max (cos x) (sin x))) := by
sorry
Nick_adfor (Feb 26 2025 at 02:10):
Zhang Qinchuan said:
Nick_adfor said:
Oh...Seems that the definition of limit in lean is a little difficult
Most people is familiar with , but Mathlib says docs#Filter is more powerful once you get used to.
You can try to the following code:
Thank you for your reply! I have briefly skimmed through the code in the Filter, and its definition does seem more complex than the traditional epsilon-delta approach I learned in my analysis course. However, its scope of application also appears to be more general even in any other topology.
Nick_adfor (Feb 26 2025 at 02:12):
Aaron Liu said:
Here's what I came up with
import Mathlib open Real Filter -- This statement simultaneously asserts that the limit exists and is equal to `max (cos x) (sin x)`. example -- forall real numbers `0 ≤ x ≤ π / 2` (x : ℝ) (hx : x ∈ Set.Icc 0 (π / 2)) : -- in the limit Tendsto -- the sequence `fₙ = ⁿ√(cos x ^ n + sin x ^ n)` (fun (n : Nat) ↦ (cos x ^ n + sin x ^ n) ^ (n⁻¹ : ℝ)) -- as `n → ∞` atTop -- approaches `max (cos x) (sin x)` (nhds (max (cos x) (sin x))) := by sorry
Thank you, too. I'll take some time to understand "nhds"
Last updated: May 02 2025 at 03:31 UTC