Skip to content

Commit

Permalink
fix(*): Fix errors caused by overly restrictive type-classes
Browse files Browse the repository at this point in the history
  • Loading branch information
eric-wieser committed Nov 7, 2020
1 parent 460b7cf commit b3fcb08
Showing 1 changed file with 9 additions and 9 deletions.
18 changes: 9 additions & 9 deletions src/group_theory/group_action/defs.lean
Original file line number Diff line number Diff line change
Expand Up @@ -114,15 +114,6 @@ by split_ifs; refl

end ite

section compatible_scalar

@[simp] lemma smul_one_smul {M} (N) [monoid N] [has_scalar M N] [mul_action N α] [has_scalar M α]
[is_scalar_tower M N α] (x : M) (y : α) :
(x • (1 : N)) • y = x • y :=
by rw [smul_assoc, one_smul]

end compatible_scalar

namespace mul_action

variables (α) [monoid α]
Expand Down Expand Up @@ -168,6 +159,15 @@ end mul_action

end

section compatible_scalar

@[simp] lemma smul_one_smul {M} (N) [monoid N] [has_scalar M N] [mul_action N α] [has_scalar M α]
[is_scalar_tower M N α] (x : M) (y : α) :
(x • (1 : N)) • y = x • y :=
by rw [smul_assoc, one_smul]

end compatible_scalar

/-- Typeclass for multiplicative actions on additive structures. This generalizes group modules. -/
class distrib_mul_action (α : Type u) (β : Type v) [monoid α] [add_monoid β]
extends mul_action α β :=
Expand Down

0 comments on commit b3fcb08

Please sign in to comment.