Skip to content

Commit

Permalink
feat(ring_theory/power_series/basic): Add rescale_X (#15397)
Browse files Browse the repository at this point in the history


Co-authored-by: Tyler Raven Billingsley <47119971+tyler-billingsley@users.noreply.github.com>
  • Loading branch information
tyler-billingsley and tyler-billingsley committed Jul 15, 2022
1 parent dc7ab9e commit 2dbbe57
Showing 1 changed file with 8 additions and 3 deletions.
11 changes: 8 additions & 3 deletions src/ring_theory/power_series/basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -1421,12 +1421,17 @@ end ring
section comm_ring
variables {A : Type*} [comm_ring A]

@[simp] lemma rescale_neg_one_X : rescale (-1 : A) X = -X :=
@[simp] lemma rescale_X (a : A) : rescale a X = C A a * X :=
begin
ext, simp only [linear_map.map_neg, coeff_rescale, coeff_X],
split_ifs with h; simp [h]
ext,
simp only [coeff_rescale, coeff_C_mul, coeff_X],
split_ifs with h;
simp [h],
end

lemma rescale_neg_one_X : rescale (-1 : A) X = -X :=
by rw [rescale_X, map_neg, map_one, neg_one_mul]

/-- The ring homomorphism taking a power series `f(X)` to `f(-X)`. -/
noncomputable def eval_neg_hom : power_series A →+* power_series A :=
rescale (-1 : A)
Expand Down

0 comments on commit 2dbbe57

Please sign in to comment.