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/direct_sum/decomposition): add an induction principle for direct_sum.decomposition class #15654

Closed
wants to merge 1 commit into from

Conversation

jjaassoonn
Copy link
Collaborator

If direct_sum.decomposition M and p : M → Prop, then to prove p m for an arbitrary m, it suffices to prove p 0 and p x for homogeneous x and p being preserved by add.


Open in Gitpod

@jjaassoonn jjaassoonn added the awaiting-review The author would like community review of the PR label Jul 24, 2022
@jjaassoonn jjaassoonn requested a review from eric-wieser July 24, 2022 00:28
@hrmacbeth hrmacbeth changed the title feat(algebra/direct_sum/decomposition): add an induction principal for direct_sum.decomposition class feat(algebra/direct_sum/decomposition): add an induction principle for direct_sum.decomposition class Jul 24, 2022
@urkud urkud added the t-algebra Algebra (groups, rings, fields etc) label Jul 24, 2022
Copy link
Member

@jcommelin jcommelin left a comment

Choose a reason for hiding this comment

The reason will be displayed to describe this comment to others. Learn more.

Thanks 🎉

bors merge

@leanprover-community-bot-assistant leanprover-community-bot-assistant 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 Jul 29, 2022
bors bot pushed a commit that referenced this pull request Jul 29, 2022
…r `direct_sum.decomposition` class (#15654)

If `direct_sum.decomposition M` and `p : M → Prop`, then to prove `p m` for an arbitrary `m`, it suffices to prove `p 0` and `p x` for homogeneous x and `p` being preserved by add.
Comment on lines +79 to +80
let ℳ' : ι → add_submonoid M :=
λ i, (⟨ℳ i, λ _ _, add_mem_class.add_mem, zero_mem_class.zero_mem _⟩ : add_submonoid M),
Copy link
Member

Choose a reason for hiding this comment

The reason will be displayed to describe this comment to others. Learn more.

This is another argument for addressing #15053 sooner rather than later; but no reason to cancel merging this PR.

@bors
Copy link

bors bot commented Jul 29, 2022

Pull request successfully merged into master.

Build succeeded:

@bors bors bot changed the title feat(algebra/direct_sum/decomposition): add an induction principle for direct_sum.decomposition class [Merged by Bors] - feat(algebra/direct_sum/decomposition): add an induction principle for direct_sum.decomposition class Jul 29, 2022
@bors bors bot closed this Jul 29, 2022
@bors bors bot deleted the jjaassoonn/homogeneous_ind branch July 29, 2022 15:19
bottine pushed a commit to bottine/mathlib that referenced this pull request Jul 30, 2022
…r `direct_sum.decomposition` class (leanprover-community#15654)

If `direct_sum.decomposition M` and `p : M → Prop`, then to prove `p m` for an arbitrary `m`, it suffices to prove `p 0` and `p x` for homogeneous x and `p` being preserved by add.
robertylewis pushed a commit that referenced this pull request Aug 2, 2022
…r `direct_sum.decomposition` class (#15654)

If `direct_sum.decomposition M` and `p : M → Prop`, then to prove `p m` for an arbitrary `m`, it suffices to prove `p 0` and `p x` for homogeneous x and `p` being preserved by add.
khwilson pushed a commit that referenced this pull request Aug 2, 2022
…r `direct_sum.decomposition` class (#15654)

If `direct_sum.decomposition M` and `p : M → Prop`, then to prove `p m` for an arbitrary `m`, it suffices to prove `p 0` and `p x` for homogeneous x and `p` being preserved by add.
bors bot pushed a commit that referenced this pull request Jan 27, 2023
By imitating the current `graded_algebra`, this pr builds `graded_module` over some `graded algebra`

Co-authored-by: Eric Wieser @eric-wieser 

- [x] depends on: #14626
- [x] depends on: #15654



Co-authored-by: Eric Wieser <[email protected]>
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.

5 participants