We read every piece of feedback, and take your input very seriously.
To see all available qualifiers, see our documentation.
There was an error while loading. Please reload this page.
Algebra.baseChange_lmul
1 parent dc0ee85 commit 9df8b6aCopy full SHA for 9df8b6a
Mathlib/RingTheory/TensorProduct/Basic.lean
@@ -1106,6 +1106,12 @@ variable {R M₁ M₂ ι ι₂ : Type*} (A : Type*)
1106
1107
end LinearMap
1108
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
+
1115
namespace LinearMap
1116
1117
variable (R A M N : Type*) [CommRing R] [CommRing A] [Algebra R A]
0 commit comments