Documentation

Mathlib.RingTheory.Unramified.Pi

Formal-unramification of finite products of rings #

Main result #

theorem Algebra.FormallyUnramified.pi_iff {R : Type (max u v)} {I : Type v} [Finite I] (f : IType (max u v)) [CommRing R] [(i : I) → CommRing (f i)] [(i : I) → Algebra R (f i)] :
FormallyUnramified R ((i : I) → f i) ∀ (i : I), FormallyUnramified R (f i)
instance Algebra.FormallyUnramified.instForall {R : Type (max u v)} {I : Type v} [Finite I] (f : IType (max u v)) [CommRing R] [(i : I) → CommRing (f i)] [(i : I) → Algebra R (f i)] [∀ (i : I), FormallyUnramified R (f i)] :
FormallyUnramified R ((i : I) → f i)