Zulip Chat Archive

Stream: Is there code for X?

Topic: no duplicates in normalized factors


Bhavik Mehta (Dec 22 2024 at 19:44):

import Mathlib.RingTheory.Nilpotent.Defs
import Mathlib.RingTheory.UniqueFactorizationDomain.NormalizedFactors

open UniqueFactorizationMonoid

variable {M : Type*} [CancelCommMonoidWithZero M] [NormalizationMonoid M] [UniqueFactorizationMonoid M]

theorem test {a : M} (ha : IsRadical a) : (normalizedFactors a).Nodup := by
  sorry

Do we have this anywhere? I'm struggling to find many lemmas to help with IsRadical

Junyan Xu (Dec 22 2024 at 19:52):

import Mathlib.Algebra.Squarefree.Basic

open UniqueFactorizationMonoid

variable {M : Type*} [CancelCommMonoidWithZero M] [NormalizationMonoid M] [UniqueFactorizationMonoid M]

theorem test {a : M} (ha : IsRadical a) : (normalizedFactors a).Nodup := by
  obtain rfl | ne := eq_or_ne a 0; · simp
  rwa [ squarefree_iff_nodup_normalizedFactors ne,
     isRadical_iff_squarefree_of_ne_zero ne]

Bhavik Mehta (Dec 22 2024 at 19:59):

Ah, thanks!


Last updated: May 02 2025 at 03:31 UTC