Skip to content
Closed
Show file tree
Hide file tree
Changes from all commits
Commits
File filter

Filter by extension

Filter by extension

Conversations
Failed to load comments.
Loading
Jump to
Jump to file
Failed to load files.
Loading
Diff view
Diff view
2 changes: 1 addition & 1 deletion Mathlib/Algebra/Algebra/Subalgebra/Lattice.lean
Original file line number Diff line number Diff line change
Expand Up @@ -754,7 +754,7 @@ theorem ext_of_adjoin_eq_top {s : Set A} (h : adjoin R s = ⊤) ⦃φ₁ φ₂ :
(hs : s.EqOn φ₁ φ₂) : φ₁ = φ₂ :=
ext fun _x => adjoin_le_equalizer φ₁ φ₂ hs <| h.symm ▸ trivial

/-- Two algebra morphisms are equal on `Algebra.span s`iff they are equal on s -/
/-- Two algebra morphisms are equal on `Algebra.span s` iff they are equal on `s`. -/
theorem eqOn_adjoin_iff {φ ψ : A →ₐ[R] B} {s : Set A} :
Set.EqOn φ ψ (adjoin R s) ↔ Set.EqOn φ ψ s := by
have (S : Set A) : S ≤ equalizer φ ψ ↔ Set.EqOn φ ψ S := Iff.rfl
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Algebra/Homology/Embedding/Connect.lean
Original file line number Diff line number Diff line change
Expand Up @@ -177,7 +177,7 @@ noncomputable def homologyIsoPos (n : ℕ) [NeZero n] (m : ℤ) (hm : m = n)
(by simp; cutsat) (by simp; cutsat) (by simp) (by simp)).symm ≪≫
HomologicalComplex.homologyMapIso h.restrictionGEIso n

