Skip to content

Commit

Permalink
Complete metrics trivially have unique limits
Browse files Browse the repository at this point in the history
  • Loading branch information
Columbus240 committed Oct 19, 2024
1 parent ed38ff6 commit d5ddabf
Showing 1 changed file with 14 additions and 0 deletions.
14 changes: 14 additions & 0 deletions theories/Topology/Completeness.v
Original file line number Diff line number Diff line change
Expand Up @@ -82,6 +82,20 @@ Proof.
eauto.
Qed.

Lemma complete_net_limit_ex_unique :
complete d ->
forall x:nat -> X, cauchy d x ->
exists! x0:X, net_limit x x0 (I:=nat_DS).
Proof.
intros Hd x Hx.
rewrite complete_net_limit_char in Hd.
specialize (Hd x Hx) as [x0 Hx0].
exists x0. split; auto.
intros x1 Hx1.
unshelve eapply (Hausdorff_impl_net_limit_unique _ _ x0 x1 Hx0 Hx1).
apply metrizable_Hausdorff. exists d; auto.
Qed.

Lemma convergent_sequence_is_cauchy:
forall (x:Net nat_DS X)
(x0:point_set X),
Expand Down

0 comments on commit d5ddabf

Please sign in to comment.