Skip to content

Commit

Permalink
feat: port RingTheory.Perfection (#4629)
Browse files Browse the repository at this point in the history
Co-authored-by: Xavier-François Roblot <46200072+xroblot@users.noreply.github.com>
Co-authored-by: int-y1 <jason_yuen2007@hotmail.com>
  • Loading branch information
3 people committed Jun 11, 2023
1 parent a01c6e8 commit b29c8d1
Show file tree
Hide file tree
Showing 3 changed files with 659 additions and 1 deletion.
1 change: 1 addition & 0 deletions Mathlib.lean
Expand Up @@ -2444,6 +2444,7 @@ import Mathlib.RingTheory.NonUnitalSubsemiring.Basic
import Mathlib.RingTheory.NonZeroDivisors
import Mathlib.RingTheory.OreLocalization.Basic
import Mathlib.RingTheory.OreLocalization.OreSet
import Mathlib.RingTheory.Perfection
import Mathlib.RingTheory.Polynomial.Basic
import Mathlib.RingTheory.Polynomial.Bernstein
import Mathlib.RingTheory.Polynomial.Chebyshev
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/RingTheory/Localization/FractionRing.lean
Expand Up @@ -302,7 +302,7 @@ instance [Nontrivial R] : Nontrivial (FractionRing R) :=

/-- Porting note: if the fields of this instance are explicitly defined as they were
in mathlib3, the last instance in this file suffers a TC timeout -/
noncomputable instance : Field (FractionRing A) := IsFractionRing.toField A
noncomputable instance field : Field (FractionRing A) := IsFractionRing.toField A

@[simp]
theorem mk_eq_div {r s} :
Expand Down

0 comments on commit b29c8d1

Please sign in to comment.