Skip to content

Commit

Permalink
feat(RingTheory/Ideal/Quotient): assume Semiring instance instead of …
Browse files Browse the repository at this point in the history
…CommRing (#9493)

Ideal.Quotient.lift only needs `Semiring S` on the target to work.

This PR only changes one line : `variable [CommRing S]` to `variable [Semiring S]`



Co-authored-by: Antoine Chambert-Loir <antoine.chambert-loir@math.univ-paris-diderot.fr>
  • Loading branch information
AntoineChambert-Loir and Antoine Chambert-Loir committed Jan 6, 2024
1 parent 1b3fb34 commit 526457f
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion Mathlib/RingTheory/Ideal/Quotient.lean
Expand Up @@ -251,7 +251,7 @@ theorem maximal_ideal_iff_isField_quotient (I : Ideal R) : I.IsMaximal ↔ IsFie
maximal_of_isField _⟩
#align ideal.quotient.maximal_ideal_iff_is_field_quotient Ideal.Quotient.maximal_ideal_iff_isField_quotient

variable [CommRing S]
variable [Semiring S]

/-- Given a ring homomorphism `f : R →+* S` sending all elements of an ideal to zero,
lift it to the quotient by this ideal. -/
Expand Down

0 comments on commit 526457f

Please sign in to comment.