Documentation

Mathlib.RingTheory.MaximalSpectrum

Maximal spectrum of a commutative ring #

The maximal spectrum of a commutative ring is the type of all maximal ideals. It is naturally a subset of the prime spectrum endowed with the subspace topology.

Main definitions #

Implementation notes #

The Zariski topology on the maximal spectrum is defined as the subspace topology induced by the natural inclusion into the prime spectrum to avoid API duplication for zero loci.

structure MaximalSpectrum (R : Type u_1) [CommSemiring R] :
Type u_1

The maximal spectrum of a commutative ring R is the type of all maximal ideals of R.

  • asIdeal : Ideal R
  • IsMaximal : self.asIdeal.IsMaximal
Instances For
    theorem MaximalSpectrum.ext {R : Type u_1} {inst✝ : CommSemiring R} {x y : MaximalSpectrum R} (asIdeal : x.asIdeal = y.asIdeal) :
    x = y

    The natural inclusion from the maximal spectrum to the prime spectrum.

    Equations
    • x.toPrimeSpectrum = { asIdeal := x.asIdeal, isPrime := }
    Instances For
      theorem MaximalSpectrum.toPrimeSpectrum_injective {R : Type u_1} [CommSemiring R] :
      Function.Injective MaximalSpectrum.toPrimeSpectrum
      theorem MaximalSpectrum.iInf_localization_eq_bot (R : Type u_4) [CommRing R] [IsDomain R] (K : Type u_5) [Field K] [Algebra R K] [IsFractionRing R K] :
      ⨅ (v : MaximalSpectrum R), Localization.subalgebra.ofField K v.asIdeal.primeCompl =

      An integral domain is equal to the intersection of its localizations at all its maximal ideals viewed as subalgebras of its field of fractions.

      theorem PrimeSpectrum.iInf_localization_eq_bot (R : Type u_4) [CommRing R] [IsDomain R] (K : Type u_5) [Field K] [Algebra R K] [IsFractionRing R K] :
      ⨅ (v : PrimeSpectrum R), Localization.subalgebra.ofField K v.asIdeal.primeCompl =

      An integral domain is equal to the intersection of its localizations at all its prime ideals viewed as subalgebras of its field of fractions.

      @[reducible, inline]

      The product of localizations at all maximal ideals of a commutative semiring.

      Equations
      Instances For

        The canonical ring homomorphism from a commutative semiring to the product of its localizations at all maximal ideals. It is always injective.

        Equations
        Instances For

          Functoriality of PiLocalization but restricted to bijective ring homs. If R and S are commutative rings, surjectivity would be enough.

          Equations
          • One or more equations did not get rendered due to their size.
          Instances For
            theorem MaximalSpectrum.toPiLocalization_not_surjective_of_infinite {ι : Type u_5} (R : ιType u_4) [(i : ι) → CommSemiring (R i)] [∀ (i : ι), Nontrivial (R i)] [Infinite ι] :
            theorem MaximalSpectrum.finite_of_toPiLocalization_pi_surjective {ι : Type u_5} {R : ιType u_4} [(i : ι) → CommSemiring (R i)] [∀ (i : ι), Nontrivial (R i)] (h : Function.Surjective (MaximalSpectrum.toPiLocalization ((i : ι) → R i))) :
            @[reducible, inline]

            The product of localizations at all prime ideals of a commutative semiring.

            Equations
            Instances For

              The canonical ring homomorphism from a commutative semiring to the product of its localizations at all prime ideals. It is always injective.

              Equations
              Instances For

                The projection from the product of localizations at primes to the product of localizations at maximal ideals.

                Equations
                Instances For

                  If R has Krull dimension ≤ 0, then piLocalizationToIsMaximal R is an isomorphism.

                  Equations
                  • One or more equations did not get rendered due to their size.
                  Instances For

                    A ring homomorphism induces a homomorphism between the products of localizations at primes.

                    Equations
                    • One or more equations did not get rendered due to their size.
                    Instances For
                      theorem PrimeSpectrum.toPiLocalization_not_surjective_of_infinite {ι : Type u_5} (R : ιType u_4) [(i : ι) → CommSemiring (R i)] [∀ (i : ι), Nontrivial (R i)] [Infinite ι] :
                      theorem PrimeSpectrum.finite_of_toPiLocalization_pi_surjective {ι : Type u_5} {R : ιType u_4} [(i : ι) → CommSemiring (R i)] [∀ (i : ι), Nontrivial (R i)] (h : Function.Surjective (PrimeSpectrum.toPiLocalization ((i : ι) → R i))) :