/-- Given `h : ConnectData K L` and `n : ℕ`non-zero, the homology
/-- Given `h : ConnectData K L` and `n : ℕ` non-zero, the homology
of `h.cochainComplex` in degree `-(n + 1)` identifies to the homology of `K` in degree `n`. -/
noncomputable def homologyIsoNeg (n : ℕ) [NeZero n] (m : ℤ) (hm : m = -(n + 1 : ℕ))
[h.cochainComplex.HasHomology m] [K.HasHomology n] :
Expand Down
6 changes: 3 additions & 3 deletions Mathlib/Analysis/Calculus/ContDiff/Operations.lean
Original file line number Diff line number Diff line change
Expand Up @@ -183,7 +183,7 @@ theorem ContDiffAt.add {f g : E → F} (hf : ContDiffAt 𝕜 n f x) (hg : ContDi
ContDiffAt 𝕜 n (fun x => f x + g x) x := by
rw [← contDiffWithinAt_univ] at *; exact hf.add hg

/-- The sum of two `C^n`functions is `C^n`. -/
/-- The sum of two `C^n` functions is `C^n`. -/
@[fun_prop]
theorem ContDiff.add {f g : E → F} (hf : ContDiff 𝕜 n f) (hg : ContDiff 𝕜 n g) :
ContDiff 𝕜 n fun x => f x + g x :=
Expand Down Expand Up @@ -264,7 +264,7 @@ theorem ContDiffWithinAt.neg {s : Set E} {f : E → F} (hf : ContDiffWithinAt
theorem ContDiffAt.neg {f : E → F} (hf : ContDiffAt 𝕜 n f x) :
ContDiffAt 𝕜 n (fun x => -f x) x := by rw [← contDiffWithinAt_univ] at *; exact hf.neg

/-- The negative of a `C^n`function is `C^n`. -/
/-- The negative of a `C^n` function is `C^n`. -/
@[fun_prop]
theorem ContDiff.neg {f : E → F} (hf : ContDiff 𝕜 n f) : ContDiff 𝕜 n fun x => -f x :=
contDiff_neg.comp hf
Expand Down Expand Up @@ -409,7 +409,7 @@ nonrec theorem ContDiffAt.mul {f g : E → 𝔸} (hf : ContDiffAt 𝕜 n f x) (h
theorem ContDiffOn.mul {f g : E → 𝔸} (hf : ContDiffOn 𝕜 n f s) (hg : ContDiffOn 𝕜 n g s) :
ContDiffOn 𝕜 n (fun x => f x * g x) s := fun x hx => (hf x hx).mul (hg x hx)

/-- The product of two `C^n`functions is `C^n`. -/
/-- The product of two `C^n` functions is `C^n`. -/
@[fun_prop]
theorem ContDiff.mul {f g : E → 𝔸} (hf : ContDiff 𝕜 n f) (hg : ContDiff 𝕜 n g) :
ContDiff 𝕜 n fun x => f x * g x :=
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Analysis/Normed/Module/FiniteDimension.lean
Original file line number Diff line number Diff line change
Expand Up @@ -46,7 +46,7 @@ linear maps are continuous. Moreover, a finite-dimensional subspace is always co
The fact that all norms are equivalent is not written explicitly, as it would mean having two norms
on a single space, which is not the way type classes work. However, if one has a
finite-dimensional vector space `E` with a norm, and a copy `E'` of this type with another norm,
then the identities from `E` to `E'` and from `E'`to `E` are continuous thanks to
then the identities from `E` to `E'` and from `E'` to `E` are continuous thanks to
`LinearMap.continuous_of_finiteDimensional`. This gives the desired norm equivalence.
-/

Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Analysis/RCLike/Inner.lean
Original file line number Diff line number Diff line change
Expand Up @@ -18,7 +18,7 @@ from `RCLike.innerProductSpace`.

* Build a non-instance `InnerProductSpace` from `wInner`.
* `cWeight` is a poor name. Can we find better? It doesn't hugely matter for typing, since it's
hidden behind the `⟪f, g⟫ₙ_[𝕝] `notation, but it does show up in lemma names
hidden behind the `⟪f, g⟫ₙ_[𝕝]` notation, but it does show up in lemma names
`⟪f, g⟫_[𝕝, cWeight]` is called `wInner_cWeight`. Maybe we should introduce some naming
convention, similarly to `MeasureTheory.average`?
-/
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Analysis/SpecialFunctions/Exponential.lean
Original file line number Diff line number Diff line change
Expand Up @@ -91,7 +91,7 @@ variable {𝕂 𝔸 : Type*} [NontriviallyNormedField 𝕂] [NormedCommRing 𝔸

/-- The exponential map in a commutative Banach algebra `𝔸` over a normed field `𝕂` of
characteristic zero has Fréchet derivative `NormedSpace.exp 𝕂 x • 1 : 𝔸 →L[𝕂] 𝔸`
at any point `x`in the disk of convergence. -/
at any point `x` in the disk of convergence. -/
theorem hasFDerivAt_exp_of_mem_ball [CharZero 𝕂] {x : 𝔸}
(hx : x ∈ EMetric.ball (0 : 𝔸) (expSeries 𝕂 𝔸).radius) :
HasFDerivAt (exp 𝕂) (exp 𝕂 x • (1 : 𝔸 →L[𝕂] 𝔸)) x := by
Expand Down
4 changes: 2 additions & 2 deletions Mathlib/CategoryTheory/Functor/KanExtension/Preserves.lean
Original file line number Diff line number Diff line change
Expand Up @@ -106,7 +106,7 @@ def LeftExtension.IsPointwiseLeftKanExtension.postcompose
LeftExtension.postcompose₂ L F G |>.obj E |>.IsPointwiseLeftKanExtension := fun c ↦
(hE c).postcompose G

/-- The cocone at a point of the whiskering right by `G`of an extension is isomorphic to the
/-- The cocone at a point of the whiskering right by `G` of an extension is isomorphic to the
action of `G` on the cocone at that point for the original extension. -/
@[simps!]
def LeftExtension.coconeAtWhiskerRightIso (E : LeftExtension L F) (c : C) :
Expand Down Expand Up @@ -358,7 +358,7 @@ def RightExtension.IsPointwiseRightKanExtension.postcompose
RightExtension.postcompose₂ L F G |>.obj E |>.IsPointwiseRightKanExtension := fun c ↦
(hE c).postcompose G

/-- The cone at a point of the whiskering right by `G`of an extension is isomorphic to the
/-- The cone at a point of the whiskering right by `G` of an extension is isomorphic to the
action of `G` on the cone at that point for the original extension. -/
@[simps!]
def RightExtension.coneAtWhiskerRightIso (E : RightExtension L F) (c : C) :
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/CategoryTheory/InducedCategory.lean
Original file line number Diff line number Diff line change
Expand Up @@ -10,7 +10,7 @@ public import Mathlib.CategoryTheory.Functor.FullyFaithful
/-!
# Induced categories and full subcategories

Given a category `D` and a function `F : C → D `from a type `C` to the
Given a category `D` and a function `F : C → D` from a type `C` to the
objects of `D`, there is an essentially unique way to give `C` a
category structure such that `F` becomes a fully faithful functor,
namely by taking $$ Hom_C(X, Y) = Hom_D(FX, FY) $$. We call this the
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/CategoryTheory/Sites/Sheaf.lean
Original file line number Diff line number Diff line change
Expand Up @@ -152,7 +152,7 @@ theorem isLimit_iff_isSheafFor :

/-- Given sieve `S` and presheaf `P : Cᵒᵖ ⥤ A`, their natural associated cone admits at most one
morphism from every cone in the same category (i.e. over the same diagram),
iff `Hom (E, P -)`is separated for the sieve `S` and all `E : A`. -/
iff `Hom (E, P -)` is separated for the sieve `S` and all `E : A`. -/
theorem subsingleton_iff_isSeparatedFor :
(∀ c, Subsingleton (c ⟶ P.mapCone S.arrows.cocone.op)) ↔
∀ E : Aᵒᵖ, IsSeparatedFor (P ⋙ coyoneda.obj E) S.arrows := by
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Combinatorics/SetFamily/Compression/Down.lean
Original file line number Diff line number Diff line change
Expand Up @@ -186,7 +186,7 @@ it suffices to prove it for
* the finset family which only contains the empty finset.
* `{s ∪ {a} | s ∈ 𝒜}` assuming the property for `𝒜` a family of finsets not containing `a`.
* `ℬ ∪ 𝒞` assuming the property for `ℬ` and `𝒞`, where `a` is an element of the ground type and
`ℬ`is a family of finsets not containing `a` and `𝒞` a family of finsets containing `a`.
`ℬ` is a family of finsets not containing `a` and `𝒞` a family of finsets containing `a`.
Note that instead of giving `ℬ` and `𝒞`, the `subfamily` case gives you `𝒜 = ℬ ∪ 𝒞`, so that
`ℬ = {s ∈ 𝒜 | a ∉ s}` and `𝒞 = {s ∈ 𝒜 | a ∈ s}`.

Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Data/NNRat/Defs.lean
Original file line number Diff line number Diff line change
Expand Up @@ -45,7 +45,7 @@ library_note2 «specialised high priority simp lemma» /--
It sometimes happens that a `@[simp]` lemma declared early in the library can be proved by `simp`
using later, more general simp lemmas. In that case, the following reasons might be arguments for
the early lemma to be tagged `@[simp high]` (rather than `@[simp, nolint simpNF]` or
un``@[simp]``ed):
un-`@[simp]`ed):
1. There is a significant portion of the library which needs the early lemma to be available via
`simp` and which doesn't have access to the more general lemmas.
2. The more general lemmas have more complicated typeclass assumptions, causing rewrites with them
Expand Down
4 changes: 2 additions & 2 deletions Mathlib/Data/PFun.lean
Original file line number Diff line number Diff line change
Expand Up @@ -42,8 +42,8 @@ Partial functions can be considered as relations, so we specialize some `Rel` de
* `PFun.ran`: Range of a partial function.
* `PFun.preimage`: Preimage of a set under a partial function.
* `PFun.core`: Core of a set under a partial function.
* `PFun.graph`: Graph of a partial function `a →. β`as a `Set (α × β)`.
* `PFun.graph'`: Graph of a partial function `a →. β`as a `Rel α β`.
* `PFun.graph`: Graph of a partial function `a →. β` as a `Set (α × β)`.
* `PFun.graph'`: Graph of a partial function `a →. β` as a `Rel α β`.

### `PFun α` as a monad

Expand Down
4 changes: 2 additions & 2 deletions Mathlib/Data/Set/Lattice.lean
Original file line number Diff line number Diff line change
Expand Up @@ -181,12 +181,12 @@ theorem subset_iUnion₂ {s : ∀ i, κ i → Set α} (i : ι) (j : κ i) : s i
theorem iInter₂_subset {s : ∀ i, κ i → Set α} (i : ι) (j : κ i) : ⋂ (i) (j), s i j ⊆ s i j :=
iInf₂_le i j

/-- This rather trivial consequence of `subset_iUnion`is convenient with `apply`, and has `i`
/-- This rather trivial consequence of `subset_iUnion` is convenient with `apply`, and has `i`
explicit for this purpose. -/
theorem subset_iUnion_of_subset {s : Set α} {t : ι → Set α} (i : ι) (h : s ⊆ t i) : s ⊆ ⋃ i, t i :=
le_iSup_of_le i h

/-- This rather trivial consequence of `iInter_subset`is convenient with `apply`, and has `i`
/-- This rather trivial consequence of `iInter_subset` is convenient with `apply`, and has `i`
explicit for this purpose. -/
theorem iInter_subset_of_subset {s : ι → Set α} {t : Set α} (i : ι) (h : s i ⊆ t) :
⋂ i, s i ⊆ t :=
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/FieldTheory/IntermediateField/Adjoin/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -663,7 +663,7 @@ theorem eq_of_root {x y : L} (hx : IsAlgebraic K x)
(h_ev : Polynomial.aeval y (minpoly K x) = 0) : minpoly K y = minpoly K x :=
((eq_iff_aeval_minpoly_eq_zero hx.isIntegral).mpr h_ev).symm

/-- The canonical `algEquiv` between `K⟮x⟯`and `K⟮y⟯`, sending `x` to `y`, where `x` and `y` have
/-- The canonical `algEquiv` between `K⟮x⟯` and `K⟮y⟯`, sending `x` to `y`, where `x` and `y` have
the same minimal polynomial over `K`. -/
noncomputable def algEquiv {x y : L} (hx : IsAlgebraic K x)
(h_mp : minpoly K x = minpoly K y) : K⟮x⟯ ≃ₐ[K] K⟮y⟯ := by
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Geometry/Manifold/ContMDiff/Defs.lean
Original file line number Diff line number Diff line change
Expand Up @@ -622,7 +622,7 @@ theorem contMDiffWithinAt_iff_le_ne_infty :
| coe n =>
exact contMDiffWithinAt_iff_nat.2 (fun m hm ↦ h _ (mod_cast hm) (by simp))

/-- A function is `C^n`at a point iff it is `C^m`at this point, for
/-- A function is `C^n` at a point iff it is `C^m` at this point, for
any `m ≤ n` which is different from `∞`. This result is useful because, when `m ≠ ∞`, being
`C^m` extends locally to a neighborhood, giving flexibility for local proofs. -/
theorem contMDiffAt_iff_le_ne_infty :
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/GroupTheory/GroupAction/Hom.lean
Original file line number Diff line number Diff line change
Expand Up @@ -801,7 +801,7 @@ class MulSemiringActionSemiHomClass (F : Type*)
extends DistribMulActionSemiHomClass F φ R S, RingHomClass F R S

/-- `MulSemiringActionHomClass F M R S` states that `F` is a type of morphisms preserving
the ring structure and equivariant with respect to a `DistribMulAction`of `M` on `R` and `S` .
the ring structure and equivariant with respect to a `DistribMulAction` of `M` on `R` and `S`.
-/
abbrev MulSemiringActionHomClass
(F : Type*)
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/GroupTheory/GroupAction/MultiplePrimitivity.lean
Original file line number Diff line number Diff line change
Expand Up @@ -158,7 +158,7 @@ theorem isMultiplyPreprimitive_ofStabilizer
aesop
exact IsPreprimitive.of_surjective ofFixingSubgroup_insert_map_bijective.surjective

/-- A pretransitive action is `n.succ-`preprimitive iff
/-- A pretransitive action is `n.succ`-preprimitive iff
the action of stabilizers is `n`-preprimitive. -/
@[to_additive]
theorem isMultiplyPreprimitive_succ_iff_ofStabilizer
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/GroupTheory/GroupAction/Pointwise.lean
Original file line number Diff line number Diff line change
Expand Up @@ -22,7 +22,7 @@ public import Mathlib.Algebra.Group.Units.Hom
It requires that `c` acts surjectively and `σ c` acts injectively and
is provided with specific versions:
- `preimage_smul_setₛₗ_of_isUnit_isUnit` when `c` and `σ c` are units
- `IsUnit.preimage_smul_setₛₗ` when `σ` belongs to a `MonoidHomClass`and `c` is a unit
- `IsUnit.preimage_smul_setₛₗ` when `σ` belongs to a `MonoidHomClass` and `c` is a unit
- `MonoidHom.preimage_smul_setₛₗ` when `σ` is a `MonoidHom` and `c` is a unit
- `Group.preimage_smul_setₛₗ` : when the types of `c` and `σ c` are groups.

Expand Down
2 changes: 1 addition & 1 deletion Mathlib/GroupTheory/GroupAction/Quotient.lean
Original file line number Diff line number Diff line change
Expand Up @@ -232,7 +232,7 @@ noncomputable def selfEquivSigmaOrbitsQuotientStabilizer : β ≃ Σ ω : Ω, α
@[to_additive AddAction.sigmaFixedByEquivOrbitsProdAddGroup
/-- **Burnside's lemma** : a (noncomputable) bijection between the disjoint union of all
`{x ∈ X | g • x = x}` for `g ∈ G` and the product `G × X/G`, where `G` is an additive group
acting on `X` and `X/G`denotes the quotient of `X` by the relation `orbitRel G X`. -/]
acting on `X` and `X/G` denotes the quotient of `X` by the relation `orbitRel G X`. -/]
noncomputable def sigmaFixedByEquivOrbitsProdGroup : (Σ a : α, fixedBy β a) ≃ Ω × α :=
calc
(Σ a : α, fixedBy β a) ≃ { ab : α × β // ab.1 • ab.2 = ab.2 } :=
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/GroupTheory/Perm/Centralizer.lean
Original file line number Diff line number Diff line change
Expand Up @@ -85,7 +85,7 @@ injectivity `Equiv.Perm.OnCycleFactors.kerParam_injective`, its range
* `Equiv.Perm.nat_card_centralizer g` computes the cardinality
of the centralizer of `g`.

* `Equiv.Perm.card_isConj_mul_eq g`computes the cardinality
* `Equiv.Perm.card_isConj_mul_eq g` computes the cardinality
of the conjugacy class of `g`.

* We now can compute the cardinality of the set of permutations with given cycle type.
Expand Down
4 changes: 2 additions & 2 deletions Mathlib/LinearAlgebra/PerfectPairing/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -41,14 +41,14 @@ class IsPerfPair (p : M →ₗ[R] N →ₗ[R] R) where
bijective_left (p) : Bijective p
bijective_right (p) : Bijective p.flip

/-- Given a perfect pairing between `M`and `N`, we may interchange the roles of `M` and `N`. -/
/-- Given a perfect pairing between `M` and `N`, we may interchange the roles of `M` and `N`. -/
protected lemma IsPerfPair.flip (hp : p.IsPerfPair) : p.flip.IsPerfPair where
bijective_left := IsPerfPair.bijective_right p
bijective_right := IsPerfPair.bijective_left p

variable [p.IsPerfPair]

/-- Given a perfect pairing between `M`and `N`, we may interchange the roles of `M` and `N`. -/
/-- Given a perfect pairing between `M` and `N`, we may interchange the roles of `M` and `N`. -/
instance flip.instIsPerfPair : p.flip.IsPerfPair := .flip ‹_›

variable (p)
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/LinearAlgebra/RootSystem/Finite/G2.lean
Original file line number Diff line number Diff line change
Expand Up @@ -35,7 +35,7 @@ stronger assumptions on the coefficients than here.
* `RootPairing.EmbeddedG2.threeShortAddTwoLong`: the long root `3α + 2β`
* `RootPairing.EmbeddedG2.span_eq_top`: a crystallographic reduced irreducible root pairing
containing two roots with pairing `-3` is spanned by this pair (thus two-dimensional).
* `RootPairing.EmbeddedG2.card_index_eq_twelve`: the `𝔤₂`root pairing has twelve roots.
* `RootPairing.EmbeddedG2.card_index_eq_twelve`: the `𝔤₂` root pairing has twelve roots.

## TODO
Once sufficient API for `RootPairing.Base` has been developed:
Expand Down
4 changes: 2 additions & 2 deletions Mathlib/Logic/Relation.lean
Original file line number Diff line number Diff line change
Expand Up @@ -36,8 +36,8 @@ the bundled version, see `Rel`.
* `Relation.EqvGen`: Equivalence closure. `EqvGen r` relates everything `ReflTransGen r` relates,
plus for all related pairs it relates them in the opposite order.
* `Relation.Comp`: Relation composition. We provide notation `∘r`. For `r : α → β → Prop` and
`s : β → γ → Prop`, `r ∘r s`relates `a : α` and `c : γ` iff there exists `b : β` that's related to
both.
`s : β → γ → Prop`, `r ∘r s` relates `a : α` and `c : γ` iff there exists `b : β` that's related
to both.
* `Relation.Map`: Image of a relation under a pair of maps. For `r : α → β → Prop`, `f : α → γ`,
`g : β → δ`, `Map r f g` is the relation `γ → δ → Prop` relating `f a` and `g b` for all `a`, `b`
related by `r`.
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/MeasureTheory/Measure/FiniteMeasureExt.lean
Original file line number Diff line number Diff line change
Expand Up @@ -14,7 +14,7 @@ public import Mathlib.MeasureTheory.Measure.HasOuterApproxClosed

The main Result is `ext_of_forall_mem_subalgebra_integral_eq_of_pseudoEMetric_complete_countable`:
Let `A` be a StarSubalgebra of `C(E, 𝕜)` that separates points and whose elements are bounded. If
the integrals of all elements of `A` with respect to two finite measures `P, P'`coincide, then the
the integrals of all elements of `A` with respect to two finite measures `P, P'` coincide, then the
measures coincide. In other words: If a Subalgebra separates points, it separates finite measures.
-/

Expand Down
2 changes: 1 addition & 1 deletion Mathlib/NumberTheory/LegendreSymbol/ZModChar.lean
Original file line number Diff line number Diff line change
Expand Up @@ -27,7 +27,7 @@ quadratic character, zmod
/-!
### Quadratic characters mod 4 and 8

We define the primitive quadratic characters `χ₄`on `ZMod 4`
We define the primitive quadratic characters `χ₄` on `ZMod 4`
and `χ₈`, `χ₈'` on `ZMod 8`.
-/

Expand Down
2 changes: 1 addition & 1 deletion Mathlib/RepresentationTheory/FiniteIndex.lean
Original file line number Diff line number Diff line change
Expand Up @@ -14,7 +14,7 @@ public import Mathlib.RepresentationTheory.Induced

Given a commutative ring `k`, a finite index subgroup `S ≤ G`, and a `k`-linear `S`-representation
`A`, this file defines an isomorphism $Ind_S^G(A) ≅ Coind_S^G(A)$. Given `g : G` and `a : A`, the
forward map sends `⟦g ⊗ₜ[k] a⟧` to the function `G → A`supported at `sg` by `ρ(s)(a)` for `s : S`
forward map sends `⟦g ⊗ₜ[k] a⟧` to the function `G → A` supported at `sg` by `ρ(s)(a)` for `s : S`
and which is 0 elsewhere. Meanwhile, the inverse sends `f : G → A` to `∑ᵢ ⟦gᵢ ⊗ₜ[k] f(gᵢ)⟧` for
`1 ≤ i ≤ n`, where `g₁, ..., gₙ` is a set of right coset representatives of `S`.

Expand Down
2 changes: 1 addition & 1 deletion Mathlib/RingTheory/Conductor.lean
Original file line number Diff line number Diff line change
Expand Up @@ -12,7 +12,7 @@ public import Mathlib.RingTheory.PowerBasis
# The conductor ideal
This file defines the conductor ideal of an element `x` of `R`-algebra `S`. This is the ideal of
`S` consisting of all elements `a` such that for all `b` in `S`, the product `a * b` lies in the
`R`subalgebra of `S` generated by `x`.
`R`-subalgebra of `S` generated by `x`.

-/

Expand Down
4 changes: 2 additions & 2 deletions Mathlib/RingTheory/DedekindDomain/AdicValuation.lean
Original file line number Diff line number Diff line change
Expand Up @@ -28,8 +28,8 @@ We define the completion of `K` with respect to the `v`-adic valuation, denoted
to its `v`-adic valuation.
- `IsDedekindDomain.HeightOneSpectrum.adicCompletionIntegers v` is the ring of integers of
`v.adicCompletion`.
- `IsDedekindDomain.HeightOneSpectrum.adicAbv v`is the `v`-adic absolute value on `K` defined as `b`
raised to negative `v`-adic valuation, for some `b` in `ℝ≥0`.
- `IsDedekindDomain.HeightOneSpectrum.adicAbv v` is the `v`-adic absolute value on `K` defined as
`b` raised to negative `v`-adic valuation, for some `b` in `ℝ≥0`.

## Main results
- `IsDedekindDomain.HeightOneSpectrum.intValuation_le_one` : The `v`-adic valuation on `R` is
Expand Down
4 changes: 2 additions & 2 deletions Mathlib/RingTheory/Ideal/Quotient/Operations.lean
Original file line number Diff line number Diff line change
Expand Up @@ -813,7 +813,7 @@ theorem ker_quotQuotMk : RingHom.ker (quotQuotMk I J) = I ⊔ J := by
comap_map_of_surjective (Ideal.Quotient.mk I) Ideal.Quotient.mk_surjective, ← RingHom.ker,
mk_ker, sup_comm]

/-- The ring homomorphism `R/(I ⊔ J) → (R/I)/J' `induced by `quotQuotMk` -/
/-- The ring homomorphism `R/(I ⊔ J) → (R/I)/J'` induced by `quotQuotMk` -/
def liftSupQuotQuotMk (I J : Ideal R) : R ⧸ I ⊔ J →+* (R ⧸ I) ⧸ J.map (Ideal.Quotient.mk I) :=
Ideal.Quotient.lift (I ⊔ J) (quotQuotMk I J) (ker_quotQuotMk I J).symm.le

Expand Down Expand Up @@ -954,7 +954,7 @@ theorem quotQuotMkₐ_toRingHom :
theorem coe_quotQuotMkₐ : ⇑(quotQuotMkₐ R I J) = quotQuotMk I J :=
rfl

/-- The injective algebra homomorphism `A / (I ⊔ J) → (A / I) / J'`induced by `quot_quot_mk`,
/-- The injective algebra homomorphism `A / (I ⊔ J) → (A / I) / J'` induced by `quotQuotMk`,
where `J'` is the projection `J` in `A / I`. -/
def liftSupQuotQuotMkₐ (I J : Ideal A) : A ⧸ I ⊔ J →ₐ[R] (A ⧸ I) ⧸ J.map (Quotient.mkₐ R I) :=
AlgHom.mk (liftSupQuotQuotMk I J) fun _ => rfl
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/RingTheory/Localization/Pi.lean
Original file line number Diff line number Diff line change
Expand Up @@ -20,7 +20,7 @@ public import Mathlib.RingTheory.KrullDimension.Zero
## Main Result

* `bijective_lift_piRingHom_algebraMap_comp_piEvalRingHom`: the canonical map from a
localization of a finite product of rings `R i `at a monoid `M` to the direct product of
localization of a finite product of rings `R i` at a monoid `M` to the direct product of
localizations `R i` at the projection of `M` onto each corresponding factor is bijective.

## Implementation notes
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Topology/Algebra/Module/Equiv.lean
Original file line number Diff line number Diff line change
Expand Up @@ -788,7 +788,7 @@ section Aut
/-!
### Automorphisms as continuous linear equivalences and as units of the ring of endomorphisms

The next theorems cover the identification between `M ≃L[R] M`and the group of units of the ring
The next theorems cover the identification between `M ≃L[R] M` and the group of units of the ring
`M →L[R] M`.
-/

Expand Down
Loading