File tree Expand file tree Collapse file tree 3 files changed +3
-3
lines changed
Algebra/Algebra/Subalgebra Expand file tree Collapse file tree 3 files changed +3
-3
lines changed Original file line number Diff line number Diff line change @@ -754,7 +754,7 @@ theorem ext_of_adjoin_eq_top {s : Set A} (h : adjoin R s = ⊤) ⦃φ₁ φ₂ :
754754 (hs : s.EqOn φ₁ φ₂) : φ₁ = φ₂ :=
755755 ext fun _x => adjoin_le_equalizer φ₁ φ₂ hs <| h.symm ▸ trivial
756756
757- /-- Two algebra morphisms are equal on `Algebra.span s` iff they are equal on s -/
757+ /-- Two algebra morphisms are equal on `Algebra.span s` iff they are equal on `s`. -/
758758theorem eqOn_adjoin_iff {φ ψ : A →ₐ[R] B} {s : Set A} :
759759 Set.EqOn φ ψ (adjoin R s) ↔ Set.EqOn φ ψ s := by
760760 have (S : Set A) : S ≤ equalizer φ ψ ↔ Set.EqOn φ ψ S := Iff.rfl
Original file line number Diff line number Diff line change @@ -801,7 +801,7 @@ class MulSemiringActionSemiHomClass (F : Type*)
801801 extends DistribMulActionSemiHomClass F φ R S, RingHomClass F R S
802802
803803/-- `MulSemiringActionHomClass F M R S` states that `F` is a type of morphisms preserving
804- the ring structure and equivariant with respect to a `DistribMulAction` of `M` on `R` and `S` .
804+ the ring structure and equivariant with respect to a `DistribMulAction` of `M` on `R` and `S`.
805805-/
806806abbrev MulSemiringActionHomClass
807807 (F : Type *)
Original file line number Diff line number Diff line change @@ -12,7 +12,7 @@ public import Mathlib.RingTheory.PowerBasis
1212# The conductor ideal
1313This file defines the conductor ideal of an element `x` of `R`-algebra `S`. This is the ideal of
1414`S` consisting of all elements `a` such that for all `b` in `S`, the product `a * b` lies in the
15- `R` subalgebra of `S` generated by `x`.
15+ `R`- subalgebra of `S` generated by `x`.
1616
1717-/
1818
You can’t perform that action at this time.
0 commit comments