Skip to content

Commit

Permalink
chore(*): add mathlib4 synchronization comments (#18139)
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.free_monoid.count`
* `algebra.order.lattice_group`
* `data.fin.basic`
* `data.int.range`
* `data.list.destutter`
* `data.list.nat_antidiagonal`
* `data.list.perm`
* `data.list.prime`
* `order.circular`
  • Loading branch information
leanprover-community-bot committed Jan 13, 2023
1 parent 0acae65 commit 044a140
Show file tree
Hide file tree
Showing 9 changed files with 27 additions and 0 deletions.
3 changes: 3 additions & 0 deletions src/algebra/free_monoid/count.lean
Original file line number Diff line number Diff line change
Expand Up @@ -9,6 +9,9 @@ import data.list.count
/-!
# `list.count` as a bundled homomorphism
> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
> Any changes to this file require a corresponding PR to mathlib4.
In this file we define `free_monoid.countp`, `free_monoid.count`, `free_add_monoid.countp`, and
`free_add_monoid.count`. These are `list.countp` and `list.count` bundled as multiplicative and
additive homomorphisms from `free_monoid` and `free_add_monoid`.
Expand Down
3 changes: 3 additions & 0 deletions src/algebra/order/lattice_group.lean
Original file line number Diff line number Diff line change
Expand Up @@ -10,6 +10,9 @@ import tactic.nth_rewrite
/-!
# Lattice ordered groups
> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
> Any changes to this file require a corresponding PR to mathlib4.
Lattice ordered groups were introduced by [Birkhoff][birkhoff1942].
They form the algebraic underpinnings of vector lattices, Banach lattices, AL-space, AM-space etc.
Expand Down
3 changes: 3 additions & 0 deletions src/data/fin/basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -12,6 +12,9 @@ import order.hom.set
/-!
# The finite type with `n` elements
> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
> Any changes to this file require a corresponding PR to mathlib4.
`fin n` is the type whose elements are natural numbers smaller than `n`.
This file expands on the development in the core library.
Expand Down
3 changes: 3 additions & 0 deletions src/data/int/range.lean
Original file line number Diff line number Diff line change
Expand Up @@ -9,6 +9,9 @@ import data.int.order.basic
/-!
# Intervals in ℤ
> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
> Any changes to this file require a corresponding PR to mathlib4.
This file defines integer ranges. `range m n` is the set of integers greater than `m` and strictly
less than `n`.
Expand Down
3 changes: 3 additions & 0 deletions src/data/list/destutter.lean
Original file line number Diff line number Diff line change
Expand Up @@ -8,6 +8,9 @@ import data.list.chain
/-!
# Destuttering of Lists
> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
> Any changes to this file require a corresponding PR to mathlib4.
This file proves theorems about `list.destutter` (in `data.list.defs`), which greedily removes all
non-related items that are adjacent in a list, e.g. `[2, 2, 3, 3, 2].destutter (≠) = [2, 3, 2]`.
Note that we make no guarantees of being the longest sublist with this property; e.g.,
Expand Down
3 changes: 3 additions & 0 deletions src/data/list/nat_antidiagonal.lean
Original file line number Diff line number Diff line change
Expand Up @@ -9,6 +9,9 @@ import data.list.range
/-!
# Antidiagonals in ℕ × ℕ as lists
> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
> Any changes to this file require a corresponding PR to mathlib4.
This file defines the antidiagonals of ℕ × ℕ as lists: the `n`-th antidiagonal is the list of
pairs `(i, j)` such that `i + j = n`. This is useful for polynomial multiplication and more
generally for sums going from `0` to `n`.
Expand Down
3 changes: 3 additions & 0 deletions src/data/list/perm.lean
Original file line number Diff line number Diff line change
Expand Up @@ -11,6 +11,9 @@ import data.nat.factorial.basic
/-!
# List Permutations
> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
> Any changes to this file require a corresponding PR to mathlib4.
This file introduces the `list.perm` relation, which is true if two lists are permutations of one
another.
Expand Down
3 changes: 3 additions & 0 deletions src/data/list/prime.lean
Original file line number Diff line number Diff line change
Expand Up @@ -11,6 +11,9 @@ import data.list.perm
/-!
# Products of lists of prime elements.
> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
> Any changes to this file require a corresponding PR to mathlib4.
This file contains some theorems relating `prime` and products of `list`s.
-/
Expand Down
3 changes: 3 additions & 0 deletions src/order/circular.lean
Original file line number Diff line number Diff line change
Expand Up @@ -8,6 +8,9 @@ import data.set.basic
/-!
# Circular order hierarchy
> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
> Any changes to this file require a corresponding PR to mathlib4.
This file defines circular preorders, circular partial orders and circular orders.
## Hierarchy
Expand Down

0 comments on commit 044a140

Please sign in to comment.