Skip to content

Commit

Permalink
fix: category_theory -> CategoryTheory in note (#2357)
Browse files Browse the repository at this point in the history
This changes the name of a library_note from
"category_theory universes" to
"CategoryTheory universes"
to be more in line with the new naming conventions.



Co-authored-by: Moritz Firsching <firsching@google.com>
  • Loading branch information
mo271 and mo271 committed Mar 2, 2023
1 parent 41b4afa commit 1640c54
Show file tree
Hide file tree
Showing 12 changed files with 12 additions and 12 deletions.
2 changes: 1 addition & 1 deletion Mathlib/CategoryTheory/Category/Basic.lean
Expand Up @@ -37,7 +37,7 @@ I am experimenting with using the `aesop` tactic as a replacement for `tidy`.
-/


library_note "category_theory universes"
library_note "CategoryTheory universes"
/--
The typeclass `Category C` describes morphisms associated to objects of type `C : Type u`.
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/CategoryTheory/Core.lean
Expand Up @@ -30,7 +30,7 @@ namespace CategoryTheory

universe v₁ v₂ u₁ u₂

-- morphism levels before object levels. See note [category_theory universes].
-- morphism levels before object levels. See note [CategoryTheory universes].
/-- The core of a category C is the groupoid whose morphisms are all the
isomorphisms of C. -/
-- Porting note: This linter does not exist yet
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/CategoryTheory/EqToHom.lean
Expand Up @@ -32,7 +32,7 @@ result in the various `eqToHom` morphisms to drop out at the appropriate moment!

universe v₁ v₂ v₃ u₁ u₂ u₃

-- morphism levels before object levels. See note [category_theory universes].
-- morphism levels before object levels. See note [CategoryTheory universes].
namespace CategoryTheory

open Opposite
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/CategoryTheory/FullSubcategory.lean
Expand Up @@ -42,7 +42,7 @@ form of `D`. This is used to set up several algebraic categories like
namespace CategoryTheory

universe v v₂ u₁ u₂
-- morphism levels before object levels. See note [category_theory universes].
-- morphism levels before object levels. See note [CategoryTheory universes].

section Induced

Expand Down
2 changes: 1 addition & 1 deletion Mathlib/CategoryTheory/Functor/Basic.lean
Expand Up @@ -25,7 +25,7 @@ but in mathlib4 we should switch to this.)

namespace CategoryTheory

-- declare the `v`'s first; see note [category_theory universes].
-- declare the `v`'s first; see note [CategoryTheory universes].
universe v v₁ v₂ v₃ u u₁ u₂ u₃

section
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/CategoryTheory/Functor/Category.lean
Expand Up @@ -26,7 +26,7 @@ this is a small category at the next higher level.

namespace CategoryTheory

-- declare the `v`'s first; see note [category_theory universes].
-- declare the `v`'s first; see note [CategoryTheory universes].
universe v₁ v₂ v₃ u₁ u₂ u₃

open NatTrans Category CategoryTheory.Functor
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/CategoryTheory/Iso.lean
Expand Up @@ -39,7 +39,7 @@ category, category theory, isomorphism

universe v u

-- morphism levels before object levels. See note [category_theory universes].
-- morphism levels before object levels. See note [CategoryTheory universes].
namespace CategoryTheory

open Category
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/CategoryTheory/NatTrans.lean
Expand Up @@ -37,7 +37,7 @@ Introduces notations

namespace CategoryTheory

-- declare the `v`'s first; see note [category_theory universes].
-- declare the `v`'s first; see note [CategoryTheory universes].
universe v₁ v₂ v₃ v₄ u₁ u₂ u₃ u₄

variable {C : Type u₁} [Category.{v₁} C] {D : Type u₂} [Category.{v₂} D]
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/CategoryTheory/Opposites.lean
Expand Up @@ -30,7 +30,7 @@ set_option autoImplicit false

universe v₁ v₂ u₁ u₂

-- morphism levels before object levels. See note [category_theory universes].
-- morphism levels before object levels. See note [CategoryTheory universes].
open Opposite

variable {C : Type u₁}
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/CategoryTheory/Types.lean
Expand Up @@ -37,7 +37,7 @@ We prove some basic facts about the category `Type`:

namespace CategoryTheory

-- morphism levels before object levels. See note [category_theory universes].
-- morphism levels before object levels. See note [CategoryTheory universes].
universe v v' w u u'

/- The `@[to_additive]` attribute is just a hint that expressions involving this instance can
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Combinatorics/Quiver/Basic.lean
Expand Up @@ -31,7 +31,7 @@ but it is also results in error-prone universe signatures when constraints requi
open Opposite

-- We use the same universe order as in category theory.
-- See note [category_theory universes]
-- See note [CategoryTheory universes]
universe v v₁ v₂ u u₁ u₂

/-- A quiver `G` on a type `V` of vertices assigns to every pair `a b : V` of vertices
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Data/Opposite.lean
Expand Up @@ -21,7 +21,7 @@ category, with all arrows reversed.

universe v u

-- morphism levels before object levels. See note [category_theory universes].
-- morphism levels before object levels. See note [CategoryTheory universes].
variable (α : Sort u)

/-- The type of objects of the opposite of `α`; used to define the opposite category.
Expand Down

0 comments on commit 1640c54

Please sign in to comment.