Skip to content

Commit 34a573b

Browse files
committed
Bump mathlib
1 parent da021ed commit 34a573b

File tree

7 files changed

+19
-21
lines changed

7 files changed

+19
-21
lines changed

LeanCamCombi/GrowthInGroups/Lecture4.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -1,4 +1,4 @@
1-
import Mathlib.Analysis.Matrix
1+
import Mathlib.Analysis.Matrix.Normed
22
import Mathlib.GroupTheory.Nilpotent
33
import Mathlib.LinearAlgebra.Matrix.GeneralLinearGroup.Defs
44
import LeanCamCombi.Mathlib.Combinatorics.Additive.ApproximateSubgroup
@@ -21,7 +21,7 @@ lemma fact_4_1 (S T : GL n ℂ) :
2121
open scoped Classical in
2222
lemma lemma_4_2 (hC₀ : Fintype.card n < C₀) (K : ℝ) :
2323
∃ δ : ℝ,
24-
(A : Finset (GL n ℂ)) (hA : IsApproximateSubgroup K A.toSet) (hC₀ : ∀ a ∈ A, ‖a.val‖ ≤ C₀),
24+
∀ A : Finset (GL n ℂ), IsApproximateSubgroup K (A : Set (GL n ℂ)) → (∀ a ∈ A, ‖a.val‖ ≤ C₀)
2525
∃ γ ∈ A ^ 2, δ * #A ≤ #{x ∈ A ^ 4 | Commute γ x} := sorry
2626

2727
lemma corollary_4_3 (K C₀ : ℝ) :

