WARNING: THIS SITE IS A MIRROR OF GITHUB.COM / IT CANNOT LOGIN OR REGISTER ACCOUNTS / THE CONTENTS ARE PROVIDED AS-IS / THIS SITE ASSUMES NO RESPONSIBILITY FOR ANY DISPLAYED CONTENT OR LINKS / IF YOU FOUND SOMETHING MAY NOT GOOD FOR EVERYONE, CONTACT ADMIN AT ilovescratch@foxmail.com
Skip to content

Commit 7ddd6dc

Browse files
chore: bump mathlib to v4.22.0 (#696)
Co-authored-by: Kevin Buzzard <[email protected]>
1 parent 1e3cb91 commit 7ddd6dc

File tree

14 files changed

+58
-120
lines changed

14 files changed

+58
-120
lines changed

FLT.lean

Lines changed: 0 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -54,8 +54,6 @@ import FLT.Mathlib.Algebra.IsQuaternionAlgebra
5454
import FLT.Mathlib.Algebra.Module.LinearMap.Defs
5555
import FLT.Mathlib.Algebra.Module.Submodule.Basic
5656
import FLT.Mathlib.Algebra.Order.AbsoluteValue.Basic
57-
import FLT.Mathlib.Algebra.Order.GroupWithZero
58-
import FLT.Mathlib.Algebra.Order.GroupWithZero.Canonical
5957
import FLT.Mathlib.Analysis.Normed.Ring.WithAbs
6058
import FLT.Mathlib.Analysis.SpecialFunctions.Stirling
6159
import FLT.Mathlib.Data.Fin.Basic

FLT/AutomorphicRepresentation/Example.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -262,10 +262,10 @@ lemma multiples (N : ℕ+) (z : ZHat) : (∃ (y : ZHat), N * y = z) ↔ z N = 0
262262
rw [h, ZMod.castHom_apply, ZMod.cast_eq_val, ZMod.natCast_eq_zero_iff] at hk
263263
have hNjk := z.prop (N * j) (N * k) (mul_dvd_mul (dvd_refl _) hjk)
264264
rw [ZMod.castHom_apply, ZMod.cast_eq_val] at hNjk
265-
simp only [PNat.mul_coe, map_natCast, ZMod.eq_iff_modEq_nat]
265+
simp only [PNat.mul_coe, map_natCast, ZMod.natCast_eq_natCast_iff]
266266
apply Nat.ModEq.mul_right_cancel' (c := N) (by simp)
267267
rw [Nat.div_mul_cancel hj, Nat.div_mul_cancel hk,
268-
mul_comm (j : ℕ) (N : ℕ), ← ZMod.eq_iff_modEq_nat, hNjk]
268+
mul_comm (j : ℕ) (N : ℕ), ← ZMod.natCast_eq_natCast_iff, hNjk]
269269
simp
270270
}
271271
refine ⟨y, ?_⟩

FLT/DedekindDomain/AdicValuation.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -6,7 +6,7 @@ Authors: Matthew Jasper
66
import FLT.Mathlib.Topology.Algebra.Valued.ValuationTopology
77
import FLT.Mathlib.RingTheory.Valuation.ValuationSubring
88
import FLT.Mathlib.RingTheory.LocalRing.MaximalIdeal.Basic
9-
import FLT.Mathlib.Algebra.Order.GroupWithZero
9+
import Mathlib.Algebra.Order.GroupWithZero.Canonical
1010
import Mathlib.RingTheory.DedekindDomain.AdicValuation
1111
import Mathlib.Algebra.Group.Int.TypeTags
1212
import Mathlib.NumberTheory.RamificationInertia.Basic

FLT/Deformations/RepresentationTheory/AbsoluteGaloisGroup.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -278,7 +278,7 @@ instance neZero_maximalIdeal_integralClosure :
278278
NeZero (𝔪 (IntegralClosure 𝒪ᵥ (Kᵥᵃˡᵍ))) := by
279279
have : 𝒪ᵥ ≠ ⊤ := by
280280
refine fun h ↦ IsDiscreteValuationRing.not_isField 𝒪ᵥ (h ▸ ?_)
281-
exact (Subring.topEquiv (R := Kᵥ)).isField _ (Semifield.toIsField Kᵥ)
281+
exact (Subring.topEquiv (R := Kᵥ)).isField (Semifield.toIsField Kᵥ)
282282
exact ⟨(Ideal.bot_lt_of_maximal (𝔪 _)
283283
(not_isField_integralClosure (L := Kᵥᵃˡᵍ) _ this)).ne'⟩
284284

FLT/Deformations/RepresentationTheory/Basic.lean

Lines changed: 1 addition & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -271,11 +271,9 @@ lemma Matrix.map_det {F α β n : Type*} [CommRing β] [CommRing α] [Fintype n]
271271
(M.map f).det = f M.det :=
272272
(RingHom.map_det (f : α →+* β) M).symm
273273

