Zulip Chat Archive
Stream: Is there code for X?
Topic: injectivity of multiplication on EReal
Ruben Van de Velde (Jan 20 2025 at 12:55):
Do we really not have either of these?
lemma mul_right_inj {a b c : EReal} (hbot : b ≠ ⊥) (htop : b ≠ ⊤) (hzero : b ≠ 0) : a * b = c * b ↔ a = c := sorry
lemma mul_right_coe_inj {a c : EReal} {b : ℝ} (hzero : b ≠ 0) : a * b = c * b ↔ a = c := sorry
(I have an ugly proof in #20293)
Edward van de Meent (Jan 20 2025 at 13:03):
from the looks of it, no... but i'm also pretty sure these'd be called something like mul_left_cancel
or something like that
Edward van de Meent (Jan 20 2025 at 13:03):
see for example docs#mul_left_cancel
Ruben Van de Velde (Jan 20 2025 at 13:31):
mul_left_cancel
is the implication; this is the iff. Though that would be fine as well
Damiano Testa (Jan 20 2025 at 13:41):
Also the analogous ones for ENNReal
appear to be missing.
Damiano Testa (Jan 20 2025 at 13:44):
Maybe the ENNReal
ones exist docs#ENNReal.mul_eq_mul_left ?
Ruben Van de Velde (Jan 20 2025 at 13:57):
Damiano Testa said:
Maybe the
ENNReal
ones exist docs#ENNReal.mul_eq_mul_left ?
I'll rename those, thanks for the pointer
Ruben Van de Velde (Jan 20 2025 at 15:31):
Last updated: May 02 2025 at 03:31 UTC