Zulip Chat Archive

Stream: Is there code for X?

Topic: pow_cancel_left


Patrick Johnson (Jan 13 2022 at 10:29):

Do we have something like this:

lemma pow_cancel_left {a b c : }
  (h₁ : 1 < c)
  (h₂ : c ^ a = c ^ b) :
  a = b

I have a very ugly proof, but I'm surprised I can't find any similar lemma in mathlib.

Yaël Dillies (Jan 13 2022 at 10:32):

Untested

lemma pow_cancel_left {a b c : } (h₁ : 1 < c) (h₂ : c ^ a = c ^ b) : a = b :=
(strict_mono_pow h₁).injective h₂

Yaël Dillies (Jan 13 2022 at 10:33):

This proof works for c in an ordered semiring, but the lemma should hold more generally.

Patrick Johnson (Jan 13 2022 at 10:37):

I totally forgot about strict_mono_pow. Thanks.


Last updated: Dec 20 2023 at 11:08 UTC