Skip to content

Conversation

@leanprover-community-bot-assistant
Copy link
Collaborator

@leanprover-community-bot-assistant leanprover-community-bot-assistant commented Oct 29, 2025

No description provided.

wlog h : p.natDegree ≤ n generalizing n
· refine Nat.decreasingInduction' (fun n hn _ ih ↦ ?_) (le_of_not_ge h) ?_
· rw [coeff_divByMonic_X_sub_C_rec, ih, eq_comm, Icc_eq_cons_Ioc (Nat.succ_le.mpr hn),
· rw [coeff_divByMonic_X_sub_C_rec, ih, eq_comm, Icc_eq_cons_Ioc (Nat.succ_le_iff.mpr hn),
Copy link
Member

Choose a reason for hiding this comment

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

Suggested change
· rw [coeff_divByMonic_X_sub_C_rec, ih, eq_comm, Icc_eq_cons_Ioc (Nat.succ_le_iff.mpr hn),
· rw [coeff_divByMonic_X_sub_C_rec, ih, eq_comm, Icc_eq_cons_Ioc (Nat.succ_le_of_lt hn),

rw [add_comm]; exact (mem_Icc.mp hi).1
· exact this _ le_rfl
rw [Icc_eq_empty (Nat.lt_succ.mpr h).not_ge, sum_empty]
rw [Icc_eq_empty (Nat.lt_succ_iff.mpr h).not_ge, sum_empty]
Copy link
Member

Choose a reason for hiding this comment

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

Suggested change
rw [Icc_eq_empty (Nat.lt_succ_iff.mpr h).not_ge, sum_empty]
rw [Icc_eq_empty (Nat.lt_succ_of_le h).not_ge, sum_empty]

lemma eval_homogenize {p : K[X]} {n : ℕ} (hn : p.natDegree ≤ n) (x : Fin 2 → K) (hx : x 10) :
MvPolynomial.eval x (p.homogenize n) = p.eval (x 0 / x 1) * x 1 ^ n := by
simp only [homogenize, Polynomial.eval_eq_sum_range' (Nat.lt_succ.mpr hn),
simp only [homogenize, Polynomial.eval_eq_sum_range' (Nat.lt_succ_iff.mpr hn),
Copy link
Member

Choose a reason for hiding this comment

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

Suggested change
simp only [homogenize, Polynomial.eval_eq_sum_range' (Nat.lt_succ_iff.mpr hn),
simp only [homogenize, Polynomial.eval_eq_sum_range' (Nat.lt_succ_of_le hn),

Copy link
Member

@kbuzzard kbuzzard left a comment

Choose a reason for hiding this comment

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

I've gone through all the diff. I think writing Nat.foo.mp or Nat.foo.2 is daft when foo is actually proved as \<one_way, the_other_way\>, not least because the individual implication lemmas typically have names which are at least as explanatory as the iff ones. I changed the first one myself and pushed, and then realised there were 10+ others so I've left them for someone else to decide.

There's a merge conflict but other than that this looks ready to go.

@kim-em
Copy link

kim-em commented Nov 3, 2025

bors merge

@mathlib-bors
Copy link

mathlib-bors bot commented Nov 3, 2025

Build failed:

@kim-em
Copy link

kim-em commented Nov 3, 2025

bors merge

@mathlib-bors
Copy link

mathlib-bors bot commented Nov 3, 2025

Pull request successfully merged into bump/v4.26.0.

Build succeeded:

@mathlib-bors mathlib-bors bot changed the title chore: adaptations for nightly-2025-10-29 [Merged by Bors] - chore: adaptations for nightly-2025-10-29 Nov 3, 2025
@mathlib-bors mathlib-bors bot closed this Nov 3, 2025
@mathlib-bors mathlib-bors bot deleted the bump/nightly-2025-10-29 branch November 3, 2025 13:01
Sign up for free to join this conversation on GitHub. Already have an account? Sign in to comment

Labels

None yet

Projects

None yet

Development

Successfully merging this pull request may close these issues.