File tree Expand file tree Collapse file tree 1 file changed +10
-0
lines changed Expand file tree Collapse file tree 1 file changed +10
-0
lines changed Original file line number Diff line number Diff line change @@ -316,6 +316,16 @@ theorem comap_op_mul (M N : Submodule R Aᵐᵒᵖ) :
316
316
simp_rw [comap_equiv_eq_map_symm, map_unop_mul]
317
317
#align submodule.comap_op_mul Submodule.comap_op_mul
318
318
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
+
319
329
section
320
330
321
331
open Pointwise
You can’t perform that action at this time.
0 commit comments