Skip to content

Commit 9df8b6a

Browse files
committed
feat(RingTheory/TensorProduct): Add Algebra.baseChange_lmul (#18424)
Co-authored-by: Andrew Yang <36414270+erdOne@users.noreply.github.com>
1 parent dc0ee85 commit 9df8b6a

File tree

1 file changed

+6
-0
lines changed

1 file changed

+6
-0
lines changed

Mathlib/RingTheory/TensorProduct/Basic.lean

Lines changed: 6 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -1106,6 +1106,12 @@ variable {R M₁ M₂ ι ι₂ : Type*} (A : Type*)
11061106

11071107
end LinearMap
11081108

1109+
lemma Algebra.baseChange_lmul {R B : Type*} [CommRing R] [CommRing B] [Algebra R B]
1110+
{A : Type*} [CommRing A] [Algebra R A] (f : B) :
1111+
(Algebra.lmul R B f).baseChange A = Algebra.lmul A (A ⊗[R] B) (1 ⊗ₜ f) := by
1112+
ext i
1113+
simp
1114+
11091115
namespace LinearMap
11101116

11111117
variable (R A M N : Type*) [CommRing R] [CommRing A] [Algebra R A]

0 commit comments

Comments
 (0)