The explicit sheaf condition for condensed sets #
We give the following three explicit descriptions of condensed objects:
Condensed.ofSheafStonean
: A finite-product-preserving presheaf onStonean
.Condensed.ofSheafProfinite
: A finite-product-preserving presheaf onProfinite
, satisfyingEqualizerCondition
.Condensed.ofSheafStonean
: A finite-product-preserving presheaf onCompHaus
, satisfyingEqualizerCondition
.
The property EqualizerCondition
is defined in Mathlib/CategoryTheory/Sites/RegularSheaves.lean
and it says that for any effective epi X ⟶ B
(in this case that is equivalent to being a
continuous surjection), the presheaf F
exhibits F(B)
as the equalizer of the two maps
F(X) ⇉ F(X ×_B X)
We also give variants for condensed objects in concrete categories whose forgetful functor reflects finite limits (resp. products), where it is enough to check the sheaf condition after postcomposing with the forgetful functor.
The condensed object associated to a finite-product-preserving presheaf on Stonean
.
Equations
- Condensed.ofSheafStonean F = (Condensed.StoneanCompHaus.equivalence A).functor.obj { val := F, cond := ⋯ }
Instances For
The condensed object associated to a presheaf on Stonean
whose postcomposition with the
forgetful functor preserves finite products.
Equations
- Condensed.ofSheafForgetStonean F = (Condensed.StoneanCompHaus.equivalence A).functor.obj { val := F, cond := ⋯ }
Instances For
The condensed object associated to a presheaf on Profinite
which preserves finite products and
satisfies the equalizer condition.
Equations
- Condensed.ofSheafProfinite F hF = (Condensed.ProfiniteCompHaus.equivalence A).functor.obj { val := F, cond := ⋯ }
Instances For
The condensed object associated to a presheaf on Profinite
whose postcomposition with the
forgetful functor preserves finite products and satisfies the equalizer condition.
Equations
- Condensed.ofSheafForgetProfinite F hF = (Condensed.ProfiniteCompHaus.equivalence A).functor.obj { val := F, cond := ⋯ }
Instances For
The condensed object associated to a presheaf on CompHaus
which preserves finite products and
satisfies the equalizer condition.
Equations
- Condensed.ofSheafCompHaus F hF = { val := F, cond := ⋯ }
Instances For
The condensed object associated to a presheaf on CompHaus
whose postcomposition with the
forgetful functor preserves finite products and satisfies the equalizer condition.
Equations
- Condensed.ofSheafForgetCompHaus F hF = { val := F, cond := ⋯ }
Instances For
A condensed object satisfies the equalizer condition.
A condensed object preserves finite products.
Equations
- ⋯ = ⋯
A condensed object regarded as a sheaf on Profinite
preserves finite products.
Equations
- ⋯ = ⋯
A condensed object regarded as a sheaf on Profinite
satisfies the equalizer condition.
A condensed object regarded as a sheaf on Stonean
preserves finite products.
Equations
- ⋯ = ⋯
A CondensedSet
version of Condensed.ofSheafStonean
.
Equations
Instances For
A CondensedSet
version of Condensed.ofSheafProfinite
.
Equations
Instances For
A CondensedSet
version of Condensed.ofSheafCompHaus
.
Equations
Instances For
A CondensedMod
version of Condensed.ofSheafStonean
.
Equations
Instances For
A CondensedMod
version of Condensed.ofSheafProfinite
.
Equations
- CondensedMod.ofSheafProfinite R F hF = Condensed.ofSheafProfinite F hF
Instances For
A CondensedMod
version of Condensed.ofSheafCompHaus
.
Equations
- CondensedMod.ofSheafCompHaus R F hF = Condensed.ofSheafCompHaus F hF