Skip to content

Commit

Permalink
chore(*): add mathlib4 synchronization comments (#18851)
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 files:
* `algebra.monoid_algebra.ideal`
* `algebra.ring_quot`
* `algebraic_topology.dold_kan.decomposition`
* `algebraic_topology.dold_kan.degeneracies`
* `algebraic_topology.dold_kan.n_reflects_iso`
* `algebraic_topology.dold_kan.split_simplicial_object`
* `category_theory.adjunction.over`
* `data.polynomial.module`
* `linear_algebra.affine_space.independent`
* `linear_algebra.matrix.adjugate`
* `linear_algebra.matrix.nondegenerate`
* `ring_theory.mv_polynomial.ideal`
  • Loading branch information
leanprover-community-bot committed Apr 22, 2023
1 parent 7dfe858 commit 4f81bc2
Show file tree
Hide file tree
Showing 12 changed files with 36 additions and 0 deletions.
3 changes: 3 additions & 0 deletions src/algebra/monoid_algebra/ideal.lean
Expand Up @@ -9,6 +9,9 @@ import ring_theory.ideal.basic

/-!
# Lemmas about ideals of `monoid_algebra` and `add_monoid_algebra`
> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
> Any changes to this file require a corresponding PR to mathlib4.
-/

variables {k A G : Type*}
Expand Down
3 changes: 3 additions & 0 deletions src/algebra/ring_quot.lean
Expand Up @@ -9,6 +9,9 @@ import ring_theory.ideal.quotient
/-!
# Quotients of non-commutative rings
> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
> Any changes to this file require a corresponding PR to mathlib4.
Unfortunately, ideals have only been developed in the commutative case as `ideal`,
and it's not immediately clear how one should formalise ideals in the non-commutative case.
Expand Down
3 changes: 3 additions & 0 deletions src/algebraic_topology/dold_kan/decomposition.lean
Expand Up @@ -10,6 +10,9 @@ import algebraic_topology.dold_kan.p_infty
# Decomposition of the Q endomorphisms
> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
> Any changes to this file require a corresponding PR to mathlib4.
In this file, we obtain a lemma `decomposition_Q` which expresses
explicitly the projection `(Q q).f (n+1) : X _[n+1] ⟶ X _[n+1]`
(`X : simplicial_object C` with `C` a preadditive category) as
Expand Down
3 changes: 3 additions & 0 deletions src/algebraic_topology/dold_kan/degeneracies.lean
Expand Up @@ -11,6 +11,9 @@ import tactic.fin_cases
# Behaviour of P_infty with respect to degeneracies
> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
> Any changes to this file require a corresponding PR to mathlib4.
For any `X : simplicial_object C` where `C` is an abelian category,
the projector `P_infty : K[X] ⟶ K[X]` is supposed to be the projection
on the normalized subcomplex, parallel to the degenerate subcomplex, i.e.
Expand Down
3 changes: 3 additions & 0 deletions src/algebraic_topology/dold_kan/n_reflects_iso.lean
Expand Up @@ -13,6 +13,9 @@ import category_theory.idempotents.karoubi_karoubi
# N₁ and N₂ reflects isomorphisms
> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
> Any changes to this file require a corresponding PR to mathlib4.
In this file, it is shown that the functors
`N₁ : simplicial_object C ⥤ karoubi (chain_complex C ℕ)` and
`N₂ : karoubi (simplicial_object C) ⥤ karoubi (chain_complex C ℕ))`
Expand Down
3 changes: 3 additions & 0 deletions src/algebraic_topology/dold_kan/split_simplicial_object.lean
Expand Up @@ -12,6 +12,9 @@ import algebraic_topology.dold_kan.functor_n
# Split simplicial objects in preadditive categories
> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
> Any changes to this file require a corresponding PR to mathlib4.
In this file we define a functor `nondeg_complex : simplicial_object.split C ⥤ chain_complex C ℕ`
when `C` is a preadditive category with finite coproducts, and get an isomorphism
`to_karoubi_nondeg_complex_iso_N₁ : nondeg_complex ⋙ to_karoubi _ ≅ forget C ⋙ dold_kan.N₁`.
Expand Down
3 changes: 3 additions & 0 deletions src/category_theory/adjunction/over.lean
Expand Up @@ -10,6 +10,9 @@ import category_theory.over
/-!
# Adjunctions related to the over category
> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
> Any changes to this file require a corresponding PR to mathlib4.
Construct the left adjoint `star X` to `over.forget X : over X ⥤ C`.
## TODO
Expand Down
3 changes: 3 additions & 0 deletions src/data/polynomial/module.lean
Expand Up @@ -9,6 +9,9 @@ import ring_theory.finite_type
/-!
# Polynomial module
> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
> Any changes to this file require a corresponding PR to mathlib4.
In this file, we define the polynomial module for an `R`-module `M`, i.e. the `R[X]`-module `M[X]`.
This is defined as an type alias `polynomial_module R M := ℕ →₀ M`, since there might be different
Expand Down
3 changes: 3 additions & 0 deletions src/linear_algebra/affine_space/independent.lean
Expand Up @@ -13,6 +13,9 @@ import linear_algebra.basis
/-!
# Affine independence
> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
> Any changes to this file require a corresponding PR to mathlib4.
This file defines affinely independent families of points.
## Main definitions
Expand Down
3 changes: 3 additions & 0 deletions src/linear_algebra/matrix/adjugate.lean
Expand Up @@ -11,6 +11,9 @@ import ring_theory.polynomial.basic
/-!
# Cramer's rule and adjugate matrices
> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
> Any changes to this file require a corresponding PR to mathlib4.
The adjugate matrix is the transpose of the cofactor matrix.
It is calculated with Cramer's rule, which we introduce first.
The vectors returned by Cramer's rule are given by the linear map `cramer`,
Expand Down
3 changes: 3 additions & 0 deletions src/linear_algebra/matrix/nondegenerate.lean
Expand Up @@ -10,6 +10,9 @@ import linear_algebra.matrix.adjugate
/-!
# Matrices associated with non-degenerate bilinear forms
> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
> Any changes to this file require a corresponding PR to mathlib4.
## Main definitions
* `matrix.nondegenerate A`: the proposition that when interpreted as a bilinear form, the matrix `A`
Expand Down
3 changes: 3 additions & 0 deletions src/ring_theory/mv_polynomial/ideal.lean
Expand Up @@ -9,6 +9,9 @@ import data.mv_polynomial.division
/-!
# Lemmas about ideals of `mv_polynomial`
> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
> Any changes to this file require a corresponding PR to mathlib4.
Notably this contains results about monomial ideals.
## Main results
Expand Down

0 comments on commit 4f81bc2

Please sign in to comment.