-
Notifications
You must be signed in to change notification settings - Fork 298
[Merged by Bors] - chore(algebra/order/with_zero): Move unrelated lemmas #15676
Conversation
@@ -49,7 +49,7 @@ A `pow` form of `nat.factorization_choose_le` | |||
lemma pow_factorization_choose_le (hn : 0 < n) : p ^ (choose n k).factorization p ≤ n := | |||
begin | |||
cases le_or_lt p 1, | |||
{ exact (pow_le_pow_of_le h).trans ((le_of_eq (one_pow _)).trans hn) }, | |||
{ exact (pow_le_pow_of_le_left' h _).trans ((le_of_eq (one_pow _)).trans hn) }, |
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.
Is this coming from a rename?
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.
No, I deleted pow_le_pow_of_le
because it duplicates pow_le_pow_of_le_left'
.
@@ -106,7 +106,7 @@ end | |||
@[simp, to_additive] | |||
lemma prod_take_mul_prod_drop : | |||
∀ (L : list M) (i : ℕ), (L.take i).prod * (L.drop i).prod = L.prod | |||
| [] i := by simp | |||
| [] i := by simp [@zero_le' ℕ] |
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.
These @zero_le' ℕ
are somewhat ugly. Can you fix that regression please?
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.
Not sure how... This is a bug in to_additive
that shows only now because of the import changes.
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.
this has come up before in #10767
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.
lgtm, hopefully @[to_additive]
can get fixed :/
@@ -106,7 +106,7 @@ end | |||
@[simp, to_additive] | |||
lemma prod_take_mul_prod_drop : | |||
∀ (L : list M) (i : ℕ), (L.take i).prod * (L.drop i).prod = L.prod | |||
| [] i := by simp | |||
| [] i := by simp [@zero_le' ℕ] |
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.
this has come up before in #10767
Thanks 🎉 bors merge |
Move a bunch of lemmas that were not about `whatever_with_zero` from `algebra.order.with_zero` to `algebra.group_power.order`. Delete `nat.le_zero_iff` in favor of `le_zero_iff`.
Pull request successfully merged into master. Build succeeded: |
Move a bunch of lemmas that were not about
whatever_with_zero
fromalgebra.order.with_zero
toalgebra.group_power.order
. Deletenat.le_zero_iff
in favor ofle_zero_iff
.This is preparatory work to be able to import
algebra.order.with_zero
earlier (in particular inalgebra.order.field
).