Skip to content

Commit

Permalink
chore: Move MulAction to under Algebra (#13140)
Browse files Browse the repository at this point in the history
Move the content of `GroupTheory.GroupAction.Defs` that doesn't depend on `GroupWithZero` to a new file `Algebra.Group.Action.Defs`.  This is part of #13027.
  • Loading branch information
YaelDillies committed May 24, 2024
1 parent 4b398c7 commit 7476a96
Show file tree
Hide file tree
Showing 11 changed files with 847 additions and 877 deletions.
1 change: 1 addition & 0 deletions Mathlib.lean
Original file line number Diff line number Diff line change
Expand Up @@ -185,6 +185,7 @@ import Mathlib.Algebra.GCDMonoid.Nat
import Mathlib.Algebra.GeomSum
import Mathlib.Algebra.GradedMonoid
import Mathlib.Algebra.GradedMulAction
import Mathlib.Algebra.Group.Action.Defs
import Mathlib.Algebra.Group.AddChar
import Mathlib.Algebra.Group.Aut
import Mathlib.Algebra.Group.Basic
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Algebra/FreeMonoid/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,8 +4,8 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Simon Hudon, Yury Kudryashov
-/
import Mathlib.Algebra.BigOperators.Group.List
import Mathlib.Algebra.Group.Action.Defs
import Mathlib.Algebra.Group.Units
import Mathlib.GroupTheory.GroupAction.Defs

#align_import algebra.free_monoid.basic from "leanprover-community/mathlib"@"657df4339ae6ceada048c8a2980fb10e393143ec"

Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Algebra/GradedMonoid.lean
Original file line number Diff line number Diff line change
Expand Up @@ -6,7 +6,7 @@ Authors: Eric Wieser
import Mathlib.Algebra.BigOperators.Group.List
import Mathlib.Algebra.Group.InjSurj
import Mathlib.Data.List.FinRange
import Mathlib.GroupTheory.GroupAction.Defs
import Mathlib.Algebra.Group.Action.Defs
import Mathlib.Data.SetLike.Basic
import Mathlib.Algebra.Group.Submonoid.Basic
import Mathlib.Data.Sigma.Basic
Expand Down
838 changes: 838 additions & 0 deletions Mathlib/Algebra/Group/Action/Defs.lean

Large diffs are not rendered by default.

2 changes: 1 addition & 1 deletion Mathlib/CategoryTheory/Endomorphism.lean
Original file line number Diff line number Diff line change
Expand Up @@ -3,12 +3,12 @@ Copyright (c) 2019 Yury Kudryashov. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Yury Kudryashov, Scott Morrison, Simon Hudon
-/
import Mathlib.Algebra.Group.Action.Defs
import Mathlib.Algebra.Group.Equiv.Basic
import Mathlib.Algebra.Group.Units
import Mathlib.Algebra.Group.Units.Hom
import Mathlib.CategoryTheory.Groupoid
import Mathlib.CategoryTheory.Opposites
import Mathlib.GroupTheory.GroupAction.Defs

#align_import category_theory.endomorphism from "leanprover-community/mathlib"@"32253a1a1071173b33dc7d6a218cf722c6feb514"

Expand Down
863 changes: 1 addition & 862 deletions Mathlib/GroupTheory/GroupAction/Defs.lean

Large diffs are not rendered by default.

8 changes: 0 additions & 8 deletions Mathlib/GroupTheory/GroupAction/Group.lean
Original file line number Diff line number Diff line change
Expand Up @@ -22,14 +22,6 @@ universe u v w
variable {α : Type u} {β : Type v} {γ : Type w}

section MulAction

/-- `Monoid.toMulAction` is faithful on cancellative monoids. -/
@[to_additive " `AddMonoid.toAddAction` is faithful on additive cancellative monoids. "]
instance RightCancelMonoid.faithfulSMul [RightCancelMonoid α] : FaithfulSMul α α :=
fun h => mul_right_cancel (h 1)⟩
#align right_cancel_monoid.to_has_faithful_smul RightCancelMonoid.faithfulSMul
#align add_right_cancel_monoid.to_has_faithful_vadd AddRightCancelMonoid.faithfulVAdd

section Group

variable [Group α] [MulAction α β]
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/GroupTheory/GroupAction/Option.lean
Original file line number Diff line number Diff line change
Expand Up @@ -3,7 +3,7 @@ Copyright (c) 2022 Yaël Dillies. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Yaël Dillies
-/
import Mathlib.GroupTheory.GroupAction.Defs
import Mathlib.Algebra.Group.Action.Defs

#align_import group_theory.group_action.option from "leanprover-community/mathlib"@"f1a2caaf51ef593799107fe9a8d5e411599f3996"

Expand Down
2 changes: 1 addition & 1 deletion Mathlib/GroupTheory/GroupAction/Ring.lean
Original file line number Diff line number Diff line change
Expand Up @@ -3,8 +3,8 @@ Copyright (c) 2022 Eric Wieser. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Eric Wieser
-/
import Mathlib.Algebra.Group.Action.Defs
import Mathlib.Algebra.Ring.Defs
import Mathlib.GroupTheory.GroupAction.Defs

/-!
# Commutativity and associativity of action of integers on rings
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/GroupTheory/GroupAction/Sigma.lean
Original file line number Diff line number Diff line change
Expand Up @@ -3,7 +3,7 @@ Copyright (c) 2022 Yaël Dillies. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Yaël Dillies
-/
import Mathlib.GroupTheory.GroupAction.Defs
import Mathlib.Algebra.Group.Action.Defs

#align_import group_theory.group_action.sigma from "leanprover-community/mathlib"@"f1a2caaf51ef593799107fe9a8d5e411599f3996"

Expand Down
2 changes: 1 addition & 1 deletion Mathlib/GroupTheory/GroupAction/Sum.lean
Original file line number Diff line number Diff line change
Expand Up @@ -3,7 +3,7 @@ Copyright (c) 2022 Yaël Dillies. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Yaël Dillies
-/
import Mathlib.GroupTheory.GroupAction.Defs
import Mathlib.Algebra.Group.Action.Defs

#align_import group_theory.group_action.sum from "leanprover-community/mathlib"@"f1a2caaf51ef593799107fe9a8d5e411599f3996"

Expand Down

0 comments on commit 7476a96

Please sign in to comment.