Skip to content
This repository has been archived by the owner on Jul 24, 2024. It is now read-only.

[Merged by Bors] - feat(algebra/triv_sq_zero_ext): lemmas about big operators #18488

Closed
wants to merge 4 commits into from

Conversation

eric-wieser
Copy link
Member

@eric-wieser eric-wieser commented Feb 23, 2023

Some more results following on from #18384.

For now this just has the list lemmas. The multiset and finset lemmas are hard to state cleanly.


Open in Gitpod

My attempt at stating the omitted multiset and finset versions can be found in the git history of this PR as

lemma snd_multiset_prod {ι} [decidable_eq ι] [comm_semiring R] [add_comm_monoid M]
  [module R M] [module Rᵐᵒᵖ M] [is_central_scalar R M]
  (s : multiset ι) (f : ι → tsze R M) :
  (s.map f).prod.snd =
    (s.map (λ i, ((s.erase i).map (λ j, (f j).fst)).prod • (f i).snd)).sum :=

lemma snd_prod {ι} [decidable_eq ι] [comm_semiring R] [add_comm_monoid M]
  [module R M] [module Rᵐᵒᵖ M] [is_central_scalar R M]
  (s : finset ι) (f : ι → tsze R M) :
  (∏ i in s, f i).snd =
    ∑ i in s, (∏ j in s.erase i, (f j).fst) • (f i).snd :=

With some extra machinery it should be possible to avoid [decidable_eq ι].

@eric-wieser eric-wieser added WIP Work in progress modifies-synchronized-file This PR touches a files that has already been ported to mathlib4, and may need a synchronization PR. labels Feb 23, 2023
@eric-wieser eric-wieser force-pushed the eric-wieser/tsze-big_operators branch from 9882aa8 to eed6456 Compare March 2, 2023 14:14
@eric-wieser eric-wieser added awaiting-review The author would like community review of the PR awaiting-CI The author would like to see what CI has to say before doing more work. and removed modifies-synchronized-file This PR touches a files that has already been ported to mathlib4, and may need a synchronization PR. WIP Work in progress labels Mar 14, 2023
@github-actions github-actions bot removed the awaiting-CI The author would like to see what CI has to say before doing more work. label Mar 14, 2023
@eric-wieser eric-wieser added the t-algebra Algebra (groups, rings, fields etc) label Mar 15, 2023
@ocfnash
Copy link
Collaborator

ocfnash commented Mar 15, 2023

Thanks!

bors merge

@github-actions github-actions bot added ready-to-merge All that is left is for bors to build and merge this PR. (Remember you need to say `bors r+`.) and removed awaiting-review The author would like community review of the PR labels Mar 15, 2023
bors bot pushed a commit that referenced this pull request Mar 15, 2023
Some more results following on from #18384.

For now this just has the list lemmas. The multiset and finset lemmas are hard to state cleanly.
@bors
Copy link

bors bot commented Mar 15, 2023

Pull request successfully merged into master.

Build succeeded:

@bors bors bot changed the title feat(algebra/triv_sq_zero_ext): lemmas about big operators [Merged by Bors] - feat(algebra/triv_sq_zero_ext): lemmas about big operators Mar 15, 2023
@bors bors bot closed this Mar 15, 2023
@bors bors bot deleted the eric-wieser/tsze-big_operators branch March 15, 2023 17:21
Sign up for free to subscribe to this conversation on GitHub. Already have an account? Sign in.
Labels
ready-to-merge All that is left is for bors to build and merge this PR. (Remember you need to say `bors r+`.) t-algebra Algebra (groups, rings, fields etc)
Projects
None yet
Development

Successfully merging this pull request may close these issues.

2 participants