Skip to content

Commit

Permalink
Add instances
Browse files Browse the repository at this point in the history
  • Loading branch information
erdOne committed Jan 6, 2025
1 parent 4af89a0 commit 4365b38
Show file tree
Hide file tree
Showing 3 changed files with 9 additions and 0 deletions.
3 changes: 3 additions & 0 deletions Mathlib/RingTheory/Etale/Pi.lean
Original file line number Diff line number Diff line change
Expand Up @@ -30,4 +30,7 @@ theorem pi_iff [Finite I] :
simp_rw [FormallyEtale.iff_unramified_and_smooth, forall_and]
rw [FormallyUnramified.pi_iff A, FormallySmooth.pi_iff A]

instance [Finite I] [∀ i, FormallyEtale R (A i)] : FormallyEtale R (Π i, A i) :=
.of_unramified_and_smooth

end Algebra.FormallyEtale
3 changes: 3 additions & 0 deletions Mathlib/RingTheory/Smooth/Pi.lean
Original file line number Diff line number Diff line change
Expand Up @@ -118,4 +118,7 @@ theorem pi_iff [Finite I] :
rwa [mul_sub, ← map_mul, mul_comm, mul_assoc, (he.idem i).eq, he', ← map_mul, ← Pi.single_mul,
one_mul, sub_eq_zero] at this

instance [Finite I] [∀ i, FormallySmooth R (A i)] : FormallySmooth R (Π i, A i) :=
(pi_iff _).mpr ‹_›

end Algebra.FormallySmooth
3 changes: 3 additions & 0 deletions Mathlib/RingTheory/Unramified/Pi.lean
Original file line number Diff line number Diff line change
Expand Up @@ -95,4 +95,7 @@ theorem pi_iff :
Ideal.Quotient.mkₐ_eq_mk]
exact Ideal.mem_map_of_mem (Ideal.Quotient.mk J') (hf (Pi.single x r))

instance [∀ i, FormallyUnramified R (f i)] : FormallyUnramified R (Π i, f i) :=
(pi_iff _).mpr ‹_›

end Algebra.FormallyUnramified

0 comments on commit 4365b38

Please sign in to comment.