Zulip Chat Archive
Stream: Is there code for X?
Topic: supremum of pointwise product of sets of real numbers
Jujian Zhang (Oct 06 2022 at 13:56):
Do we have that where are sets of real number?
import data.real.basic
open_locale pointwise
example
(s : set ℝ) (hs : ∀ (a : ℝ), a ∈ s → 0 ≤ a)
(t : set ℝ) (ht : ∀ (a : ℝ), a ∈ t → 0 ≤ a): Sup s * Sup t = Sup (s * t) :=
sorry
Sebastien Gouezel (Oct 06 2022 at 14:00):
What about s = t = [-2, -1]
?
Jujian Zhang (Oct 06 2022 at 14:01):
Good point! but in my case s
and t
are all nonnegative, let me change the code.
Yaël Dillies (Oct 06 2022 at 14:09):
Last updated: Dec 20 2023 at 11:08 UTC