Documentation

Mathlib.RingTheory.LocalRing.Quotient

We gather results about the quotients of local rings.

noncomputable def IsLocalRing.basisQuotient {R : Type u_1} {S : Type u_2} [CommRing R] [CommRing S] [Algebra R S] [IsLocalRing R] [Module.Finite R S] [Module.Free R S] {ι : Type u_3} [Fintype ι] (b : Basis ι R S) :

Given a basis of S, the induced basis of S / Ideal.map (algebraMap R S) p.

Equations
Instances For
    theorem IsLocalRing.basisQuotient_apply {R : Type u_1} {S : Type u_2} [CommRing R] [CommRing S] [Algebra R S] [IsLocalRing R] [Module.Finite R S] [Module.Free R S] {ι : Type u_3} [Fintype ι] (b : Basis ι R S) (i : ι) :
    theorem IsLocalRing.basisQuotient_repr {R : Type u_1} {S : Type u_2} [CommRing R] [CommRing S] [Algebra R S] [IsLocalRing R] [Module.Finite R S] [Module.Free R S] {ι : Type u_4} [Fintype ι] (b : Basis ι R S) (x : S) (i : ι) :
    @[deprecated IsLocalRing.quotient_span_eq_top_iff_span_eq_top (since := "2024-11-11")]

    Alias of IsLocalRing.quotient_span_eq_top_iff_span_eq_top.

    @[deprecated IsLocalRing.finrank_quotient_map (since := "2024-11-11")]

    Alias of IsLocalRing.finrank_quotient_map.

    @[deprecated IsLocalRing.basisQuotient (since := "2024-11-11")]
    def LocalRing.basisQuotient {R : Type u_1} {S : Type u_2} [CommRing R] [CommRing S] [Algebra R S] [IsLocalRing R] [Module.Finite R S] [Module.Free R S] {ι : Type u_3} [Fintype ι] (b : Basis ι R S) :

    Alias of IsLocalRing.basisQuotient.


    Given a basis of S, the induced basis of S / Ideal.map (algebraMap R S) p.

    Equations
    Instances For
      @[deprecated IsLocalRing.basisQuotient_apply (since := "2024-11-11")]
      theorem LocalRing.basisQuotient_apply {R : Type u_1} {S : Type u_2} [CommRing R] [CommRing S] [Algebra R S] [IsLocalRing R] [Module.Finite R S] [Module.Free R S] {ι : Type u_3} [Fintype ι] (b : Basis ι R S) (i : ι) :

      Alias of IsLocalRing.basisQuotient_apply.

      @[deprecated IsLocalRing.basisQuotient_repr (since := "2024-11-11")]
      theorem LocalRing.basisQuotient_repr {R : Type u_1} {S : Type u_2} [CommRing R] [CommRing S] [Algebra R S] [IsLocalRing R] [Module.Finite R S] [Module.Free R S] {ι : Type u_4} [Fintype ι] (b : Basis ι R S) (x : S) (i : ι) :

      Alias of IsLocalRing.basisQuotient_repr.