Skip to content

Commit e26f972

Browse files
committed
chore(Algebra/Group/Action/Basic): merge two sections (#22509)
1 parent 692313e commit e26f972

File tree

1 file changed

+12
-14
lines changed

1 file changed

+12
-14
lines changed

Mathlib/Algebra/Group/Action/Basic.lean

Lines changed: 12 additions & 14 deletions
Original file line numberDiff line numberDiff line change
@@ -80,11 +80,12 @@ end Monoid
8080
end MulAction
8181

8282
section Arrow
83+
variable {G A B : Type*} [DivisionMonoid G] [MulAction G A]
8384

8485
/-- If `G` acts on `A`, then it acts also on `A → B`, by `(g • F) a = F (g⁻¹ • a)`. -/
8586
@[to_additive (attr := simps) arrowAddAction
86-
"If `G` acts on `A`, then it acts also on `A → B`, by `(g +ᵥ F) a = F (g⁻¹ +ᵥ a)`"]
87-
def arrowAction {G A B : Type*} [DivisionMonoid G] [MulAction G A] : MulAction G (A → B) where
87+
"If `G` acts on `A`, then it acts also on `A → B`, by `(g +ᵥ F) a = F (g⁻¹ +ᵥ a)`"]
88+
def arrowAction : MulAction G (A → B) where
8889
smul g F a := F (g⁻¹ • a)
8990
one_smul f := by
9091
show (fun x => f ((1 : G)⁻¹ • x)) = f
@@ -93,6 +94,15 @@ def arrowAction {G A B : Type*} [DivisionMonoid G] [MulAction G A] : MulAction G
9394
show (fun a => f ((x*y)⁻¹ • a)) = (fun a => f (y⁻¹ • x⁻¹ • a))
9495
simp only [mul_smul, mul_inv_rev]
9596

97+
attribute [local instance] arrowAction
98+
99+
variable [Monoid M]
100+
101+
/-- When `M` is a monoid, `ArrowAction` is additionally a `MulDistribMulAction`. -/
102+
def arrowMulDistribMulAction : MulDistribMulAction G (A → M) where
103+
smul_one _ := rfl
104+
smul_mul _ _ _ := rfl
105+
96106
end Arrow
97107

98108
namespace IsUnit
@@ -179,15 +189,3 @@ lemma smul_div' (r : M) (x y : A) : r • (x / y) = r • x / r • y :=
179189
map_div (MulDistribMulAction.toMonoidHom A r) x y
180190

181191
end MulDistribMulAction
182-
183-
section Arrow
184-
variable [Group G] [MulAction G A] [Monoid M]
185-
186-
attribute [local instance] arrowAction
187-
188-
/-- When `M` is a monoid, `ArrowAction` is additionally a `MulDistribMulAction`. -/
189-
def arrowMulDistribMulAction : MulDistribMulAction G (A → M) where
190-
smul_one _ := rfl
191-
smul_mul _ _ _ := rfl
192-
193-
end Arrow

0 commit comments

Comments
 (0)