Documentation

Mathlib.RingTheory.Smooth.Pi

Formal-smoothness of finite products of rings #

Main result #

theorem Algebra.FormallySmooth.of_pi {R : Type (max u v)} {I : Type u} (A : IType (max u v)) [CommRing R] [(i : I) → CommRing (A i)] [(i : I) → Algebra R (A i)] [FormallySmooth R ((i : I) → A i)] (i : I) :
theorem Algebra.FormallySmooth.pi_iff {R : Type (max u v)} {I : Type u} (A : IType (max u v)) [CommRing R] [(i : I) → CommRing (A i)] [(i : I) → Algebra R (A i)] [Finite I] :
FormallySmooth R ((i : I) → A i) ∀ (i : I), FormallySmooth R (A i)
instance Algebra.FormallySmooth.instForallOfFinite {R : Type (max u v)} {I : Type u} (A : IType (max u v)) [CommRing R] [(i : I) → CommRing (A i)] [(i : I) → Algebra R (A i)] [Finite I] [∀ (i : I), FormallySmooth R (A i)] :
FormallySmooth R ((i : I) → A i)