mathlib4
mathlib4 copied to clipboard
Feat(LinearAlgebra/TensorProduct/RightExactness): Tensoring with a quotient of the ring
Informally we show (R⧸I) ⊗ M = M/IM.
- [ ] depends on: #13119
If someone can golf away this dependency I'd be happy! The existing proof that Submodule.map (TensorProduct.lid R M) (range (rTensor M (Submodule.subtype I))) = I • ⊤ isn't great.
This PR/issue depends on:
- ~~leanprover-community/mathlib4#13119~~ By Dependent Issues (🤖). Happy coding!
Also can you provide _ ∘ₗ TensorProduct.mk R _ M 1 = Submodule.mkQ _? Just found out that I needed them :D
Also can you provide
_ ∘ₗ TensorProduct.mk R _ M 1 = Submodule.mkQ _? Just found out that I needed them :D
I'm not sure what you have in mind exactly. I added four new lemmas in terms of composition of linear maps, do any of them fit your use case?
Edit: Oh I see, you want (LinearEquiv.toLinearMap_symm_comp_eq _ _).mp (quotTensorEquivQuotSMul_symm_comp_mkQ I). I'll add a lemma for that
Thanks a lot! maintainer merge
🚀 Pull request has been placed on the maintainer queue by erdOne.
Pull request successfully merged into master.
Build succeeded: