Documentation

Mathlib.RingTheory.AdicCompletion.Topology

Connection between adic properties and topological properties #

Main results #

theorem IsAdic.isHausdorff_iff {R : Type u_1} [CommRing R] [TopologicalSpace R] {I : Ideal R} (hI : IsAdic I) :

IsHausdorff I R is equivalent to being Hausdorff in the adic topology.

IsPrecomplete I R is equivalent to being complete in the adic topology.

IsAdicComplete I R is equivalent to being complete and hausdorff in the adic topology.