Skip to content

Commit dd72118

Browse files
authored
Merge pull request #134 from Ruben-VandeVelde/bump
Bump mathlib
2 parents f36b001 + 5f0dcee commit dd72118

File tree

5 files changed

+10
-34
lines changed

5 files changed

+10
-34
lines changed

FLT/ForMathlib/MiscLemmas.lean

-24
Original file line numberDiff line numberDiff line change
@@ -60,30 +60,6 @@ theorem coinduced_prod_eq_prod_coinduced {X Y S T : Type*} [AddCommGroup X] [Add
6060

6161
end elsewhere
6262

63-
section missing_API
64-
65-
variable {R : Type*} [Semiring R] {P : Type*} [AddCommMonoid P] [Module R P]
66-
67-
namespace Module
68-
69-
-- the below is all done for rings but it should be semirings
70-
/-- Free modules are projective. -/
71-
theorem Projective.of_basis' {ι : Type*} (b : Basis ι R P) : Projective R P := by
72-
-- need P →ₗ (P →₀ R) for definition of projective.
73-
-- get it from `ι → (P →₀ R)` coming from `b`.
74-
use b.constr ℕ fun i => Finsupp.single (b i) (1 : R)
75-
intro m
76-
simp only [b.constr_apply, mul_one, id, Finsupp.smul_single', Finsupp.linearCombination_single,
77-
map_finsupp_sum]
78-
exact b.linearCombination_repr m
79-
80-
instance (priority := 100) Projective.of_free' [Module.Free R P] : Module.Projective R P :=
81-
.of_basis' <| Module.Free.chooseBasis R P
82-
83-
end Module
84-
85-
end missing_API
86-
8763
theorem TopologicalSpace.prod_mono {α β : Type*} {σ₁ σ₂ : TopologicalSpace α}
8864
{τ₁ τ₂ : TopologicalSpace β} (hσ : σ₁ ≤ σ₂) (hτ : τ₁ ≤ τ₂) :
8965
@instTopologicalSpaceProd α β σ₁ τ₁ ≤ @instTopologicalSpaceProd α β σ₂ τ₂ :=

FLT/MathlibExperiments/Frobenius.lean

+1-1
Original file line numberDiff line numberDiff line change
@@ -488,7 +488,7 @@ theorem gal_smul_F_eq (σ : L ≃ₐ[K] L) :
488488
∏ τ : L ≃ₐ[K] L,
489489
(X - C (galRestrict A K L B σ
490490
(galRestrict A K L B τ α))):= by
491-
simp [Finset.smul_prod, smul_sub, smul_X, smul_C, AlgEquiv.smul_def]
491+
simp [Finset.smul_prod', smul_sub, smul_X, smul_C, AlgEquiv.smul_def]
492492

493493
/-- use `Finset.prod_bij` to show
494494
`(galRestrict A K L B σ • (∏ τ : L ≃ₐ[K] L, (X - C (galRestrict A K L B τ α))) =

FLT/MathlibExperiments/Frobenius2.lean

+1-1
Original file line numberDiff line numberDiff line change
@@ -167,7 +167,7 @@ variable {A Q} in
167167
open Finset in
168168
lemma F.smul_eq_self (σ : B ≃ₐ[A] B) : σ • (F A Q) = F A Q := calc
169169
σ • F A Q = σ • ∏ τ : B ≃ₐ[A] B, (X - C (τ • (y A Q))) := by rw [F_spec]
170-
_ = ∏ τ : B ≃ₐ[A] B, σ • (X - C (τ • (y A Q))) := smul_prod
170+
_ = ∏ τ : B ≃ₐ[A] B, σ • (X - C (τ • (y A Q))) := smul_prod'
171171
_ = ∏ τ : B ≃ₐ[A] B, (X - C ((σ * τ) • (y A Q))) := by simp [smul_sub]
172172
_ = ∏ τ' : B ≃ₐ[A] B, (X - C (τ' • (y A Q))) := Fintype.prod_bijective (fun τ ↦ σ * τ)
173173
(Group.mulLeft_bijective σ) _ _ (fun _ ↦ rfl)

FLT/MathlibExperiments/FrobeniusRiou.lean

+2-2
Original file line numberDiff line numberDiff line change
@@ -66,7 +66,7 @@ variable (P Q : Ideal B) [P.IsPrime] [Q.IsPrime]
6666
open scoped Pointwise
6767

6868
private theorem norm_fixed (b : B) (g : G) : g • (∏ᶠ σ : G, σ • b) = ∏ᶠ σ : G, σ • b := calc
69-
g • (∏ᶠ σ : G, σ • b) = ∏ᶠ σ : G, g • (σ • b) := smul_finprod _
69+
g • (∏ᶠ σ : G, σ • b) = ∏ᶠ σ : G, g • (σ • b) := smul_finprod' _
7070
_ = ∏ᶠ σ : G, σ • b := finprod_eq_of_bijective (g • ·) (MulAction.bijective g)
7171
fun x ↦ smul_smul g x b
7272

@@ -243,7 +243,7 @@ private theorem F_spec (b : B) : F G b = ∏ᶠ τ : G, (X - C (τ • b)) := rf
243243

244244
private theorem F_smul_eq_self (σ : G) (b : B) : σ • (F G b) = F G b := calc
245245
σ • F G b = σ • ∏ᶠ τ : G, (X - C (τ • b)) := by rw [F_spec]
246-
_ = ∏ᶠ τ : G, σ • (X - C (τ • b)) := smul_finprod _
246+
_ = ∏ᶠ τ : G, σ • (X - C (τ • b)) := smul_finprod' _
247247
_ = ∏ᶠ τ : G, (X - C ((σ * τ) • b)) := by simp [smul_sub, smul_smul]
248248
_ = ∏ᶠ τ' : G, (X - C (τ' • b)) := finprod_eq_of_bijective (fun τ ↦ σ * τ)
249249
(Group.mulLeft_bijective σ) (fun _ ↦ rfl)

lake-manifest.json

+6-6
Original file line numberDiff line numberDiff line change
@@ -5,7 +5,7 @@
55
"type": "git",
66
"subDir": null,
77
"scope": "leanprover-community",
8-
"rev": "46fed98b5cac2b1ea64e363b420c382ed1af0d85",
8+
"rev": "2ce0037d487217469a1efeb9ea8196fe15ab9c46",
99
"name": "batteries",
1010
"manifestFile": "lake-manifest.json",
1111
"inputRev": "main",
@@ -25,7 +25,7 @@
2525
"type": "git",
2626
"subDir": null,
2727
"scope": "leanprover-community",
28-
"rev": "662f986ad3c5ad6ab1a1726b3c04f5ec425aa9f7",
28+
"rev": "2c39748d927749624f480b641f1d2d77b8632b92",
2929
"name": "aesop",
3030
"manifestFile": "lake-manifest.json",
3131
"inputRev": "master",
@@ -61,11 +61,11 @@
6161
"inputRev": "main",
6262
"inherited": true,
6363
"configFile": "lakefile.toml"},
64-
{"url": "https://github.com/siddhartha-gadgil/LeanSearchClient.git",
64+
{"url": "https://github.com/leanprover-community/LeanSearchClient",
6565
"type": "git",
6666
"subDir": null,
67-
"scope": "",
68-
"rev": "c260ed920e2ebd23ef9fc8ca3fd24115e04c18b1",
67+
"scope": "leanprover-community",
68+
"rev": "3e9460c40e09457b2fd079ef55316535536425fc",
6969
"name": "LeanSearchClient",
7070
"manifestFile": "lake-manifest.json",
7171
"inputRev": "main",
@@ -75,7 +75,7 @@
7575
"type": "git",
7676
"subDir": null,
7777
"scope": "",
78-
"rev": "7eb3f52a4fc12036cb1c4a953dd0f497b57a2434",
78+
"rev": "95af9be74f8b9d98505d9900fe8f563a89e5e667",
7979
"name": "mathlib",
8080
"manifestFile": "lake-manifest.json",
8181
"inputRev": null,

0 commit comments

Comments
 (0)