Skip to content

Commit

Permalink
feat(group_theory/group_action/opposite): Add smul_eq_mul_unop (#12995
Browse files Browse the repository at this point in the history
)

This PR adds a simp-lemma `smul_eq_mul_unop`, similar to `op_smul_eq_mul` and `smul_eq_mul`.



Co-authored-by: tb65536 <tb65536@users.noreply.github.com>
  • Loading branch information
tb65536 and tb65536 committed Mar 28, 2022
1 parent 6fe0c3b commit 261a195
Showing 1 changed file with 4 additions and 1 deletion.
5 changes: 4 additions & 1 deletion src/group_theory/group_action/opposite.lean
Expand Up @@ -79,7 +79,10 @@ See also `monoid.to_opposite_mul_action` and `monoid_with_zero.to_opposite_mul_a
@[to_additive] instance has_mul.to_has_opposite_scalar [has_mul α] : has_scalar αᵐᵒᵖ α :=
{ smul := λ c x, x * c.unop }

@[simp, to_additive] lemma op_smul_eq_mul [has_mul α] {a a' : α} : op a • a' = a' * a := rfl
@[to_additive] lemma op_smul_eq_mul [has_mul α] {a a' : α} : op a • a' = a' * a := rfl

@[simp, to_additive] lemma mul_opposite.smul_eq_mul_unop [has_mul α] {a : αᵐᵒᵖ} {a' : α} :
a • a' = a' * a.unop := rfl

/-- The right regular action of a group on itself is transitive. -/
@[to_additive] instance mul_action.opposite_regular.is_pretransitive {G : Type*} [group G] :
Expand Down

0 comments on commit 261a195

Please sign in to comment.