Skip to content

Commit

Permalink
chore(category_theory/*): reduce imports (#13305)
Browse files Browse the repository at this point in the history
An unnecessary import of `tactic.monotonicity` earlier in the hierarchy was pulling in quite a lot. A few compensatory imports are needed later.



Co-authored-by: Scott Morrison <scott.morrison@gmail.com>
  • Loading branch information
semorrison and semorrison committed Apr 11, 2022
1 parent 5e8d6bb commit a447dae
Show file tree
Hide file tree
Showing 3 changed files with 3 additions and 2 deletions.
1 change: 1 addition & 0 deletions src/algebra/category/Semigroup/basic.lean
Expand Up @@ -4,6 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Julian Kuelshammer
-/
import algebra.pempty_instances
import algebra.hom.equiv
import category_theory.concrete_category.bundled_hom
import category_theory.functor.reflects_isomorphisms

Expand Down
1 change: 1 addition & 0 deletions src/category_theory/essential_image.lean
Expand Up @@ -5,6 +5,7 @@ Authors: Bhavik Mehta
-/
import category_theory.natural_isomorphism
import category_theory.full_subcategory
import data.set.basic

/-!
# Essential image of a functor
Expand Down
3 changes: 1 addition & 2 deletions src/category_theory/functor/basic.lean
Expand Up @@ -4,7 +4,6 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Tim Baumann, Stephen Morgan, Scott Morrison
-/
import tactic.reassoc_axiom
import tactic.monotonicity
import category_theory.category.basic

/-!
Expand All @@ -13,7 +12,7 @@ import category_theory.category.basic
Defines a functor between categories, extending a `prefunctor` between quivers.
Introduces notation `C ⥤ D` for the type of all functors from `C` to `D`.
(Unfortunately the `⇒` arrow (`\functor`) is taken by core,
(Unfortunately the `⇒` arrow (`\functor`) is taken by core,
but in mathlib4 we should switch to this.)
-/

Expand Down

0 comments on commit a447dae

Please sign in to comment.