Restricted products of sets, groups and rings, and their topology #
We define the restricted product of R : ι → Type*
of types, relative to
a family of subsets A : (i : ι) → Set (R i)
and a filter 𝓕 : Filter ι
. This
is the set of all x : Π i, R i
such that the set {j | x j ∈ A j}
belongs to 𝓕
.
We denote it by Πʳ i, [R i, A i]_[𝓕]
.
The main case of interest, which we shall refer to as the "classical restricted product",
is that of 𝓕 = cofinite
. Recall that this is the filter of all subsets of ι
, which are
cofinite in the sense that they have finite complement.
Hence, the associated restricted product is the set of all x : Π i, R i
such that
x j ∈ A j
for all but finitely many j
s. We denote it simply by Πʳ i, [R i, A i]
.
Another notable case is that of the principal filter 𝓕 = 𝓟 s
corresponding to some subset s
of ι
. The associated restricted product Πʳ i, [R i, A i]_[𝓟 s]
is the set of all
x : Π i, R i
such that x j ∈ A j
for all j ∈ s
. Put another way, this is just
(Π i ∈ s, A i) × (Π i ∉ s, R i)
, modulo the obvious isomorphism.
We endow these types with the obvious algebraic structures, as well as their natural topology, which we describe below. We also show various compatibility results.
In particular, with the theory of adeles in mind, we show that if each R i
is a locally compact
topological ring with open subring A i
, and if all but finitely many of the A i
s are also
compact, then Πʳ i, [R i, A i]
is a locally compact topological ring.
Main definitions #
RestrictedProduct
: the restricted product of a familyR
of types, relative to a familyA
of subsets and a filter𝓕
on the indexing set. This is denotedΠʳ i, [R i, A i]_[𝓕]
, or simplyΠʳ i, [R i, A i]
when𝓕 = cofinite
.RestrictedProduct.instDFunLike
: interpret an element ofΠʳ i, [R i, A i]_[𝓕]
as an element ofΠ i, R i
using theDFunLike
machinery.RestrictedProduct.structureMap
: the inclusion map fromΠ i, A i
toΠʳ i, [R i, A i]_[𝓕]
.RestrictedProduct.topologicalSpace
: theTopologicalSpace
instance onΠʳ i, [R i, A i]_[𝓕]
.
Topology on the restricted product #
The topology on the restricted product Πʳ i, [R i, A i]_[𝓕]
is defined in the following way:
- If
𝓕
is some principal filter𝓟 s
, recall thatΠʳ i, [R i, A i]_[𝓟 s]
is canonically identified with(Π i ∈ s, A i) × (Π i ∉ s, R i)
. We endow it with the product topology, which is also the topology induced from the full productΠ i, R i
. - In general, we note that
𝓕
is the infimum of the principal filters coarser than𝓕
. We then endowΠʳ i, [R i, A i]_[𝓕]
with the inductive limit / final topology associated to the inclusion mapsΠʳ i, [R i, A i]_[𝓟 s] → Πʳ i, [R i, A i]_[𝓕]
where𝓕 ≤ 𝓟 s
.
In particular:
- On the classical restricted product, with respect to the cofinite filter, this corresponds to
taking the inductive limit of the
Πʳ i, [R i, A i]_[𝓟 s]
over all cofinite setss : Set ι
. - If
𝓕 = 𝓟 s
is a principal filter, this second step clearly does not change the topology, sinces
belongs to the indexing set of the inductive limit.
Taking advantage of that second remark, we do not actually declare an instance specific to
principal filters. Instead, we provide directly the general instance (corresponding to step 2 above)
as RestrictedProduct.topologicalSpace
. We then prove that, for a principal filter, the
map to the full product is an inducing (RestrictedProduct.isEmbedding_coe_of_principal
),
and that the topology for a general 𝓕
is indeed the expected inductive limit
(RestrictedProduct.topologicalSpace_eq_iSup
).
Main statements #
RestrictedProduct.isEmbedding_coe_of_principal
: for any setS
,Πʳ i, [R i, A i]_[𝓟 S]
is endowed with the subset topology coming fromΠ i, R i
.RestrictedProduct.topologicalSpace_eq_iSup
: the topology onΠʳ i, [R i, A i]_[𝓕]
is the inductive limit / final topology associated to the natural mapsΠʳ i, [R i, A i]_[𝓟 S] → Πʳ i, [R i, A i]_[𝓕]
, where𝓕 ≤ 𝓟 S
.RestrictedProduct.continuous_dom
: a map fromΠʳ i, [R i, A i]_[𝓕]
is continuous if and only if its restriction to eachΠʳ i, [R i, A i]_[𝓟 s]
(with𝓕 ≤ 𝓟 s
) is continuous.RestrictedProduct.continuous_dom_prod_left
: assume that eachA i
is an open subset ofR i
. Then, for any topological spaceY
, a map fromY × Πʳ i, [R i, A i]
is continuous if and only if its restriction to eachY × Πʳ i, [R i, A i]_[𝓟 S]
(withS
cofinite) is continuous.RestrictedProduct.isTopologicalGroup
: if eachR i
is a topological group and eachA i
is an open subgroup ofR i
, thenΠʳ i, [R i, A i]
is a topological group.RestrictedProduct.isTopologicalRing
: if eachR i
is a topological ring and eachA i
is an open subring ofR i
, thenΠʳ i, [R i, A i]
is a topological ring.RestrictedProduct.continuousSMul
: if some topological monoidG
acts on eachM i
, and eachA i
is stable for that action, then the natural action ofG
onΠʳ i, [M i, A i]
is also continuous. In particular, if eachM i
is a topologicalR
-module and eachA i
is an open sub-R
-module ofM i
, thenΠʳ i, [M i, A i]
is a topologicalR
-module.RestrictedProduct.weaklyLocallyCompactSpace_of_cofinite
: if eachR i
is weakly locally compact, eachA i
is open, and all but finitely manyA i
s are also compact, then the restricted productΠʳ i, [R i, A i]
is weakly locally compact.RestrictedProduct.locallyCompactSpace_of_group
: assume that eachR i
is a locally compact group withA i
an open subgroup. Assume also that all but finitely manyA i
s are compact. Then the restricted productΠʳ i, [R i, A i]
is a locally compact group.
Notation #
Πʳ i, [R i, A i]_[𝓕]
isRestrictedProduct R A 𝓕
.Πʳ i, [R i, A i]
isRestrictedProduct R A cofinite
.
Implementation details #
Outside of principal filters and the cofinite filter, the topology we define on the restricted product does not seem well-behaved. While declaring a single instance is practical, it may conflict with more interesting topologies in some other cases. Thus, future contributions should not restrain from specializing these instances to principal and cofinite filters if necessary.
Tags #
restricted product, adeles, ideles
Definition and elementary maps #
The restricted product of a family R : ι → Type*
of types, relative to subsets
A : (i : ι) → Set (R i)
and the filter 𝓕 : Filter ι
, is the set of all x : Π i, R i
such that the set {j | x j ∈ A j}
belongs to 𝓕
. We denote it by Πʳ i, [R i, A i]_[𝓕]
.
The most common use case is with 𝓕 = cofinite
, in which case the restricted product is the set
of all x : Π i, R i
such that x j ∈ A j
for all but finitely many j
. We denote it simply
by Πʳ i, [R i, A i]
.
Similarly, if S
is a principal filter, the restricted product Πʳ i, [R i, A i]_[𝓟 s]
is the set of all x : Π i, R i
such that ∀ j ∈ S, x j ∈ A j
.
Instances For
Πʳ i, [R i, A i]_[𝓕]
is RestrictedProduct R A 𝓕
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Pretty printer defined by notation3
command.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Pretty printer defined by notation3
command.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Πʳ i, [R i, A i]
is RestrictedProduct R A cofinite
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- RestrictedProduct.instDFunLike R A = { coe := fun (x : RestrictedProduct (fun (i : ι) => R i) (fun (i : ι) => A i) 𝓕) (i : ι) => ↑x i, coe_injective' := ⋯ }
The structure map of the restricted product is the obvious inclusion from Π i, A i
into Πʳ i, [R i, A i]_[𝓕]
.
Equations
- RestrictedProduct.structureMap R A 𝓕 x = ⟨fun (i : ι) => ↑(x i), ⋯⟩
Instances For
If 𝓕 ≤ 𝓖
, the restricted product Πʳ i, [R i, A i]_[𝓖]
is naturally included in
Πʳ i, [R i, A i]_[𝓕]
. This is the corresponding map.
Equations
- RestrictedProduct.inclusion R A h x = ⟨⇑x, ⋯⟩
Instances For
Algebraic instances on restricted products #
In this section, we endow the restricted product with its algebraic instances.
To avoid any unnecessary coercions, we use subobject classes for the subset B i
of each R i
.
Equations
- RestrictedProduct.instOneCoeOfOneMemClass R = { one := ⟨fun (x : ι) => 1, ⋯⟩ }
Equations
- RestrictedProduct.instZeroCoeOfZeroMemClass R = { zero := ⟨fun (x : ι) => 0, ⋯⟩ }
Equations
- RestrictedProduct.instInvCoeOfInvMemClass R = { inv := fun (x : RestrictedProduct (fun (i : ι) => R i) (fun (i : ι) => ↑(B i)) 𝓕) => ⟨fun (i : ι) => (x i)⁻¹, ⋯⟩ }
Equations
- RestrictedProduct.instNegCoeOfNegMemClass R = { neg := fun (x : RestrictedProduct (fun (i : ι) => R i) (fun (i : ι) => ↑(B i)) 𝓕) => ⟨fun (i : ι) => -x i, ⋯⟩ }
Equations
- RestrictedProduct.instMulCoeOfMulMemClass R = { mul := fun (x y : RestrictedProduct (fun (i : ι) => R i) (fun (i : ι) => ↑(B i)) 𝓕) => ⟨fun (i : ι) => x i * y i, ⋯⟩ }
Equations
- RestrictedProduct.instAddCoeOfAddMemClass R = { add := fun (x y : RestrictedProduct (fun (i : ι) => R i) (fun (i : ι) => ↑(B i)) 𝓕) => ⟨fun (i : ι) => x i + y i, ⋯⟩ }
Equations
- RestrictedProduct.instSMulCoeOfSMulMemClass R = { smul := fun (g : G) (x : RestrictedProduct (fun (i : ι) => R i) (fun (i : ι) => ↑(B i)) 𝓕) => ⟨fun (i : ι) => g • x i, ⋯⟩ }
Equations
- RestrictedProduct.instVAddCoeOfVAddMemClass R = { vadd := fun (g : G) (x : RestrictedProduct (fun (i : ι) => R i) (fun (i : ι) => ↑(B i)) 𝓕) => ⟨fun (i : ι) => g +ᵥ x i, ⋯⟩ }
Equations
- RestrictedProduct.instDivCoeOfSubgroupClass R = { div := fun (x y : RestrictedProduct (fun (i : ι) => R i) (fun (i : ι) => ↑(B i)) 𝓕) => ⟨fun (i : ι) => x i / y i, ⋯⟩ }
Equations
- RestrictedProduct.instSubCoeOfAddSubgroupClass R = { sub := fun (x y : RestrictedProduct (fun (i : ι) => R i) (fun (i : ι) => ↑(B i)) 𝓕) => ⟨fun (i : ι) => x i - y i, ⋯⟩ }
Equations
- RestrictedProduct.instPowCoeNatOfSubmonoidClass R = { pow := fun (x : RestrictedProduct (fun (i : ι) => R i) (fun (i : ι) => ↑(B i)) 𝓕) (n : ℕ) => ⟨fun (i : ι) => x i ^ n, ⋯⟩ }
Equations
- RestrictedProduct.instPowCoeIntOfSubgroupClass R = { pow := fun (x : RestrictedProduct (fun (i : ι) => R i) (fun (i : ι) => ↑(B i)) 𝓕) (n : ℤ) => ⟨fun (i : ι) => x i ^ n, ⋯⟩ }
Equations
- RestrictedProduct.instNatCastCoeOfAddSubmonoidWithOneClass R = { natCast := fun (n : ℕ) => ⟨fun (x : ι) => ↑n, ⋯⟩ }
Equations
- RestrictedProduct.instIntCastCoeOfSubringClass R = { intCast := fun (n : ℤ) => ⟨fun (x : ι) => ↑n, ⋯⟩ }
Equations
- RestrictedProduct.instAddGroupCoeOfAddSubgroupClass R = Function.Injective.addGroup (fun (f : RestrictedProduct (fun (i : ι) => R i) (fun (i : ι) => ↑(B i)) 𝓕) => ⇑f) ⋯ ⋯ ⋯ ⋯ ⋯ ⋯ ⋯
Equations
- RestrictedProduct.instGroupCoeOfSubgroupClass R = Function.Injective.group (fun (f : RestrictedProduct (fun (i : ι) => R i) (fun (i : ι) => ↑(B i)) 𝓕) => ⇑f) ⋯ ⋯ ⋯ ⋯ ⋯ ⋯ ⋯
Equations
- RestrictedProduct.instRingCoeOfSubringClass R = Function.Injective.ring (fun (f : RestrictedProduct (fun (i : ι) => R i) (fun (i : ι) => ↑(B i)) 𝓕) => ⇑f) ⋯ ⋯ ⋯ ⋯ ⋯ ⋯ ⋯ ⋯ ⋯ ⋯ ⋯ ⋯
Topology on the restricted product #
The topology on the restricted product Πʳ i, [R i, A i]_[𝓕]
is defined in the following way:
- If
𝓕
is some principal filter𝓟 s
, recall thatΠʳ i, [R i, A i]_[𝓟 s]
is canonically identified with(Π i ∈ s, A i) × (Π i ∉ s, R i)
. We endow it with the product topology, which is also the topology induced from the full productΠ i, R i
. - In general, we note that
𝓕
is the infimum of the principal filters coarser than𝓕
. We then endowΠʳ i, [R i, A i]_[𝓕]
with the inductive limit / final topology associated to the inclusion mapsΠʳ i, [R i, A i]_[𝓟 s] → Πʳ i, [R i, A i]_[𝓕]
where𝓕 ≤ 𝓟 s
.
In particular:
- On the classical restricted product, with respect to the cofinite filter, this corresponds to
taking the inductive limit of the
Πʳ i, [R i, A i]_[𝓟 s]
over all cofinite setss : Set ι
. - If
𝓕 = 𝓟 s
is a principal filter, this second step clearly does not change the topology, sinces
belongs to the indexing set of the inductive limit.
Taking advantage of that second remark, we do not actually declare an instance specific to
principal filters. Instead, we provide directly the general instance (corresponding to step 2 above)
as RestrictedProduct.topologicalSpace
. We then prove that, for a principal filter, the
map to the full product is an inducing (RestrictedProduct.isEmbedding_coe_of_principal
),
and that the topology for a general 𝓕
is indeed the expected inductive limit
(RestrictedProduct.topologicalSpace_eq_iSup
).
Note: outside of these two cases, this topology on the restricted product does not seem well-behaved. While declaring a single instance is practical, it may conflict with more interesting topologies in some other cases. Thus, future contributions should not restrain from specializing these instances to principal and cofinite filters if necessary.
Definition of the topology #
Equations
- One or more equations did not get rendered due to their size.
Topological facts in the principal case #
The obvious bijection between Πʳ i, [R i, A i]_[⊤]
and Π i, A i
is a homeomorphism.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The obvious bijection between Πʳ i, [R i, A i]_[⊥]
and Π i, R i
is a homeomorphism.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Assume that S
is a subset of ι
with finite complement, that each R i
is weakly locally
compact, and that A i
is compact for all i ∈ S
. Then the restricted product
Πʳ i, [R i, A i]_[𝓟 S]
is locally compact.
Note: we spell "S
has finite complement" as cofinite ≤ 𝓟 S
.
Topological facts in the general case #
The universal property of the topology on the restricted product: a map from
Πʳ i, [R i, A i]_[𝓕]
is continuous iff its restriction to each Πʳ i, [R i, A i]_[𝓟 s]
(with 𝓕 ≤ 𝓟 s
) is continuous.
Π i, A i
has the subset topology from the restricted product.
Topological facts in the case where 𝓕 = cofinite
and all A i
s are open #
The classical restricted product, associated to the cofinite filter, satisfies more topological
properties when each A i
is an open subset of R i
. The key fact is that each
Πʳ i, [R i, A i]_[𝓟 S]
(with S
cofinite) then embeds as an open subset in
Πʳ i, [R i, A i]
.
This allows us to prove a "universal property with parameters", expressing that for any
arbitrary topolgical space X
(of "parameters"), the product X × Πʳ i, [R i, A i]
is still the inductive limit of the X × Πʳ i, [R i, A i]_[𝓟 S]
for S
cofinite.
This fact, which is not true for a general inductive limit, will allow us to prove continuity of functions of two variables (e.g algebraic operations), which would otherwise be inaccessible.
Π i, A i
is homeomorphic to an open subset of the restricted product.
If each R i
is weakly locally compact, each A i
is open, and all but finitely many A i
s
are also compact, then the restricted product Πʳ i, [R i, A i]
is weakly locally compact.
The universal property with parameters of the topology on the restricted product:
for any topological space Y
of "parameters", a map from (Πʳ i, [R i, A i]) × Y
is continuous
iff its restriction to each (Πʳ i, [R i, A i]_[𝓟 S]) × Y
(with S
cofinite) is continuous.
The universal property with parameters of the topology on the restricted product:
for any topological space Y
of "parameters", a map from Y × Πʳ i, [R i, A i]
is continuous
iff its restriction to each Y × Πʳ i, [R i, A i]_[𝓟 S]
(with S
cofinite) is continuous.
A map from Πʳ i, [R i, A i] × Πʳ i, [R' i, A' i]
is continuous
iff its restriction to each Πʳ i, [R i, A i]_[𝓟 S] × Πʳ i, [R' i, A' i]_[𝓟 S]
(with S
cofinite) is continuous.
This is the key result for continuity of multiplication and addition.
Compatibility properties between algebra and topology #
Assume that each R i
is a locally compact group with A i
an open subgroup.
Assume also that all but finitely many A i
s are compact.
Then the restricted product Πʳ i, [R i, A i]
is a locally compact group.
Assume that each R i
is a locally compact additive group with A i
an open subgroup.
Assume also that all but finitely many A i
s are compact.
Then the restricted product Πʳ i, [R i, A i]
is a locally compact additive group.