Skip to content

Commit

Permalink
chore(ring_theory/unique_factorization_domain): drop simp annotation …
Browse files Browse the repository at this point in the history
…for factors_pow (#14646)

Followup to #14555.
  • Loading branch information
Ruben-VandeVelde committed Jun 9, 2022
1 parent 7b4680f commit 4d4de43
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion src/ring_theory/unique_factorization_domain.lean
Expand Up @@ -461,7 +461,7 @@ begin
exact (associated.mul_mul (factors_prod hx) (factors_prod hy)).symm,
end

@[simp] lemma factors_pow {x : α} (n : ℕ) :
lemma factors_pow {x : α} (n : ℕ) :
multiset.rel associated (factors (x ^ n)) (n • factors x) :=
begin
induction n with n ih,
Expand Down

0 comments on commit 4d4de43

Please sign in to comment.