Skip to content

Commit

Permalink
feat (RingTheory/Localization/LocalizationLocalization): Generalize f…
Browse files Browse the repository at this point in the history
…rom CommRing to CommSemiring (#9112)

Change hypothesis CommRing to CommSemiring in the first section of the file
  • Loading branch information
XavierXarles committed Dec 16, 2023
1 parent 4160b2a commit c014896
Showing 1 changed file with 8 additions and 4 deletions.
12 changes: 8 additions & 4 deletions Mathlib/RingTheory/Localization/LocalizationLocalization.lean
Expand Up @@ -22,17 +22,19 @@ commutative ring, field of fractions
-/


variable {R : Type*} [CommRing R] (M : Submonoid R) {S : Type*} [CommRing S]

variable [Algebra R S] {P : Type*} [CommRing P]

open Function BigOperators

namespace IsLocalization

section LocalizationLocalization

variable (N : Submonoid S) (T : Type*) [CommRing T] [Algebra R T]
variable {R : Type*} [CommSemiring R] (M : Submonoid R) {S : Type*} [CommSemiring S]

variable [Algebra R S] {P : Type*} [CommSemiring P]

variable (N : Submonoid S) (T : Type*) [CommSemiring T] [Algebra R T]


section

Expand Down Expand Up @@ -254,6 +256,8 @@ end IsLocalization

namespace IsFractionRing

variable {R : Type*} [CommRing R] (M : Submonoid R) {S : Type*} [CommRing S]

open IsLocalization

theorem isFractionRing_of_isLocalization (S T : Type*) [CommRing S] [CommRing T] [Algebra R S]
Expand Down

0 comments on commit c014896

Please sign in to comment.