Zulip Chat Archive

Stream: Is there code for X?

Topic: Is Nilpotent if a power is Nilpotent


Xavier Xarles (Dec 04 2023 at 18:45):

I don't find in mathlib4

import Mathlib.RingTheory.Nilpotent

variable {R : Type*}

theorem  IsNilpotent.if_pow [MonoidWithZero R] (x : R)(m:)(h:IsNilpotent (x ^ m)): IsNilpotent x := by
  obtain n, h := h
  use (m*n)
  rw [ h, pow_mul x m n]

Ruben Van de Velde (Dec 04 2023 at 18:59):

I think you're right. Want to make a PR? Call it of_pow, though

Ruben Van de Velde (Dec 04 2023 at 19:01):

And the iff version assuming n ne 0

Jireh Loreaux (Dec 05 2023 at 01:26):

And while you're at it maybe you can rename docs#IsNilpotent.pow to IsNilpotent.pow_succ and make the argument n explicit.


Last updated: Dec 20 2023 at 11:08 UTC