Skip to content

Commit

Permalink
feat(data/polynomial/div): a - b ∣ p.eval a - p.eval b (#13021)
Browse files Browse the repository at this point in the history
Co-authored-by: Eric Rodriguez <@ericrbg>
  • Loading branch information
vihdzp committed Mar 29, 2022
1 parent 111d3a4 commit 66509e1
Showing 1 changed file with 7 additions and 0 deletions.
7 changes: 7 additions & 0 deletions src/data/polynomial/div.lean
Expand Up @@ -413,6 +413,13 @@ begin
(sum_monomial_eq _)
end

lemma sub_dvd_eval_sub (a b : R) (p : R[X]) : a - b ∣ p.eval a - p.eval b :=
begin
suffices : X - C b ∣ p - C (p.eval b),
{ simpa only [coe_eval_ring_hom, eval_sub, eval_X, eval_C] using (eval_ring_hom a).map_dvd this },
simp [dvd_iff_is_root]
end

variable (R)

lemma not_is_field : ¬ is_field R[X] :=
Expand Down

0 comments on commit 66509e1

Please sign in to comment.