Skip to content

Commit 88c789e

Browse files
chore: update SHA of already forward-ported files (#2181)
Update some SHAs of files that changed in mathlib3. These 17 files need mainly only updated SHA as they've been only touched by backports or already have been forward-ported. The relevant changes are: * [Algebra.Group.Defs (#17884)](https://leanprover-community.github.io/mathlib-port-status/file/algebra/group/defs?range=41cf0cc2f528dd40a8f2db167ea4fb37b8fde7f3..2e0975f6a25dd3fbfb9e41556a77f075f6269748) * #945 * [Algebra.Group.WithOne.Defs (#18081)](https://leanprover-community.github.io/mathlib-port-status/file/algebra/group/with_one/defs?range=e574b1a4e891376b0ef974b926da39e05da12a06..995b47e555f1b6297c7cf16855f1023e355219fb) * #1439 * [Algebra.Module.Submodule.Basic (#18291) : backport](https://leanprover-community.github.io/mathlib-port-status/file/algebra/module/submodule/basic?range=f7fc89d5d5ff1db2d1242c7bb0e9062ce47ef47c..feb99064803fd3108e37c18b0f77d0a8344677a3) * [Algebra.Order.Monoid.WithTop (#18149, #18081)](https://leanprover-community.github.io/mathlib-port-status/file/algebra/order/monoid/with_top?range=2258b40dacd2942571c8ce136215350c702dc78f..e7e2ba8aa216a5833b5ed85a93317263711a36b5) * #1508 * #1439 * [Algebra.Order.Ring.WithTop (#18149, #18081)](https://leanprover-community.github.io/mathlib-port-status/file/algebra/order/ring/with_top?range=550b58538991c8977703fdeb7c9d51a5aa27df11..e7e2ba8aa216a5833b5ed85a93317263711a36b5) * #1508 * #1439 * [Data.Finset.NAry (#18081)](https://leanprover-community.github.io/mathlib-port-status/file/data/finset/n_ary?range=9003f28797c0664a49e4179487267c494477d853..995b47e555f1b6297c7cf16855f1023e355219fb) * #1439 * [Data.Option.NAry (#18081)](https://leanprover-community.github.io/mathlib-port-status/file/data/option/n_ary?range=2258b40dacd2942571c8ce136215350c702dc78f..995b47e555f1b6297c7cf16855f1023e355219fb) * #1439 * [Data.Set.NAry (#18081)](https://leanprover-community.github.io/mathlib-port-status/file/data/set/n_ary?range=2ed7e4aec72395b6a7c3ac4ac7873a7a43ead17c..995b47e555f1b6297c7cf16855f1023e355219fb) * #1439 * [Data.SetLike.Basic (#18291) : backport](https://leanprover-community.github.io/mathlib-port-status/file/data/set_like/basic?range=fc2ed6f838ce7c9b7c7171e58d78eaf7b438fb0e..feb99064803fd3108e37c18b0f77d0a8344677a3) * [Data.Sum.Basic (#18184)](https://leanprover-community.github.io/mathlib-port-status/file/data/sum/basic?range=d6aae1bcbd04b8de2022b9b83a5b5b10e10c777d..f4ecb599422baaf39055d8278c7d9ef3b5b72b88) * #1583 * [GroupTheory.GroupAction.SubMulAction (#18291) : backport](https://leanprover-community.github.io/mathlib-port-status/file/group_theory/group_action/sub_mul_action?range=f93c11933efbc3c2f0299e47b8ff83e9b539cbf6..feb99064803fd3108e37c18b0f77d0a8344677a3) * [GroupTheory.Submonoid.Basic (#18291) : backport](https://leanprover-community.github.io/mathlib-port-status/file/group_theory/submonoid/basic?range=207cfac9fcd06138865b5d04f7091e46d9320432..feb99064803fd3108e37c18b0f77d0a8344677a3) * [ Logic.Basic (#18291): backport](https://leanprover-community.github.io/mathlib-port-status/file/logic/basic?range=1c521b4fb909320eca16b2bb6f8b5b0490b1cb5e..feb99064803fd3108e37c18b0f77d0a8344677a3) * #1509 * [Order.InitialSeg (#18198): backport](https://leanprover-community.github.io/mathlib-port-status/file/order/initial_seg?range=ee0c179cd3c8a45aa5bffbf1b41d8dbede452865..7c3269ca3fa4c0c19e4d127cd7151edbdbf99ed4) * [Order.RelClasses (#17957)](https://leanprover-community.github.io/mathlib-port-status/file/order/rel_classes?range=c4658a649d216f57e99621708b09dcb3dcccbd23..bc7d81beddb3d6c66f71449c5bc76c38cb77cf9e) * #1047 * [Order.WithBot (#18081)](https://leanprover-community.github.io/mathlib-port-status/file/order/with_bot?range=70d50ecfd4900dd6d328da39ab7ebd516abe4025..995b47e555f1b6297c7cf16855f1023e355219fb) * #1439 * [RingTheory.Subsemiring.Basic (#18291) : backport](https://leanprover-community.github.io/mathlib-port-status/file/ring_theory/subsemiring/basic?range=f93c11933efbc3c2f0299e47b8ff83e9b539cbf6..feb99064803fd3108e37c18b0f77d0a8344677a3) Co-authored-by: Eric Wieser <wieser.eric@gmail.com>
1 parent bc5bc3c commit 88c789e

File tree

17 files changed

+84
-33
lines changed

17 files changed

+84
-33
lines changed

Mathlib/Algebra/Group/Defs.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Jeremy Avigad, Leonardo de Moura, Simon Hudon, Mario Carneiro
55
66
! This file was ported from Lean 3 source module algebra.group.defs
7-
! leanprover-community/mathlib commit 41cf0cc2f528dd40a8f2db167ea4fb37b8fde7f3
7+
! leanprover-community/mathlib commit 2e0975f6a25dd3fbfb9e41556a77f075f6269748
88
! Please do not edit these lines, except to modify the commit id
99
! if you have ported upstream changes.
1010
-/

Mathlib/Algebra/Group/WithOne/Defs.lean

Lines changed: 3 additions & 8 deletions
Original file line numberDiff line numberDiff line change
@@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Mario Carneiro, Johan Commelin
55
66
! This file was ported from Lean 3 source module algebra.group.with_one.defs
7-
! leanprover-community/mathlib commit e574b1a4e891376b0ef974b926da39e05da12a06
7+
! leanprover-community/mathlib commit 995b47e555f1b6297c7cf16855f1023e355219fb
88
! Please do not edit these lines, except to modify the commit id
99
! if you have ported upstream changes.
1010
-/
@@ -98,7 +98,7 @@ instance inhabited : Inhabited (WithOne α) :=
9898
instance nontrivial [Nonempty α] : Nontrivial (WithOne α) :=
9999
Option.nontrivial
100100

101-
-- porting note: this new declaration is here to make `((a : α): WithOne α)` have type `WithOne α` ;
101+
-- porting note: this new declaration is here to make `((a : α): WithOne α)` have type `WithOne α`;
102102
-- otherwise the coercion kicks in and it becomes `Option.some a : WithOne α` which
103103
-- becomes `Option.some a : Option α`.
104104
/-- The canonical map from `α` into `WithOne α` -/
@@ -190,11 +190,6 @@ protected theorem cases_on {P : WithOne α → Prop} : ∀ x : WithOne α, P 1
190190
-- port note: I don't know if `elab_as_elim` is being added to the additivised declaration.
191191
attribute [elab_as_elim] WithZero.cases_on
192192

193-
-- porting note: in Lean 3 there was the following comment:
194-
-- the `show` statements in the proofs are important, because otherwise the generated lemmas
195-
-- `WithOne.mulOneClass._proof_{1,2}` have an ill-typed statement after `WithOne` is made
196-
-- irreducible. Maybe one day when mathlib is ported to Lean 4 we can experiment
197-
-- to see if these `show` comments can be removed.
198193
@[to_additive]
199194
instance mulOneClass [Mul α] : MulOneClass (WithOne α) where
200195
mul := (· * ·)
@@ -290,7 +285,7 @@ instance commMonoidWithZero [CommMonoid α] : CommMonoidWithZero (WithZero α) :
290285
{ WithZero.monoidWithZero, WithZero.commSemigroup with }
291286

292287
/-- Given an inverse operation on `α` there is an inverse operation
293-
on `WithZero α` sending `0` to `0`-/
288+
on `WithZero α` sending `0` to `0`. -/
294289
instance inv [Inv α] : Inv (WithZero α) :=
295290
fun a => Option.map Inv.inv a⟩
296291

Mathlib/Algebra/Module/Submodule/Basic.lean

Lines changed: 6 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Nathaniel Thomas, Jeremy Avigad, Johannes Hölzl, Mario Carneiro
55
66
! This file was ported from Lean 3 source module algebra.module.submodule.basic
7-
! leanprover-community/mathlib commit f7fc89d5d5ff1db2d1242c7bb0e9062ce47ef47c
7+
! leanprover-community/mathlib commit feb99064803fd3108e37c18b0f77d0a8344677a3
88
! Please do not edit these lines, except to modify the commit id
99
! if you have ported upstream changes.
1010
-/
@@ -38,7 +38,11 @@ universe u'' u' u v w
3838

3939
variable {G : Type u''} {S : Type u'} {R : Type u} {M : Type v} {ι : Type w}
4040

41-
/-- `SubmoduleClass S R M` says `S` is a type of submodules `s ≤ M`. -/
41+
/--
42+
`SubmoduleClass S R M` says `S` is a type of submodules `s ≤ M`.
43+
44+
Note that only `R` is marked as `outParam` since `M` is already supplied by the `SetLike` class.
45+
-/
4246
class SubmoduleClass (S : Type _) (R : outParam <| Type _) (M : Type _) [AddZeroClass M] [SMul R M]
4347
[SetLike S M] [AddSubmonoidClass S M] extends SMulMemClass S R M
4448
#align submodule_class SubmoduleClass

Mathlib/Algebra/Order/Monoid/WithTop.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -5,7 +5,7 @@ Authors: Jeremy Avigad, Leonardo de Moura, Mario Carneiro, Johannes Hölzl
55
Ported by: Jon Eugster
66
77
! This file was ported from Lean 3 source module algebra.order.monoid.with_top
8-
! leanprover-community/mathlib commit 2258b40dacd2942571c8ce136215350c702dc78f
8+
! leanprover-community/mathlib commit e7e2ba8aa216a5833b5ed85a93317263711a36b5
99
! Please do not edit these lines, except to modify the commit id
1010
! if you have ported upstream changes.
1111
-/

Mathlib/Algebra/Order/Ring/WithTop.lean

Lines changed: 4 additions & 4 deletions
Original file line numberDiff line numberDiff line change
@@ -3,7 +3,7 @@ Copyright (c) 2016 Jeremy Avigad. All rights reserved.
33
Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Jeremy Avigad, Leonardo de Moura, Mario Carneiro
55
! This file was ported from Lean 3 source module algebra.order.ring.with_top
6-
! leanprover-community/mathlib commit 550b58538991c8977703fdeb7c9d51a5aa27df11
6+
! leanprover-community/mathlib commit e7e2ba8aa216a5833b5ed85a93317263711a36b5
77
! Please do not edit these lines, except to modify the commit id
88
! if you have ported upstream changes.
99
-/
@@ -425,9 +425,9 @@ instance [MulZeroClass α] [Preorder α] [MulPosMonoRev α] : MulPosMonoRev (Wit
425425
exact le_of_mul_le_mul_right h x0 ⟩
426426

427427
instance orderedCommSemiring [CanonicallyOrderedCommSemiring α] [Nontrivial α] :
428-
OrderedCommSemiring (WithBot α) :=
428+
OrderedCommSemiring (WithBot α) :=
429429
{ WithBot.zeroLEOneClass, WithBot.orderedAddCommMonoid, WithBot.commSemiring with
430-
mul_le_mul_of_nonneg_left := fun _ _ _ => mul_le_mul_of_nonneg_left,
431-
mul_le_mul_of_nonneg_right := fun _ _ _ => mul_le_mul_of_nonneg_right, }
430+
mul_le_mul_of_nonneg_left := fun _ _ _ => mul_le_mul_of_nonneg_left
431+
mul_le_mul_of_nonneg_right := fun _ _ _ => mul_le_mul_of_nonneg_right }
432432

433433
end WithBot

Mathlib/Data/Finset/NAry.lean

Lines changed: 14 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Yaël Dillies
55
66
! This file was ported from Lean 3 source module data.finset.n_ary
7-
! leanprover-community/mathlib commit 9003f28797c0664a49e4179487267c494477d853
7+
! leanprover-community/mathlib commit 995b47e555f1b6297c7cf16855f1023e355219fb
88
! Please do not edit these lines, except to modify the commit id
99
! if you have ported upstream changes.
1010
-/
@@ -475,4 +475,17 @@ theorem image_image₂_right_anticomm {f : α → β' → γ} {g : β → β'} {
475475
(image_image₂_antidistrib_right fun a b => (h_right_anticomm b a).symm).symm
476476
#align finset.image_image₂_right_anticomm Finset.image_image₂_right_anticomm
477477

478+
/-- If `a` is a left identity for `f : α → β → β`, then `{a}` is a left identity for
479+
`Finset.image₂ f`. -/
480+
theorem image₂_left_identity {f : α → γ → γ} {a : α} (h : ∀ b, f a b = b) (t : Finset γ) :
481+
image₂ f {a} t = t :=
482+
coe_injective <| by rw [coe_image₂, coe_singleton, Set.image2_left_identity h]
483+
#align finset.image₂_left_identity Finset.image₂_left_identity
484+
485+
/-- If `b` is a right identity for `f : α → β → α`, then `{b}` is a right identity for
486+
`Finset.image₂ f`. -/
487+
theorem image₂_right_identity {f : γ → β → γ} {b : β} (h : ∀ a, f a b = a) (s : Finset γ) :
488+
image₂ f s {b} = s := by rw [image₂_singleton_right, funext h, image_id']
489+
#align finset.image₂_right_identity Finset.image₂_right_identity
490+
478491
end Finset

Mathlib/Data/Option/NAry.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Yaël Dillies
55
66
! This file was ported from Lean 3 source module data.option.n_ary
7-
! leanprover-community/mathlib commit 2258b40dacd2942571c8ce136215350c702dc78f
7+
! leanprover-community/mathlib commit 995b47e555f1b6297c7cf16855f1023e355219fb
88
! Please do not edit these lines, except to modify the commit id
99
! if you have ported upstream changes.
1010
-/

Mathlib/Data/Set/NAry.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Floris van Doorn
55
66
! This file was ported from Lean 3 source module data.set.n_ary
7-
! leanprover-community/mathlib commit 2ed7e4aec72395b6a7c3ac4ac7873a7a43ead17c
7+
! leanprover-community/mathlib commit 995b47e555f1b6297c7cf16855f1023e355219fb
88
! Please do not edit these lines, except to modify the commit id
99
! if you have ported upstream changes.
1010
-/

Mathlib/Data/SetLike/Basic.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Eric Wieser
55
66
! This file was ported from Lean 3 source module data.set_like.basic
7-
! leanprover-community/mathlib commit fc2ed6f838ce7c9b7c7171e58d78eaf7b438fb0e
7+
! leanprover-community/mathlib commit feb99064803fd3108e37c18b0f77d0a8344677a3
88
! Please do not edit these lines, except to modify the commit id
99
! if you have ported upstream changes.
1010
-/

Mathlib/Data/Sum/Basic.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Mario Carneiro, Yury G. Kudryashov
55
66
! This file was ported from Lean 3 source module data.sum.basic
7-
! leanprover-community/mathlib commit d6aae1bcbd04b8de2022b9b83a5b5b10e10c777d
7+
! leanprover-community/mathlib commit f4ecb599422baaf39055d8278c7d9ef3b5b72b88
88
! Please do not edit these lines, except to modify the commit id
99
! if you have ported upstream changes.
1010
-/

0 commit comments

Comments
 (0)