Formal-étaleness of finite products of rings #
Main result #
Algebra.FormallyEtale.pi_iff
: IfI
is finite,Π i : I, A i
isR
-formally-étale if and only if eachA i
isR
-formally-étale.
theorem
Algebra.FormallyEtale.pi_iff
{R : Type (max u v)}
{I : Type u}
(A : I → Type (max u v))
[CommRing R]
[(i : I) → CommRing (A i)]
[(i : I) → Algebra R (A i)]
[Finite I]
:
FormallyEtale R ((i : I) → A i) ↔ ∀ (i : I), FormallyEtale R (A i)
instance
Algebra.FormallyEtale.instForallOfFinite
{R : Type (max u v)}
{I : Type u}
(A : I → Type (max u v))
[CommRing R]
[(i : I) → CommRing (A i)]
[(i : I) → Algebra R (A i)]
[Finite I]
[∀ (i : I), FormallyEtale R (A i)]
:
FormallyEtale R ((i : I) → A i)