Skip to content

Commit b5f6488

Browse files
committed
chore(RingTheory/TensorProduct/Basic): relax the condition of Subalgebra.finite_sup to CommSemiring (#12323)
1 parent 23844d2 commit b5f6488

File tree

1 file changed

+1
-1
lines changed

1 file changed

+1
-1
lines changed

Mathlib/RingTheory/TensorProduct/Basic.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -1222,7 +1222,7 @@ theorem endTensorEndAlgHom_apply (f : End A M) (g : End R N) :
12221222

12231223
end Module
12241224

1225-
theorem Subalgebra.finite_sup {K L : Type*} [CommRing K] [CommRing L] [Algebra K L]
1225+
theorem Subalgebra.finite_sup {K L : Type*} [CommSemiring K] [CommSemiring L] [Algebra K L]
12261226
(E1 E2 : Subalgebra K L) [Module.Finite K E1] [Module.Finite K E2] :
12271227
Module.Finite K ↥(E1 ⊔ E2) := by
12281228
rw [← E1.range_val, ← E2.range_val, ← Algebra.TensorProduct.productMap_range]

0 commit comments

Comments
 (0)