Skip to content

Commit

Permalink
shake
Browse files Browse the repository at this point in the history
  • Loading branch information
YaelDillies committed Jan 25, 2025
1 parent 5115a0a commit d043cb3
Show file tree
Hide file tree
Showing 5 changed files with 9 additions and 6 deletions.
2 changes: 1 addition & 1 deletion Mathlib/Algebra/Category/MonCat/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -3,9 +3,9 @@ Copyright (c) 2018 Kim Morrison. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Kim Morrison
-/
import Mathlib.Algebra.Group.PUnit
import Mathlib.Algebra.Group.ULift
import Mathlib.Algebra.Ring.Action.Group
import Mathlib.Algebra.Ring.PUnit
import Mathlib.CategoryTheory.ConcreteCategory.BundledHom
import Mathlib.CategoryTheory.Functor.ReflectsIso

Expand Down
3 changes: 2 additions & 1 deletion Mathlib/Algebra/Category/Ring/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,8 +4,9 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Kim Morrison, Johannes Hölzl, Yury Kudryashov
-/
import Mathlib.Algebra.Category.Grp.Basic
import Mathlib.CategoryTheory.ConcreteCategory.ReflectsIso
import Mathlib.Algebra.Ring.Equiv
import Mathlib.Algebra.Ring.PUnit
import Mathlib.CategoryTheory.ConcreteCategory.ReflectsIso

/-!
# Category instances for `Semiring`, `Ring`, `CommSemiring`, and `CommRing`.
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Analysis/Normed/Group/Constructions.lean
Original file line number Diff line number Diff line change
Expand Up @@ -3,8 +3,8 @@ Copyright (c) 2018 Patrick Massot. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Patrick Massot, Johannes Hölzl, Yaël Dillies
-/
import Mathlib.Algebra.Group.PUnit
import Mathlib.Algebra.Group.ULift
import Mathlib.Algebra.Ring.PUnit
import Mathlib.Analysis.Normed.Group.Basic

/-!
Expand Down
7 changes: 4 additions & 3 deletions Mathlib/CategoryTheory/Action/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,11 +4,12 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Kim Morrison
-/
import Mathlib.Algebra.Category.Grp.Basic
import Mathlib.CategoryTheory.SingleObj
import Mathlib.CategoryTheory.Limits.FunctorCategory.Basic
import Mathlib.CategoryTheory.Limits.Preserves.Basic
import Mathlib.Algebra.Ring.PUnit
import Mathlib.CategoryTheory.Adjunction.Limits
import Mathlib.CategoryTheory.Conj
import Mathlib.CategoryTheory.Limits.FunctorCategory.Basic
import Mathlib.CategoryTheory.Limits.Preserves.Basic
import Mathlib.CategoryTheory.SingleObj

/-!
# `Action V G`, the category of actions of a monoid `G` inside some category `V`.
Expand Down
1 change: 1 addition & 0 deletions Mathlib/CategoryTheory/Monoidal/Internal/Types.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,6 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Kim Morrison
-/
import Mathlib.Algebra.Category.MonCat.Basic
import Mathlib.Algebra.Ring.PUnit
import Mathlib.CategoryTheory.Monoidal.CommMon_
import Mathlib.CategoryTheory.Monoidal.Types.Symmetric

Expand Down

0 comments on commit d043cb3

Please sign in to comment.