LeanCamCombi/Mathlib/Combinatorics/Additive/ApproximateSubgroup.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -39,7 +39,7 @@ lemma exists_isApproximateSubgroup_of_small_doubling [DecidableEq G] {A : Finset
3939
have hS₁ : 1 ∈ S := by simp [S, hA₀.ne_empty]; bound
4040
have hS₀ : S.Nonempty := ⟨1, hS₁⟩
4141
have hSA : S ⊆ A⁻¹ * A := filter_subset ..
42-
have hSsymm : S⁻¹ = S := by ext; simp [S]; simp [← mem_inv']; sorry
42+
have hSsymm : S⁻¹ = S := by ext; simp [S]; sorry
4343
have hScard := calc
4444
(#S : ℝ) ≤ #(A⁻¹ * A) := by gcongr
4545
_ ≤ K ^ 2 * #A := sorry

LeanCamCombi/PlainCombi/LittlewoodOfford.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -3,7 +3,7 @@ Copyright (c) 2022 Yaël Dillies. All rights reserved.
33
Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Yaël Dillies
55
-/
6-
import Mathlib.Analysis.NormedSpace.HahnBanach.Extension
6+
import Mathlib.Analysis.Normed.Module.HahnBanach
77
import Mathlib.Combinatorics.Enumerative.DoubleCounting
88
import Mathlib.Order.Partition.Finpartition
99

LeanCamCombi/PlainCombi/ProbLYM.lean

Lines changed: 1 addition & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -11,8 +11,6 @@ import LeanCamCombi.PlainCombi.KatonaCircle
1111
1212
This file proves the LYM inequality using (very elementary) probability theory.
1313
14-
15-
1614
## References
1715
1816
This proof formalizes Section 1.2 of Prof. Yufei Zhao's lecture notes for MIT 18.226:
@@ -35,7 +33,7 @@ open Finset Fintype Numbering
3533
variable {α : Type*} [Fintype α] {𝒜 : Finset (Finset α)}
3634

3735
/-- The **Lubell-Yamamoto-Meshalkin inequality**, proved using the Katona circle method. -/
38-
theorem LYM_inequality (h𝒜 : IsAntichain (· ⊆ ·) 𝒜.toSet) :
36+
theorem LYM_inequality (h𝒜 : IsAntichain (· ⊆ ·) (𝒜 : Set (Finset α))) :
3937
∑ s ∈ 𝒜, ((card α).choose #s : ℚ≥0)⁻¹ ≤ 1 := by
4038
classical
4139
calc

lake-manifest.json

Lines changed: 12 additions & 12 deletions
Original file line numberDiff line numberDiff line change
@@ -5,17 +5,17 @@
55
"type": "git",
66
"subDir": null,
77
"scope": "",
8-
"rev": "f897ebcf72cd16f89ab4577d0c826cd14afaafc7",
8+
"rev": "029db123ddaa7f8fd0d18cea3b1b33bf84dacd1e",
99
"name": "mathlib",
1010
"manifestFile": "lake-manifest.json",
11-
"inputRev": "v4.24.0",
11+
"inputRev": "v4.25.0",
1212
"inherited": false,
1313
"configFile": "lakefile.lean"},
1414
{"url": "https://github.com/leanprover-community/plausible",
1515
"type": "git",
1616
"subDir": null,
1717
"scope": "leanprover-community",
18-
"rev": "dfd06ebfe8d0e8fa7faba9cb5e5a2e74e7bd2805",
18+
"rev": "2503bfb5e2d4d8202165f5bd2cc39e44a3be31c3",
1919
"name": "plausible",
2020
"manifestFile": "lake-manifest.json",
2121
"inputRev": "main",
@@ -25,7 +25,7 @@
2525
"type": "git",
2626
"subDir": null,
2727
"scope": "leanprover-community",
28-
"rev": "99657ad92e23804e279f77ea6dbdeebaa1317b98",
28+
"rev": "2ed4ba69b6127de8f5c2af83cccacd3c988b06bf",
2929
"name": "LeanSearchClient",
3030
"manifestFile": "lake-manifest.json",
3131
"inputRev": "main",
@@ -35,7 +35,7 @@
3535
"type": "git",
3636
"subDir": null,
3737
"scope": "leanprover-community",
38-
"rev": "d768126816be17600904726ca7976b185786e6b9",
38+
"rev": "009064c21bad4d7f421f2901c5e817c8bf3468cb",
3939
"name": "importGraph",
4040
"manifestFile": "lake-manifest.json",
4141
"inputRev": "main",
@@ -45,17 +45,17 @@
4545
"type": "git",
4646
"subDir": null,
4747
"scope": "leanprover-community",
48-
"rev": "556caed0eadb7901e068131d1be208dd907d07a2",
48+
"rev": "fb8ed0a85a96e3176f6e94b20d413ea72d92576d",
4949
"name": "proofwidgets",
5050
"manifestFile": "lake-manifest.json",
51-
"inputRev": "v0.0.74",
51+
"inputRev": "v0.0.77",
5252
"inherited": true,
5353
"configFile": "lakefile.lean"},
5454
{"url": "https://github.com/leanprover-community/aesop",
5555
"type": "git",
5656
"subDir": null,
5757
"scope": "leanprover-community",
58-
"rev": "725ac8cd67acd70a7beaf47c3725e23484c1ef50",
58+
"rev": "26e4c7c0e63eb3e6cce3cf7faba27b8526ea8349",
5959
"name": "aesop",
6060
"manifestFile": "lake-manifest.json",
6161
"inputRev": "master",
@@ -65,7 +65,7 @@
6565
"type": "git",
6666
"subDir": null,
6767
"scope": "leanprover-community",
68-
"rev": "dea6a3361fa36d5a13f87333dc506ada582e025c",
68+
"rev": "2781d8ad404303b2fe03710ac7db946ddfe3539f",
6969
"name": "Qq",
7070
"manifestFile": "lake-manifest.json",
7171
"inputRev": "master",
@@ -75,7 +75,7 @@
7575
"type": "git",
7676
"subDir": null,
7777
"scope": "leanprover-community",
78-
"rev": "8da40b72fece29b7d3fe3d768bac4c8910ce9bee",
78+
"rev": "39260e31b7b3f7f05643da95242463b462dc05f1",
7979
"name": "batteries",
8080
"manifestFile": "lake-manifest.json",
8181
"inputRev": "main",
@@ -85,10 +85,10 @@
8585
"type": "git",
8686
"subDir": null,
8787
"scope": "leanprover",
88-
"rev": "91c18fa62838ad0ab7384c03c9684d99d306e1da",
88+
"rev": "1dae8b12f8ba27576ffe5ddee78bebf6458157b0",
8989
"name": "Cli",
9090
"manifestFile": "lake-manifest.json",
91-
"inputRev": "main",
91+
"inputRev": "v4.25.0",
9292
"inherited": true,
9393
"configFile": "lakefile.toml"}],
9494
"name": "LeanCamCombi",

lakefile.toml

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -39,7 +39,7 @@ linter.style.setOption = true
3939
[[require]]
4040
name = "mathlib"
4141
git = "https://github.com/leanprover-community/mathlib4.git"
42-
rev = "v4.24.0"
42+
rev = "v4.25.0"
4343

4444
[[lean_lib]]
4545
name = "LeanCamCombi"

lean-toolchain

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

0 commit comments

Comments
 (0)