Skip to content

Commit

Permalink
fix(*): Lemma rename
Browse files Browse the repository at this point in the history
  • Loading branch information
eric-wieser committed Nov 7, 2020
1 parent 63315a3 commit 208af0f
Showing 1 changed file with 2 additions and 2 deletions.
4 changes: 2 additions & 2 deletions src/algebra/polynomial/group_ring_action.lean
Expand Up @@ -67,11 +67,11 @@ variables (G : Type*) [group G]

theorem eval_smul' [mul_semiring_action G S] (g : G) (f : polynomial S) (x : S) :
f.eval (g • x) = g • (g⁻¹ • f).eval x :=
by rw [← smul_eval_smul, mul_action.smul_inv_smul]
by rw [← smul_eval_smul, smul_inv_smul]

theorem smul_eval [mul_semiring_action G S] (g : G) (f : polynomial S) (x : S) :
(g • f).eval x = g • f.eval (g⁻¹ • x) :=
by rw [← smul_eval_smul, mul_action.smul_inv_smul]
by rw [← smul_eval_smul, smul_inv_smul]

end polynomial

Expand Down

0 comments on commit 208af0f

Please sign in to comment.