url
stringclasses 147
values | commit
stringclasses 147
values | file_path
stringlengths 7
101
| full_name
stringlengths 1
94
| start
stringlengths 6
10
| end
stringlengths 6
11
| tactic
stringlengths 1
11.2k
| state_before
stringlengths 3
2.09M
| state_after
stringlengths 6
2.09M
|
---|---|---|---|---|---|---|---|---|
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Order/SupClosed.lean | supClosure_prod | [16, 1] | [23, 32] | rintro ⟨_, _⟩ ⟨⟨u, hu, hus, rfl⟩, v, hv, hvt, rfl⟩ | α : Type u_1
β : Type u_2
inst✝¹ : SemilatticeSup α
inst✝ : SemilatticeSup β
s✝ t✝ : Set α
a b : α
s : Set α
t : Set β
⊢ supClosure s ×ˢ supClosure t ≤ supClosure (s ×ˢ t) | case mk.intro.intro.intro.intro.intro.intro.intro
α : Type u_1
β : Type u_2
inst✝¹ : SemilatticeSup α
inst✝ : SemilatticeSup β
s✝ t✝ : Set α
a b : α
s : Set α
t : Set β
u : Finset α
hu : u.Nonempty
hus : ↑u ⊆ s
v : Finset β
hv : v.Nonempty
hvt : ↑v ⊆ t
⊢ (u.sup' hu id, v.sup' hv id) ∈ supClosure (s ×ˢ t) |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Order/SupClosed.lean | supClosure_prod | [16, 1] | [23, 32] | refine ⟨u ×ˢ v, hu.product hv, ?_, ?_⟩ | case mk.intro.intro.intro.intro.intro.intro.intro
α : Type u_1
β : Type u_2
inst✝¹ : SemilatticeSup α
inst✝ : SemilatticeSup β
s✝ t✝ : Set α
a b : α
s : Set α
t : Set β
u : Finset α
hu : u.Nonempty
hus : ↑u ⊆ s
v : Finset β
hv : v.Nonempty
hvt : ↑v ⊆ t
⊢ (u.sup' hu id, v.sup' hv id) ∈ supClosure (s ×ˢ t) | case mk.intro.intro.intro.intro.intro.intro.intro.refine_1
α : Type u_1
β : Type u_2
inst✝¹ : SemilatticeSup α
inst✝ : SemilatticeSup β
s✝ t✝ : Set α
a b : α
s : Set α
t : Set β
u : Finset α
hu : u.Nonempty
hus : ↑u ⊆ s
v : Finset β
hv : v.Nonempty
hvt : ↑v ⊆ t
⊢ ↑(u ×ˢ v) ⊆ s ×ˢ t
case mk.intro.intro.intro.intro.intro.intro.intro.refine_2
α : Type u_1
β : Type u_2
inst✝¹ : SemilatticeSup α
inst✝ : SemilatticeSup β
s✝ t✝ : Set α
a b : α
s : Set α
t : Set β
u : Finset α
hu : u.Nonempty
hus : ↑u ⊆ s
v : Finset β
hv : v.Nonempty
hvt : ↑v ⊆ t
⊢ (u ×ˢ v).sup' ⋯ id = (u.sup' hu id, v.sup' hv id) |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Order/SupClosed.lean | supClosure_prod | [16, 1] | [23, 32] | simpa only [coe_product] using Set.prod_mono hus hvt | case mk.intro.intro.intro.intro.intro.intro.intro.refine_1
α : Type u_1
β : Type u_2
inst✝¹ : SemilatticeSup α
inst✝ : SemilatticeSup β
s✝ t✝ : Set α
a b : α
s : Set α
t : Set β
u : Finset α
hu : u.Nonempty
hus : ↑u ⊆ s
v : Finset β
hv : v.Nonempty
hvt : ↑v ⊆ t
⊢ ↑(u ×ˢ v) ⊆ s ×ˢ t | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Order/SupClosed.lean | supClosure_prod | [16, 1] | [23, 32] | simp [prodMk_sup'_sup'] | case mk.intro.intro.intro.intro.intro.intro.intro.refine_2
α : Type u_1
β : Type u_2
inst✝¹ : SemilatticeSup α
inst✝ : SemilatticeSup β
s✝ t✝ : Set α
a b : α
s : Set α
t : Set β
u : Finset α
hu : u.Nonempty
hus : ↑u ⊆ s
v : Finset β
hv : v.Nonempty
hvt : ↑v ⊆ t
⊢ (u ×ˢ v).sup' ⋯ id = (u.sup' hu id, v.sup' hv id) | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Order/SupClosed.lean | infClosure_prod | [32, 1] | [39, 32] | rintro ⟨_, _⟩ ⟨⟨u, hu, hus, rfl⟩, v, hv, hvt, rfl⟩ | α : Type u_1
β : Type u_2
inst✝¹ : SemilatticeInf α
inst✝ : SemilatticeInf β
s✝ t✝ : Set α
a b : α
s : Set α
t : Set β
⊢ infClosure s ×ˢ infClosure t ≤ infClosure (s ×ˢ t) | case mk.intro.intro.intro.intro.intro.intro.intro
α : Type u_1
β : Type u_2
inst✝¹ : SemilatticeInf α
inst✝ : SemilatticeInf β
s✝ t✝ : Set α
a b : α
s : Set α
t : Set β
u : Finset α
hu : u.Nonempty
hus : ↑u ⊆ s
v : Finset β
hv : v.Nonempty
hvt : ↑v ⊆ t
⊢ (u.inf' hu id, v.inf' hv id) ∈ infClosure (s ×ˢ t) |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Order/SupClosed.lean | infClosure_prod | [32, 1] | [39, 32] | refine ⟨u ×ˢ v, hu.product hv, ?_, ?_⟩ | case mk.intro.intro.intro.intro.intro.intro.intro
α : Type u_1
β : Type u_2
inst✝¹ : SemilatticeInf α
inst✝ : SemilatticeInf β
s✝ t✝ : Set α
a b : α
s : Set α
t : Set β
u : Finset α
hu : u.Nonempty
hus : ↑u ⊆ s
v : Finset β
hv : v.Nonempty
hvt : ↑v ⊆ t
⊢ (u.inf' hu id, v.inf' hv id) ∈ infClosure (s ×ˢ t) | case mk.intro.intro.intro.intro.intro.intro.intro.refine_1
α : Type u_1
β : Type u_2
inst✝¹ : SemilatticeInf α
inst✝ : SemilatticeInf β
s✝ t✝ : Set α
a b : α
s : Set α
t : Set β
u : Finset α
hu : u.Nonempty
hus : ↑u ⊆ s
v : Finset β
hv : v.Nonempty
hvt : ↑v ⊆ t
⊢ ↑(u ×ˢ v) ⊆ s ×ˢ t
case mk.intro.intro.intro.intro.intro.intro.intro.refine_2
α : Type u_1
β : Type u_2
inst✝¹ : SemilatticeInf α
inst✝ : SemilatticeInf β
s✝ t✝ : Set α
a b : α
s : Set α
t : Set β
u : Finset α
hu : u.Nonempty
hus : ↑u ⊆ s
v : Finset β
hv : v.Nonempty
hvt : ↑v ⊆ t
⊢ (u ×ˢ v).inf' ⋯ id = (u.inf' hu id, v.inf' hv id) |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Order/SupClosed.lean | infClosure_prod | [32, 1] | [39, 32] | simpa only [coe_product] using Set.prod_mono hus hvt | case mk.intro.intro.intro.intro.intro.intro.intro.refine_1
α : Type u_1
β : Type u_2
inst✝¹ : SemilatticeInf α
inst✝ : SemilatticeInf β
s✝ t✝ : Set α
a b : α
s : Set α
t : Set β
u : Finset α
hu : u.Nonempty
hus : ↑u ⊆ s
v : Finset β
hv : v.Nonempty
hvt : ↑v ⊆ t
⊢ ↑(u ×ˢ v) ⊆ s ×ˢ t | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Order/SupClosed.lean | infClosure_prod | [32, 1] | [39, 32] | simp [prodMk_inf'_inf'] | case mk.intro.intro.intro.intro.intro.intro.intro.refine_2
α : Type u_1
β : Type u_2
inst✝¹ : SemilatticeInf α
inst✝ : SemilatticeInf β
s✝ t✝ : Set α
a b : α
s : Set α
t : Set β
u : Finset α
hu : u.Nonempty
hus : ↑u ⊆ s
v : Finset β
hv : v.Nonempty
hvt : ↑v ⊆ t
⊢ (u ×ˢ v).inf' ⋯ id = (u.inf' hu id, v.inf' hv id) | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Order/SupClosed.lean | latticeClosure_prod | [48, 1] | [50, 42] | simp_rw [← supClosure_infClosure] | α : Type u_1
β : Type u_2
inst✝¹ : DistribLattice α
inst✝ : DistribLattice β
s✝ s : Set α
t : Set β
⊢ latticeClosure (s ×ˢ t) = latticeClosure s ×ˢ latticeClosure t | α : Type u_1
β : Type u_2
inst✝¹ : DistribLattice α
inst✝ : DistribLattice β
s✝ s : Set α
t : Set β
⊢ supClosure (infClosure (s ×ˢ t)) = supClosure (infClosure s) ×ˢ supClosure (infClosure t) |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Order/SupClosed.lean | latticeClosure_prod | [48, 1] | [50, 42] | simp | α : Type u_1
β : Type u_2
inst✝¹ : DistribLattice α
inst✝ : DistribLattice β
s✝ s : Set α
t : Set β
⊢ supClosure (infClosure (s ×ˢ t)) = supClosure (infClosure s) ×ˢ supClosure (infClosure t) | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Combinatorics/SimpleGraph/Degree.lean | SimpleGraph.degOn_empty | [16, 1] | [17, 63] | simp [degOn] | α : Type u_1
inst✝² : Fintype α
inst✝¹ : DecidableEq α
G : SimpleGraph α
inst✝ : DecidableRel G.Adj
s t : Finset α
a✝ a : α
⊢ G.degOn ∅ a = 0 | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Combinatorics/SimpleGraph/Degree.lean | SimpleGraph.degOn_univ | [19, 1] | [20, 92] | rw [degOn, degree, univ_inter] | α : Type u_1
inst✝² : Fintype α
inst✝¹ : DecidableEq α
G : SimpleGraph α
inst✝ : DecidableRel G.Adj
s t : Finset α
a✝ a : α
⊢ G.degOn univ a = G.degree a | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Combinatorics/SimpleGraph/Degree.lean | SimpleGraph.degOn_union | [23, 1] | [26, 51] | unfold degOn | α : Type u_1
inst✝² : Fintype α
inst✝¹ : DecidableEq α
G : SimpleGraph α
inst✝ : DecidableRel G.Adj
s t : Finset α
a✝ : α
h : Disjoint s t
a : α
⊢ G.degOn (s ∪ t) a = G.degOn s a + G.degOn t a | α : Type u_1
inst✝² : Fintype α
inst✝¹ : DecidableEq α
G : SimpleGraph α
inst✝ : DecidableRel G.Adj
s t : Finset α
a✝ : α
h : Disjoint s t
a : α
⊢ ((s ∪ t) ∩ G.neighborFinset a).card = (s ∩ G.neighborFinset a).card + (t ∩ G.neighborFinset a).card |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Combinatorics/SimpleGraph/Degree.lean | SimpleGraph.degOn_union | [23, 1] | [26, 51] | rw [← card_union_of_disjoint, ← union_inter_distrib_right] | α : Type u_1
inst✝² : Fintype α
inst✝¹ : DecidableEq α
G : SimpleGraph α
inst✝ : DecidableRel G.Adj
s t : Finset α
a✝ : α
h : Disjoint s t
a : α
⊢ ((s ∪ t) ∩ G.neighborFinset a).card = (s ∩ G.neighborFinset a).card + (t ∩ G.neighborFinset a).card | α : Type u_1
inst✝² : Fintype α
inst✝¹ : DecidableEq α
G : SimpleGraph α
inst✝ : DecidableRel G.Adj
s t : Finset α
a✝ : α
h : Disjoint s t
a : α
⊢ Disjoint (s ∩ G.neighborFinset a) (t ∩ G.neighborFinset a) |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Combinatorics/SimpleGraph/Degree.lean | SimpleGraph.degOn_union | [23, 1] | [26, 51] | exact h.mono inter_subset_left inter_subset_left | α : Type u_1
inst✝² : Fintype α
inst✝¹ : DecidableEq α
G : SimpleGraph α
inst✝ : DecidableRel G.Adj
s t : Finset α
a✝ : α
h : Disjoint s t
a : α
⊢ Disjoint (s ∩ G.neighborFinset a) (t ∩ G.neighborFinset a) | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Combinatorics/SimpleGraph/Degree.lean | SimpleGraph.sum_degOn_comm | [29, 1] | [32, 39] | simp_rw [degOn, card_eq_sum_ones, ← sum_indicator_eq_sum_inter] | α : Type u_1
inst✝² : Fintype α
inst✝¹ : DecidableEq α
G : SimpleGraph α
inst✝ : DecidableRel G.Adj
s✝ t✝ : Finset α
a : α
s t : Finset α
⊢ ∑ a ∈ s, G.degOn t a = ∑ a ∈ t, G.degOn s a | α : Type u_1
inst✝² : Fintype α
inst✝¹ : DecidableEq α
G : SimpleGraph α
inst✝ : DecidableRel G.Adj
s✝ t✝ : Finset α
a : α
s t : Finset α
⊢ ∑ x ∈ s, ∑ i ∈ t, (↑(G.neighborFinset x)).indicator (fun x => 1) i =
∑ x ∈ t, ∑ i ∈ s, (↑(G.neighborFinset x)).indicator (fun x => 1) i |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Combinatorics/SimpleGraph/Degree.lean | SimpleGraph.sum_degOn_comm | [29, 1] | [32, 39] | rw [sum_comm] | α : Type u_1
inst✝² : Fintype α
inst✝¹ : DecidableEq α
G : SimpleGraph α
inst✝ : DecidableRel G.Adj
s✝ t✝ : Finset α
a : α
s t : Finset α
⊢ ∑ x ∈ s, ∑ i ∈ t, (↑(G.neighborFinset x)).indicator (fun x => 1) i =
∑ x ∈ t, ∑ i ∈ s, (↑(G.neighborFinset x)).indicator (fun x => 1) i | α : Type u_1
inst✝² : Fintype α
inst✝¹ : DecidableEq α
G : SimpleGraph α
inst✝ : DecidableRel G.Adj
s✝ t✝ : Finset α
a : α
s t : Finset α
⊢ ∑ y ∈ t, ∑ x ∈ s, (↑(G.neighborFinset x)).indicator (fun x => 1) y =
∑ x ∈ t, ∑ i ∈ s, (↑(G.neighborFinset x)).indicator (fun x => 1) i |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Combinatorics/SimpleGraph/Degree.lean | SimpleGraph.sum_degOn_comm | [29, 1] | [32, 39] | simp [Set.indicator_apply, adj_comm] | α : Type u_1
inst✝² : Fintype α
inst✝¹ : DecidableEq α
G : SimpleGraph α
inst✝ : DecidableRel G.Adj
s✝ t✝ : Finset α
a : α
s t : Finset α
⊢ ∑ y ∈ t, ∑ x ∈ s, (↑(G.neighborFinset x)).indicator (fun x => 1) y =
∑ x ∈ t, ∑ i ∈ s, (↑(G.neighborFinset x)).indicator (fun x => 1) i | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Data/Nat/Defs.lean | Nat.eq_of_dvd_of_lt_two_mul | [6, 1] | [11, 67] | obtain ⟨_ | _ | c, rfl⟩ := hdvd | a b : ℕ
ha : a ≠ 0
hdvd : b ∣ a
hlt : a < 2 * b
⊢ a = b | case intro.zero
b : ℕ
ha : b * 0 ≠ 0
hlt : b * 0 < 2 * b
⊢ b * 0 = b
case intro.succ.zero
b : ℕ
ha : b * (0 + 1) ≠ 0
hlt : b * (0 + 1) < 2 * b
⊢ b * (0 + 1) = b
case intro.succ.succ
b c : ℕ
ha : b * (c + 1 + 1) ≠ 0
hlt : b * (c + 1 + 1) < 2 * b
⊢ b * (c + 1 + 1) = b |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Data/Nat/Defs.lean | Nat.eq_of_dvd_of_lt_two_mul | [6, 1] | [11, 67] | simp at ha | case intro.zero
b : ℕ
ha : b * 0 ≠ 0
hlt : b * 0 < 2 * b
⊢ b * 0 = b | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Data/Nat/Defs.lean | Nat.eq_of_dvd_of_lt_two_mul | [6, 1] | [11, 67] | exact Nat.mul_one _ | case intro.succ.zero
b : ℕ
ha : b * (0 + 1) ≠ 0
hlt : b * (0 + 1) < 2 * b
⊢ b * (0 + 1) = b | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Data/Nat/Defs.lean | Nat.eq_of_dvd_of_lt_two_mul | [6, 1] | [11, 67] | rw [Nat.mul_comm] at hlt | case intro.succ.succ
b c : ℕ
ha : b * (c + 1 + 1) ≠ 0
hlt : b * (c + 1 + 1) < 2 * b
⊢ b * (c + 1 + 1) = b | case intro.succ.succ
b c : ℕ
ha : b * (c + 1 + 1) ≠ 0
hlt : (c + 1 + 1) * b < 2 * b
⊢ b * (c + 1 + 1) = b |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Data/Nat/Defs.lean | Nat.eq_of_dvd_of_lt_two_mul | [6, 1] | [11, 67] | cases Nat.not_le_of_lt hlt (Nat.mul_le_mul_right _ (by omega)) | case intro.succ.succ
b c : ℕ
ha : b * (c + 1 + 1) ≠ 0
hlt : (c + 1 + 1) * b < 2 * b
⊢ b * (c + 1 + 1) = b | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Data/Nat/Defs.lean | Nat.eq_of_dvd_of_lt_two_mul | [6, 1] | [11, 67] | omega | b c : ℕ
ha : b * (c + 1 + 1) ≠ 0
hlt : (c + 1 + 1) * b < 2 * b
⊢ 2 ≤ c + 1 + 1 | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/LittlewoodOfford.lean | Finset.exists_littlewood_offord_partition | [20, 1] | [35, 8] | induction' s using Finset.induction with i s hi ih | ι : Type u_1
E : Type u_2
inst✝² : NormedAddCommGroup E
inst✝¹ : NormedSpace ℝ E
𝒜 : Finset (Finset ι)
s : Finset ι
f : ι → E
r : ℝ
inst✝ : DecidableEq ι
hr : 0 < r
hf : ∀ i ∈ s, r ≤ ‖f i‖
⊢ ∃ P,
P.parts.card = s.card.choose (s.card / 2) ∧
(∀ 𝒜 ∈ P.parts, ∀ t ∈ 𝒜, t ⊆ s) ∧ ∀ 𝒜 ∈ P.parts, (↑𝒜).Pairwise fun u v => r ≤ dist (∑ i ∈ u, f i) (∑ i ∈ v, f i) | case empty
ι : Type u_1
E : Type u_2
inst✝² : NormedAddCommGroup E
inst✝¹ : NormedSpace ℝ E
𝒜 : Finset (Finset ι)
s : Finset ι
f : ι → E
r : ℝ
inst✝ : DecidableEq ι
hr : 0 < r
hf : ∀ i ∈ ∅, r ≤ ‖f i‖
⊢ ∃ P,
P.parts.card = ∅.card.choose (∅.card / 2) ∧
(∀ 𝒜 ∈ P.parts, ∀ t ∈ 𝒜, t ⊆ ∅) ∧ ∀ 𝒜 ∈ P.parts, (↑𝒜).Pairwise fun u v => r ≤ dist (∑ i ∈ u, f i) (∑ i ∈ v, f i)
case insert
ι : Type u_1
E : Type u_2
inst✝² : NormedAddCommGroup E
inst✝¹ : NormedSpace ℝ E
𝒜 : Finset (Finset ι)
s✝ : Finset ι
f : ι → E
r : ℝ
inst✝ : DecidableEq ι
hr : 0 < r
i : ι
s : Finset ι
hi : i ∉ s
ih :
(∀ i ∈ s, r ≤ ‖f i‖) →
∃ P,
P.parts.card = s.card.choose (s.card / 2) ∧
(∀ 𝒜 ∈ P.parts, ∀ t ∈ 𝒜, t ⊆ s) ∧ ∀ 𝒜 ∈ P.parts, (↑𝒜).Pairwise fun u v => r ≤ dist (∑ i ∈ u, f i) (∑ i ∈ v, f i)
hf : ∀ i_1 ∈ insert i s, r ≤ ‖f i_1‖
⊢ ∃ P,
P.parts.card = (insert i s).card.choose ((insert i s).card / 2) ∧
(∀ 𝒜 ∈ P.parts, ∀ t ∈ 𝒜, t ⊆ insert i s) ∧
∀ 𝒜 ∈ P.parts, (↑𝒜).Pairwise fun u v => r ≤ dist (∑ i ∈ u, f i) (∑ i ∈ v, f i) |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/LittlewoodOfford.lean | Finset.exists_littlewood_offord_partition | [20, 1] | [35, 8] | obtain ⟨P, hP, hs, hPr⟩ := ih fun j hj ↦ hf _ $ mem_insert_of_mem hj | case insert
ι : Type u_1
E : Type u_2
inst✝² : NormedAddCommGroup E
inst✝¹ : NormedSpace ℝ E
𝒜 : Finset (Finset ι)
s✝ : Finset ι
f : ι → E
r : ℝ
inst✝ : DecidableEq ι
hr : 0 < r
i : ι
s : Finset ι
hi : i ∉ s
ih :
(∀ i ∈ s, r ≤ ‖f i‖) →
∃ P,
P.parts.card = s.card.choose (s.card / 2) ∧
(∀ 𝒜 ∈ P.parts, ∀ t ∈ 𝒜, t ⊆ s) ∧ ∀ 𝒜 ∈ P.parts, (↑𝒜).Pairwise fun u v => r ≤ dist (∑ i ∈ u, f i) (∑ i ∈ v, f i)
hf : ∀ i_1 ∈ insert i s, r ≤ ‖f i_1‖
⊢ ∃ P,
P.parts.card = (insert i s).card.choose ((insert i s).card / 2) ∧
(∀ 𝒜 ∈ P.parts, ∀ t ∈ 𝒜, t ⊆ insert i s) ∧
∀ 𝒜 ∈ P.parts, (↑𝒜).Pairwise fun u v => r ≤ dist (∑ i ∈ u, f i) (∑ i ∈ v, f i) | case insert.intro.intro.intro
ι : Type u_1
E : Type u_2
inst✝² : NormedAddCommGroup E
inst✝¹ : NormedSpace ℝ E
𝒜 : Finset (Finset ι)
s✝ : Finset ι
f : ι → E
r : ℝ
inst✝ : DecidableEq ι
hr : 0 < r
i : ι
s : Finset ι
hi : i ∉ s
ih :
(∀ i ∈ s, r ≤ ‖f i‖) →
∃ P,
P.parts.card = s.card.choose (s.card / 2) ∧
(∀ 𝒜 ∈ P.parts, ∀ t ∈ 𝒜, t ⊆ s) ∧ ∀ 𝒜 ∈ P.parts, (↑𝒜).Pairwise fun u v => r ≤ dist (∑ i ∈ u, f i) (∑ i ∈ v, f i)
hf : ∀ i_1 ∈ insert i s, r ≤ ‖f i_1‖
P : Finpartition s.powerset
hP : P.parts.card = s.card.choose (s.card / 2)
hs : ∀ 𝒜 ∈ P.parts, ∀ t ∈ 𝒜, t ⊆ s
hPr : ∀ 𝒜 ∈ P.parts, (↑𝒜).Pairwise fun u v => r ≤ dist (∑ i ∈ u, f i) (∑ i ∈ v, f i)
⊢ ∃ P,
P.parts.card = (insert i s).card.choose ((insert i s).card / 2) ∧
(∀ 𝒜 ∈ P.parts, ∀ t ∈ 𝒜, t ⊆ insert i s) ∧
∀ 𝒜 ∈ P.parts, (↑𝒜).Pairwise fun u v => r ≤ dist (∑ i ∈ u, f i) (∑ i ∈ v, f i) |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/LittlewoodOfford.lean | Finset.exists_littlewood_offord_partition | [20, 1] | [35, 8] | clear ih | case insert.intro.intro.intro
ι : Type u_1
E : Type u_2
inst✝² : NormedAddCommGroup E
inst✝¹ : NormedSpace ℝ E
𝒜 : Finset (Finset ι)
s✝ : Finset ι
f : ι → E
r : ℝ
inst✝ : DecidableEq ι
hr : 0 < r
i : ι
s : Finset ι
hi : i ∉ s
ih :
(∀ i ∈ s, r ≤ ‖f i‖) →
∃ P,
P.parts.card = s.card.choose (s.card / 2) ∧
(∀ 𝒜 ∈ P.parts, ∀ t ∈ 𝒜, t ⊆ s) ∧ ∀ 𝒜 ∈ P.parts, (↑𝒜).Pairwise fun u v => r ≤ dist (∑ i ∈ u, f i) (∑ i ∈ v, f i)
hf : ∀ i_1 ∈ insert i s, r ≤ ‖f i_1‖
P : Finpartition s.powerset
hP : P.parts.card = s.card.choose (s.card / 2)
hs : ∀ 𝒜 ∈ P.parts, ∀ t ∈ 𝒜, t ⊆ s
hPr : ∀ 𝒜 ∈ P.parts, (↑𝒜).Pairwise fun u v => r ≤ dist (∑ i ∈ u, f i) (∑ i ∈ v, f i)
⊢ ∃ P,
P.parts.card = (insert i s).card.choose ((insert i s).card / 2) ∧
(∀ 𝒜 ∈ P.parts, ∀ t ∈ 𝒜, t ⊆ insert i s) ∧
∀ 𝒜 ∈ P.parts, (↑𝒜).Pairwise fun u v => r ≤ dist (∑ i ∈ u, f i) (∑ i ∈ v, f i) | case insert.intro.intro.intro
ι : Type u_1
E : Type u_2
inst✝² : NormedAddCommGroup E
inst✝¹ : NormedSpace ℝ E
𝒜 : Finset (Finset ι)
s✝ : Finset ι
f : ι → E
r : ℝ
inst✝ : DecidableEq ι
hr : 0 < r
i : ι
s : Finset ι
hi : i ∉ s
hf : ∀ i_1 ∈ insert i s, r ≤ ‖f i_1‖
P : Finpartition s.powerset
hP : P.parts.card = s.card.choose (s.card / 2)
hs : ∀ 𝒜 ∈ P.parts, ∀ t ∈ 𝒜, t ⊆ s
hPr : ∀ 𝒜 ∈ P.parts, (↑𝒜).Pairwise fun u v => r ≤ dist (∑ i ∈ u, f i) (∑ i ∈ v, f i)
⊢ ∃ P,
P.parts.card = (insert i s).card.choose ((insert i s).card / 2) ∧
(∀ 𝒜 ∈ P.parts, ∀ t ∈ 𝒜, t ⊆ insert i s) ∧
∀ 𝒜 ∈ P.parts, (↑𝒜).Pairwise fun u v => r ≤ dist (∑ i ∈ u, f i) (∑ i ∈ v, f i) |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/LittlewoodOfford.lean | Finset.exists_littlewood_offord_partition | [20, 1] | [35, 8] | obtain ⟨g, hg, hgf⟩ :=
exists_dual_vector ℝ (f i) (norm_pos_iff.1 $ hr.trans_le $ hf _ $ mem_insert_self _ _) | case insert.intro.intro.intro
ι : Type u_1
E : Type u_2
inst✝² : NormedAddCommGroup E
inst✝¹ : NormedSpace ℝ E
𝒜 : Finset (Finset ι)
s✝ : Finset ι
f : ι → E
r : ℝ
inst✝ : DecidableEq ι
hr : 0 < r
i : ι
s : Finset ι
hi : i ∉ s
hf : ∀ i_1 ∈ insert i s, r ≤ ‖f i_1‖
P : Finpartition s.powerset
hP : P.parts.card = s.card.choose (s.card / 2)
hs : ∀ 𝒜 ∈ P.parts, ∀ t ∈ 𝒜, t ⊆ s
hPr : ∀ 𝒜 ∈ P.parts, (↑𝒜).Pairwise fun u v => r ≤ dist (∑ i ∈ u, f i) (∑ i ∈ v, f i)
⊢ ∃ P,
P.parts.card = (insert i s).card.choose ((insert i s).card / 2) ∧
(∀ 𝒜 ∈ P.parts, ∀ t ∈ 𝒜, t ⊆ insert i s) ∧
∀ 𝒜 ∈ P.parts, (↑𝒜).Pairwise fun u v => r ≤ dist (∑ i ∈ u, f i) (∑ i ∈ v, f i) | case insert.intro.intro.intro.intro.intro
ι : Type u_1
E : Type u_2
inst✝² : NormedAddCommGroup E
inst✝¹ : NormedSpace ℝ E
𝒜 : Finset (Finset ι)
s✝ : Finset ι
f : ι → E
r : ℝ
inst✝ : DecidableEq ι
hr : 0 < r
i : ι
s : Finset ι
hi : i ∉ s
hf : ∀ i_1 ∈ insert i s, r ≤ ‖f i_1‖
P : Finpartition s.powerset
hP : P.parts.card = s.card.choose (s.card / 2)
hs : ∀ 𝒜 ∈ P.parts, ∀ t ∈ 𝒜, t ⊆ s
hPr : ∀ 𝒜 ∈ P.parts, (↑𝒜).Pairwise fun u v => r ≤ dist (∑ i ∈ u, f i) (∑ i ∈ v, f i)
g : E →L[ℝ] ℝ
hg : ‖g‖ = 1
hgf : g (f i) = ↑‖f i‖
⊢ ∃ P,
P.parts.card = (insert i s).card.choose ((insert i s).card / 2) ∧
(∀ 𝒜 ∈ P.parts, ∀ t ∈ 𝒜, t ⊆ insert i s) ∧
∀ 𝒜 ∈ P.parts, (↑𝒜).Pairwise fun u v => r ≤ dist (∑ i ∈ u, f i) (∑ i ∈ v, f i) |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/LittlewoodOfford.lean | Finset.exists_littlewood_offord_partition | [20, 1] | [35, 8] | choose t ht using fun 𝒜 (h𝒜 : 𝒜 ∈ P.parts) ↦
Finset.exists_max_image _ (fun t ↦ g (∑ i in t, f i)) (P.nonempty_of_mem_parts h𝒜) | case insert.intro.intro.intro.intro.intro
ι : Type u_1
E : Type u_2
inst✝² : NormedAddCommGroup E
inst✝¹ : NormedSpace ℝ E
𝒜 : Finset (Finset ι)
s✝ : Finset ι
f : ι → E
r : ℝ
inst✝ : DecidableEq ι
hr : 0 < r
i : ι
s : Finset ι
hi : i ∉ s
hf : ∀ i_1 ∈ insert i s, r ≤ ‖f i_1‖
P : Finpartition s.powerset
hP : P.parts.card = s.card.choose (s.card / 2)
hs : ∀ 𝒜 ∈ P.parts, ∀ t ∈ 𝒜, t ⊆ s
hPr : ∀ 𝒜 ∈ P.parts, (↑𝒜).Pairwise fun u v => r ≤ dist (∑ i ∈ u, f i) (∑ i ∈ v, f i)
g : E →L[ℝ] ℝ
hg : ‖g‖ = 1
hgf : g (f i) = ↑‖f i‖
⊢ ∃ P,
P.parts.card = (insert i s).card.choose ((insert i s).card / 2) ∧
(∀ 𝒜 ∈ P.parts, ∀ t ∈ 𝒜, t ⊆ insert i s) ∧
∀ 𝒜 ∈ P.parts, (↑𝒜).Pairwise fun u v => r ≤ dist (∑ i ∈ u, f i) (∑ i ∈ v, f i) | case insert.intro.intro.intro.intro.intro
ι : Type u_1
E : Type u_2
inst✝² : NormedAddCommGroup E
inst✝¹ : NormedSpace ℝ E
𝒜 : Finset (Finset ι)
s✝ : Finset ι
f : ι → E
r : ℝ
inst✝ : DecidableEq ι
hr : 0 < r
i : ι
s : Finset ι
hi : i ∉ s
hf : ∀ i_1 ∈ insert i s, r ≤ ‖f i_1‖
P : Finpartition s.powerset
hP : P.parts.card = s.card.choose (s.card / 2)
hs : ∀ 𝒜 ∈ P.parts, ∀ t ∈ 𝒜, t ⊆ s
hPr : ∀ 𝒜 ∈ P.parts, (↑𝒜).Pairwise fun u v => r ≤ dist (∑ i ∈ u, f i) (∑ i ∈ v, f i)
g : E →L[ℝ] ℝ
hg : ‖g‖ = 1
hgf : g (f i) = ↑‖f i‖
t : (𝒜 : Finset (Finset ι)) → 𝒜 ∈ P.parts → Finset ι
ht : ∀ (𝒜 : Finset (Finset ι)) (h𝒜 : 𝒜 ∈ P.parts), t 𝒜 h𝒜 ∈ 𝒜 ∧ ∀ x' ∈ 𝒜, g (∑ i ∈ x', f i) ≤ g (∑ i ∈ t 𝒜 h𝒜, f i)
⊢ ∃ P,
P.parts.card = (insert i s).card.choose ((insert i s).card / 2) ∧
(∀ 𝒜 ∈ P.parts, ∀ t ∈ 𝒜, t ⊆ insert i s) ∧
∀ 𝒜 ∈ P.parts, (↑𝒜).Pairwise fun u v => r ≤ dist (∑ i ∈ u, f i) (∑ i ∈ v, f i) |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/LittlewoodOfford.lean | Finset.exists_littlewood_offord_partition | [20, 1] | [35, 8] | sorry | case insert.intro.intro.intro.intro.intro
ι : Type u_1
E : Type u_2
inst✝² : NormedAddCommGroup E
inst✝¹ : NormedSpace ℝ E
𝒜 : Finset (Finset ι)
s✝ : Finset ι
f : ι → E
r : ℝ
inst✝ : DecidableEq ι
hr : 0 < r
i : ι
s : Finset ι
hi : i ∉ s
hf : ∀ i_1 ∈ insert i s, r ≤ ‖f i_1‖
P : Finpartition s.powerset
hP : P.parts.card = s.card.choose (s.card / 2)
hs : ∀ 𝒜 ∈ P.parts, ∀ t ∈ 𝒜, t ⊆ s
hPr : ∀ 𝒜 ∈ P.parts, (↑𝒜).Pairwise fun u v => r ≤ dist (∑ i ∈ u, f i) (∑ i ∈ v, f i)
g : E →L[ℝ] ℝ
hg : ‖g‖ = 1
hgf : g (f i) = ↑‖f i‖
t : (𝒜 : Finset (Finset ι)) → 𝒜 ∈ P.parts → Finset ι
ht : ∀ (𝒜 : Finset (Finset ι)) (h𝒜 : 𝒜 ∈ P.parts), t 𝒜 h𝒜 ∈ 𝒜 ∧ ∀ x' ∈ 𝒜, g (∑ i ∈ x', f i) ≤ g (∑ i ∈ t 𝒜 h𝒜, f i)
⊢ ∃ P,
P.parts.card = (insert i s).card.choose ((insert i s).card / 2) ∧
(∀ 𝒜 ∈ P.parts, ∀ t ∈ 𝒜, t ⊆ insert i s) ∧
∀ 𝒜 ∈ P.parts, (↑𝒜).Pairwise fun u v => r ≤ dist (∑ i ∈ u, f i) (∑ i ∈ v, f i) | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/LittlewoodOfford.lean | Finset.exists_littlewood_offord_partition | [20, 1] | [35, 8] | exact ⟨Finpartition.indiscrete $ singleton_ne_empty _, by simp⟩ | case empty
ι : Type u_1
E : Type u_2
inst✝² : NormedAddCommGroup E
inst✝¹ : NormedSpace ℝ E
𝒜 : Finset (Finset ι)
s : Finset ι
f : ι → E
r : ℝ
inst✝ : DecidableEq ι
hr : 0 < r
hf : ∀ i ∈ ∅, r ≤ ‖f i‖
⊢ ∃ P,
P.parts.card = ∅.card.choose (∅.card / 2) ∧
(∀ 𝒜 ∈ P.parts, ∀ t ∈ 𝒜, t ⊆ ∅) ∧ ∀ 𝒜 ∈ P.parts, (↑𝒜).Pairwise fun u v => r ≤ dist (∑ i ∈ u, f i) (∑ i ∈ v, f i) | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/LittlewoodOfford.lean | Finset.exists_littlewood_offord_partition | [20, 1] | [35, 8] | simp | ι : Type u_1
E : Type u_2
inst✝² : NormedAddCommGroup E
inst✝¹ : NormedSpace ℝ E
𝒜 : Finset (Finset ι)
s : Finset ι
f : ι → E
r : ℝ
inst✝ : DecidableEq ι
hr : 0 < r
hf : ∀ i ∈ ∅, r ≤ ‖f i‖
⊢ (Finpartition.indiscrete ⋯).parts.card = ∅.card.choose (∅.card / 2) ∧
(∀ 𝒜 ∈ (Finpartition.indiscrete ⋯).parts, ∀ t ∈ 𝒜, t ⊆ ∅) ∧
∀ 𝒜 ∈ (Finpartition.indiscrete ⋯).parts, (↑𝒜).Pairwise fun u v => r ≤ dist (∑ i ∈ u, f i) (∑ i ∈ v, f i) | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/LittlewoodOfford.lean | Finset.card_le_of_forall_dist_sum_le | [37, 1] | [47, 73] | obtain ⟨P, hP, _hs, hr⟩ := exists_littlewood_offord_partition hr hf | ι : Type u_1
E : Type u_2
inst✝¹ : NormedAddCommGroup E
inst✝ : NormedSpace ℝ E
𝒜 : Finset (Finset ι)
s : Finset ι
f : ι → E
r : ℝ
hr : 0 < r
h𝒜 : ∀ t ∈ 𝒜, t ⊆ s
hf : ∀ i ∈ s, r ≤ ‖f i‖
h𝒜r : ∀ u ∈ 𝒜, ∀ v ∈ 𝒜, dist (∑ i ∈ u, f i) (∑ i ∈ v, f i) < r
⊢ 𝒜.card ≤ s.card.choose (s.card / 2) | case intro.intro.intro
ι : Type u_1
E : Type u_2
inst✝¹ : NormedAddCommGroup E
inst✝ : NormedSpace ℝ E
𝒜 : Finset (Finset ι)
s : Finset ι
f : ι → E
r : ℝ
hr✝ : 0 < r
h𝒜 : ∀ t ∈ 𝒜, t ⊆ s
hf : ∀ i ∈ s, r ≤ ‖f i‖
h𝒜r : ∀ u ∈ 𝒜, ∀ v ∈ 𝒜, dist (∑ i ∈ u, f i) (∑ i ∈ v, f i) < r
P : Finpartition s.powerset
hP : P.parts.card = s.card.choose (s.card / 2)
_hs : ∀ 𝒜 ∈ P.parts, ∀ t ∈ 𝒜, t ⊆ s
hr : ∀ 𝒜 ∈ P.parts, (↑𝒜).Pairwise fun u v => r ≤ dist (∑ i ∈ u, f i) (∑ i ∈ v, f i)
⊢ 𝒜.card ≤ s.card.choose (s.card / 2) |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/LittlewoodOfford.lean | Finset.card_le_of_forall_dist_sum_le | [37, 1] | [47, 73] | rw [← hP] | case intro.intro.intro
ι : Type u_1
E : Type u_2
inst✝¹ : NormedAddCommGroup E
inst✝ : NormedSpace ℝ E
𝒜 : Finset (Finset ι)
s : Finset ι
f : ι → E
r : ℝ
hr✝ : 0 < r
h𝒜 : ∀ t ∈ 𝒜, t ⊆ s
hf : ∀ i ∈ s, r ≤ ‖f i‖
h𝒜r : ∀ u ∈ 𝒜, ∀ v ∈ 𝒜, dist (∑ i ∈ u, f i) (∑ i ∈ v, f i) < r
P : Finpartition s.powerset
hP : P.parts.card = s.card.choose (s.card / 2)
_hs : ∀ 𝒜 ∈ P.parts, ∀ t ∈ 𝒜, t ⊆ s
hr : ∀ 𝒜 ∈ P.parts, (↑𝒜).Pairwise fun u v => r ≤ dist (∑ i ∈ u, f i) (∑ i ∈ v, f i)
⊢ 𝒜.card ≤ s.card.choose (s.card / 2) | case intro.intro.intro
ι : Type u_1
E : Type u_2
inst✝¹ : NormedAddCommGroup E
inst✝ : NormedSpace ℝ E
𝒜 : Finset (Finset ι)
s : Finset ι
f : ι → E
r : ℝ
hr✝ : 0 < r
h𝒜 : ∀ t ∈ 𝒜, t ⊆ s
hf : ∀ i ∈ s, r ≤ ‖f i‖
h𝒜r : ∀ u ∈ 𝒜, ∀ v ∈ 𝒜, dist (∑ i ∈ u, f i) (∑ i ∈ v, f i) < r
P : Finpartition s.powerset
hP : P.parts.card = s.card.choose (s.card / 2)
_hs : ∀ 𝒜 ∈ P.parts, ∀ t ∈ 𝒜, t ⊆ s
hr : ∀ 𝒜 ∈ P.parts, (↑𝒜).Pairwise fun u v => r ≤ dist (∑ i ∈ u, f i) (∑ i ∈ v, f i)
⊢ 𝒜.card ≤ P.parts.card |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/LittlewoodOfford.lean | Finset.card_le_of_forall_dist_sum_le | [37, 1] | [47, 73] | simpa only [exists_prop] using P.exists_mem (mem_powerset.2 $ h𝒜 _ ht) | case intro.intro.intro
ι : Type u_1
E : Type u_2
inst✝¹ : NormedAddCommGroup E
inst✝ : NormedSpace ℝ E
𝒜 : Finset (Finset ι)
s : Finset ι
f : ι → E
r : ℝ
hr✝ : 0 < r
h𝒜 : ∀ t ∈ 𝒜, t ⊆ s
hf : ∀ i ∈ s, r ≤ ‖f i‖
h𝒜r : ∀ u ∈ 𝒜, ∀ v ∈ 𝒜, dist (∑ i ∈ u, f i) (∑ i ∈ v, f i) < r
P : Finpartition s.powerset
hP : P.parts.card = s.card.choose (s.card / 2)
_hs : ∀ 𝒜 ∈ P.parts, ∀ t ∈ 𝒜, t ⊆ s
hr : ∀ 𝒜 ∈ P.parts, (↑𝒜).Pairwise fun u v => r ≤ dist (∑ i ∈ u, f i) (∑ i ∈ v, f i)
t : Finset ι
ht : t ∈ 𝒜
⊢ ∃ b ∈ P.parts, (fun x x_1 => x ∈ x_1) t b | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Combinatorics/SimpleGraph/Degree.lean | SimpleGraph.degOn_empty | [16, 1] | [17, 63] | simp [degOn] | α : Type u_1
inst✝² : Fintype α
inst✝¹ : DecidableEq α
G : SimpleGraph α
inst✝ : DecidableRel G.Adj
s t : Finset α
a✝ a : α
⊢ G.degOn ∅ a = 0 | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Combinatorics/SimpleGraph/Degree.lean | SimpleGraph.degOn_univ | [19, 1] | [20, 92] | rw [degOn, degree, univ_inter] | α : Type u_1
inst✝² : Fintype α
inst✝¹ : DecidableEq α
G : SimpleGraph α
inst✝ : DecidableRel G.Adj
s t : Finset α
a✝ a : α
⊢ G.degOn univ a = G.degree a | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Combinatorics/SimpleGraph/Degree.lean | SimpleGraph.degOn_union | [23, 1] | [26, 51] | unfold degOn | α : Type u_1
inst✝² : Fintype α
inst✝¹ : DecidableEq α
G : SimpleGraph α
inst✝ : DecidableRel G.Adj
s t : Finset α
a✝ : α
h : Disjoint s t
a : α
⊢ G.degOn (s ∪ t) a = G.degOn s a + G.degOn t a | α : Type u_1
inst✝² : Fintype α
inst✝¹ : DecidableEq α
G : SimpleGraph α
inst✝ : DecidableRel G.Adj
s t : Finset α
a✝ : α
h : Disjoint s t
a : α
⊢ ((s ∪ t) ∩ G.neighborFinset a).card = (s ∩ G.neighborFinset a).card + (t ∩ G.neighborFinset a).card |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Combinatorics/SimpleGraph/Degree.lean | SimpleGraph.degOn_union | [23, 1] | [26, 51] | rw [← card_union_of_disjoint, ← union_inter_distrib_right] | α : Type u_1
inst✝² : Fintype α
inst✝¹ : DecidableEq α
G : SimpleGraph α
inst✝ : DecidableRel G.Adj
s t : Finset α
a✝ : α
h : Disjoint s t
a : α
⊢ ((s ∪ t) ∩ G.neighborFinset a).card = (s ∩ G.neighborFinset a).card + (t ∩ G.neighborFinset a).card | α : Type u_1
inst✝² : Fintype α
inst✝¹ : DecidableEq α
G : SimpleGraph α
inst✝ : DecidableRel G.Adj
s t : Finset α
a✝ : α
h : Disjoint s t
a : α
⊢ Disjoint (s ∩ G.neighborFinset a) (t ∩ G.neighborFinset a) |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Combinatorics/SimpleGraph/Degree.lean | SimpleGraph.degOn_union | [23, 1] | [26, 51] | exact h.mono inter_subset_left inter_subset_left | α : Type u_1
inst✝² : Fintype α
inst✝¹ : DecidableEq α
G : SimpleGraph α
inst✝ : DecidableRel G.Adj
s t : Finset α
a✝ : α
h : Disjoint s t
a : α
⊢ Disjoint (s ∩ G.neighborFinset a) (t ∩ G.neighborFinset a) | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Combinatorics/SimpleGraph/Degree.lean | SimpleGraph.sum_degOn_comm | [29, 1] | [32, 39] | simp_rw [degOn, card_eq_sum_ones, ← sum_indicator_eq_sum_inter] | α : Type u_1
inst✝² : Fintype α
inst✝¹ : DecidableEq α
G : SimpleGraph α
inst✝ : DecidableRel G.Adj
s✝ t✝ : Finset α
a : α
s t : Finset α
⊢ ∑ a ∈ s, G.degOn t a = ∑ a ∈ t, G.degOn s a | α : Type u_1
inst✝² : Fintype α
inst✝¹ : DecidableEq α
G : SimpleGraph α
inst✝ : DecidableRel G.Adj
s✝ t✝ : Finset α
a : α
s t : Finset α
⊢ ∑ x ∈ s, ∑ i ∈ t, (↑(G.neighborFinset x)).indicator (fun x => 1) i =
∑ x ∈ t, ∑ i ∈ s, (↑(G.neighborFinset x)).indicator (fun x => 1) i |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Combinatorics/SimpleGraph/Degree.lean | SimpleGraph.sum_degOn_comm | [29, 1] | [32, 39] | rw [sum_comm] | α : Type u_1
inst✝² : Fintype α
inst✝¹ : DecidableEq α
G : SimpleGraph α
inst✝ : DecidableRel G.Adj
s✝ t✝ : Finset α
a : α
s t : Finset α
⊢ ∑ x ∈ s, ∑ i ∈ t, (↑(G.neighborFinset x)).indicator (fun x => 1) i =
∑ x ∈ t, ∑ i ∈ s, (↑(G.neighborFinset x)).indicator (fun x => 1) i | α : Type u_1
inst✝² : Fintype α
inst✝¹ : DecidableEq α
G : SimpleGraph α
inst✝ : DecidableRel G.Adj
s✝ t✝ : Finset α
a : α
s t : Finset α
⊢ ∑ y ∈ t, ∑ x ∈ s, (↑(G.neighborFinset x)).indicator (fun x => 1) y =
∑ x ∈ t, ∑ i ∈ s, (↑(G.neighborFinset x)).indicator (fun x => 1) i |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Combinatorics/SimpleGraph/Degree.lean | SimpleGraph.sum_degOn_comm | [29, 1] | [32, 39] | simp [Set.indicator_apply, adj_comm] | α : Type u_1
inst✝² : Fintype α
inst✝¹ : DecidableEq α
G : SimpleGraph α
inst✝ : DecidableRel G.Adj
s✝ t✝ : Finset α
a : α
s t : Finset α
⊢ ∑ y ∈ t, ∑ x ∈ s, (↑(G.neighborFinset x)).indicator (fun x => 1) y =
∑ x ∈ t, ∑ i ∈ s, (↑(G.neighborFinset x)).indicator (fun x => 1) i | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/BernoulliSeq.lean | ProbabilityTheory.IsBernoulliSeq.ne_zero | [44, 1] | [46, 41] | rw [← hX.map a, h, Measure.map_zero] | α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : Nonempty α
a : α
h : μ = 0
⊢ (PMF.bernoulli' p ⋯).toMeasure = 0 | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/BernoulliSeq.lean | ProbabilityTheory.IsBernoulliSeq.aemeasurable | [48, 1] | [55, 19] | classical
have : (PMF.bernoulli' p hX.le_one).toMeasure ≠ 0 := NeZero.ne _
rw [← hX.map a, Measure.map] at this
refine' (Ne.dite_ne_right_iff fun hX' ↦ _).1 this
rw [Measure.mapₗ_ne_zero_iff hX'.measurable_mk]
haveI : Nonempty α := ⟨a⟩
exact hX.ne_zero | α : Type u_1
Ω : Type u_2
inst✝ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
a : α
⊢ AEMeasurable (fun ω => a ∈ X ω) μ | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/BernoulliSeq.lean | ProbabilityTheory.IsBernoulliSeq.aemeasurable | [48, 1] | [55, 19] | have : (PMF.bernoulli' p hX.le_one).toMeasure ≠ 0 := NeZero.ne _ | α : Type u_1
Ω : Type u_2
inst✝ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
a : α
⊢ AEMeasurable (fun ω => a ∈ X ω) μ | α : Type u_1
Ω : Type u_2
inst✝ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
a : α
this : (PMF.bernoulli' p ⋯).toMeasure ≠ 0
⊢ AEMeasurable (fun ω => a ∈ X ω) μ |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/BernoulliSeq.lean | ProbabilityTheory.IsBernoulliSeq.aemeasurable | [48, 1] | [55, 19] | rw [← hX.map a, Measure.map] at this | α : Type u_1
Ω : Type u_2
inst✝ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
a : α
this : (PMF.bernoulli' p ⋯).toMeasure ≠ 0
⊢ AEMeasurable (fun ω => a ∈ X ω) μ | α : Type u_1
Ω : Type u_2
inst✝ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
a : α
this :
(if hf : AEMeasurable (fun ω => a ∈ X ω) μ then (Measure.mapₗ (AEMeasurable.mk (fun ω => a ∈ X ω) hf)) μ else 0) ≠ 0
⊢ AEMeasurable (fun ω => a ∈ X ω) μ |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/BernoulliSeq.lean | ProbabilityTheory.IsBernoulliSeq.aemeasurable | [48, 1] | [55, 19] | refine' (Ne.dite_ne_right_iff fun hX' ↦ _).1 this | α : Type u_1
Ω : Type u_2
inst✝ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
a : α
this :
(if hf : AEMeasurable (fun ω => a ∈ X ω) μ then (Measure.mapₗ (AEMeasurable.mk (fun ω => a ∈ X ω) hf)) μ else 0) ≠ 0
⊢ AEMeasurable (fun ω => a ∈ X ω) μ | α : Type u_1
Ω : Type u_2
inst✝ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
a : α
this :
(if hf : AEMeasurable (fun ω => a ∈ X ω) μ then (Measure.mapₗ (AEMeasurable.mk (fun ω => a ∈ X ω) hf)) μ else 0) ≠ 0
hX' : AEMeasurable (fun ω => a ∈ X ω) μ
⊢ (Measure.mapₗ (AEMeasurable.mk (fun ω => a ∈ X ω) hX')) μ ≠ 0 |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/BernoulliSeq.lean | ProbabilityTheory.IsBernoulliSeq.aemeasurable | [48, 1] | [55, 19] | rw [Measure.mapₗ_ne_zero_iff hX'.measurable_mk] | α : Type u_1
Ω : Type u_2
inst✝ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
a : α
this :
(if hf : AEMeasurable (fun ω => a ∈ X ω) μ then (Measure.mapₗ (AEMeasurable.mk (fun ω => a ∈ X ω) hf)) μ else 0) ≠ 0
hX' : AEMeasurable (fun ω => a ∈ X ω) μ
⊢ (Measure.mapₗ (AEMeasurable.mk (fun ω => a ∈ X ω) hX')) μ ≠ 0 | α : Type u_1
Ω : Type u_2
inst✝ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
a : α
this :
(if hf : AEMeasurable (fun ω => a ∈ X ω) μ then (Measure.mapₗ (AEMeasurable.mk (fun ω => a ∈ X ω) hf)) μ else 0) ≠ 0
hX' : AEMeasurable (fun ω => a ∈ X ω) μ
⊢ μ ≠ 0 |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/BernoulliSeq.lean | ProbabilityTheory.IsBernoulliSeq.aemeasurable | [48, 1] | [55, 19] | haveI : Nonempty α := ⟨a⟩ | α : Type u_1
Ω : Type u_2
inst✝ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
a : α
this :
(if hf : AEMeasurable (fun ω => a ∈ X ω) μ then (Measure.mapₗ (AEMeasurable.mk (fun ω => a ∈ X ω) hf)) μ else 0) ≠ 0
hX' : AEMeasurable (fun ω => a ∈ X ω) μ
⊢ μ ≠ 0 | α : Type u_1
Ω : Type u_2
inst✝ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
a : α
this✝ :
(if hf : AEMeasurable (fun ω => a ∈ X ω) μ then (Measure.mapₗ (AEMeasurable.mk (fun ω => a ∈ X ω) hf)) μ else 0) ≠ 0
hX' : AEMeasurable (fun ω => a ∈ X ω) μ
this : Nonempty α
⊢ μ ≠ 0 |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/BernoulliSeq.lean | ProbabilityTheory.IsBernoulliSeq.aemeasurable | [48, 1] | [55, 19] | exact hX.ne_zero | α : Type u_1
Ω : Type u_2
inst✝ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
a : α
this✝ :
(if hf : AEMeasurable (fun ω => a ∈ X ω) μ then (Measure.mapₗ (AEMeasurable.mk (fun ω => a ∈ X ω) hf)) μ else 0) ≠ 0
hX' : AEMeasurable (fun ω => a ∈ X ω) μ
this : Nonempty α
⊢ μ ≠ 0 | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/BernoulliSeq.lean | ProbabilityTheory.IsBernoulliSeq.nullMeasurableSet | [57, 1] | [59, 89] | rw [(by ext; simp : {ω | a ∈ X ω} = (fun ω ↦ a ∈ X ω) ⁻¹' {True})] | α : Type u_1
Ω : Type u_2
inst✝ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
a : α
⊢ NullMeasurableSet {ω | a ∈ X ω} μ | α : Type u_1
Ω : Type u_2
inst✝ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
a : α
⊢ NullMeasurableSet ((fun ω => a ∈ X ω) ⁻¹' {True}) μ |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/BernoulliSeq.lean | ProbabilityTheory.IsBernoulliSeq.nullMeasurableSet | [57, 1] | [59, 89] | exact (hX.aemeasurable a).nullMeasurableSet_preimage MeasurableSpace.measurableSet_top | α : Type u_1
Ω : Type u_2
inst✝ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
a : α
⊢ NullMeasurableSet ((fun ω => a ∈ X ω) ⁻¹' {True}) μ | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/BernoulliSeq.lean | ProbabilityTheory.IsBernoulliSeq.nullMeasurableSet | [57, 1] | [59, 89] | ext | α : Type u_1
Ω : Type u_2
inst✝ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
a : α
⊢ {ω | a ∈ X ω} = (fun ω => a ∈ X ω) ⁻¹' {True} | case h
α : Type u_1
Ω : Type u_2
inst✝ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
a : α
x✝ : Ω
⊢ x✝ ∈ {ω | a ∈ X ω} ↔ x✝ ∈ (fun ω => a ∈ X ω) ⁻¹' {True} |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/BernoulliSeq.lean | ProbabilityTheory.IsBernoulliSeq.nullMeasurableSet | [57, 1] | [59, 89] | simp | case h
α : Type u_1
Ω : Type u_2
inst✝ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
a : α
x✝ : Ω
⊢ x✝ ∈ {ω | a ∈ X ω} ↔ x✝ ∈ (fun ω => a ∈ X ω) ⁻¹' {True} | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/BernoulliSeq.lean | ProbabilityTheory.IsBernoulliSeq.meas_apply | [66, 1] | [71, 9] | rw [(_ : {ω | a ∈ X ω} = (fun ω ↦ a ∈ X ω) ⁻¹' {True}),
← Measure.map_apply_of_aemeasurable (hX.aemeasurable a) MeasurableSpace.measurableSet_top] | α : Type u_1
Ω : Type u_2
inst✝ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
a : α
⊢ μ {ω | a ∈ X ω} = ↑p | α : Type u_1
Ω : Type u_2
inst✝ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
a : α
⊢ (Measure.map (fun ω => a ∈ X ω) μ) {True} = ↑p
α : Type u_1
Ω : Type u_2
inst✝ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
a : α
⊢ {ω | a ∈ X ω} = (fun ω => a ∈ X ω) ⁻¹' {True} |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/BernoulliSeq.lean | ProbabilityTheory.IsBernoulliSeq.meas_apply | [66, 1] | [71, 9] | simp [hX.map] | α : Type u_1
Ω : Type u_2
inst✝ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
a : α
⊢ (Measure.map (fun ω => a ∈ X ω) μ) {True} = ↑p | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/BernoulliSeq.lean | ProbabilityTheory.IsBernoulliSeq.meas_apply | [66, 1] | [71, 9] | ext ω | α : Type u_1
Ω : Type u_2
inst✝ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
a : α
⊢ {ω | a ∈ X ω} = (fun ω => a ∈ X ω) ⁻¹' {True} | case h
α : Type u_1
Ω : Type u_2
inst✝ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
a : α
ω : Ω
⊢ ω ∈ {ω | a ∈ X ω} ↔ ω ∈ (fun ω => a ∈ X ω) ⁻¹' {True} |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/BernoulliSeq.lean | ProbabilityTheory.IsBernoulliSeq.meas_apply | [66, 1] | [71, 9] | simp | case h
α : Type u_1
Ω : Type u_2
inst✝ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
a : α
ω : Ω
⊢ ω ∈ {ω | a ∈ X ω} ↔ ω ∈ (fun ω => a ∈ X ω) ⁻¹' {True} | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/BernoulliSeq.lean | ProbabilityTheory.IsBernoulliSeq.meas | [75, 1] | [92, 43] | simp_rw [ext_iff, setOf_forall] | α : Type u_1
Ω : Type u_2
inst✝² : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝¹ : IsProbabilityMeasure μ
inst✝ : Fintype α
s : Finset α
⊢ μ {ω | {a | a ∈ X ω} = ↑s} = ↑p ^ s.card * (1 - ↑p) ^ (card α - s.card) | α : Type u_1
Ω : Type u_2
inst✝² : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝¹ : IsProbabilityMeasure μ
inst✝ : Fintype α
s : Finset α
⊢ μ (⋂ i, {x | i ∈ {a | a ∈ X x} ↔ i ∈ ↑s}) = ↑p ^ s.card * (1 - ↑p) ^ (card α - s.card) |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/BernoulliSeq.lean | ProbabilityTheory.IsBernoulliSeq.meas | [75, 1] | [92, 43] | rw [hX.iIndepFun.meas_iInter, ← s.prod_mul_prod_compl, Finset.prod_eq_pow_card,
Finset.prod_eq_pow_card, Finset.card_compl] | α : Type u_1
Ω : Type u_2
inst✝² : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝¹ : IsProbabilityMeasure μ
inst✝ : Fintype α
s : Finset α
⊢ μ (⋂ i, {x | i ∈ {a | a ∈ X x} ↔ i ∈ ↑s}) = ↑p ^ s.card * (1 - ↑p) ^ (card α - s.card) | α : Type u_1
Ω : Type u_2
inst✝² : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝¹ : IsProbabilityMeasure μ
inst✝ : Fintype α
s : Finset α
⊢ ∀ a ∈ sᶜ, μ {x | a ∈ {a | a ∈ X x} ↔ a ∈ ↑s} = 1 - ↑p
α : Type u_1
Ω : Type u_2
inst✝² : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝¹ : IsProbabilityMeasure μ
inst✝ : Fintype α
s : Finset α
⊢ ∀ a ∈ s, μ {x | a ∈ {a | a ∈ X x} ↔ a ∈ ↑s} = ↑p
α : Type u_1
Ω : Type u_2
inst✝² : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝¹ : IsProbabilityMeasure μ
inst✝ : Fintype α
s : Finset α
⊢ ∀ (i : α), MeasurableSet {x | i ∈ {a | a ∈ X x} ↔ i ∈ ↑s} |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/BernoulliSeq.lean | ProbabilityTheory.IsBernoulliSeq.meas | [75, 1] | [92, 43] | rintro a | α : Type u_1
Ω : Type u_2
inst✝² : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝¹ : IsProbabilityMeasure μ
inst✝ : Fintype α
s : Finset α
⊢ ∀ (i : α), MeasurableSet {x | i ∈ {a | a ∈ X x} ↔ i ∈ ↑s} | α : Type u_1
Ω : Type u_2
inst✝² : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝¹ : IsProbabilityMeasure μ
inst✝ : Fintype α
s : Finset α
a : α
⊢ MeasurableSet {x | a ∈ {a | a ∈ X x} ↔ a ∈ ↑s} |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/BernoulliSeq.lean | ProbabilityTheory.IsBernoulliSeq.meas | [75, 1] | [92, 43] | by_cases a ∈ s | α : Type u_1
Ω : Type u_2
inst✝² : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝¹ : IsProbabilityMeasure μ
inst✝ : Fintype α
s : Finset α
a : α
⊢ MeasurableSet {x | a ∈ {a | a ∈ X x} ↔ a ∈ ↑s} | case pos
α : Type u_1
Ω : Type u_2
inst✝² : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝¹ : IsProbabilityMeasure μ
inst✝ : Fintype α
s : Finset α
a : α
h✝ : a ∈ s
⊢ MeasurableSet {x | a ∈ {a | a ∈ X x} ↔ a ∈ ↑s}
case neg
α : Type u_1
Ω : Type u_2
inst✝² : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝¹ : IsProbabilityMeasure μ
inst✝ : Fintype α
s : Finset α
a : α
h✝ : a ∉ s
⊢ MeasurableSet {x | a ∈ {a | a ∈ X x} ↔ a ∈ ↑s} |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/BernoulliSeq.lean | ProbabilityTheory.IsBernoulliSeq.meas | [75, 1] | [92, 43] | rintro a hi | α : Type u_1
Ω : Type u_2
inst✝² : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝¹ : IsProbabilityMeasure μ
inst✝ : Fintype α
s : Finset α
⊢ ∀ a ∈ sᶜ, μ {x | a ∈ {a | a ∈ X x} ↔ a ∈ ↑s} = 1 - ↑p | α : Type u_1
Ω : Type u_2
inst✝² : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝¹ : IsProbabilityMeasure μ
inst✝ : Fintype α
s : Finset α
a : α
hi : a ∈ sᶜ
⊢ μ {x | a ∈ {a | a ∈ X x} ↔ a ∈ ↑s} = 1 - ↑p |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/BernoulliSeq.lean | ProbabilityTheory.IsBernoulliSeq.meas | [75, 1] | [92, 43] | rw [Finset.mem_compl] at hi | α : Type u_1
Ω : Type u_2
inst✝² : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝¹ : IsProbabilityMeasure μ
inst✝ : Fintype α
s : Finset α
a : α
hi : a ∈ sᶜ
⊢ μ {x | a ∈ {a | a ∈ X x} ↔ a ∈ ↑s} = 1 - ↑p | α : Type u_1
Ω : Type u_2
inst✝² : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝¹ : IsProbabilityMeasure μ
inst✝ : Fintype α
s : Finset α
a : α
hi : a ∉ s
⊢ μ {x | a ∈ {a | a ∈ X x} ↔ a ∈ ↑s} = 1 - ↑p |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/BernoulliSeq.lean | ProbabilityTheory.IsBernoulliSeq.meas | [75, 1] | [92, 43] | simp only [hi, ← compl_setOf, prob_compl_eq_one_sub₀, mem_setOf_eq, Finset.mem_coe,
iff_false_iff, hX.nullMeasurableSet, hX.meas_apply] | α : Type u_1
Ω : Type u_2
inst✝² : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝¹ : IsProbabilityMeasure μ
inst✝ : Fintype α
s : Finset α
a : α
hi : a ∉ s
⊢ μ {x | a ∈ {a | a ∈ X x} ↔ a ∈ ↑s} = 1 - ↑p | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/BernoulliSeq.lean | ProbabilityTheory.IsBernoulliSeq.meas | [75, 1] | [92, 43] | rintro a hi | α : Type u_1
Ω : Type u_2
inst✝² : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝¹ : IsProbabilityMeasure μ
inst✝ : Fintype α
s : Finset α
⊢ ∀ a ∈ s, μ {x | a ∈ {a | a ∈ X x} ↔ a ∈ ↑s} = ↑p | α : Type u_1
Ω : Type u_2
inst✝² : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝¹ : IsProbabilityMeasure μ
inst✝ : Fintype α
s : Finset α
a : α
hi : a ∈ s
⊢ μ {x | a ∈ {a | a ∈ X x} ↔ a ∈ ↑s} = ↑p |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/BernoulliSeq.lean | ProbabilityTheory.IsBernoulliSeq.meas | [75, 1] | [92, 43] | simp only [hi, mem_setOf_eq, Finset.mem_coe, iff_true_iff, hX.meas_apply] | α : Type u_1
Ω : Type u_2
inst✝² : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝¹ : IsProbabilityMeasure μ
inst✝ : Fintype α
s : Finset α
a : α
hi : a ∈ s
⊢ μ {x | a ∈ {a | a ∈ X x} ↔ a ∈ ↑s} = ↑p | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/BernoulliSeq.lean | ProbabilityTheory.IsBernoulliSeq.meas | [75, 1] | [92, 43] | simp only [mem_setOf_eq, Finset.mem_coe, iff_true_iff, *] | case pos
α : Type u_1
Ω : Type u_2
inst✝² : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝¹ : IsProbabilityMeasure μ
inst✝ : Fintype α
s : Finset α
a : α
h✝ : a ∈ s
⊢ MeasurableSet {x | a ∈ {a | a ∈ X x} ↔ a ∈ ↑s} | case pos
α : Type u_1
Ω : Type u_2
inst✝² : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝¹ : IsProbabilityMeasure μ
inst✝ : Fintype α
s : Finset α
a : α
h✝ : a ∈ s
⊢ MeasurableSet {x | a ∈ X x} |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/BernoulliSeq.lean | ProbabilityTheory.IsBernoulliSeq.meas | [75, 1] | [92, 43] | exact ⟨{True}, trivial, by ext; simp⟩ | case pos
α : Type u_1
Ω : Type u_2
inst✝² : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝¹ : IsProbabilityMeasure μ
inst✝ : Fintype α
s : Finset α
a : α
h✝ : a ∈ s
⊢ MeasurableSet {x | a ∈ X x} | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/BernoulliSeq.lean | ProbabilityTheory.IsBernoulliSeq.meas | [75, 1] | [92, 43] | ext | α : Type u_1
Ω : Type u_2
inst✝² : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝¹ : IsProbabilityMeasure μ
inst✝ : Fintype α
s : Finset α
a : α
h✝ : a ∈ s
⊢ (fun ω => a ∈ X ω) ⁻¹' {True} = {x | a ∈ X x} | case h
α : Type u_1
Ω : Type u_2
inst✝² : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝¹ : IsProbabilityMeasure μ
inst✝ : Fintype α
s : Finset α
a : α
h✝ : a ∈ s
x✝ : Ω
⊢ x✝ ∈ (fun ω => a ∈ X ω) ⁻¹' {True} ↔ x✝ ∈ {x | a ∈ X x} |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/BernoulliSeq.lean | ProbabilityTheory.IsBernoulliSeq.meas | [75, 1] | [92, 43] | simp | case h
α : Type u_1
Ω : Type u_2
inst✝² : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝¹ : IsProbabilityMeasure μ
inst✝ : Fintype α
s : Finset α
a : α
h✝ : a ∈ s
x✝ : Ω
⊢ x✝ ∈ (fun ω => a ∈ X ω) ⁻¹' {True} ↔ x✝ ∈ {x | a ∈ X x} | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/BernoulliSeq.lean | ProbabilityTheory.IsBernoulliSeq.meas | [75, 1] | [92, 43] | simp only [mem_setOf_eq, Finset.mem_coe, iff_false_iff, *] | case neg
α : Type u_1
Ω : Type u_2
inst✝² : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝¹ : IsProbabilityMeasure μ
inst✝ : Fintype α
s : Finset α
a : α
h✝ : a ∉ s
⊢ MeasurableSet {x | a ∈ {a | a ∈ X x} ↔ a ∈ ↑s} | case neg
α : Type u_1
Ω : Type u_2
inst✝² : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝¹ : IsProbabilityMeasure μ
inst✝ : Fintype α
s : Finset α
a : α
h✝ : a ∉ s
⊢ MeasurableSet {x | a ∉ X x} |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/BernoulliSeq.lean | ProbabilityTheory.IsBernoulliSeq.meas | [75, 1] | [92, 43] | exact ⟨{False}, trivial, by ext; simp⟩ | case neg
α : Type u_1
Ω : Type u_2
inst✝² : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝¹ : IsProbabilityMeasure μ
inst✝ : Fintype α
s : Finset α
a : α
h✝ : a ∉ s
⊢ MeasurableSet {x | a ∉ X x} | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/BernoulliSeq.lean | ProbabilityTheory.IsBernoulliSeq.meas | [75, 1] | [92, 43] | ext | α : Type u_1
Ω : Type u_2
inst✝² : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝¹ : IsProbabilityMeasure μ
inst✝ : Fintype α
s : Finset α
a : α
h✝ : a ∉ s
⊢ (fun ω => a ∈ X ω) ⁻¹' {False} = {x | a ∉ X x} | case h
α : Type u_1
Ω : Type u_2
inst✝² : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝¹ : IsProbabilityMeasure μ
inst✝ : Fintype α
s : Finset α
a : α
h✝ : a ∉ s
x✝ : Ω
⊢ x✝ ∈ (fun ω => a ∈ X ω) ⁻¹' {False} ↔ x✝ ∈ {x | a ∉ X x} |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/BernoulliSeq.lean | ProbabilityTheory.IsBernoulliSeq.meas | [75, 1] | [92, 43] | simp | case h
α : Type u_1
Ω : Type u_2
inst✝² : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝¹ : IsProbabilityMeasure μ
inst✝ : Fintype α
s : Finset α
a : α
h✝ : a ∉ s
x✝ : Ω
⊢ x✝ ∈ (fun ω => a ∈ X ω) ⁻¹' {False} ↔ x✝ ∈ {x | a ∉ X x} | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/BernoulliSeq.lean | ProbabilityTheory.IsBernoulliSeq.compl | [94, 1] | [104, 66] | simp only [iIndepFun_iff, mem_compl_iff, MeasurableSpace.comap_not] | α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
⊢ iIndepFun inferInstance (fun a ω => a ∈ (X ω)ᶜ) μ | α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
⊢ ∀ (s : Finset α) {f' : α → Set Ω}, (∀ i ∈ s, MeasurableSet (f' i)) → μ (⋂ i ∈ s, f' i) = ∏ i ∈ s, μ (f' i) |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/BernoulliSeq.lean | ProbabilityTheory.IsBernoulliSeq.compl | [94, 1] | [104, 66] | exact (iIndepFun_iff _ _ _).1 hX.iIndepFun | α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
⊢ ∀ (s : Finset α) {f' : α → Set Ω}, (∀ i ∈ s, MeasurableSet (f' i)) → μ (⋂ i ∈ s, f' i) = ∏ i ∈ s, μ (f' i) | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/BernoulliSeq.lean | ProbabilityTheory.IsBernoulliSeq.compl | [94, 1] | [104, 66] | have : Measurable Not := fun _ _ ↦ trivial | α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
a : α
⊢ Measure.map (fun ω => a ∈ (X ω)ᶜ) μ = (PMF.bernoulli' (1 - p) ⋯).toMeasure | α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
a : α
this : Measurable Not
⊢ Measure.map (fun ω => a ∈ (X ω)ᶜ) μ = (PMF.bernoulli' (1 - p) ⋯).toMeasure |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/BernoulliSeq.lean | ProbabilityTheory.IsBernoulliSeq.compl | [94, 1] | [104, 66] | refine' (this.aemeasurable.map_map_of_aemeasurable (hX.aemeasurable _)).symm.trans _ | α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
a : α
this : Measurable Not
⊢ Measure.map (fun ω => a ∈ (X ω)ᶜ) μ = (PMF.bernoulli' (1 - p) ⋯).toMeasure | α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
a : α
this : Measurable Not
⊢ Measure.map Not (Measure.map (fun ω => a ∈ X ω) μ) = (PMF.bernoulli' (1 - p) ⋯).toMeasure |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/BernoulliSeq.lean | ProbabilityTheory.IsBernoulliSeq.compl | [94, 1] | [104, 66] | rw [hX.map, PMF.map_toMeasure _ this, PMF.map_not_bernoulli'] | α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
a : α
this : Measurable Not
⊢ Measure.map Not (Measure.map (fun ω => a ∈ X ω) μ) = (PMF.bernoulli' (1 - p) ⋯).toMeasure | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/BernoulliSeq.lean | ProbabilityTheory.IsBernoulliSeq.inter | [106, 1] | [128, 17] | refine' iIndepSet.Indep_comap ((iIndepSet_iff_meas_iInter fun i ↦ _).2 _) | α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
⊢ iIndepFun inferInstance (fun a ω => a ∈ X ω ∩ Y ω) μ | case refine'_1
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
i : α
⊢ MeasurableSet fun ω => (X ω ∩ Y ω) i
case refine'_2
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
⊢ ∀ (t : Finset α), μ (⋂ i ∈ t, fun ω => (X ω ∩ Y ω) i) = ∏ i ∈ t, μ fun ω => (X ω ∩ Y ω) i |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/BernoulliSeq.lean | ProbabilityTheory.IsBernoulliSeq.inter | [106, 1] | [128, 17] | refine' MeasurableSet.inter _ _ | case refine'_1
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
i : α
⊢ MeasurableSet fun ω => (X ω ∩ Y ω) i
case refine'_2
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
⊢ ∀ (t : Finset α), μ (⋂ i ∈ t, fun ω => (X ω ∩ Y ω) i) = ∏ i ∈ t, μ fun ω => (X ω ∩ Y ω) i | case refine'_1.refine'_1
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
i : α
⊢ MeasurableSet fun ω => X ω i
case refine'_1.refine'_2
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
i : α
⊢ MeasurableSet fun ω => Y ω i
case refine'_2
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
⊢ ∀ (t : Finset α), μ (⋂ i ∈ t, fun ω => (X ω ∩ Y ω) i) = ∏ i ∈ t, μ fun ω => (X ω ∩ Y ω) i |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/BernoulliSeq.lean | ProbabilityTheory.IsBernoulliSeq.inter | [106, 1] | [128, 17] | sorry | case refine'_1.refine'_1
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
i : α
⊢ MeasurableSet fun ω => X ω i
case refine'_1.refine'_2
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
i : α
⊢ MeasurableSet fun ω => Y ω i
case refine'_2
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
⊢ ∀ (t : Finset α), μ (⋂ i ∈ t, fun ω => (X ω ∩ Y ω) i) = ∏ i ∈ t, μ fun ω => (X ω ∩ Y ω) i | case refine'_1.refine'_2
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
i : α
⊢ MeasurableSet fun ω => Y ω i
case refine'_2
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
⊢ ∀ (t : Finset α), μ (⋂ i ∈ t, fun ω => (X ω ∩ Y ω) i) = ∏ i ∈ t, μ fun ω => (X ω ∩ Y ω) i |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/BernoulliSeq.lean | ProbabilityTheory.IsBernoulliSeq.inter | [106, 1] | [128, 17] | sorry | case refine'_1.refine'_2
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
i : α
⊢ MeasurableSet fun ω => Y ω i
case refine'_2
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
⊢ ∀ (t : Finset α), μ (⋂ i ∈ t, fun ω => (X ω ∩ Y ω) i) = ∏ i ∈ t, μ fun ω => (X ω ∩ Y ω) i | case refine'_2
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
⊢ ∀ (t : Finset α), μ (⋂ i ∈ t, fun ω => (X ω ∩ Y ω) i) = ∏ i ∈ t, μ fun ω => (X ω ∩ Y ω) i |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/BernoulliSeq.lean | ProbabilityTheory.IsBernoulliSeq.inter | [106, 1] | [128, 17] | refine' fun s ↦ _ | case refine'_2
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
⊢ ∀ (t : Finset α), μ (⋂ i ∈ t, fun ω => (X ω ∩ Y ω) i) = ∏ i ∈ t, μ fun ω => (X ω ∩ Y ω) i | case refine'_2
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
s : Finset α
⊢ μ (⋂ i ∈ s, fun ω => (X ω ∩ Y ω) i) = ∏ i ∈ s, μ fun ω => (X ω ∩ Y ω) i |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/BernoulliSeq.lean | ProbabilityTheory.IsBernoulliSeq.inter | [106, 1] | [128, 17] | change μ (⋂ i ∈ s, {ω | X ω i} ∩ {ω | Y ω i}) = s.prod fun i ↦ μ ({ω | X ω i} ∩ {ω | Y ω i}) | case refine'_2
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
s : Finset α
⊢ μ (⋂ i ∈ s, fun ω => (X ω ∩ Y ω) i) = ∏ i ∈ s, μ fun ω => (X ω ∩ Y ω) i | case refine'_2
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
s : Finset α
⊢ μ (⋂ i ∈ s, {ω | X ω i} ∩ {ω | Y ω i}) = ∏ i ∈ s, μ ({ω | X ω i} ∩ {ω | Y ω i}) |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/BernoulliSeq.lean | ProbabilityTheory.IsBernoulliSeq.inter | [106, 1] | [128, 17] | simp_rw [iInter_inter_distrib] | case refine'_2
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
s : Finset α
⊢ μ (⋂ i ∈ s, {ω | X ω i} ∩ {ω | Y ω i}) = ∏ i ∈ s, μ ({ω | X ω i} ∩ {ω | Y ω i}) | case refine'_2
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
s : Finset α
⊢ μ ((⋂ i ∈ s, {ω | X ω i}) ∩ ⋂ i ∈ s, {ω | Y ω i}) = ∏ i ∈ s, μ ({ω | X ω i} ∩ {ω | Y ω i}) |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/BernoulliSeq.lean | ProbabilityTheory.IsBernoulliSeq.inter | [106, 1] | [128, 17] | rw [h.meas_inter, hX.iIndepFun.meas_biInter, hY.iIndepFun.meas_biInter,
← Finset.prod_mul_distrib] | case refine'_2
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
s : Finset α
⊢ μ ((⋂ i ∈ s, {ω | X ω i}) ∩ ⋂ i ∈ s, {ω | Y ω i}) = ∏ i ∈ s, μ ({ω | X ω i} ∩ {ω | Y ω i}) | case refine'_2
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
s : Finset α
⊢ ∏ x ∈ s, μ {ω | X ω x} * μ {ω | Y ω x} = ∏ i ∈ s, μ ({ω | X ω i} ∩ {ω | Y ω i})
case refine'_2
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
s : Finset α
⊢ ∀ i ∈ s, MeasurableSet {ω | Y ω i}
case refine'_2
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
s : Finset α
⊢ ∀ i ∈ s, MeasurableSet {ω | X ω i}
case refine'_2.hs
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
s : Finset α
⊢ MeasurableSet (⋂ i ∈ s, {ω | X ω i})
case refine'_2.ht
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
s : Finset α
⊢ MeasurableSet (⋂ i ∈ s, {ω | Y ω i}) |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/BernoulliSeq.lean | ProbabilityTheory.IsBernoulliSeq.inter | [106, 1] | [128, 17] | refine' Finset.prod_congr rfl fun i hi ↦ (h.meas_inter _ _).symm | case refine'_2
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
s : Finset α
⊢ ∏ x ∈ s, μ {ω | X ω x} * μ {ω | Y ω x} = ∏ i ∈ s, μ ({ω | X ω i} ∩ {ω | Y ω i})
case refine'_2
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
s : Finset α
⊢ ∀ i ∈ s, MeasurableSet {ω | Y ω i}
case refine'_2
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
s : Finset α
⊢ ∀ i ∈ s, MeasurableSet {ω | X ω i}
case refine'_2.hs
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
s : Finset α
⊢ MeasurableSet (⋂ i ∈ s, {ω | X ω i})
case refine'_2.ht
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
s : Finset α
⊢ MeasurableSet (⋂ i ∈ s, {ω | Y ω i}) | case refine'_2.refine'_1
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
s : Finset α
i : α
hi : i ∈ s
⊢ MeasurableSet {ω | X ω i}
case refine'_2.refine'_2
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
s : Finset α
i : α
hi : i ∈ s
⊢ MeasurableSet {ω | Y ω i}
case refine'_2
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
s : Finset α
⊢ ∀ i ∈ s, MeasurableSet {ω | Y ω i}
case refine'_2
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
s : Finset α
⊢ ∀ i ∈ s, MeasurableSet {ω | X ω i}
case refine'_2.hs
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
s : Finset α
⊢ MeasurableSet (⋂ i ∈ s, {ω | X ω i})
case refine'_2.ht
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
s : Finset α
⊢ MeasurableSet (⋂ i ∈ s, {ω | Y ω i}) |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/BernoulliSeq.lean | ProbabilityTheory.IsBernoulliSeq.inter | [106, 1] | [128, 17] | sorry | case refine'_2.refine'_1
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
s : Finset α
i : α
hi : i ∈ s
⊢ MeasurableSet {ω | X ω i}
case refine'_2.refine'_2
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
s : Finset α
i : α
hi : i ∈ s
⊢ MeasurableSet {ω | Y ω i}
case refine'_2
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
s : Finset α
⊢ ∀ i ∈ s, MeasurableSet {ω | Y ω i}
case refine'_2
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
s : Finset α
⊢ ∀ i ∈ s, MeasurableSet {ω | X ω i}
case refine'_2.hs
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
s : Finset α
⊢ MeasurableSet (⋂ i ∈ s, {ω | X ω i})
case refine'_2.ht
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
s : Finset α
⊢ MeasurableSet (⋂ i ∈ s, {ω | Y ω i}) | case refine'_2.refine'_2
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
s : Finset α
i : α
hi : i ∈ s
⊢ MeasurableSet {ω | Y ω i}
case refine'_2
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
s : Finset α
⊢ ∀ i ∈ s, MeasurableSet {ω | Y ω i}
case refine'_2
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
s : Finset α
⊢ ∀ i ∈ s, MeasurableSet {ω | X ω i}
case refine'_2.hs
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
s : Finset α
⊢ MeasurableSet (⋂ i ∈ s, {ω | X ω i})
case refine'_2.ht
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
s : Finset α
⊢ MeasurableSet (⋂ i ∈ s, {ω | Y ω i}) |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/BernoulliSeq.lean | ProbabilityTheory.IsBernoulliSeq.inter | [106, 1] | [128, 17] | sorry | case refine'_2.refine'_2
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
s : Finset α
i : α
hi : i ∈ s
⊢ MeasurableSet {ω | Y ω i}
case refine'_2
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
s : Finset α
⊢ ∀ i ∈ s, MeasurableSet {ω | Y ω i}
case refine'_2
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
s : Finset α
⊢ ∀ i ∈ s, MeasurableSet {ω | X ω i}
case refine'_2.hs
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
s : Finset α
⊢ MeasurableSet (⋂ i ∈ s, {ω | X ω i})
case refine'_2.ht
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
s : Finset α
⊢ MeasurableSet (⋂ i ∈ s, {ω | Y ω i}) | case refine'_2
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
s : Finset α
⊢ ∀ i ∈ s, MeasurableSet {ω | Y ω i}
case refine'_2
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
s : Finset α
⊢ ∀ i ∈ s, MeasurableSet {ω | X ω i}
case refine'_2.hs
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
s : Finset α
⊢ MeasurableSet (⋂ i ∈ s, {ω | X ω i})
case refine'_2.ht
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
s : Finset α
⊢ MeasurableSet (⋂ i ∈ s, {ω | Y ω i}) |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/BernoulliSeq.lean | ProbabilityTheory.IsBernoulliSeq.inter | [106, 1] | [128, 17] | sorry | case refine'_2
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
s : Finset α
⊢ ∀ i ∈ s, MeasurableSet {ω | Y ω i}
case refine'_2
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
s : Finset α
⊢ ∀ i ∈ s, MeasurableSet {ω | X ω i}
case refine'_2.hs
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
s : Finset α
⊢ MeasurableSet (⋂ i ∈ s, {ω | X ω i})
case refine'_2.ht
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
s : Finset α
⊢ MeasurableSet (⋂ i ∈ s, {ω | Y ω i}) | case refine'_2
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
s : Finset α
⊢ ∀ i ∈ s, MeasurableSet {ω | X ω i}
case refine'_2.hs
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
s : Finset α
⊢ MeasurableSet (⋂ i ∈ s, {ω | X ω i})
case refine'_2.ht
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
s : Finset α
⊢ MeasurableSet (⋂ i ∈ s, {ω | Y ω i}) |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/BernoulliSeq.lean | ProbabilityTheory.IsBernoulliSeq.inter | [106, 1] | [128, 17] | sorry | case refine'_2
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
s : Finset α
⊢ ∀ i ∈ s, MeasurableSet {ω | X ω i}
case refine'_2.hs
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
s : Finset α
⊢ MeasurableSet (⋂ i ∈ s, {ω | X ω i})
case refine'_2.ht
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
s : Finset α
⊢ MeasurableSet (⋂ i ∈ s, {ω | Y ω i}) | case refine'_2.hs
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
s : Finset α
⊢ MeasurableSet (⋂ i ∈ s, {ω | X ω i})
case refine'_2.ht
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
s : Finset α
⊢ MeasurableSet (⋂ i ∈ s, {ω | Y ω i}) |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/BernoulliSeq.lean | ProbabilityTheory.IsBernoulliSeq.inter | [106, 1] | [128, 17] | sorry | case refine'_2.hs
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
s : Finset α
⊢ MeasurableSet (⋂ i ∈ s, {ω | X ω i})
case refine'_2.ht
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
s : Finset α
⊢ MeasurableSet (⋂ i ∈ s, {ω | Y ω i}) | case refine'_2.ht
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
s : Finset α
⊢ MeasurableSet (⋂ i ∈ s, {ω | Y ω i}) |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/BernoulliSeq.lean | ProbabilityTheory.IsBernoulliSeq.inter | [106, 1] | [128, 17] | sorry | case refine'_2.ht
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
s : Finset α
⊢ MeasurableSet (⋂ i ∈ s, {ω | Y ω i}) | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/BernoulliSeq.lean | ProbabilityTheory.IsBernoulliSeq.union | [130, 1] | [141, 68] | convert (hX.compl.inter hY.compl _).compl using 1 | α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
⊢ IsBernoulliSeq (fun ω => X ω ∪ Y ω) (p + q - p * q) μ | case h.e'_4
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
⊢ (fun ω => X ω ∪ Y ω) = fun ω => ((X ω)ᶜ ∩ (Y ω)ᶜ)ᶜ
case h.e'_5
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
⊢ p + q - p * q = 1 - (1 - p) * (1 - q)
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
⊢ IndepFun (fun ω => (X ω)ᶜ) (fun ω => (Y ω)ᶜ) μ |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/BernoulliSeq.lean | ProbabilityTheory.IsBernoulliSeq.union | [130, 1] | [141, 68] | simp [compl_inter] | case h.e'_4
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
⊢ (fun ω => X ω ∪ Y ω) = fun ω => ((X ω)ᶜ ∩ (Y ω)ᶜ)ᶜ | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/BernoulliSeq.lean | ProbabilityTheory.IsBernoulliSeq.union | [130, 1] | [141, 68] | rw [mul_tsub, mul_one, tsub_tsub, tsub_tsub_cancel_of_le, tsub_mul, one_mul,
add_tsub_assoc_of_le (mul_le_of_le_one_left' $ hX.le_one)] | case h.e'_5
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
⊢ p + q - p * q = 1 - (1 - p) * (1 - q) | case h.e'_5
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
⊢ p + (1 - p) * q ≤ 1 |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/BernoulliSeq.lean | ProbabilityTheory.IsBernoulliSeq.union | [130, 1] | [141, 68] | exact (add_le_add_left (mul_le_of_le_one_right' $ hY.le_one) _).trans_eq
(add_tsub_cancel_of_le hX.le_one) | case h.e'_5
α : Type u_1
Ω : Type u_2
inst✝¹ : MeasurableSpace Ω
X Y : Ω → Set α
μ : Measure Ω
p q : ℝ≥0
hX : IsBernoulliSeq X p μ
hY : IsBernoulliSeq Y q μ
inst✝ : IsProbabilityMeasure μ
h : IndepFun X Y μ
⊢ p + (1 - p) * q ≤ 1 | no goals |
Subsets and Splits
No community queries yet
The top public SQL queries from the community will appear here once available.