Zulip Chat Archive
Stream: Is there code for X?
Topic: Boundedness Theorem for Continuous Functions
rtertr (Sonia) (Jun 12 2023 at 12:07):
Hi, is there a theorem stating that if a function is continuous and
lim(x-->infinity) f(x) < infinity
and lim(x-->-infinity) f(x) < infinity
, then f(x) < infinity
? :)
Kevin Buzzard (Jun 12 2023 at 12:12):
What does f(x)<infinity even mean? What is the codomain of your function?
rtertr (Sonia) (Jun 12 2023 at 12:16):
Oh yeah it is real. I wanna show that the function is bounded ∃C:ℝ, ∀x:E, ‖f x‖ ≤ C
Jireh Loreaux (Jun 12 2023 at 13:20):
What is E
?
Kevin Buzzard (Jun 12 2023 at 13:23):
I think that what you're asking is how to prove that if you know is continuous, and and then there exists such that (because is continuous and hence bounded on ). But this conversation is demonstrating that the best way to ask a question is to formalise the question in Lean and not hope that the readers can do so.
rtertr (Sonia) (Jun 12 2023 at 13:29):
Yes, thank you. Sorry if I was a bit vague :smile:
Eric Rodriguez (Jun 12 2023 at 13:37):
and for that, docs#continuous.exists_forall_le' could help but may be a bit hard to use without understanding of filters. formalising using docs#is_compact.exists_forall_ge may be easier
rtertr (Sonia) (Jun 12 2023 at 13:43):
Ah, thank you :smile: The thing is I already proved what I wanted, so I don't technically need the theorem. But I was just writing about my process, and I wanted to see if such theorem actually existed, and I had just not been able to find it when I first started working. :smiley_cat:
Jireh Loreaux (Jun 12 2023 at 15:54):
Note: I don't think we have your result as stated. If I try some formalizations of your statement, it would look something like this:
import analysis.normed.field.basic
open filter bornology
example (f : C(ℝ, ℝ)) (hf_lt₁ : is_bounded_under (<) at_top f)
(hf_lt₂ : is_bounded_under (<) at_bot f) :
bdd_above (set.range f) := sorry
-- you can put the two properties at `∞` and `-∞` together using `⊔` on the respective filters.
example (f : C(ℝ, ℝ)) (hf_lt : is_bounded_under (<) (at_top ⊔ at_bot ) f) :
bdd_above (set.range f) := sorry
-- here is another filter that represents the idea "at +∞ or -∞"
example (f : C(ℝ, ℝ)) (hf_lt : is_bounded_under (<) (comap norm at_top) f) :
bdd_above (set.range f) := sorry
-- yet another filter using `bornology.cobounded`
example (f : C(ℝ, ℝ)) (hf_lt : is_bounded_under (<) (cobounded ℝ) f) :
bdd_above (set.range f) := sorry
I don't think we have any of these (or similar statements) explicitly in mathlib, but I could be wrong.
rtertr (Sonia) (Jun 12 2023 at 16:28):
Ah, okay, thank you very much! That is good to know! :D
Last updated: Dec 20 2023 at 11:08 UTC