Skip to content

Commit

Permalink
chore(*): add mathlib4 synchronization comments
Browse files Browse the repository at this point in the history
  • Loading branch information
leanprover-community-bot committed Oct 17, 2023
1 parent b1abe23 commit 95aad47
Show file tree
Hide file tree
Showing 4 changed files with 12 additions and 0 deletions.
3 changes: 3 additions & 0 deletions src/algebraic_topology/dold_kan/equivalence.lean
Original file line number Diff line number Diff line change
Expand Up @@ -11,6 +11,9 @@ import algebraic_topology.dold_kan.normalized
# The Dold-Kan correspondence
> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
> Any changes to this file require a corresponding PR to mathlib4.
The Dold-Kan correspondence states that for any abelian category `A`, there is
an equivalence between the category of simplicial objects in `A` and the
category of chain complexes in `A` (with degrees indexed by `ℕ` and the
Expand Down
Original file line number Diff line number Diff line change
Expand Up @@ -12,6 +12,9 @@ import category_theory.idempotents.simplicial_object
# The Dold-Kan correspondence for pseudoabelian categories
> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
> Any changes to this file require a corresponding PR to mathlib4.
In this file, for any idempotent complete additive category `C`,
the Dold-Kan equivalence
`idempotents.dold_kan.equivalence C : simplicial_object C ≌ chain_complex C ℕ`
Expand Down
3 changes: 3 additions & 0 deletions src/combinatorics/quiver/covering.lean
Original file line number Diff line number Diff line change
Expand Up @@ -11,6 +11,9 @@ import logic.equiv.basic
/-!
# Covering
> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
> Any changes to this file require a corresponding PR to mathlib4.
This file defines coverings of quivers as prefunctors that are bijective on the
so-called stars and costars at each vertex of the domain.
Expand Down
3 changes: 3 additions & 0 deletions src/linear_algebra/quadratic_form/dual.lean
Original file line number Diff line number Diff line change
Expand Up @@ -9,6 +9,9 @@ import linear_algebra.quadratic_form.prod
/-!
# Quadratic form structures related to `module.dual`
> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
> Any changes to this file require a corresponding PR to mathlib4.
## Main definitions
* `bilin_form.dual_prod R M`, the bilinear form on `(f, x) : module.dual R M × M` defined as
Expand Down

0 comments on commit 95aad47

Please sign in to comment.