Skip to content

Commit

Permalink
feat(algebra/hom/equiv/basic): Add to_additive to Pi_congr_right
Browse files Browse the repository at this point in the history
…lemmas (#17827)

Add `to_additive` attribute to three lemmas about `mul_equiv.Pi_congr_right`.
  • Loading branch information
winstonyin committed Dec 6, 2022
1 parent 10ee5ed commit e753057
Showing 1 changed file with 3 additions and 3 deletions.
6 changes: 3 additions & 3 deletions src/algebra/hom/equiv/basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -450,16 +450,16 @@ def Pi_congr_right {η : Type*}
map_mul' := λ x y, funext $ λ j, (es j).map_mul (x j) (y j),
.. equiv.Pi_congr_right (λ j, (es j).to_equiv) }

@[simp]
@[simp, to_additive]
lemma Pi_congr_right_refl {η : Type*} {Ms : η → Type*} [Π j, has_mul (Ms j)] :
Pi_congr_right (λ j, mul_equiv.refl (Ms j)) = mul_equiv.refl _ := rfl

@[simp]
@[simp, to_additive]
lemma Pi_congr_right_symm {η : Type*}
{Ms Ns : η → Type*} [Π j, has_mul (Ms j)] [Π j, has_mul (Ns j)]
(es : ∀ j, Ms j ≃* Ns j) : (Pi_congr_right es).symm = (Pi_congr_right $ λ i, (es i).symm) := rfl

@[simp]
@[simp, to_additive]
lemma Pi_congr_right_trans {η : Type*}
{Ms Ns Ps : η → Type*} [Π j, has_mul (Ms j)] [Π j, has_mul (Ns j)]
[Π j, has_mul (Ps j)]
Expand Down

0 comments on commit e753057

Please sign in to comment.