Skip to content

Commit

Permalink
chore: fix docstring of IsLocalization (#7234)
Browse files Browse the repository at this point in the history
  • Loading branch information
ADedecker committed Sep 18, 2023
1 parent 3882a68 commit 00fdd1f
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion Mathlib/RingTheory/Localization/Basic.lean
Expand Up @@ -94,7 +94,7 @@ variable {R : Type*} [CommSemiring R] (M : Submonoid R) (S : Type*) [CommSemirin

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

/-- The typeclass `IsLocalization (M : Submodule R) S` where `S` is an `R`-algebra
/-- The typeclass `IsLocalization (M : Submonoid R) S` where `S` is an `R`-algebra
expresses that `S` is isomorphic to the localization of `R` at `M`. -/
class IsLocalization : Prop where
--Porting note: add ' to fields, and made new versions of these with either `S` or `M` explicit.
Expand Down

0 comments on commit 00fdd1f

Please sign in to comment.