Skip to content

Commit 96f5ac1

Browse files
authored
chore: bump mathlib (#759)
Also, change `lakefile.toml` to point to the master branch of mathlib.
1 parent 9ae0a89 commit 96f5ac1

File tree

10 files changed

+23
-28
lines changed

10 files changed

+23
-28
lines changed

FLT/Data/QHat.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -690,7 +690,7 @@ lemma unitsrat_join_unitszHat : unitsratsub ⊔ unitszHatsub = ⊤ := by
690690
have h : (M : QHat) = (M : ℚ) ⊗ₜ[ℤ] 1 := by norm_cast
691691
rw [Algebra.TensorProduct.includeRight_apply, hxinv, h, Algebra.TensorProduct.tmul_mul_tmul,
692692
mul_one, one_div, inv_mul_cancel₀]
693-
simp only [ne_eq, Rat.natCast_eq_zero, PNat.ne_zero, not_false_eq_true]
693+
simp only [ne_eq, Rat.natCast_eq_zero_iff, PNat.ne_zero, not_false_eq_true]
694694
rcases hx with ⟨X, hX⟩
695695
let I := Ideal.span {X}
696696
let J := I.comap (Int.castRingHom ZHat)
@@ -729,7 +729,7 @@ lemma unitsrat_join_unitszHat : unitsratsub ⊔ unitszHatsub = ⊤ := by
729729
set G : ℚ := 1 / g with G_def
730730
have gG : g * G = 1 := by
731731
rw [G_def, one_div, mul_inv_cancel₀]
732-
simp only [ne_eq, Rat.intCast_eq_zero, Int.ne_of_gt gpos, not_false_eq_true]
732+
simp only [ne_eq, Rat.intCast_eq_zero_iff, Int.ne_of_gt gpos, not_false_eq_true]
733733
use ⟨g, G, gG, mul_comm _ G ▸ gG⟩
734734
use ⟨z, y, by rw[mul_comm]; exact this, this⟩
735735
simp only [← Units.val_inj, ← hX, Units.map_mk, MonoidHom.coe_coe, map_intCast,

FLT/DedekindDomain/AdicValuation.lean

Lines changed: 5 additions & 5 deletions
Original file line numberDiff line numberDiff line change
@@ -89,8 +89,8 @@ lemma emultiplicity_eq_of_valuation_eq_ofAdd {a : A} {k : ℕ}
8989
have hnz : a ≠ 0 := ne_zero_of_some_le_intValuation _ (le_of_eq hv.symm)
9090
have hnb : Ideal.span {a} ≠ ⊥ := by
9191
rwa [ne_eq, Ideal.span_singleton_eq_bot]
92-
simp only [intValuation_if_neg _ hnz, ofAdd_neg, WithZero.coe_inv, inv_inj, WithZero.coe_inj,
93-
EmbeddingLike.apply_eq_iff_eq, Nat.cast_inj] at hv
92+
simp only [intValuation_if_neg _ hnz, WithZero.exp, ofAdd_neg, WithZero.coe_inv, inv_inj,
93+
WithZero.coe_inj, EmbeddingLike.apply_eq_iff_eq, Nat.cast_inj] at hv
9494
rw [← hv, UniqueFactorizationMonoid.emultiplicity_eq_count_normalizedFactors v.irreducible hnb,
9595
count_associates_factors_eq hnb v.isPrime v.ne_bot, normalize_eq]
9696

@@ -117,7 +117,7 @@ lemma exists_adicValued_mul_sub_le {a b : A} {γ : WithZero (Multiplicative ℤ)
117117
(emultiplicity_eq_of_valuation_eq_ofAdd v <| intValuation_eq_coe_neg_multiplicity v hnz)
118118
(ENat.coe_le_coe.mpr hle)
119119
have hb : b ∈ v.asIdeal ^ multiplicity v.asIdeal (Ideal.span {a}) := by
120-
rwa [← intValuation_le_pow_iff_mem, ← intValuation_eq_coe_neg_multiplicity _ hnz]
120+
rwa [← intValuation_le_pow_iff_mem, WithZero.exp, ← intValuation_eq_coe_neg_multiplicity _ hnz]
121121
-- Now make use of
122122
-- `v.asIdeal ^ multiplicity v.asIdeal (Ideal.span {a}) = v.asIdeal ^ n ⊔ Ideal.span {a}`
123123
-- (this is where we need `IsDedekindDomain A`)
@@ -127,7 +127,7 @@ lemma exists_adicValued_mul_sub_le {a b : A} {γ : WithZero (Multiplicative ℤ)
127127
obtain ⟨y, hy⟩ := Ideal.mem_span_singleton'.mp hz
128128
use y
129129
-- And again prove the result about valuations by turning into one about ideals.
130-
rwa [hy, ← hxz, sub_add_cancel_right, intValuation_le_pow_iff_mem, neg_mem_iff]
130+
rwa [hy, ← hxz, sub_add_cancel_right, ← WithZero.exp, intValuation_le_pow_iff_mem, neg_mem_iff]
131131

132132
lemma exists_adicValued_sub_lt_of_adicValued_le_one {x : (WithVal (v.valuation K))}
133133
(γ : (WithZero (Multiplicative ℤ))ˣ) (hx : Valued.v x ≤ 1) :
@@ -432,7 +432,7 @@ theorem exists_uniformizer (v : HeightOneSpectrum A) :
432432
∃ π : v.adicCompletionIntegers K, Valued.v π.1 = Multiplicative.ofAdd (- 1 : ℤ) := by
433433
obtain ⟨π, hπ⟩ := v.intValuation_exists_uniformizer
434434
use π
435-
rw [← hπ, ← ValuationSubring.algebraMap_apply, ← IsScalarTower.algebraMap_apply,
435+
rw [← WithZero.exp, ← hπ, ← ValuationSubring.algebraMap_apply, ← IsScalarTower.algebraMap_apply,
436436
v.valuedAdicCompletion_eq_valuation, v.valuation_of_algebraMap]
437437

438438
variable {K} in

FLT/DedekindDomain/IntegralClosure.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -109,7 +109,7 @@ lemma intValuation_comap (hAB : Function.Injective (algebraMap A B))
109109
simp only [intValuation, Valuation.coe_mk, MonoidWithZeroHom.coe_mk, ZeroHom.coe_mk]
110110
change (ite _ _ _) ^ _ = ite _ _ _
111111
rw [map_eq_zero_iff _ hAB, if_neg hx, if_neg hx, ← Set.image_singleton, ← Ideal.map_span,
112-
mk_count_factors_map _ _ hAB, mul_comm]
112+
mk_count_factors_map _ _ hAB, mul_comm, WithZero.exp, WithZero.exp]
113113
simp
114114

115115
omit [IsIntegralClosure B A L] in

FLT/Deformations/Lemmas.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -81,7 +81,7 @@ instance IsTopologicalGroup.discreteUniformity
8181
{G : Type*} [Group G] [TopologicalSpace G] [IsTopologicalGroup G] [DiscreteTopology G] :
8282
letI := IsTopologicalGroup.toUniformSpace G
8383
DiscreteUniformity G := by
84-
simp only [discreteUniformity_iff_idRel_mem_uniformity]
84+
simp only [discreteUniformity_iff_relId_mem_uniformity]
8585
exact ⟨{1}, by simp [Set.subset_def, div_eq_one]⟩
8686

8787
lemma IsLocalRing.map_maximalIdeal {R S} [CommRing R] [CommRing S]

FLT/Mathlib/Algebra/Algebra/Hom.lean

Lines changed: 0 additions & 5 deletions
Original file line numberDiff line numberDiff line change
@@ -81,8 +81,3 @@ theorem SemialgHom.algebraMap_apply {A B : Type*} [CommSemiring A] [CommSemiring
8181
algebraMap A B a = f a := rfl
8282

8383
end semialghom
84-
85-
@[simp]
86-
theorem AlgHom.coe_toLinearMap {R A B : Type*} [CommSemiring R] [Semiring A] [Semiring B]
87-
[Algebra R A] [Algebra R B] (f : A →ₐ[R] B) :
88-
⇑(f : A →ₗ[R] B) = ⇑f := rfl

FLT/Mathlib/Topology/Algebra/Valued/WithZeroMulInt.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -114,11 +114,11 @@ theorem finite_cover_of_uniformity_basis [IsDiscreteValuationRing 𝒪[K]] {γ :
114114
let ⟨m, hm⟩ := exists_pow_lt_of_le_neg_one (irreducible_valuation_le_ofAdd_neg_one hϖ) γ
115115
letI := finite_quotient_maximalIdeal_pow_of_finite_residueField h m
116116
have h := Fintype.ofFinite (𝒪[K] ⧸ 𝓂[K] ^ m)
117-
let T := Subtype.val '' (h.elems.image Quotient.out).toSet
117+
let T := Subtype.val '' (h.elems.image Quotient.out : Set 𝒪[K])
118118
refine ⟨T, (Set.Finite.image _ (Finset.finite_toSet _)), fun x hx => ?_⟩
119119
simp only [Set.mem_iUnion]
120120
let y := (Ideal.Quotient.mk (𝓂[K] ^ m) ⟨x, hx⟩).out
121-
refine ⟨y, Set.mem_image_of_mem _ <| Finset.mem_image_of_mem _ (h.complete _),
121+
refine ⟨y, Set.mem_image_of_mem _ <| Finset.mem_image_of_mem Quotient.out (h.complete _),
122122
lt_of_le_of_lt (mem_maximalIdeal_pow_valuation (Ideal.Quotient.out_sub _ _) hϖ) hm⟩
123123

124124
variable (K)

FLT/NumberField/AdeleRing.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -480,7 +480,7 @@ theorem Rat.AdeleRing.cocompact :
480480
simpa using HeightOneSpectrum.coe_algebraMap_mem (𝓞 ℚ) ℚ v xi
481481
refine ⟨b, hb, ?_⟩
482482
unfold b; unfold a
483-
simp [c]
483+
simp [-algebraMap.coe_inj, c]
484484
{ isCompact_univ := h_W_image ▸ IsCompact.image h_W_compact continuous_quot_mk }
485485

486486
variable (K L : Type*) [Field K] [Field L] [NumberField K] [NumberField L] [Algebra K L]

lake-manifest.json

Lines changed: 9 additions & 9 deletions
Original file line numberDiff line numberDiff line change
@@ -15,17 +15,17 @@
1515
"type": "git",
1616
"subDir": null,
1717
"scope": "",
18-
"rev": "da2fd30c91aa177fc00c364d00e2c55334a5b32b",
18+
"rev": "9003b8fbd74a577536c5e79a21854807a31a793d",
1919
"name": "mathlib",
2020
"manifestFile": "lake-manifest.json",
21-
"inputRev": "v4.25.0-rc1",
21+
"inputRev": "master",
2222
"inherited": false,
2323
"configFile": "lakefile.lean"},
2424
{"url": "https://github.com/leanprover-community/plausible",
2525
"type": "git",
2626
"subDir": null,
2727
"scope": "leanprover-community",
28-
"rev": "7607162f5a1c1eb23c23027629a418b3a160670e",
28+
"rev": "8864a73bf79aad549e34eff972c606343935106d",
2929
"name": "plausible",
3030
"manifestFile": "lake-manifest.json",
3131
"inputRev": "main",
@@ -45,7 +45,7 @@
4545
"type": "git",
4646
"subDir": null,
4747
"scope": "leanprover-community",
48-
"rev": "e5c37730d22634ee0169c164f25dac49918ed951",
48+
"rev": "451499ea6e97cee4c8979b507a9af5581a849161",
4949
"name": "importGraph",
5050
"manifestFile": "lake-manifest.json",
5151
"inputRev": "main",
@@ -65,7 +65,7 @@
6565
"type": "git",
6666
"subDir": null,
6767
"scope": "leanprover-community",
68-
"rev": "cbe864cd5177966c9e005418cfdc1fb36db62e13",
68+
"rev": "1fa48c6a63b4c4cda28be61e1037192776e77ac0",
6969
"name": "aesop",
7070
"manifestFile": "lake-manifest.json",
7171
"inputRev": "master",
@@ -75,7 +75,7 @@
7575
"type": "git",
7676
"subDir": null,
7777
"scope": "leanprover-community",
78-
"rev": "593aa51c4aa07ee81e9233b53e1f61a5b4d9f761",
78+
"rev": "95c2f8afe09d9e49d3cacca667261da04f7f93f7",
7979
"name": "Qq",
8080
"manifestFile": "lake-manifest.json",
8181
"inputRev": "master",
@@ -85,7 +85,7 @@
8585
"type": "git",
8686
"subDir": null,
8787
"scope": "leanprover-community",
88-
"rev": "5bd478197f2e5d2a4fde527cf3581d83f49baa9b",
88+
"rev": "c029ceb9956ef9d567fc034e5403ec829f8d0d87",
8989
"name": "batteries",
9090
"manifestFile": "lake-manifest.json",
9191
"inputRev": "main",
@@ -95,10 +95,10 @@
9595
"type": "git",
9696
"subDir": null,
9797
"scope": "leanprover",
98-
"rev": "f75f4926aff7ba19949e16c19094d7298806b1a6",
98+
"rev": "72ae7004d9f0ddb422aec5378204fdd7828c5672",
9999
"name": "Cli",
100100
"manifestFile": "lake-manifest.json",
101-
"inputRev": "v4.25.0-rc1",
101+
"inputRev": "v4.25.0-rc2",
102102
"inherited": true,
103103
"configFile": "lakefile.toml"}],
104104
"name": "FLT",

lakefile.toml

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -15,7 +15,7 @@ warn.sorry = false
1515
[[require]]
1616
name = "mathlib"
1717
git = "https://github.com/leanprover-community/mathlib4.git"
18-
rev = "v4.25.0-rc1"
18+
rev = "master"
1919

2020
[[require]]
2121
name = "checkdecls"

lean-toolchain

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -1 +1 @@
1-
leanprover/lean4:v4.25.0-rc1
1+
leanprover/lean4:v4.25.0-rc2

0 commit comments

Comments
 (0)