mathlib4 icon indicating copy to clipboard operation
mathlib4 copied to clipboard

feat(RingTheory/TwoSidedIdeal/Basic): two-sided-ideal as a bimodule

Open jjaassoonn opened this issue 1 year ago • 1 comments


Open in Gitpod

jjaassoonn avatar Jul 05 '24 16:07 jjaassoonn

PR summary 24700a44cc

Import changes for modified files

Dependency changes

File Base Count Head Count Change
Mathlib.RingTheory.TwoSidedIdeal.Basic 560 563 +3 (+0.54%)
Import changes for all files
Files Import difference
Mathlib.RingTheory.TwoSidedIdeal.Basic 3

Declarations diff

+ coeAddMonoidHom + coe_mop_smul + coe_smul + instance : SMul R I where smul r x := ⟨r • x.1, I.mul_mem_left _ _ x.2⟩ + instance : SMul Rᵐᵒᵖ I where smul r x := ⟨r • x.1, I.mul_mem_right _ _ x.2⟩ + instance : SMulCommClass R Rᵐᵒᵖ I + leftModule + rightModule + subtype + subtypeMop

You can run this locally as follows
## summary with just the declaration names:
./scripts/no_lost_declarations.sh short <optional_commit>

## more verbose report:
./scripts/no_lost_declarations.sh <optional_commit>

github-actions[bot] avatar Jul 05 '24 16:07 github-actions[bot]

Thanks!

maintainer merge

kbuzzard avatar Jul 07 '24 19:07 kbuzzard

🚀 Pull request has been placed on the maintainer queue by kbuzzard.

github-actions[bot] avatar Jul 07 '24 19:07 github-actions[bot]

!bench

mattrobball avatar Jul 07 '24 19:07 mattrobball

Here are the benchmark results for commit 24700a44cc5105d4d63f0d4d17910de09d2b78be. There were no significant changes against commit d2e8846f9bb14855a6d84e36552bc60e38bab88f.

leanprover-bot avatar Jul 07 '24 19:07 leanprover-bot

bors merge

kim-em avatar Jul 07 '24 21:07 kim-em

Pull request successfully merged into master.

Build succeeded:

mathlib-bors[bot] avatar Jul 07 '24 22:07 mathlib-bors[bot]