Completion of a module with respect to an ideal. #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
In this file we define the notions of Hausdorff, precomplete, and complete for an R
-module M
with respect to an ideal I
:
Main definitions #
is_Hausdorff I M
: this says that the intersection ofI^n M
is0
.is_precomplete I M
: this says that every Cauchy sequence converges.is_adic_complete I M
: this says thatM
is Hausdorff and precomplete.Hausdorffification I M
: this is the universal Hausdorff module with a map fromM
.completion I M
: ifI
is finitely generated, then this is the universal complete module (TODO) with a map fromM
. This map is injective iffM
is Hausdorff and surjective iffM
is precomplete.
A module M
is Hausdorff with respect to an ideal I
if ⋂ I^n M = 0
.
- prec' : ∀ (f : ℕ → M), (∀ {m n : ℕ}, m ≤ n → f m ≡ f n [SMOD I ^ m • ⊤]) → (∃ (L : M), ∀ (n : ℕ), f n ≡ L [SMOD I ^ n • ⊤])
A module M
is precomplete with respect to an ideal I
if every Cauchy sequence converges.
Instances of this typeclass
- to_is_Hausdorff : is_Hausdorff I M
- to_is_precomplete : is_precomplete I M
A module M
is I
-adically complete if it is Hausdorff and precomplete.
Instances of this typeclass
The completion of a module with respect to an ideal. This is not necessarily Hausdorff. In fact, this is only complete if the ideal is finitely generated.
Equations
Instances for ↥adic_completion
The canonical linear map to the Hausdorffification.
universal property of Hausdorffification: any linear map to a Hausdorff module extends to a unique map from the Hausdorffification.
Uniqueness of lift.
The canonical linear map to the completion.
Linearly evaluating a sequence in the completion at a given input.
Equations
- adic_completion.eval I M n = {to_fun := λ (f : ↥(adic_completion I M)), f.val n, map_add' := _, map_smul' := _}