Skip to content
This repository has been archived by the owner on Jul 24, 2024. It is now read-only.

Commit

Permalink
chore(*): add mathlib4 synchronization comments (#17790)
Browse files Browse the repository at this point in the history
Regenerated from the [port status wiki page](https://github.com/leanprover-community/mathlib/wiki/mathlib4-port-status).
Relates to the following PRs:
* `algebra.order.sub.canonical`: leanprover-community/mathlib4#814
* `category_theory.category.Rel`: leanprover-community/mathlib4#822
* `category_theory.category.basic`: leanprover-community/mathlib4#749
* `category_theory.functor.basic`: leanprover-community/mathlib4#749
* `category_theory.functor.category`: leanprover-community/mathlib4#749
* `category_theory.functor.functorial`: leanprover-community/mathlib4#822
* `category_theory.isomorphism`: leanprover-community/mathlib4#749
* `category_theory.natural_transformation`: leanprover-community/mathlib4#749
* `category_theory.thin`: leanprover-community/mathlib4#822
* `combinatorics.quiver.basic`: leanprover-community/mathlib4#749
* `combinatorics.quiver.path`: leanprover-community/mathlib4#811
* `data.psigma.order`: leanprover-community/mathlib4#815
* `data.stream.defs`: leanprover-community/mathlib4#665
* `order.boolean_algebra`: leanprover-community/mathlib4#794
* `order.heyting.basic`: leanprover-community/mathlib4#793
* `order.rel_iso.group`: leanprover-community/mathlib4#813
  • Loading branch information
leanprover-community-bot committed Dec 3, 2022
1 parent e469260 commit 308f6d0
Show file tree
Hide file tree
Showing 16 changed files with 64 additions and 0 deletions.
4 changes: 4 additions & 0 deletions src/algebra/order/sub/canonical.lean
Original file line number Diff line number Diff line change
Expand Up @@ -8,6 +8,10 @@ import algebra.order.sub.defs

/-!
# Lemmas about subtraction in canonically ordered monoids
> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
> https://github.com/leanprover-community/mathlib4/pull/814
> Any changes to this file require a corresponding PR to mathlib4.
-/

variables {α : Type*}
Expand Down
4 changes: 4 additions & 0 deletions src/category_theory/category/Rel.lean
Original file line number Diff line number Diff line change
Expand Up @@ -6,6 +6,10 @@ Authors: Scott Morrison
import category_theory.category.basic

/-!
> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
> https://github.com/leanprover-community/mathlib4/pull/822
> Any changes to this file require a corresponding PR to mathlib4.
The category of types with binary relations as morphisms.
-/

Expand Down
4 changes: 4 additions & 0 deletions src/category_theory/category/basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -8,6 +8,10 @@ import combinatorics.quiver.basic
/-!
# Categories
> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
> https://github.com/leanprover-community/mathlib4/pull/749
> Any changes to this file require a corresponding PR to mathlib4.
Defines a category, as a type class parametrised by the type of objects.
## Notations
Expand Down
4 changes: 4 additions & 0 deletions src/category_theory/functor/basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -9,6 +9,10 @@ import category_theory.category.basic
/-!
# Functors
> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
> https://github.com/leanprover-community/mathlib4/pull/749
> Any changes to this file require a corresponding PR to mathlib4.
Defines a functor between categories, extending a `prefunctor` between quivers.
Introduces notation `C ⥤ D` for the type of all functors from `C` to `D`.
Expand Down
4 changes: 4 additions & 0 deletions src/category_theory/functor/category.lean
Original file line number Diff line number Diff line change
Expand Up @@ -9,6 +9,10 @@ import category_theory.isomorphism
/-!
# The category of functors and natural transformations between two fixed categories.
> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
> https://github.com/leanprover-community/mathlib4/pull/749
> Any changes to this file require a corresponding PR to mathlib4.
We provide the category instance on `C ⥤ D`, with morphisms the natural transformations.
## Universes
Expand Down
4 changes: 4 additions & 0 deletions src/category_theory/functor/functorial.lean
Original file line number Diff line number Diff line change
Expand Up @@ -7,6 +7,10 @@ import category_theory.functor.basic

/-!
# Unbundled functors, as a typeclass decorating the object-level function.
> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
> https://github.com/leanprover-community/mathlib4/pull/822
> Any changes to this file require a corresponding PR to mathlib4.
-/

namespace category_theory
Expand Down
4 changes: 4 additions & 0 deletions src/category_theory/isomorphism.lean
Original file line number Diff line number Diff line change
Expand Up @@ -8,6 +8,10 @@ import category_theory.functor.basic
/-!
# Isomorphisms
> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
> https://github.com/leanprover-community/mathlib4/pull/749
> Any changes to this file require a corresponding PR to mathlib4.
This file defines isomorphisms between objects of a category.
## Main definitions
Expand Down
4 changes: 4 additions & 0 deletions src/category_theory/natural_transformation.lean
Original file line number Diff line number Diff line change
Expand Up @@ -8,6 +8,10 @@ import category_theory.functor.basic
/-!
# Natural transformations
> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
> https://github.com/leanprover-community/mathlib4/pull/749
> Any changes to this file require a corresponding PR to mathlib4.
Defines natural transformations between functors.
A natural transformation `α : nat_trans F G` consists of morphisms `α.app X : F.obj X ⟶ G.obj X`,
Expand Down
4 changes: 4 additions & 0 deletions src/category_theory/thin.lean
Original file line number Diff line number Diff line change
Expand Up @@ -9,6 +9,10 @@ import category_theory.isomorphism
/-!
# Thin categories
> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
> https://github.com/leanprover-community/mathlib4/pull/822
> Any changes to this file require a corresponding PR to mathlib4.
A thin category (also known as a sparse category) is a category with at most one morphism between
each pair of objects.
Expand Down
4 changes: 4 additions & 0 deletions src/combinatorics/quiver/basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -8,6 +8,10 @@ import data.opposite
/-!
# Quivers
> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
> https://github.com/leanprover-community/mathlib4/pull/749
> Any changes to this file require a corresponding PR to mathlib4.
This module defines quivers. A quiver on a type `V` of vertices assigns to every
pair `a b : V` of vertices a type `a ⟶ b` of arrows from `a` to `b`. This
is a very permissive notion of directed graph.
Expand Down
4 changes: 4 additions & 0 deletions src/combinatorics/quiver/path.lean
Original file line number Diff line number Diff line change
Expand Up @@ -9,6 +9,10 @@ import logic.lemmas
/-!
# Paths in quivers
> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
> https://github.com/leanprover-community/mathlib4/pull/811
> Any changes to this file require a corresponding PR to mathlib4.
Given a quiver `V`, we define the type of paths from `a : V` to `b : V` as an inductive
family. We define composition of paths and the action of prefunctors on paths.
-/
Expand Down
4 changes: 4 additions & 0 deletions src/data/psigma/order.lean
Original file line number Diff line number Diff line change
Expand Up @@ -9,6 +9,10 @@ import order.bounded_order
/-!
# Lexicographic order on a sigma type
> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
> https://github.com/leanprover-community/mathlib4/pull/815
> Any changes to this file require a corresponding PR to mathlib4.
This file defines the lexicographic order on `Σₗ' i, α i`. `a` is less than `b` if its summand is
strictly less than the summand of `b` or they are in the same summand and `a` is less than `b`
there.
Expand Down
4 changes: 4 additions & 0 deletions src/data/stream/defs.lean
Original file line number Diff line number Diff line change
Expand Up @@ -7,6 +7,10 @@ Authors: Leonardo de Moura
/-!
# Definition of `stream` and functions on streams
> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
> https://github.com/leanprover-community/mathlib4/pull/665
> Any changes to this file require a corresponding PR to mathlib4.
A stream `stream α` is an infinite sequence of elements of `α`. One can also think about it as an
infinite list. In this file we define `stream` and some functions that take and/or return streams.
-/
Expand Down
4 changes: 4 additions & 0 deletions src/order/boolean_algebra.lean
Original file line number Diff line number Diff line change
Expand Up @@ -8,6 +8,10 @@ import order.heyting.basic
/-!
# (Generalized) Boolean algebras
> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
> https://github.com/leanprover-community/mathlib4/pull/794
> Any changes to this file require a corresponding PR to mathlib4.
A Boolean algebra is a bounded distributive lattice with a complement operator. Boolean algebras
generalize the (classical) logic of propositions and the lattice of subsets of a set.
Expand Down
4 changes: 4 additions & 0 deletions src/order/heyting/basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -8,6 +8,10 @@ import order.prop_instances
/-!
# Heyting algebras
> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
> https://github.com/leanprover-community/mathlib4/pull/793
> Any changes to this file require a corresponding PR to mathlib4.
This file defines Heyting, co-Heyting and bi-Heyting algebras.
An Heyting algebra is a bounded distributive lattice with an implication operation `⇨` such that
Expand Down
4 changes: 4 additions & 0 deletions src/order/rel_iso/group.lean
Original file line number Diff line number Diff line change
Expand Up @@ -8,6 +8,10 @@ import order.rel_iso.basic

/-!
# Relation isomorphisms form a group
> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
> https://github.com/leanprover-community/mathlib4/pull/813
> Any changes to this file require a corresponding PR to mathlib4.
-/

variables {α: Type*}
Expand Down

0 comments on commit 308f6d0

Please sign in to comment.