Collapsing covers #
We define the endofunctor on Scheme.Cover P
that collapses a cover to a single object cover.
noncomputable def
AlgebraicGeometry.Scheme.Cover.sigma
{P : CategoryTheory.MorphismProperty Scheme}
{S : Scheme}
[IsLocalAtSource P]
[UnivLE.{v, u}]
(𝒰 : Cover P S)
:
Cover P S
If 𝒰
is a cover of S
, this is the single object cover where the covering
object is the disjoint union.
Equations
- One or more equations did not get rendered due to their size.
Instances For
@[simp]
theorem
AlgebraicGeometry.Scheme.Cover.sigma_J
{P : CategoryTheory.MorphismProperty Scheme}
{S : Scheme}
[IsLocalAtSource P]
[UnivLE.{v, u}]
(𝒰 : Cover P S)
:
@[simp]
theorem
AlgebraicGeometry.Scheme.Cover.sigma_obj
{P : CategoryTheory.MorphismProperty Scheme}
{S : Scheme}
[IsLocalAtSource P]
[UnivLE.{v, u}]
(𝒰 : Cover P S)
(x✝ : PUnit.{v + 1})
:
@[simp]
theorem
AlgebraicGeometry.Scheme.Cover.sigma_f
{P : CategoryTheory.MorphismProperty Scheme}
{S : Scheme}
[IsLocalAtSource P]
[UnivLE.{v, u}]
(𝒰 : Cover P S)
(x✝ : ↥S)
:
@[simp]
theorem
AlgebraicGeometry.Scheme.Cover.sigma_map
{P : CategoryTheory.MorphismProperty Scheme}
{S : Scheme}
[IsLocalAtSource P]
[UnivLE.{v, u}]
(𝒰 : Cover P S)
(x✝ : PUnit.{v + 1})
:
instance
AlgebraicGeometry.Scheme.Cover.instUniqueJSigma
{P : CategoryTheory.MorphismProperty Scheme}
{S : Scheme}
[IsLocalAtSource P]
[UnivLE.{v, u}]
(𝒰 : Cover P S)
:
Equations
noncomputable def
AlgebraicGeometry.Scheme.Cover.toSigma
{P : CategoryTheory.MorphismProperty Scheme}
{S : Scheme}
[IsLocalAtSource P]
[UnivLE.{v, u}]
[P.IsMultiplicative]
(𝒰 : Cover P S)
:
𝒰
refines the single object cover defined by 𝒰
.
Equations
Instances For
@[simp]
theorem
AlgebraicGeometry.Scheme.Cover.toSigma_idx
{P : CategoryTheory.MorphismProperty Scheme}
{S : Scheme}
[IsLocalAtSource P]
[UnivLE.{v, u}]
[P.IsMultiplicative]
(𝒰 : Cover P S)
(x✝ : 𝒰.J)
:
@[simp]
theorem
AlgebraicGeometry.Scheme.Cover.toSigma_app
{P : CategoryTheory.MorphismProperty Scheme}
{S : Scheme}
[IsLocalAtSource P]
[UnivLE.{v, u}]
[P.IsMultiplicative]
(𝒰 : Cover P S)
(i : 𝒰.J)
:
noncomputable def
AlgebraicGeometry.Scheme.Cover.Hom.sigma
{P : CategoryTheory.MorphismProperty Scheme}
{S : Scheme}
[IsLocalAtSource P]
[UnivLE.{v, u}]
[P.IsMultiplicative]
{𝒰 𝒱 : Cover P S}
(f : 𝒰 ⟶ 𝒱)
:
A refinement of coverings induces a refinement on the single object coverings.
Equations
- One or more equations did not get rendered due to their size.
Instances For
@[simp]
theorem
AlgebraicGeometry.Scheme.Cover.Hom.sigma_idx
{P : CategoryTheory.MorphismProperty Scheme}
{S : Scheme}
[IsLocalAtSource P]
[UnivLE.{v, u}]
[P.IsMultiplicative]
{𝒰 𝒱 : Cover P S}
(f : 𝒰 ⟶ 𝒱)
(x✝ : 𝒰.sigma.J)
:
@[simp]
theorem
AlgebraicGeometry.Scheme.Cover.Hom.sigma_app
{P : CategoryTheory.MorphismProperty Scheme}
{S : Scheme}
[IsLocalAtSource P]
[UnivLE.{v, u}]
[P.IsMultiplicative]
{𝒰 𝒱 : Cover P S}
(f : 𝒰 ⟶ 𝒱)
(x✝ : 𝒰.sigma.J)
:
(sigma f).app x✝ = CategoryTheory.Limits.Sigma.desc fun (j : 𝒰.J) =>
CategoryTheory.CategoryStruct.comp (f.app j) (CategoryTheory.Limits.Sigma.ι 𝒱.obj (f.idx j))
noncomputable def
AlgebraicGeometry.Scheme.Cover.sigmaFunctor
{P : CategoryTheory.MorphismProperty Scheme}
{S : Scheme}
[IsLocalAtSource P]
[UnivLE.{v, u}]
[P.IsMultiplicative]
:
CategoryTheory.Functor (Cover P S) (Cover P S)
Collapsing a cover to a single object cover is functorial.
Equations
- One or more equations did not get rendered due to their size.
Instances For
@[simp]
theorem
AlgebraicGeometry.Scheme.Cover.sigmaFunctor_obj
{P : CategoryTheory.MorphismProperty Scheme}
{S : Scheme}
[IsLocalAtSource P]
[UnivLE.{v, u}]
[P.IsMultiplicative]
(𝒰 : Cover P S)
:
@[simp]
theorem
AlgebraicGeometry.Scheme.Cover.sigmaFunctor_map
{P : CategoryTheory.MorphismProperty Scheme}
{S : Scheme}
[IsLocalAtSource P]
[UnivLE.{v, u}]
[P.IsMultiplicative]
{X✝ Y✝ : Cover P S}
(f : X✝ ⟶ Y✝)
: