Zulip Chat Archive

Stream: new members

Topic: content


vxctyxeha (Apr 30 2025 at 13:20):

is there simpler way to solve this

import Mathlib

open Polynomial
lemma p_content : ( X^3 +  3 * X^2 - 3 : Polynomial ).content = 1 := by sorry

vxctyxeha (Apr 30 2025 at 14:46):

sometimes a good tactic is worthy 100 lines

Riccardo Brasca (Apr 30 2025 at 14:56):

We know that primitive polynomials have content equal to 1, and that monic polynomials are primitive. Using monicity! to prove that the polynomial is monic this is probably a one-liner.


Last updated: May 02 2025 at 03:31 UTC