274-
@[simp]
275274
lemma LinearMap.trace_toLin' {R n : Type*} [CommSemiring R] [DecidableEq n]
276275
[Fintype n] (M : Matrix n n R) : LinearMap.trace _ _ M.toLin' = M.trace := by
277-
rw [LinearMap.trace_eq_matrix_trace _ (Pi.basisFun ..), LinearMap.toMatrix_eq_toMatrix',
278-
LinearMap.toMatrix'_toLin']
276+
simp
279277

280278
omit [NumberField K] in
281279
lemma FramedGaloisRep.det_baseChange [IsTopologicalRing B]

FLT/HaarMeasure/HaarChar/AddEquiv.lean

Lines changed: 12 additions & 8 deletions
Original file line numberDiff line numberDiff line change
@@ -41,8 +41,9 @@ variable [BorelSpace G] [IsTopologicalGroup G] [LocallyCompactSpace G]
4141

4242
/-- If `φ : G ≃ₜ* G` then `mulEquivHaarChar φ` is the positive real factor by which
4343
`φ` scales Haar measure on `G`. -/
44-
@[to_additive "If `φ : A ≃ₜ+ A` then `addEquivAddHaarChar φ` is the positive
45-
real factor by which `φ` scales Haar measure on `A`."]
44+
@[to_additive
45+
/-- If `φ : A ≃ₜ+ A` then `addEquivAddHaarChar φ` is the positive real factor by which
46+
`φ` scales Haar measure on `A`. -/]
4647
noncomputable def mulEquivHaarChar (φ : G ≃ₜ* G) : ℝ≥0 :=
4748
haarScalarFactor haar (map φ haar)
4849

@@ -240,8 +241,9 @@ lemma mulEquivHaarChar_eq_mulEquivHaarChar_of_isOpenEmbedding {X Y : Type*}
240241

241242
/-- A version of `mulEquivHaarChar_eq_mulEquivHaarChar_of_isOpenEmbedding` with the stronger
242243
assumption that `f` is a `ContinuousMulEquiv`, for convenience. -/
243-
@[to_additive "A version of `addEquivAddHaarChar_eq_addEquivAddHaarChar_of_isOpenEmbedding`
244-
with the stronger assumption that `f` is a `ContinuousAddEquiv`, for convenience."]
244+
@[to_additive
245+
/-- A version of `addEquivAddHaarChar_eq_addEquivAddHaarChar_of_isOpenEmbedding` with the stronger
246+
assumption that `f` is a `ContinuousAddEquiv`, for convenience. -/]
245247
lemma mulEquivHaarChar_eq_mulEquivHaarChar_of_continuousMulEquiv {X Y : Type*}
246248
[TopologicalSpace X] [Group X] [IsTopologicalGroup X] [LocallyCompactSpace X]
247249
[MeasurableSpace X] [BorelSpace X]
@@ -260,8 +262,9 @@ variable {A B C D : Type*} [Group A] [Group B] [Group C] [Group D]
260262

261263
/-- The product of two multiplication-preserving homeomorphisms is
262264
a multiplication-preserving homeomorphism. -/
263-
@[to_additive "The product of
264-
two addition-preserving homeomorphisms is an addition-preserving homeomorphism."]
265+
@[to_additive
266+
/-- The product of two addition-preserving homeomorphisms is
267+
an addition-preserving homeomorphism. -/]
265268
def _root_.ContinuousMulEquiv.prodCongr (φ : A ≃ₜ* B) (ψ : C ≃ₜ* D) : A × C ≃ₜ* B × D where
266269
__ := φ.toMulEquiv.prodCongr ψ
267270
continuous_toFun := Continuous.prodMap φ.continuous_toFun ψ.continuous_toFun
@@ -388,8 +391,9 @@ variable {ι : Type*} {G H : ι → Type*}
388391
/-- An arbitrary product of multiplication-preserving homeomorphisms
389392
is a multiplication-preserving homeomorphism.
390393
-/
391-
@[to_additive "An arbitrary product of
392-
addition-preserving homeomorphisms is an addition-preserving homeomorphism."]
394+
@[to_additive
395+
/-- An arbitrary product of addition-preserving homeomorphisms
396+
is an addition-preserving homeomorphism. -/]
393397
def _root_.ContinuousMulEquiv.piCongrRight (ψ : Π i, (G i) ≃ₜ* (H i)) :
394398
(∀ i, G i) ≃ₜ* (∀ i, H i) where
395399
__ := MulEquiv.piCongrRight (fun i ↦ ψ i)

FLT/Mathlib/Algebra/Order/GroupWithZero.lean

Lines changed: 0 additions & 28 deletions
This file was deleted.

FLT/Mathlib/Algebra/Order/GroupWithZero/Canonical.lean

Lines changed: 0 additions & 41 deletions
This file was deleted.

FLT/Mathlib/Topology/Algebra/ContinuousMonoidHom.lean

Lines changed: 4 additions & 4 deletions
Original file line numberDiff line numberDiff line change
@@ -21,8 +21,8 @@ def ContinuousAddEquiv.quotientPi {ι : Type*} {G : ι → Type*} [(i : ι) →
2121
/-- A family indexed by a type with a unique element
2222
is `ContinuousMulEquiv` to the element at the single index. -/
2323
@[to_additive
24-
"A family indexed by a type with a unique element
25-
is `ContinuousAddEquiv` to the element at the single index."]
24+
/-- A family indexed by a type with a unique element
25+
is `ContinuousAddEquiv` to the element at the single index. -/]
2626
def ContinuousMulEquiv.piUnique {ι : Type*} (M : ι → Type*) [(j : ι) → Mul (M j)]
2727
[(j : ι) → TopologicalSpace (M j)] [Unique ι] :
2828
((j : ι) → M j) ≃ₜ* M default where
@@ -33,8 +33,8 @@ def ContinuousMulEquiv.piUnique {ι : Type*} (M : ι → Type*) [(j : ι) → Mu
3333
/-- Splits the indices of `∀ (i : ι), Y i` along the predicate `p`.
3434
This is `Equiv.piEquivPiSubtypeProd` as a `ContinuousMulEquiv`. -/
3535
@[to_additive piEquivPiSubtypeProd
36-
"Splits the indices of `∀ (i : ι), Y i` along the predicate `p`.
37-
This is `Equiv.piEquivPiSubtypeProd` as a `ContinuousAddEquiv`."]
36+
/-- Splits the indices of `∀ (i : ι), Y i` along the predicate `p`.
37+
This is `Equiv.piEquivPiSubtypeProd` as a `ContinuousAddEquiv`. -/]
3838
def ContinuousMulEquiv.piEquivPiSubtypeProd {ι : Type*} (p : ι → Prop) (Y : ι → Type*)
3939
[(i : ι) → TopologicalSpace (Y i)] [(i : ι) → Mul (Y i)] [DecidablePred p] :
4040
((i : ι) → Y i) ≃ₜ* ((i : { x : ι // p x }) → Y i) × ((i : { x : ι // ¬p x }) → Y i) :=

FLT/Mathlib/Topology/Algebra/RestrictedProduct/Basic.lean

Lines changed: 8 additions & 5 deletions
Original file line numberDiff line numberDiff line change
@@ -66,8 +66,9 @@ variable [Π i, Monoid (G i)] [Π i, SubmonoidClass (S i) (G i)]
6666
[Π i, Monoid (H i)] [Π i, SubmonoidClass (T i) (H i)] in
6767
/-- The monoid homomorphism between restricted products over a fixed index type,
6868
given monoid homomorphisms on the factors. -/
69-
@[to_additive "The additive monoid homomorphism between restricted products over a fixed index type,
70-
given additive monoid homomorphisms on the factors."]
69+
@[to_additive
70+
/-- The additive monoid homomorphism between restricted products over a fixed index type,
71+
given additive monoid homomorphisms on the factors. -/]
7172
def MonoidHom.restrictedProductCongrRight (φ : (i : ι) → G i →* H i)
7273
(hφ : ∀ᶠ i in ℱ, Set.MapsTo (φ i) (A i) (B i)) :
7374
Πʳ i, [G i, A i]_[ℱ] →* Πʳ i, [H i, B i]_[ℱ] where
@@ -109,8 +110,9 @@ variable [(i : ι) → One (G i)] in
109110
/-- The support of an element of a restricted product of monoids (or more generally,
110111
objects with a 1. The support is the components which aren't 1.)
111112
-/
112-
@[to_additive "The support of an element of a restricted product of additive monoids
113-
(or more generally, objects with a 0. The support is the components which aren't 0."]
113+
@[to_additive
114+
/-- The support of an element of a restricted product of additive monoids (or more generally,
115+
objects with a 0. The support is the components which aren't 0. -/]
114116
def mulSupport (u : Πʳ i, [G i, A i]) : Set ι :=
115117
{i : ι | u i ≠ 1}
116118

@@ -328,7 +330,8 @@ variable (A : (i : ι) → (S i))
328330
variable [DecidableEq ι]
329331

330332
/-- The function supported at `i`, with value `x` there, and `1` elsewhere. -/
331-
@[to_additive "The function supported at `i`, with value `x` there, and `0` elsewhere."]
333+
@[to_additive
334+
/-- The function supported at `i`, with value `x` there, and `0` elsewhere. -/]
332335
def mulSingle [∀ i, One (G i)] [∀ i, OneMemClass (S i) (G i)] (i : ι) (x : G i) :
333336
Πʳ i, [G i, A i] where
334337
val := Pi.mulSingle i x

0 commit comments

Comments
 (0)