Inverse limits of schemes with affine transition maps #
In this file, we develop API for inverse limits of schemes with affine transition maps, following EGA IV 8 and https://stacks.math.columbia.edu/tag/01YT.
Suppose we have a cofiltered diagram of nonempty quasi-compact schemes, whose transition maps are affine. Then the limit is also nonempty.
Suppose we have a cofiltered diagram of schemes whose transition maps are affine. The limit of a family of compatible nonempty quasicompact closed sets in the diagram is also nonempty.
A variant of exists_mem_of_isClosed_of_nonempty where the closed sets are only defined
for the objects over a given j : I.
Let { Dᵢ } be a cofiltered diagram of compact schemes with affine transition maps.
If U ⊆ Dⱼ contains the image of limᵢ Dᵢ ⟶ Dⱼ, then it contains the image of some Dₖ ⟶ Dⱼ.
Given a diagram { Dᵢ } of schemes and a open U ⊆ Dᵢ,
this is the diagram of { Dⱼᵢ⁻¹ U }_{j ≤ i}.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The map Dⱼᵢ⁻¹ U ⟶ Dᵢ from the restricted diagram to the original diagram.
Equations
- AlgebraicGeometry.opensDiagramι D i U = { app := fun (j : CategoryTheory.Over i) => ((TopologicalSpace.Opens.map (D.map j.hom).base).obj U).ι, naturality := ⋯ }
Instances For
Given a diagram { Dᵢ } of schemes and a open U ⊆ Dᵢ,
the preimage of U ⊆ Dᵢ under the map lim Dᵢ ⟶ Dᵢ is the limit of { Dⱼᵢ⁻¹ U }_{j ≤ i}.
This is the underlying cone, and it is limiting as witnessed by isLimitOpensCone below.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Given a diagram { Dᵢ }_{i ∈ I} of schemes and a open U ⊆ Dᵢ,
the preimage of U ⊆ Dᵢ under the map lim Dᵢ ⟶ Dᵢ is the limit of { Dⱼᵢ⁻¹ U }_{j ≤ i}.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Cofiltered Limits and Schemes of Finite Type #
Given a cofiltered diagram D of quasi-compact S-schemes with affine transition maps,
and another scheme X of finite type over S.
Then the canonical map colim Homₛ(Dᵢ, X) ⟶ Homₛ(lim Dᵢ, X) is injective.
In other words, for each pair of a : Homₛ(Dᵢ, X) and b : Homₛ(Dⱼ, X) that give rise to the
same map Homₛ(lim Dᵢ, X), there exists a k with fᵢ : k ⟶ i and fⱼ : k ⟶ j such that
D(fᵢ) ≫ a = D(fⱼ) ≫ b.
This results is formalized in Scheme.exists_hom_hom_comp_eq_comp_of_locallyOfFiniteType.
We first reduce to the case i = j, and the goal is to reduce to the case where X and S
are affine, where the result follows from commutative algebra.
To achieve this, we show that there exists some i₀ ⟶ i such that for each x, a x and b x
are contained in the same component (i.e. given an open cover 𝒰ₛ of S,
and 𝒰ₓ of X refining 𝒰ₛ, the range of x ↦ (a x, b x) falls in the diagonal part
⋃ᵢⱼ 𝒰ₓⱼ ×[𝒰ₛᵢ] 𝒰ₓⱼ).
Then we may restrict to the sub-diagram over i₀ (which is cofinal because D is cofiltered),
and check locally on X, reducing to the affine case.
For the actual implementation, we wrap i, a, b, the limit cone lim Dᵢ, and open covers
of X and S into a structure ExistsHomHomCompEqCompAux for convenience.
See the injective part of (1) => (3) of https://stacks.math.columbia.edu/tag/01ZC.
(Implementation)
An auxiliary structure used to prove Scheme.exists_hom_hom_comp_eq_comp_of_locallyOfFiniteType.
See the section docstring.
(Implementation) The limit cone. See the section docstring.
- hc : CategoryTheory.Limits.IsLimit self.c
(Implementation) The limit cone is a limit. See the section docstring.
- i : I
(Implementation)
a. See the section docstring.(Implementation)
b. See the section docstring.- 𝒰S : S.OpenCover
(Implementation) An open cover on
S. See the section docstring. - 𝒰X (i : (CategoryTheory.Precoverage.ZeroHypercover.pullback₁ f self.𝒰S).I₀) : ((CategoryTheory.Precoverage.ZeroHypercover.pullback₁ f self.𝒰S).X i).OpenCover
(Implementation) A family of open covers refining
𝒰S. See the section docstring.
Instances For
(Implementation)
The index i' such that a and b restricted onto i' maps into the diagonal components.
See the section docstring.
Instances For
(Implementation) The map from i' to i. See the section docstring.
Instances For
(Implementation)
The map sending x to (a x, b x), which should fall in the diagonal component.
See the section docstring.
Equations
- A.g = CategoryTheory.CategoryStruct.comp (D.map A.hii') (CategoryTheory.Limits.pullback.lift A.a A.b ⋯)
Instances For
(Implementation)
The covering of D(i') by the pullback of the diagonal components of X ×ₛ X.
See the section docstring.
Equations
- One or more equations did not get rendered due to their size.
Instances For
(Implementation) An affine open cover refining 𝒰D₀. See the section docstring.
Equations
- A.𝒰D = CategoryTheory.Precoverage.ZeroHypercover.bind A.𝒰D₀ fun (x : A.𝒰D₀.I₀) => (A.𝒰D₀.X x).affineCover
Instances For
(Implementation) The diagram restricted to Over i'. See the section docstring.
Equations
- A.D' j = (CategoryTheory.Over.post D).comp ((CategoryTheory.Over.pullback (A.𝒰D.f j)).comp (CategoryTheory.Over.forget (A.𝒰D.X j)))
Instances For
(Implementation) The limit cone restricted to Over i'. See the section docstring.
Equations
- A.c' j = ((CategoryTheory.Over.pullback (A.𝒰D.f j)).comp (CategoryTheory.Over.forget (A.𝒰D.X j))).mapCone ((CategoryTheory.Over.conePost D A.i').obj A.c)
Instances For
(Implementation)
The limit cone restricted to Over i' is still a limit because the diagram is cofiltered.
See the section docstring.
Equations
- A.hc' j = CategoryTheory.Limits.isLimitOfPreserves ((CategoryTheory.Over.pullback (A.𝒰D.f j)).comp (CategoryTheory.Over.forget (A.𝒰D.X j))) (CategoryTheory.Over.isLimitConePost A.i' A.hc)
Instances For
Given a cofiltered diagram D of quasi-compact S-schemes with affine transition maps,
and another scheme X of finite type over S.
Then the canonical map colim Homₛ(Dᵢ, X) ⟶ Homₛ(lim Dᵢ, X) is injective.
In other words, for each pair of a : Homₛ(Dᵢ, X) and b : Homₛ(Dⱼ, X) that give rise to the
same map Homₛ(lim Dᵢ, X), there exists a k with fᵢ : k ⟶ i and fⱼ : k ⟶ j such that
D(fᵢ) ≫ a = D(fⱼ) ≫ b.
Sections of the limit #
Let D be a cofiltered diagram schemes with affine transition map.
Consider the canonical map colim Γ(Dᵢ, ⊤) ⟶ Γ(lim Dᵢ, ⊤).
If D consists of quasicompact schemes, then this map is injective. More generally, we show
that if s t : Γ(Dᵢ, U) have equal image in lim Dᵢ, then they are equal at some Γ(Dⱼ, Dⱼᵢ⁻¹U).
See AlgebraicGeometry.exists_app_map_eq_map_of_isLimit.
If D consists of qcqs schemes, then this map is surjective. Specifically, we show that
any s : Γ(lim Dᵢ, ⊤) comes from Γ(Dᵢ, ⊤) for some i.
See AlgebraicGeometry.exists_appTop_π_eq_of_isLimit.
These two results imply that PreservesLimit D Scheme.Γ.rightOp, which is available as an instance.