-
Notifications
You must be signed in to change notification settings - Fork 298
[Merged by Bors] - feat(data/mv_polynomial/*): Simple •
lemmas
#18084
Conversation
There was a problem hiding this 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₁} : |
There was a problem hiding this comment.
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.
There was a problem hiding this comment.
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.
✌️ YaelDillies can now approve this pull request. To approve and merge a pull request, simply reply with |
bors merge |
Pull request successfully merged into master. Build succeeded: |
•
lemmas•
lemmas
A handful of missing lemmas about
a • f
wheref
is a multivariate polynomial.