Skip to content

Commit c314029

Browse files
committed
Bump mathlib to v4.23.0
1 parent 99a77d1 commit c314029

File tree

6 files changed

+23
-25
lines changed

6 files changed

+23
-25
lines changed

LeanCamCombi/Mathlib/Probability/ProbabilityMassFunction/Constructions.lean

Lines changed: 1 addition & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -38,9 +38,7 @@ lemma mem_support_bernoulli'_iff : b ∈ (bernoulli' p hp).support ↔ if b then
3838
ext q
3939
by_cases p <;> by_cases q <;> simp [*]
4040
refine (map_ofFintype _ _ _).trans ?_
41-
simp only [this, bernoulli', Finset.mem_filter, Finset.mem_univ, true_and,
42-
Finset.mem_disjiUnion, tsub_le_self, eq_iff_iff, Finset.sum_singleton, WithTop.coe_sub,
43-
ENNReal.coe_one]
41+
simp only [eq_iff_iff, this, Finset.sum_singleton, bernoulli']
4442
congr 1 with q
4543
split_ifs <;> simp [ENNReal.sub_sub_cancel WithTop.one_ne_top (ENNReal.coe_le_coe.2 hp)]
4644

LeanCamCombi/PlainCombi/KatonaCircle.lean

Lines changed: 2 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -82,12 +82,11 @@ def prefixedEquiv (s : Finset α) : prefixed s ≃ Numbering s × Numbering ↑(
8282
by_cases hx : x ∈ s
8383
· have : g ⟨x, hx⟩ < #s := by simpa using (g ⟨x, hx⟩).2
8484
simp [hx, this]
85-
· simp [hx, Equiv.symm_apply_eq]
85+
· simp [hx]
8686
val.right_inv n := by
8787
obtain hns | hsn := lt_or_ge n.1 #s
8888
· simp [hns]
89-
· simp [hsn.not_gt, hsn, dif_neg (mem_compl.1 <| Subtype.prop _), Fin.ext_iff,
90-
Fintype.card_subtype_le]
89+
· simp [hsn.not_gt, hsn, dif_neg (mem_compl.1 <| Subtype.prop _)]
9190
property := mem_prefixed.2 fun x ↦ by
9291
constructor
9392
· intro hx

LeanCamCombi/PlainCombi/LittlewoodOfford.lean

Lines changed: 3 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -22,8 +22,9 @@ lemma exists_littlewood_offord_partition [DecidableEq ι] (hr : 0 < r) (hf : ∀
2222
#P.parts = (#s).choose (#s / 2) ∧ (∀ 𝒜 ∈ P.parts, ∀ t ∈ 𝒜, t ⊆ s) ∧ ∀ 𝒜 ∈ P.parts,
2323
(𝒜 : Set (Finset ι)).Pairwise fun u v ↦ r ≤ dist (∑ i ∈ u, f i) (∑ i ∈ v, f i) := by
2424
classical
25-
induction' s using Finset.induction with i s hi ih
26-
· exact ⟨Finpartition.indiscrete <| singleton_ne_empty _, by simp⟩
25+
induction s using Finset.induction with
26+
| empty => exact ⟨Finpartition.indiscrete <| singleton_ne_empty _, by simp⟩
27+
| insert i s hi ih =>
2728
obtain ⟨P, hP, hs, hPr⟩ := ih fun j hj ↦ hf _ <| mem_insert_of_mem hj
2829
clear ih
2930
obtain ⟨g, hg, hgf⟩ :=

lake-manifest.json

Lines changed: 15 additions & 15 deletions
Original file line numberDiff line numberDiff line change
@@ -5,20 +5,20 @@
55
"type": "git",
66
"subDir": null,
77
"scope": "",
8-
"rev": "79e94a093aff4a60fb1b1f92d9681e407124c2ca",
8+
"rev": "37df177aaa770670452312393d4e84aaad56e7b6",
99
"name": "mathlib",
1010
"manifestFile": "lake-manifest.json",
11-
"inputRev": "v4.22.0",
11+
"inputRev": "v4.23.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": "b100ad4c5d74a464f497aaa8e7c74d86bf39a56f",
18+
"rev": "a22e7c1fa7707fb7ea75f2f9fd6b14de2b7b87a9",
1919
"name": "plausible",
2020
"manifestFile": "lake-manifest.json",
21-
"inputRev": "v4.22.0",
21+
"inputRev": "main",
2222
"inherited": true,
2323
"configFile": "lakefile.toml"},
2424
{"url": "https://github.com/leanprover-community/LeanSearchClient",
@@ -35,57 +35,57 @@
3535
"type": "git",
3636
"subDir": null,
3737
"scope": "leanprover-community",
38-
"rev": "eb164a46de87078f27640ee71e6c3841defc2484",
38+
"rev": "7fca1d4a190761bac0028848f73dc9a59fcb4957",
3939
"name": "importGraph",
4040
"manifestFile": "lake-manifest.json",
41-
"inputRev": "v4.22.0",
41+
"inputRev": "main",
4242
"inherited": true,
4343
"configFile": "lakefile.toml"},
4444
{"url": "https://github.com/leanprover-community/ProofWidgets4",
4545
"type": "git",
4646
"subDir": null,
4747
"scope": "leanprover-community",
48-
"rev": "1253a071e6939b0faf5c09d2b30b0bfc79dae407",
48+
"rev": "6e47cc88cfbf1601ab364e9a4de5f33f13401ff8",
4949
"name": "proofwidgets",
5050
"manifestFile": "lake-manifest.json",
51-
"inputRev": "v0.0.68",
51+
"inputRev": "v0.0.71",
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": "1256a18522728c2eeed6109b02dd2b8f207a2a3c",
58+
"rev": "247ff80701c76760523b5d7c180b27b7708faf38",
5959
"name": "aesop",
6060
"manifestFile": "lake-manifest.json",
61-
"inputRev": "v4.22.0",
61+
"inputRev": "master",
6262
"inherited": true,
6363
"configFile": "lakefile.toml"},
6464
{"url": "https://github.com/leanprover-community/quote4",
6565
"type": "git",
6666
"subDir": null,
6767
"scope": "leanprover-community",
68-
"rev": "917bfa5064b812b7fbd7112d018ea0b4def25ab3",
68+
"rev": "9b703a545097978aef0e7e243ab8b71c32a9ff65",
6969
"name": "Qq",
7070
"manifestFile": "lake-manifest.json",
71-
"inputRev": "v4.22.0",
71+
"inputRev": "master",
7272
"inherited": true,
7373
"configFile": "lakefile.toml"},
7474
{"url": "https://github.com/leanprover-community/batteries",
7575
"type": "git",
7676
"subDir": null,
7777
"scope": "leanprover-community",
78-
"rev": "240676e9568c254a69be94801889d4b13f3b249f",
78+
"rev": "d117e2c28cba42e974bc22568ac999492a34e812",
7979
"name": "batteries",
8080
"manifestFile": "lake-manifest.json",
81-
"inputRev": "v4.22.0",
81+
"inputRev": "main",
8282
"inherited": true,
8383
"configFile": "lakefile.toml"},
8484
{"url": "https://github.com/leanprover/lean4-cli",
8585
"type": "git",
8686
"subDir": null,
8787
"scope": "leanprover",
88-
"rev": "c682c91d2d4dd59a7187e2ab977ac25bd1f87329",
88+
"rev": "41c5d0b8814dec559e2e1441171db434fe2281cc",
8989
"name": "Cli",
9090
"manifestFile": "lake-manifest.json",
9191
"inputRev": "main",

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.22.0"
42+
rev = "v4.23.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.22.0
1+
leanprover/lean4:v4.23.0

0 commit comments

Comments
 (0)