Completeness in terms of cauchy
filters vs is_cau_seq
sequences
In this file we apply metric.complete_of_cauchy_seq_tendsto
to prove that a normed_ring
is complete in terms of cauchy
filter if and only if it is complete in terms
of cau_seq
Cauchy sequences.
theorem
cau_seq.tendsto_limit
{β : Type v}
[normed_ring β]
[hn : is_absolute_value norm]
(f : cau_seq β norm)
[cau_seq.is_complete β norm] :
filter.tendsto ⇑f filter.at_top (𝓝 f.lim)
@[instance]
theorem
cau_seq_iff_cauchy_seq
{α : Type u}
[normed_field α]
{u : ℕ → α} :
is_cau_seq norm u ↔ cauchy_seq u
In a normed field, cau_seq
coincides with the usual notion of Cauchy sequences.
@[instance]
A complete normed field is complete as a metric space, as Cauchy sequences converge by assumption and this suffices to characterize completeness.