File tree Expand file tree Collapse file tree 1 file changed +1
-2
lines changed Expand file tree Collapse file tree 1 file changed +1
-2
lines changed Original file line number Diff line number Diff line change @@ -216,8 +216,7 @@ theorem inftyValuation.X_inv : inftyValuation Fq (1 / RatFunc.X) = exp (-1) := b
216216-- https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/.60synthInstance.2EmaxHeartbeats.60.20error.20but.20only.20in.20.60simpNF.60
217217theorem inftyValuation.polynomial {p : Fq[X]} (hp : p ≠ 0 ) :
218218 inftyValuationDef Fq (algebraMap Fq[X] (RatFunc Fq) p) = exp (p.natDegree : ℤ) := by
219- have hp' : algebraMap Fq[X] (RatFunc Fq) p ≠ 0 := by simpa
220- rw [inftyValuationDef, if_neg hp', RatFunc.intDegree_polynomial]
219+ rw [inftyValuationDef, if_neg (by simpa), RatFunc.intDegree_polynomial]
221220
222221/-- The valued field `Fq(t)` with the valuation at infinity. -/
223222def inftyValuedFqt : Valued (RatFunc Fq) ℤᵐ⁰ :=
You can’t perform that action at this time.
0 commit comments