File tree Expand file tree Collapse file tree 1 file changed +1
-7
lines changed
Mathlib/RingTheory/WittVector Expand file tree Collapse file tree 1 file changed +1
-7
lines changed Original file line number Diff line number Diff line change @@ -140,15 +140,9 @@ theorem exists_eq_pow_p_mul' (a : 𝕎 k) (ha : a ≠ 0) :
140
140
have hb₀ : b.coeff 0 = b₀ := rfl
141
141
exact ⟨m, mkUnit hb₀, h₂⟩
142
142
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
- -/
149
143
/-- The ring of Witt Vectors of a perfect field of positive characteristic is a DVR.
150
144
-/
151
- theorem isDiscreteValuationRing : IsDiscreteValuationRing (𝕎 k) :=
145
+ instance isDiscreteValuationRing : IsDiscreteValuationRing (𝕎 k) :=
152
146
IsDiscreteValuationRing.ofHasUnitMulPowIrreducibleFactorization (by
153
147
refine ⟨p, irreducible p, fun {x} hx => ?_⟩
154
148
obtain ⟨n, b, hb⟩ := exists_eq_pow_p_mul' x hx
You can’t perform that action at this time.
0 commit comments