Skip to content

Commit fa1d892

Browse files
committed
feat: Add Submodule.restrictScalars_mul. (#8649)
Co-authored-by: Andrew Yang <36414270+erdOne@users.noreply.github.com>
1 parent 27d3a24 commit fa1d892

File tree

1 file changed

+10
-0
lines changed

1 file changed

+10
-0
lines changed

Mathlib/Algebra/Algebra/Operations.lean

Lines changed: 10 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -316,6 +316,16 @@ theorem comap_op_mul (M N : Submodule R Aᵐᵒᵖ) :
316316
simp_rw [comap_equiv_eq_map_symm, map_unop_mul]
317317
#align submodule.comap_op_mul Submodule.comap_op_mul
318318

319+
lemma restrictScalars_mul {A B C} [CommSemiring A] [CommSemiring B] [Semiring C]
320+
[Algebra A B] [Algebra A C] [Algebra B C] [IsScalarTower A B C] {I J : Submodule B C} :
321+
(I * J).restrictScalars A = I.restrictScalars A * J.restrictScalars A := by
322+
apply le_antisymm
323+
· intro x (hx : x ∈ I * J)
324+
refine Submodule.mul_induction_on hx ?_ ?_
325+
· exact fun m hm n hn ↦ mul_mem_mul hm hn
326+
· exact fun _ _ ↦ add_mem
327+
· exact mul_le.mpr (fun _ hm _ hn ↦ mul_mem_mul hm hn)
328+
319329
section
320330

321331
open Pointwise

0 commit comments

Comments
 (0)