Skip to content

Commit 7c47eb5

Browse files
committed
Bump mathlib
1 parent 4e5cfa9 commit 7c47eb5

File tree

8 files changed

+18
-68
lines changed

8 files changed

+18
-68
lines changed

LeanCamCombi.lean

Lines changed: 0 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -15,8 +15,6 @@ import LeanCamCombi.Mathlib.Combinatorics.Additive.ApproximateSubgroup
1515
import LeanCamCombi.Mathlib.Combinatorics.SetFamily.LYM
1616
import LeanCamCombi.Mathlib.Combinatorics.SimpleGraph.Density
1717
import LeanCamCombi.Mathlib.Combinatorics.SimpleGraph.Subgraph
18-
import LeanCamCombi.Mathlib.Data.Fintype.Card
19-
import LeanCamCombi.Mathlib.Data.Nat.Choose.Cast
2018
import LeanCamCombi.Mathlib.Probability.ProbabilityMassFunction.Constructions
2119
import LeanCamCombi.PlainCombi.KatonaCircle
2220
import LeanCamCombi.PlainCombi.LittlewoodOfford

LeanCamCombi/ExtrProbCombi/BernoulliSeq.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -33,7 +33,7 @@ variable {α Ω : Type*} [MeasurableSpace Ω]
3333
structure IsBernoulliSeq (X : Ω → Set α) (p : outParam ℝ≥0) (μ : Measure Ω := by volume_tac) : Prop
3434
where
3535
protected le_one : p ≤ 1
36-
protected iIndepFun : iIndepFun inferInstance (fun a ω ↦ a ∈ X ω) μ
36+
protected iIndepFun : iIndepFun (fun a ω ↦ a ∈ X ω) μ
3737
protected map : ∀ a, Measure.map (fun ω ↦ a ∈ X ω) μ = (PMF.bernoulli' p le_one).toMeasure
3838

3939
variable {X Y : Ω → Set α} {μ : Measure Ω} {p q : ℝ≥0} (hX : IsBernoulliSeq X p μ)

LeanCamCombi/ExtrProbCombi/BinomialRandomGraph.lean

Lines changed: 2 additions & 4 deletions
Original file line numberDiff line numberDiff line change
@@ -41,11 +41,9 @@ include hG
4141
protected nonrec lemma le_one : p ≤ 1 := hG.le_one
4242

4343
lemma iIndepFun_mem_edgeSet_not_isDiag :
44-
iIndepFun inferInstance (fun (e : {e : Sym2 α // ¬ e.IsDiag}) ω ↦ ↑e ∈ (G ω).edgeSet) μ :=
45-
hG.iIndepFun
44+
iIndepFun (fun (e : {e : Sym2 α // ¬ e.IsDiag}) ω ↦ ↑e ∈ (G ω).edgeSet) μ := hG.iIndepFun
4645

47-
lemma iIndepFun_mem_edgeSet : iIndepFun inferInstance (fun e ω ↦ e ∈ (G ω).edgeSet) μ :=
48-
sorry
46+
lemma iIndepFun_mem_edgeSet : iIndepFun (fun e ω ↦ e ∈ (G ω).edgeSet) μ := sorry
4947

5048
lemma map_mem_edgeSet (he : ¬ e.IsDiag) :
5149
Measure.map (fun ω ↦ e ∈ (G ω).edgeSet) μ = (PMF.bernoulli' p hG.le_one).toMeasure :=

LeanCamCombi/Mathlib/Data/Fintype/Card.lean

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

LeanCamCombi/Mathlib/Data/Nat/Choose/Cast.lean

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

LeanCamCombi/PlainCombi/KatonaCircle.lean

Lines changed: 4 additions & 5 deletions
Original file line numberDiff line numberDiff line change
@@ -3,11 +3,10 @@ Copyright (c) 2024 Ching-Tsun Chou, Chris Wong. All rights reserved.
33
Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Ching-Tsun Chou, Chris Wong
55
-/
6-
import LeanCamCombi.Mathlib.Data.Fintype.Card
7-
import LeanCamCombi.Mathlib.Data.Nat.Choose.Cast
86
import Mathlib.Data.Finset.Density
97
import Mathlib.Data.Fintype.Prod
108
import Mathlib.Data.Fintype.Perm
9+
import Mathlib.Data.Nat.Choose.Cast
1110

1211
/-!
1312
# The Katona circle method
@@ -71,7 +70,7 @@ def prefixedEquiv (s : Finset α) : prefixed s ≃ Numbering s × Numbering ↑(
7170
invFun := fun (g, g') ↦
7271
{ val.toFun x :=
7372
if hx : x ∈ s then
74-
g ⟨x, hx⟩ |>.castLE Fintype.card_subtype_le'
73+
g ⟨x, hx⟩ |>.castLE (Fintype.card_subtype_le _)
7574
else
7675
g' ⟨x, by simpa⟩ |>.addNat #s |>.cast (by simp [card_le_univ])
7776
val.invFun n :=
@@ -88,7 +87,7 @@ def prefixedEquiv (s : Finset α) : prefixed s ≃ Numbering s × Numbering ↑(
8887
obtain hns | hsn := lt_or_le n.1 #s
8988
· simp [hns]
9089
· simp [hsn.not_lt, hsn, dif_neg (mem_compl.1 <| Subtype.prop _), Fin.ext_iff,
91-
Fintype.card_subtype_le']
90+
Fintype.card_subtype_le]
9291
property := mem_prefixed.2 fun x ↦ by
9392
constructor
9493
· intro hx
@@ -107,7 +106,7 @@ lemma card_prefixed (s : Finset α) : #(prefixed s) = (#s)! * (card α - #s)! :=
107106

108107
@[simp]
109108
lemma dens_prefixed (s : Finset α) : (prefixed s).dens = ((card α).choose #s : ℚ≥0)⁻¹ := by
110-
simp [dens, card_prefixed, Nat.cast_choose' _ s.card_le_univ]
109+
simp [dens, card_prefixed, Nat.cast_choose _ s.card_le_univ]
111110

112111
-- TODO: This can be strengthened to an iff
113112
lemma disjoint_prefixed_prefixed (hst : ¬ s ⊆ t) (hts : ¬ t ⊆ s) :

lake-manifest.json

Lines changed: 10 additions & 10 deletions
Original file line numberDiff line numberDiff line change
@@ -5,17 +5,17 @@
55
"type": "git",
66
"subDir": null,
77
"scope": "",
8-
"rev": "5269898d6a51d047931107c8d72d934d8d5d3753",
8+
"rev": "3800f46f4b3baed8f14b0cd3a90963c5a453667b",
99
"name": "mathlib",
1010
"manifestFile": "lake-manifest.json",
11-
"inputRev": "v4.17.0",
11+
"inputRev": null,
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": "c708be04267e3e995a14ac0d08b1530579c1525a",
18+
"rev": "ebfb31672ab0a5b6d00a018ff67d2ec51ed66f3a",
1919
"name": "plausible",
2020
"manifestFile": "lake-manifest.json",
2121
"inputRev": "main",
@@ -35,7 +35,7 @@
3535
"type": "git",
3636
"subDir": null,
3737
"scope": "leanprover-community",
38-
"rev": "0447b0a7b7f41f0a1749010db3f222e4a96f9d30",
38+
"rev": "08372f1ec11df288ff76621ead7b0b575cb29355",
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": "799f6986de9f61b784ff7be8f6a8b101045b8ffd",
48+
"rev": "a602d13aca2913724c7d47b2d7df0353620c4ee8",
4949
"name": "proofwidgets",
5050
"manifestFile": "lake-manifest.json",
51-
"inputRev": "v0.0.52",
51+
"inputRev": "v0.0.53",
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": "56a2c80b209c253e0281ac4562a92122b457dcc0",
58+
"rev": "ec060e0e10c685be8af65f288e23d026c9fde245",
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": "95561f7a5811fae6a309e4a1bbe22a0a4a98bf03",
68+
"rev": "d892d7a88ad0ccf748fb8e651308ccd13426ba73",
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": "efcc7d9bd9936ecdc625baf0d033b60866565cd5",
78+
"rev": "cce013731b5b355ff4528ac9717ae3e0cc5c4519",
7979
"name": "batteries",
8080
"manifestFile": "lake-manifest.json",
8181
"inputRev": "main",
@@ -85,7 +85,7 @@
8585
"type": "git",
8686
"subDir": null,
8787
"scope": "leanprover",
88-
"rev": "e7fd1a415c80985ade02a021172834ca2139b0ca",
88+
"rev": "dd423cf2b153b5b14cb017ee4beae788565a3925",
8989
"name": "Cli",
9090
"manifestFile": "lake-manifest.json",
9191
"inputRev": "main",

lean-toolchain

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

0 commit comments

Comments
 (0)