Skip to content

Commit

Permalink
change order of commRing and divisionRing in field
Browse files Browse the repository at this point in the history
  • Loading branch information
alreadydone authored Dec 22, 2024
1 parent 49dbf9e commit 53313de
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion Mathlib/RingTheory/Ideal/Quotient/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -138,8 +138,8 @@ will have computable inverses (and `qsmul`, `ratCast`) in some applications.
See note [reducible non-instances]. -/
protected noncomputable abbrev field {R} [CommRing R] (I : Ideal R) [I.IsMaximal] :
Field (R ⧸ I) where
__ := Quotient.divisionRing I
__ := commRing _
__ := Quotient.divisionRing I

/-- If the quotient by an ideal is a field, then the ideal is maximal. -/
theorem maximal_of_isField {R} [CommRing R] (I : Ideal R) (hqf : IsField (R ⧸ I)) :
Expand Down

0 comments on commit 53313de

Please sign in to comment.