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

[Merged by Bors] - feat(data/mv_polynomial/*): Simple lemmas #18084

Closed
wants to merge 2 commits into from

Conversation

YaelDillies
Copy link
Collaborator

A handful of missing lemmas about a • f where f is a multivariate polynomial.


Open in Gitpod

@YaelDillies YaelDillies added awaiting-review The author would like community review of the PR t-algebra Algebra (groups, rings, fields etc) labels Jan 7, 2023
Copy link
Member

@riccardobrasca riccardobrasca 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 d+

@@ -419,6 +419,10 @@ by rw [X_pow_eq_monomial, support_monomial, if_neg (one_ne_zero' R)]

@[simp] lemma support_zero : (0 : mv_polynomial σ R).support = ∅ := rfl

lemma support_smul [distrib_mul_action R S₁] {a : R} {f : mv_polynomial σ S₁} :
Copy link
Member

Choose a reason for hiding this comment

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

I think a and f should be explicit here, unless you have a reason to keep them implicit.

Copy link
Collaborator Author

Choose a reason for hiding this comment

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

I am matching finsupp.support_smul, which has them implicit. And I am happy to keep it like that because I noticed that we tend to never use the explicit arguments of , <, , lemmas.

src/data/mv_polynomial/variables.lean Outdated Show resolved Hide resolved
@bors
Copy link

bors bot commented Jan 10, 2023

✌️ YaelDillies can now approve this pull request. To approve and merge a pull request, simply reply with bors r+. More detailed instructions are available here.

@leanprover-community-bot-assistant leanprover-community-bot-assistant added delegated The PR author may merge after reviewing final suggestions. and removed awaiting-review The author would like community review of the PR labels Jan 10, 2023
@YaelDillies
Copy link
Collaborator Author

bors merge

bors bot pushed a commit that referenced this pull request Jan 10, 2023
A handful of missing lemmas about `a • f` where `f` is a multivariate polynomial.
@bors
Copy link

bors bot commented Jan 10, 2023

Pull request successfully merged into master.

Build succeeded:

@bors bors bot changed the title feat(data/mv_polynomial/*): Simple lemmas [Merged by Bors] - feat(data/mv_polynomial/*): Simple lemmas Jan 10, 2023
@bors bors bot closed this Jan 10, 2023
@bors bors bot deleted the total_degree_smul_le branch January 10, 2023 16:52
Sign up for free to subscribe to this conversation on GitHub. Already have an account? Sign in.
Labels
delegated The PR author may merge after reviewing final suggestions. t-algebra Algebra (groups, rings, fields etc)
Projects
None yet
Development

Successfully merging this pull request may close these issues.

3 participants