Skip to content

Commit 3743527

Browse files
committed
Bump mathlib
1 parent 533b686 commit 3743527

File tree

5 files changed

+14
-333
lines changed

5 files changed

+14
-333
lines changed

LeanCamCombi.lean

Lines changed: 0 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -11,7 +11,6 @@ import LeanCamCombi.GrowthInGroups.Lecture3
1111
import LeanCamCombi.GrowthInGroups.Lecture4
1212
import LeanCamCombi.Mathlib.Combinatorics.Additive.ApproximateSubgroup
1313
import LeanCamCombi.Mathlib.Combinatorics.SetFamily.LYM
14-
import LeanCamCombi.Mathlib.Combinatorics.SimpleGraph.Copy
1514
import LeanCamCombi.Mathlib.Combinatorics.SimpleGraph.Density
1615
import LeanCamCombi.Mathlib.Probability.ProbabilityMassFunction.Constructions
1716
import LeanCamCombi.PlainCombi.KatonaCircle

LeanCamCombi/ExtrProbCombi/BinomialRandomGraph.lean

Lines changed: 9 additions & 7 deletions
Original file line numberDiff line numberDiff line change
@@ -69,12 +69,14 @@ protected nonrec lemma meas [IsProbabilityMeasure μ] [Fintype α] [DecidableEq
6969
[DecidableRel H.Adj] :
7070
μ {ω | G ω = H} =
7171
p ^ #H.edgeFinset * (1 - p) ^ (Fintype.card {e : Sym2 α // ¬ e.IsDiag} - #H.edgeFinset) := by
72-
have := hG.meas
73-
(H.edgeFinset.attach.map <| ⟨Set.inclusion fun e he ↦
74-
not_isDiag_of_mem_edgeSet _ <| mem_edgeFinset.1 he, Set.inclusion_injective _⟩)
75-
simp at this
76-
rw [Finset.card_attach, ← Fintype.card_subtype_compl] at this
77-
convert this
78-
sorry
72+
have hHaux : H.edgeFinset = ({e | e ∈ H.edgeSet} : Finset _) := by ext; simp
73+
have hGHaux ω : G ω = H ↔ {e : {e : Sym2 α // ¬ e.IsDiag} | e.1 ∈ (G ω).edgeSet} =
74+
Set.range fun a : H.edgeFinset ↦
75+
Set.inclusion (fun e he ↦ not_isDiag_of_mem_edgeSet H (mem_edgeFinset.mp he)) a := by
76+
simp only [Set.ext_iff, ← edgeSet_inj]
77+
simpa [Sym2.forall] using forall₂_congr fun u v ↦ by simp +contextual [or_iff_not_imp_left]
78+
simpa [hGHaux, hHaux, ← Fintype.card_subtype_compl] using
79+
hG.meas <| H.edgeFinset.attach.map <| ⟨Set.inclusion fun e he ↦
80+
not_isDiag_of_mem_edgeSet _ <| mem_edgeFinset.1 he, Set.inclusion_injective _⟩
7981

8082
end IsBinomialRandomGraph

LeanCamCombi/ExtrProbCombi/BollobasContainment.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -4,10 +4,10 @@ Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Yaël Dillies
55
-/
66
import Mathlib.Analysis.SpecialFunctions.Pow.Real
7+
import Mathlib.Combinatorics.SimpleGraph.Copy
78
import Mathlib.MeasureTheory.Measure.Typeclasses
89
import LeanCamCombi.Mathlib.Combinatorics.SimpleGraph.Density
910
import LeanCamCombi.ExtrProbCombi.BinomialRandomGraph
10-
import LeanCamCombi.Mathlib.Combinatorics.SimpleGraph.Copy
1111

1212
/-!
1313
# Bollobás' graph containment lemma

LeanCamCombi/Mathlib/Combinatorics/SimpleGraph/Copy.lean

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

lake-manifest.json

Lines changed: 4 additions & 4 deletions
Original file line numberDiff line numberDiff line change
@@ -5,7 +5,7 @@
55
"type": "git",
66
"subDir": null,
77
"scope": "",
8-
"rev": "d22bd4f990c36ec29867ef381dc67f43c3d40520",
8+
"rev": "6d323eaab8473e64720e30cd8e879e31d3817932",
99
"name": "mathlib",
1010
"manifestFile": "lake-manifest.json",
1111
"inputRev": null,
@@ -25,7 +25,7 @@
2525
"type": "git",
2626
"subDir": null,
2727
"scope": "leanprover-community",
28-
"rev": "ba020ed434b9c5877eb62ff072a28f5ec56eb871",
28+
"rev": "8d29bc2c3ebe1f863c2f02df816b4f3dd1b65226",
2929
"name": "LeanSearchClient",
3030
"manifestFile": "lake-manifest.json",
3131
"inputRev": "main",
@@ -55,7 +55,7 @@
5555
"type": "git",
5656
"subDir": null,
5757
"scope": "leanprover-community",
58-
"rev": "471ff276892c3451a1d693477107e9c3a0c8ab85",
58+
"rev": "ecaaeb0b44a8d5784f17bd417e83f44c906804ab",
5959
"name": "aesop",
6060
"manifestFile": "lake-manifest.json",
6161
"inputRev": "master",
@@ -75,7 +75,7 @@
7575
"type": "git",
7676
"subDir": null,
7777
"scope": "leanprover-community",
78-
"rev": "71c64425f2f76c4ffcf4a2f12b17c083976caaa0",
78+
"rev": "7ad3747bf6cb10bfe96a40186ca8970ee851eb3b",
7979
"name": "batteries",
8080
"manifestFile": "lake-manifest.json",
8181
"inputRev": "main",

0 commit comments

Comments
 (0)