Skip to content

Commit

Permalink
move(category_theory/category/default): rename to `category_theory.ba…
Browse files Browse the repository at this point in the history
…sic` (#9412)
  • Loading branch information
YaelDillies committed Sep 30, 2021
1 parent 4091f72 commit 6e6fe1f
Show file tree
Hide file tree
Showing 10 changed files with 7 additions and 10 deletions.
2 changes: 1 addition & 1 deletion src/category_theory/category/Kleisli.lean
Expand Up @@ -3,7 +3,7 @@ Copyright (c) 2018 Simon Hudon. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Simon Hudon
-/
import category_theory.category
import category_theory.category.basic

/-!
# The Kleisli construction on the Type category
Expand Down
2 changes: 1 addition & 1 deletion src/category_theory/category/Rel.lean
Expand Up @@ -3,7 +3,7 @@ Copyright (c) 2019 Scott Morrison. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Scott Morrison
-/
import category_theory.category
import category_theory.category.basic

/-!
The category of types with binary relations as morphisms.
Expand Down
File renamed without changes.
2 changes: 0 additions & 2 deletions src/category_theory/category/preorder.lean
Expand Up @@ -5,8 +5,6 @@ Authors: Stephen Morgan, Scott Morrison, Johannes Hölzl, Reid Barton
-/

import category_theory.category.Cat
import category_theory.category.default
import category_theory.opposites
import order.category.Preorder

/-!
Expand Down
2 changes: 1 addition & 1 deletion src/category_theory/category/ulift.lean
Expand Up @@ -3,7 +3,7 @@ Copyright (c) 2021 Adam Topaz. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Adam Topaz
-/
import category_theory.category
import category_theory.category.basic
import category_theory.equivalence
import category_theory.filtered

Expand Down
2 changes: 1 addition & 1 deletion src/category_theory/concrete_category/bundled.lean
Expand Up @@ -3,7 +3,7 @@ Copyright (c) 2018 Scott Morrison. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Scott Morrison, Johannes Hölzl, Reid Barton, Sean Leather
-/
import category_theory.category
import category_theory.category.basic

/-!
# Bundled types
Expand Down
2 changes: 1 addition & 1 deletion src/control/equiv_functor.lean
Expand Up @@ -3,7 +3,7 @@ Copyright (c) 2020 Scott Morrison. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Scott Morrison
-/
import category_theory.category
import category_theory.category.basic
import data.equiv.functor

/-!
Expand Down
1 change: 0 additions & 1 deletion src/control/fold.lean
Expand Up @@ -7,7 +7,6 @@ import algebra.free_monoid
import algebra.opposites
import control.traversable.instances
import control.traversable.lemmas
import category_theory.category
import category_theory.endomorphism
import category_theory.types
import category_theory.category.Kleisli
Expand Down
2 changes: 1 addition & 1 deletion src/tactic/reassoc_axiom.lean
Expand Up @@ -3,7 +3,7 @@ Copyright (c) 2019 Simon Hudon. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Simon Hudon
-/
import category_theory.category
import category_theory.category.basic

/-!
# Tools to reformulate category-theoretic axioms in a more associativity-friendly way
Expand Down
2 changes: 1 addition & 1 deletion src/tactic/slice.lean
Expand Up @@ -3,7 +3,7 @@ Copyright (c) 2018 Scott Morrison. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Scott Morrison
-/
import category_theory.category
import category_theory.category.basic

open category_theory

Expand Down

0 comments on commit 6e6fe1f

Please sign in to comment.