Skip to content

Commit 3267bd7

Browse files
committed
chore: remove note about non-instance (#29525)
The linked issue has been closed, let's see if this is okay now.
1 parent 9fe6658 commit 3267bd7

File tree

1 file changed

+1
-7
lines changed

1 file changed

+1
-7
lines changed

Mathlib/RingTheory/WittVector/DiscreteValuationRing.lean

Lines changed: 1 addition & 7 deletions
Original file line numberDiff line numberDiff line change
@@ -140,15 +140,9 @@ theorem exists_eq_pow_p_mul' (a : 𝕎 k) (ha : a ≠ 0) :
140140
have hb₀ : b.coeff 0 = b₀ := rfl
141141
exact ⟨m, mkUnit hb₀, h₂⟩
142142

143-
/-
144-
Note: The following lemma should be an instance, but it seems to cause some
145-
exponential blowups in certain typeclass resolution problems.
146-
See the following Lean4 issue as well as the zulip discussion linked there:
147-
https://github.com/leanprover/lean4/issues/1102
148-
-/
149143
/-- The ring of Witt Vectors of a perfect field of positive characteristic is a DVR.
150144
-/
151-
theorem isDiscreteValuationRing : IsDiscreteValuationRing (𝕎 k) :=
145+
instance isDiscreteValuationRing : IsDiscreteValuationRing (𝕎 k) :=
152146
IsDiscreteValuationRing.ofHasUnitMulPowIrreducibleFactorization (by
153147
refine ⟨p, irreducible p, fun {x} hx => ?_⟩
154148
obtain ⟨n, b, hb⟩ := exists_eq_pow_p_mul' x hx

0 commit comments

Comments
 (0)