Skip to content

Commit

Permalink
chore: sync some sha sums (#2116)
Browse files Browse the repository at this point in the history
Part of the `List.repeat` -> `List.replicate` refactor. On Mathlib 4 side, I removed mentions of `List.repeat` in #1475 and #1579

* [`algebra.big_operators.basic`@`9003f28797c0664a49e4179487267c494477d853`..`47adfab39a11a072db552f47594bf8ed2cf8a722`](https://leanprover-community.github.io/mathlib-port-status/file/algebra/big_operators/basic?from=9003f28797c0664a49e4179487267c494477d853&to=47adfab39a11a072db552f47594bf8ed2cf8a722)
* [`algebra.big_operators.multiset.basic`@`9003f28797c0664a49e4179487267c494477d853`..`47adfab39a11a072db552f47594bf8ed2cf8a722`](https://leanprover-community.github.io/mathlib-port-status/file/algebra/big_operators/multiset/basic?from=9003f28797c0664a49e4179487267c494477d853&to=47adfab39a11a072db552f47594bf8ed2cf8a722)
* [`algebra.gcd_monoid.multiset`@`9003f28797c0664a49e4179487267c494477d853`..`f694c7dead66f5d4c80f446c796a5aad14707f0e`](https://leanprover-community.github.io/mathlib-port-status/file/algebra/gcd_monoid/multiset?from=9003f28797c0664a49e4179487267c494477d853&to=f694c7dead66f5d4c80f446c796a5aad14707f0e)
* [`algebra.hom.freiman`@`9003f28797c0664a49e4179487267c494477d853`..`f694c7dead66f5d4c80f446c796a5aad14707f0e`](https://leanprover-community.github.io/mathlib-port-status/file/algebra/hom/freiman?from=9003f28797c0664a49e4179487267c494477d853&to=f694c7dead66f5d4c80f446c796a5aad14707f0e)
* [`data.list.big_operators.basic`@`26f081a2fb920140ed5bc5cc5344e84bcc7cb2b2`..`47adfab39a11a072db552f47594bf8ed2cf8a722`](https://leanprover-community.github.io/mathlib-port-status/file/data/list/big_operators/basic?from=26f081a2fb920140ed5bc5cc5344e84bcc7cb2b2&to=47adfab39a11a072db552f47594bf8ed2cf8a722)
* [`data.list.dedup`@`6133ae2da6ae6693248bb5451de703f1ef154cc8`..`f694c7dead66f5d4c80f446c796a5aad14707f0e`](https://leanprover-community.github.io/mathlib-port-status/file/data/list/dedup?from=6133ae2da6ae6693248bb5451de703f1ef154cc8&to=f694c7dead66f5d4c80f446c796a5aad14707f0e)
  • Loading branch information
urkud committed Feb 7, 2023
1 parent 52c04a3 commit e37d93e
Show file tree
Hide file tree
Showing 6 changed files with 6 additions and 6 deletions.
2 changes: 1 addition & 1 deletion Mathlib/Algebra/BigOperators/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Johannes Hölzl
! This file was ported from Lean 3 source module algebra.big_operators.basic
! leanprover-community/mathlib commit 9003f28797c0664a49e4179487267c494477d853
! leanprover-community/mathlib commit 47adfab39a11a072db552f47594bf8ed2cf8a722
! Please do not edit these lines, except to modify the commit id
! if you have ported upstream changes.
-/
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Algebra/BigOperators/Multiset/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Mario Carneiro
! This file was ported from Lean 3 source module algebra.big_operators.multiset.basic
! leanprover-community/mathlib commit 9003f28797c0664a49e4179487267c494477d853
! leanprover-community/mathlib commit 47adfab39a11a072db552f47594bf8ed2cf8a722
! Please do not edit these lines, except to modify the commit id
! if you have ported upstream changes.
-/
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Algebra/GCDMonoid/Multiset.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Aaron Anderson
! This file was ported from Lean 3 source module algebra.gcd_monoid.multiset
! leanprover-community/mathlib commit 9003f28797c0664a49e4179487267c494477d853
! leanprover-community/mathlib commit f694c7dead66f5d4c80f446c796a5aad14707f0e
! Please do not edit these lines, except to modify the commit id
! if you have ported upstream changes.
-/
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Algebra/Hom/Freiman.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Yaël Dillies
! This file was ported from Lean 3 source module algebra.hom.freiman
! leanprover-community/mathlib commit 9003f28797c0664a49e4179487267c494477d853
! leanprover-community/mathlib commit f694c7dead66f5d4c80f446c796a5aad14707f0e
! Please do not edit these lines, except to modify the commit id
! if you have ported upstream changes.
-/
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Data/List/BigOperators/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Johannes Hölzl, Floris van Doorn, Sébastien Gouëzel, Alex J. Best
! This file was ported from Lean 3 source module data.list.big_operators.basic
! leanprover-community/mathlib commit 26f081a2fb920140ed5bc5cc5344e84bcc7cb2b2
! leanprover-community/mathlib commit 47adfab39a11a072db552f47594bf8ed2cf8a722
! Please do not edit these lines, except to modify the commit id
! if you have ported upstream changes.
-/
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Data/List/Dedup.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Mario Carneiro
! This file was ported from Lean 3 source module data.list.dedup
! leanprover-community/mathlib commit 6133ae2da6ae6693248bb5451de703f1ef154cc8
! leanprover-community/mathlib commit f694c7dead66f5d4c80f446c796a5aad14707f0e
! Please do not edit these lines, except to modify the commit id
! if you have ported upstream changes.
-/
Expand Down

0 comments on commit e37d93e

Please sign in to comment.