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.
Subalgebra.finite_sup
CommSemiring
1 parent 23844d2 commit b5f6488Copy full SHA for b5f6488
Mathlib/RingTheory/TensorProduct/Basic.lean
@@ -1222,7 +1222,7 @@ theorem endTensorEndAlgHom_apply (f : End A M) (g : End R N) :
1222
1223
end Module
1224
1225
-theorem Subalgebra.finite_sup {K L : Type*} [CommRing K] [CommRing L] [Algebra K L]
+theorem Subalgebra.finite_sup {K L : Type*} [CommSemiring K] [CommSemiring L] [Algebra K L]
1226
(E1 E2 : Subalgebra K L) [Module.Finite K E1] [Module.Finite K E2] :
1227
Module.Finite K ↥(E1 ⊔ E2) := by
1228
rw [← E1.range_val, ← E2.range_val, ← Algebra.TensorProduct.productMap_range]
0 commit comments