Skip to content

Commit

Permalink
chore(*): add mathlib4 synchronization comments (#19132)
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.category.Module.adjunctions`
* `analysis.calculus.darboux`
* `analysis.calculus.deriv.inv`
* `analysis.calculus.diff_cont_on_cl`
* `analysis.calculus.dslope`
* `analysis.inner_product_space.gram_schmidt_ortho`
* `category_theory.abelian.ext`
* `category_theory.abelian.left_derived`
* `category_theory.bicategory.single_obj`
* `data.real.golden_ratio`
* `measure_theory.category.Meas`
* `measure_theory.decomposition.jordan`
* `measure_theory.decomposition.signed_hahn`
* `measure_theory.group.action`
* `measure_theory.group.measure`
* `number_theory.arithmetic_function`
* `number_theory.l_series`
* `number_theory.von_mangoldt`
* `topology.algebra.continuous_monoid_hom`
* `topology.instances.discrete`
* `topology.sheaves.stalks`
* `topology.tietze_extension`
  • Loading branch information
leanprover-community-bot committed May 31, 2023
1 parent 12a85fa commit 61b5e27
Show file tree
Hide file tree
Showing 22 changed files with 66 additions and 0 deletions.
3 changes: 3 additions & 0 deletions src/algebra/category/Module/adjunctions.lean
Expand Up @@ -10,6 +10,9 @@ import linear_algebra.direct_sum.finsupp
import category_theory.linear.linear_functor

/-!
> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
> Any changes to this file require a corresponding PR to mathlib4.
The functor of forming finitely supported functions on a type with values in a `[ring R]`
is the left adjoint of
the forgetful functor from `R`-modules to types.
Expand Down
3 changes: 3 additions & 0 deletions src/analysis/calculus/darboux.lean
Expand Up @@ -8,6 +8,9 @@ import analysis.calculus.local_extr
/-!
# Darboux's theorem
> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
> Any changes to this file require a corresponding PR to mathlib4.
In this file we prove that the derivative of a differentiable function on an interval takes all
intermediate values. The proof is based on the
[Wikipedia](https://en.wikipedia.org/wiki/Darboux%27s_theorem_(analysis)) page about this theorem.
Expand Down
3 changes: 3 additions & 0 deletions src/analysis/calculus/deriv/inv.lean
Expand Up @@ -9,6 +9,9 @@ import analysis.calculus.deriv.comp
/-!
# Derivatives of `x ↦ x⁻¹` and `f x / g x`
> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
> Any changes to this file require a corresponding PR to mathlib4.
In this file we prove `(x⁻¹)' = -1 / x ^ 2`, `((f x)⁻¹)' = -f' x / (f x) ^ 2`, and
`(f x / g x)' = (f' x * g x - f x * g' x) / (g x) ^ 2` for different notions of derivative.
Expand Down
3 changes: 3 additions & 0 deletions src/analysis/calculus/diff_cont_on_cl.lean
Expand Up @@ -8,6 +8,9 @@ import analysis.calculus.deriv.inv
/-!
# Functions differentiable on a domain and continuous on its closure
> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
> Any changes to this file require a corresponding PR to mathlib4.
Many theorems in complex analysis assume that a function is complex differentiable on a domain and
is continuous on its closure. In this file we define a predicate `diff_cont_on_cl` that expresses
this property and prove basic facts about this predicate.
Expand Down
3 changes: 3 additions & 0 deletions src/analysis/calculus/dslope.lean
Expand Up @@ -9,6 +9,9 @@ import analysis.calculus.deriv.inv
/-!
# Slope of a differentiable function
> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
> Any changes to this file require a corresponding PR to mathlib4.
Given a function `f : 𝕜 → E` from a nontrivially normed field to a normed space over this field,
`dslope f a b` is defined as `slope f a b = (b - a)⁻¹ • (f b - f a)` for `a ≠ b` and as `deriv f a`
for `a = b`.
Expand Down
3 changes: 3 additions & 0 deletions src/analysis/inner_product_space/gram_schmidt_ortho.lean
Expand Up @@ -10,6 +10,9 @@ import linear_algebra.matrix.block
/-!
# Gram-Schmidt Orthogonalization and Orthonormalization
> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
> Any changes to this file require a corresponding PR to mathlib4.
In this file we introduce Gram-Schmidt Orthogonalization and Orthonormalization.
The Gram-Schmidt process takes a set of vectors as input
Expand Down
3 changes: 3 additions & 0 deletions src/category_theory/abelian/ext.lean
Expand Up @@ -12,6 +12,9 @@ import category_theory.abelian.projective
/-!
# Ext
> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
> Any changes to this file require a corresponding PR to mathlib4.
We define `Ext R C n : Cᵒᵖ ⥤ C ⥤ Module R` for any `R`-linear abelian category `C`
by (left) deriving in the first argument of the bifunctor `(X, Y) ↦ Module.of R (unop X ⟶ Y)`.
Expand Down
3 changes: 3 additions & 0 deletions src/category_theory/abelian/left_derived.lean
Expand Up @@ -12,6 +12,9 @@ import category_theory.limits.constructions.epi_mono
/-!
# Zeroth left derived functors
> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
> Any changes to this file require a corresponding PR to mathlib4.
If `F : C ⥤ D` is an additive right exact functor between abelian categories, where `C` has enough
projectives, we provide the natural isomorphism `F.left_derived 0 ≅ F`.
Expand Down
3 changes: 3 additions & 0 deletions src/category_theory/bicategory/single_obj.lean
Expand Up @@ -9,6 +9,9 @@ import category_theory.monoidal.functor
/-!
# Promoting a monoidal category to a single object bicategory.
> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
> Any changes to this file require a corresponding PR to mathlib4.
A monoidal category can be thought of as a bicategory with a single object.
The objects of the monoidal category become the 1-morphisms,
Expand Down
3 changes: 3 additions & 0 deletions src/data/real/golden_ratio.lean
Expand Up @@ -13,6 +13,9 @@ import algebra.linear_recurrence
/-!
# The golden ratio and its conjugate
> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
> Any changes to this file require a corresponding PR to mathlib4.
This file defines the golden ratio `φ := (1 + √5)/2` and its conjugate
`ψ := (1 - √5)/2`, which are the two real roots of `X² - X - 1`.
Expand Down
3 changes: 3 additions & 0 deletions src/measure_theory/category/Meas.lean
Expand Up @@ -11,6 +11,9 @@ import topology.category.Top.basic
/-!
# The category of measurable spaces
> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
> Any changes to this file require a corresponding PR to mathlib4.
Measurable spaces and measurable functions form a (concrete) category `Meas`.
## Main definitions
Expand Down
3 changes: 3 additions & 0 deletions src/measure_theory/decomposition/jordan.lean
Expand Up @@ -9,6 +9,9 @@ import measure_theory.measure.mutually_singular
/-!
# Jordan decomposition
> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
> Any changes to this file require a corresponding PR to mathlib4.
This file proves the existence and uniqueness of the Jordan decomposition for signed measures.
The Jordan decomposition theorem states that, given a signed measure `s`, there exists a
unique pair of mutually singular measures `μ` and `ν`, such that `s = μ - ν`.
Expand Down
3 changes: 3 additions & 0 deletions src/measure_theory/decomposition/signed_hahn.lean
Expand Up @@ -9,6 +9,9 @@ import order.symm_diff
/-!
# Hahn decomposition
> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
> Any changes to this file require a corresponding PR to mathlib4.
This file proves the Hahn decomposition theorem (signed version). The Hahn decomposition theorem
states that, given a signed measure `s`, there exist complementary, measurable sets `i` and `j`,
such that `i` is positive and `j` is negative with respect to `s`; that is, `s` restricted on `i`
Expand Down
3 changes: 3 additions & 0 deletions src/measure_theory/group/action.lean
Expand Up @@ -11,6 +11,9 @@ import dynamics.minimal
/-!
# Measures invariant under group actions
> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
> Any changes to this file require a corresponding PR to mathlib4.
A measure `μ : measure α` is said to be *invariant* under an action of a group `G` if scalar
multiplication by `c : G` is a measure preserving map for all `c`. In this file we define a
typeclass for measures invariant under action of an (additive or multiplicative) group and prove
Expand Down
3 changes: 3 additions & 0 deletions src/measure_theory/group/measure.lean
Expand Up @@ -14,6 +14,9 @@ import topology.continuous_function.cocompact_map
/-!
# Measures on Groups
> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
> Any changes to this file require a corresponding PR to mathlib4.
We develop some properties of measures on (topological) groups
* We define properties on measures: measures that are left or right invariant w.r.t. multiplication.
Expand Down
3 changes: 3 additions & 0 deletions src/number_theory/arithmetic_function.lean
Expand Up @@ -14,6 +14,9 @@ import data.nat.factorization.basic
/-!
# Arithmetic Functions and Dirichlet Convolution
> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
> Any changes to this file require a corresponding PR to mathlib4.
This file defines arithmetic functions, which are functions from `ℕ` to a specified type that map 0
to 0. In the literature, they are often instead defined as functions from `ℕ+`. These arithmetic
functions are endowed with a multiplication, given by Dirichlet convolution, and pointwise addition,
Expand Down
3 changes: 3 additions & 0 deletions src/number_theory/l_series.lean
Expand Up @@ -11,6 +11,9 @@ import topology.algebra.infinite_sum.basic
/-!
# L-series
> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
> Any changes to this file require a corresponding PR to mathlib4.
Given an arithmetic function, we define the corresponding L-series.
## Main Definitions
Expand Down
3 changes: 3 additions & 0 deletions src/number_theory/von_mangoldt.lean
Expand Up @@ -11,6 +11,9 @@ import analysis.special_functions.log.basic
/-!
# The von Mangoldt Function
> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
> Any changes to this file require a corresponding PR to mathlib4.
In this file we define the von Mangoldt function: the function on natural numbers that returns
`log p` if the input can be expressed as `p^k` for a prime `p`.
Expand Down
3 changes: 3 additions & 0 deletions src/topology/algebra/continuous_monoid_hom.lean
Expand Up @@ -10,6 +10,9 @@ import topology.continuous_function.algebra
# Continuous Monoid Homs
> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
> Any changes to this file require a corresponding PR to mathlib4.
This file defines the space of continuous homomorphisms between two topological groups.
## Main definitions
Expand Down
3 changes: 3 additions & 0 deletions src/topology/instances/discrete.lean
Expand Up @@ -11,6 +11,9 @@ import topology.metric_space.metrizable_uniformity
/-!
# Instances related to the discrete topology
> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
> Any changes to this file require a corresponding PR to mathlib4.
We prove that the discrete topology is
* first-countable,
* second-countable for an encodable type,
Expand Down
3 changes: 3 additions & 0 deletions src/topology/sheaves/stalks.lean
Expand Up @@ -17,6 +17,9 @@ import category_theory.sites.pushforward
/-!
# Stalks
> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
> Any changes to this file require a corresponding PR to mathlib4.
For a presheaf `F` on a topological space `X`, valued in some category `C`, the *stalk* of `F`
at the point `x : X` is defined as the colimit of the composition of the inclusion of categories
`(nhds x)ᵒᵖ ⥤ (opens X)ᵒᵖ` and the functor `F : (opens X)ᵒᵖ ⥤ C`.
Expand Down
3 changes: 3 additions & 0 deletions src/topology/tietze_extension.lean
Expand Up @@ -11,6 +11,9 @@ import topology.urysohns_bounded
/-!
# Tietze extension theorem
> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
> Any changes to this file require a corresponding PR to mathlib4.
In this file we prove a few version of the Tietze extension theorem. The theorem says that a
continuous function `s → ℝ` defined on a closed set in a normal topological space `Y` can be
extended to a continuous function on the whole space. Moreover, if all values of the original
Expand Down

0 comments on commit 61b5e27

Please sign in to comment.