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/Kneser/Kneser.lean
Finset.mulStab_mul_ssubset_mulStab
[36, 1]
[82, 79]
intro x hx y hy
case a α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hab : ¬(a * b) • C.mulStab ⊆ s * t hCne : C.Nonempty x : α hx : x ∈ s ∩ a • C.mulStab y : α hy : y ∈ t ∩ b • C.mulStab c : α hc : c ∈ C.mulStab hac : a • c = x d : α hd : d ∈ C.mulStab had : b • d = y hxymem : x * y ∈ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) ⊢ ∀ x ∈ C.mulStab, ∀ y ∈ C.mulStab, x * y ∈ c • d • C.mulStab
case a α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hab : ¬(a * b) • C.mulStab ⊆ s * t hCne : C.Nonempty x✝ : α hx✝ : x✝ ∈ s ∩ a • C.mulStab y✝ : α hy✝ : y✝ ∈ t ∩ b • C.mulStab c : α hc : c ∈ C.mulStab hac : a • c = x✝ d : α hd : d ∈ C.mulStab had : b • d = y✝ hxymem : x✝ * y✝ ∈ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) x : α hx : x ∈ C.mulStab y : α hy : y ∈ C.mulStab ⊢ x * y ∈ c • d • C.mulStab
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.mulStab_mul_ssubset_mulStab
[36, 1]
[82, 79]
rw [smul_mulStab hd, smul_mulStab hc, mem_mulStab hCne, ← smul_smul, (mem_mulStab hCne).mp hy, (mem_mulStab hCne).mp hx]
case a α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hab : ¬(a * b) • C.mulStab ⊆ s * t hCne : C.Nonempty x✝ : α hx✝ : x✝ ∈ s ∩ a • C.mulStab y✝ : α hy✝ : y✝ ∈ t ∩ b • C.mulStab c : α hc : c ∈ C.mulStab hac : a • c = x✝ d : α hd : d ∈ C.mulStab had : b • d = y✝ hxymem : x✝ * y✝ ∈ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) x : α hx : x ∈ C.mulStab y : α hy : y ∈ C.mulStab ⊢ x * y ∈ c • d • C.mulStab
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.mulStab_mul_ssubset_mulStab
[36, 1]
[82, 79]
rw [singleton_mul]
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hab : ¬(a * b) • C.mulStab ⊆ s * t hCne : C.Nonempty x : α hx : x ∈ s ∩ a • C.mulStab y : α hy : y ∈ t ∩ b • C.mulStab c : α hc : c ∈ C.mulStab hac : a • c = x d : α hd : d ∈ C.mulStab had : b • d = y hxymem : x * y ∈ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) this : s ∩ a • C.mulStab * (t ∩ b • C.mulStab) ⊆ (x * y) • C.mulStab ⊢ (x * y) • C.mulStab = {x * y} * C.mulStab
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hab : ¬(a * b) • C.mulStab ⊆ s * t hCne : C.Nonempty x : α hx : x ∈ s ∩ a • C.mulStab y : α hy : y ∈ t ∩ b • C.mulStab c : α hc : c ∈ C.mulStab hac : a • c = x d : α hd : d ∈ C.mulStab had : b • d = y hxymem : x * y ∈ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) this : s ∩ a • C.mulStab * (t ∩ b • C.mulStab) ⊆ (x * y) • C.mulStab ⊢ (x * y) • C.mulStab = image (fun x_1 => x * y * x_1) C.mulStab
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.mulStab_mul_ssubset_mulStab
[36, 1]
[82, 79]
rfl
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hab : ¬(a * b) • C.mulStab ⊆ s * t hCne : C.Nonempty x : α hx : x ∈ s ∩ a • C.mulStab y : α hy : y ∈ t ∩ b • C.mulStab c : α hc : c ∈ C.mulStab hac : a • c = x d : α hd : d ∈ C.mulStab had : b • d = y hxymem : x * y ∈ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) this : s ∩ a • C.mulStab * (t ∩ b • C.mulStab) ⊆ (x * y) • C.mulStab ⊢ (x * y) • C.mulStab = image (fun x_1 => x * y * x_1) C.mulStab
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.mulStab_mul_ssubset_mulStab
[36, 1]
[82, 79]
rw [smul_eq_iff_eq_inv_smul, ← smul_assoc, smul_eq_mul, mul_assoc, mul_comm c _, ← mul_assoc, ← mul_assoc, ← mul_assoc, mul_assoc _ a b, inv_mul_self (a * b), one_mul, ← smul_eq_mul, smul_assoc, smul_mulStab hc, smul_mulStab hd]
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hab : ¬(a * b) • C.mulStab ⊆ s * t hCne : C.Nonempty x : α hx : x ∈ s ∩ a • C.mulStab y : α hy : y ∈ t ∩ b • C.mulStab c : α hc : c ∈ C.mulStab hac : a • c = x d : α hd : d ∈ C.mulStab had : b • d = y hsubset : (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊆ C.mulStab ⊢ (a * b) • C.mulStab = (a * c * (b * d)) • C.mulStab
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.mulStab_mul_ssubset_mulStab
[36, 1]
[82, 79]
apply subset_trans (mul_subset_mul inter_subset_right inter_subset_right)
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hab : ¬(a * b) • C.mulStab ⊆ s * t hCne : C.Nonempty x : α hx : x ∈ s ∩ a • C.mulStab y : α hy : y ∈ t ∩ b • C.mulStab c : α hc : c ∈ C.mulStab hac : a • c = x d : α hd : d ∈ C.mulStab had : b • d = y hsubset : (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊆ C.mulStab this : (a * b) • C.mulStab = (a * c * (b * d)) • C.mulStab ⊢ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) ⊆ (a * b) • C.mulStab
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hab : ¬(a * b) • C.mulStab ⊆ s * t hCne : C.Nonempty x : α hx : x ∈ s ∩ a • C.mulStab y : α hy : y ∈ t ∩ b • C.mulStab c : α hc : c ∈ C.mulStab hac : a • c = x d : α hd : d ∈ C.mulStab had : b • d = y hsubset : (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊆ C.mulStab this : (a * b) • C.mulStab = (a * c * (b * d)) • C.mulStab ⊢ a • C.mulStab * b • C.mulStab ⊆ (a * b) • C.mulStab
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.mulStab_mul_ssubset_mulStab
[36, 1]
[82, 79]
simp only [smul_mul_smul, mulStab_mul_mulStab, subset_refl]
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hab : ¬(a * b) • C.mulStab ⊆ s * t hCne : C.Nonempty x : α hx : x ∈ s ∩ a • C.mulStab y : α hy : y ∈ t ∩ b • C.mulStab c : α hc : c ∈ C.mulStab hac : a • c = x d : α hd : d ∈ C.mulStab had : b • d = y hsubset : (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊆ C.mulStab this : (a * b) • C.mulStab = (a * c * (b * d)) • C.mulStab ⊢ a • C.mulStab * b • C.mulStab ⊆ (a * b) • C.mulStab
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.mulStab_mul_ssubset_mulStab
[36, 1]
[82, 79]
convert hxy
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hCne : C.Nonempty x : α hx : x ∈ s ∩ a • C.mulStab y : α hy : y ∈ t ∩ b • C.mulStab c : α hc : c ∈ C.mulStab hac : a • c = x d : α hab : ¬(a * c * (b * d)) • C.mulStab ⊆ s * t hd : d ∈ C.mulStab had : b • d = y hsubset : (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊆ C.mulStab this : (a * b) • C.mulStab = (a * c * (b * d)) • C.mulStab hsub : s ∩ a • C.mulStab * (t ∩ b • C.mulStab) ⊆ (a * c * (b * d)) • C.mulStab hxy : x * y ∈ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) z : α hz : z ∈ (a * c * (b * d)) • C.mulStab hzst : z ∉ s * t w : α hw : w ∈ C.mulStab hwz : (a * c * (b * d)) • w = z ⊢ a * c * (b * d) ∈ s ∩ a • C.mulStab * (t ∩ b • C.mulStab)
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.mulStab_union
[84, 1]
[131, 73]
obtain rfl | hCne := C.eq_empty_or_nonempty
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hs₁ : (s ∩ a • C.mulStab).Nonempty ht₁ : (t ∩ b • C.mulStab).Nonempty hab : ¬(a * b) • C.mulStab ⊆ s * t hC : Disjoint C (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) ⊢ (C ∪ s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab = (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab
case inl α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' : Finset α a b : α hs₁ : (s ∩ a • ∅.mulStab).Nonempty ht₁ : (t ∩ b • ∅.mulStab).Nonempty hab : ¬(a * b) • ∅.mulStab ⊆ s * t hC : Disjoint ∅ (s ∩ a • ∅.mulStab * (t ∩ b • ∅.mulStab)) ⊢ (∅ ∪ s ∩ a • ∅.mulStab * (t ∩ b • ∅.mulStab)).mulStab = (s ∩ a • ∅.mulStab * (t ∩ b • ∅.mulStab)).mulStab case inr α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hs₁ : (s ∩ a • C.mulStab).Nonempty ht₁ : (t ∩ b • C.mulStab).Nonempty hab : ¬(a * b) • C.mulStab ⊆ s * t hC : Disjoint C (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) hCne : C.Nonempty ⊢ (C ∪ s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab = (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.mulStab_union
[84, 1]
[131, 73]
refine' ((subset_inter (mulStab_mul_ssubset_mulStab hs₁ ht₁ hab).subset Subset.rfl).trans inter_mulStab_subset_mulStab_union).antisymm' fun x hx => _
case inr α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hs₁ : (s ∩ a • C.mulStab).Nonempty ht₁ : (t ∩ b • C.mulStab).Nonempty hab : ¬(a * b) • C.mulStab ⊆ s * t hC : Disjoint C (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) hCne : C.Nonempty ⊢ (C ∪ s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab = (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab
case inr α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hs₁ : (s ∩ a • C.mulStab).Nonempty ht₁ : (t ∩ b • C.mulStab).Nonempty hab : ¬(a * b) • C.mulStab ⊆ s * t hC : Disjoint C (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) hCne : C.Nonempty x : α hx : x ∈ (C ∪ s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊢ x ∈ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.mulStab_union
[84, 1]
[131, 73]
replace hx := (mem_mulStab $ (hs₁.mul ht₁).mono subset_union_right).mp hx
case inr α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hs₁ : (s ∩ a • C.mulStab).Nonempty ht₁ : (t ∩ b • C.mulStab).Nonempty hab : ¬(a * b) • C.mulStab ⊆ s * t hC : Disjoint C (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) hCne : C.Nonempty x : α hx : x ∈ (C ∪ s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊢ x ∈ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab
case inr α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hs₁ : (s ∩ a • C.mulStab).Nonempty ht₁ : (t ∩ b • C.mulStab).Nonempty hab : ¬(a * b) • C.mulStab ⊆ s * t hC : Disjoint C (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) hCne : C.Nonempty x : α hx : x • (C ∪ s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) = C ∪ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) ⊢ x ∈ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.mulStab_union
[84, 1]
[131, 73]
rw [smul_finset_union] at hx
case inr α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hs₁ : (s ∩ a • C.mulStab).Nonempty ht₁ : (t ∩ b • C.mulStab).Nonempty hab : ¬(a * b) • C.mulStab ⊆ s * t hC : Disjoint C (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) hCne : C.Nonempty x : α hx : x • (C ∪ s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) = C ∪ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) ⊢ x ∈ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab
case inr α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hs₁ : (s ∩ a • C.mulStab).Nonempty ht₁ : (t ∩ b • C.mulStab).Nonempty hab : ¬(a * b) • C.mulStab ⊆ s * t hC : Disjoint C (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) hCne : C.Nonempty x : α hx : x • C ∪ x • (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) = C ∪ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) ⊢ x ∈ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.mulStab_union
[84, 1]
[131, 73]
suffices hxC : x ∈ C.mulStab by rw [(mem_mulStab hCne).mp hxC] at hx rw [mem_mulStab_iff_subset_smul_finset (hs₁.mul ht₁)] exact hC.symm.left_le_of_le_sup_left (le_sup_right.trans hx.ge)
case inr α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hs₁ : (s ∩ a • C.mulStab).Nonempty ht₁ : (t ∩ b • C.mulStab).Nonempty hab : ¬(a * b) • C.mulStab ⊆ s * t hC : Disjoint C (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) hCne : C.Nonempty x : α hx : x • C ∪ x • (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) = C ∪ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) ⊢ x ∈ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab
case inr α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hs₁ : (s ∩ a • C.mulStab).Nonempty ht₁ : (t ∩ b • C.mulStab).Nonempty hab : ¬(a * b) • C.mulStab ⊆ s * t hC : Disjoint C (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) hCne : C.Nonempty x : α hx : x • C ∪ x • (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) = C ∪ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) ⊢ x ∈ C.mulStab
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.mulStab_union
[84, 1]
[131, 73]
rw [mem_mulStab_iff_smul_finset_subset hCne]
case inr α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hs₁ : (s ∩ a • C.mulStab).Nonempty ht₁ : (t ∩ b • C.mulStab).Nonempty hab : ¬(a * b) • C.mulStab ⊆ s * t hC : Disjoint C (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) hCne : C.Nonempty x : α hx : x • C ∪ x • (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) = C ∪ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) ⊢ x ∈ C.mulStab
case inr α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hs₁ : (s ∩ a • C.mulStab).Nonempty ht₁ : (t ∩ b • C.mulStab).Nonempty hab : ¬(a * b) • C.mulStab ⊆ s * t hC : Disjoint C (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) hCne : C.Nonempty x : α hx : x • C ∪ x • (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) = C ∪ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) ⊢ x • C ⊆ C
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.mulStab_union
[84, 1]
[131, 73]
obtain h | h := disjoint_or_nonempty_inter (x • C) (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))
case inr α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hs₁ : (s ∩ a • C.mulStab).Nonempty ht₁ : (t ∩ b • C.mulStab).Nonempty hab : ¬(a * b) • C.mulStab ⊆ s * t hC : Disjoint C (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) hCne : C.Nonempty x : α hx : x • C ∪ x • (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) = C ∪ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) ⊢ x • C ⊆ C
case inr.inl α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hs₁ : (s ∩ a • C.mulStab).Nonempty ht₁ : (t ∩ b • C.mulStab).Nonempty hab : ¬(a * b) • C.mulStab ⊆ s * t hC : Disjoint C (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) hCne : C.Nonempty x : α hx : x • C ∪ x • (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) = C ∪ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) h : Disjoint (x • C) (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) ⊢ x • C ⊆ C case inr.inr α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hs₁ : (s ∩ a • C.mulStab).Nonempty ht₁ : (t ∩ b • C.mulStab).Nonempty hab : ¬(a * b) • C.mulStab ⊆ s * t hC : Disjoint C (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) hCne : C.Nonempty x : α hx : x • C ∪ x • (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) = C ∪ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) h : (x • C ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty ⊢ x • C ⊆ C
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.mulStab_union
[84, 1]
[131, 73]
have hUn : ((C.biUnion fun y => x • y • C.mulStab) ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty := by have : (x • C.biUnion fun y => y • C.mulStab) = C.biUnion fun y => x • y • C.mulStab := biUnion_image simpa [← this]
case inr.inr α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hs₁ : (s ∩ a • C.mulStab).Nonempty ht₁ : (t ∩ b • C.mulStab).Nonempty hab : ¬(a * b) • C.mulStab ⊆ s * t hC : Disjoint C (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) hCne : C.Nonempty x : α hx : x • C ∪ x • (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) = C ∪ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) h : (x • C ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty ⊢ x • C ⊆ C
case inr.inr α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hs₁ : (s ∩ a • C.mulStab).Nonempty ht₁ : (t ∩ b • C.mulStab).Nonempty hab : ¬(a * b) • C.mulStab ⊆ s * t hC : Disjoint C (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) hCne : C.Nonempty x : α hx : x • C ∪ x • (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) = C ∪ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) h : (x • C ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty hUn : ((C.biUnion fun y => x • y • C.mulStab) ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty ⊢ x • C ⊆ C
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.mulStab_union
[84, 1]
[131, 73]
simp_rw [biUnion_inter, biUnion_nonempty, ← smul_assoc, smul_eq_mul] at hUn
case inr.inr α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hs₁ : (s ∩ a • C.mulStab).Nonempty ht₁ : (t ∩ b • C.mulStab).Nonempty hab : ¬(a * b) • C.mulStab ⊆ s * t hC : Disjoint C (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) hCne : C.Nonempty x : α hx : x • C ∪ x • (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) = C ∪ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) h : (x • C ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty hUn : ((C.biUnion fun y => x • y • C.mulStab) ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty ⊢ x • C ⊆ C
case inr.inr α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hs₁ : (s ∩ a • C.mulStab).Nonempty ht₁ : (t ∩ b • C.mulStab).Nonempty hab : ¬(a * b) • C.mulStab ⊆ s * t hC : Disjoint C (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) hCne : C.Nonempty x : α hx : x • C ∪ x • (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) = C ∪ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) h : (x • C ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty hUn : ∃ x_1 ∈ C, ((x * x_1) • C.mulStab ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty ⊢ x • C ⊆ C
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.mulStab_union
[84, 1]
[131, 73]
obtain ⟨y, hy, hyne⟩ := hUn
case inr.inr α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hs₁ : (s ∩ a • C.mulStab).Nonempty ht₁ : (t ∩ b • C.mulStab).Nonempty hab : ¬(a * b) • C.mulStab ⊆ s * t hC : Disjoint C (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) hCne : C.Nonempty x : α hx : x • C ∪ x • (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) = C ∪ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) h : (x • C ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty hUn : ∃ x_1 ∈ C, ((x * x_1) • C.mulStab ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty ⊢ x • C ⊆ C
case inr.inr.intro.intro α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hs₁ : (s ∩ a • C.mulStab).Nonempty ht₁ : (t ∩ b • C.mulStab).Nonempty hab : ¬(a * b) • C.mulStab ⊆ s * t hC : Disjoint C (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) hCne : C.Nonempty x : α hx : x • C ∪ x • (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) = C ∪ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) h : (x • C ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty y : α hy : y ∈ C hyne : ((x * y) • C.mulStab ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty ⊢ x • C ⊆ C
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.mulStab_union
[84, 1]
[131, 73]
have hxyCsubC : (x * y) • C.mulStab ⊆ x • C := by rw [← smul_eq_mul, smul_assoc, smul_finset_subset_smul_finset_iff] exact smul_finset_mulStab_subset hy
case inr.inr.intro.intro α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hs₁ : (s ∩ a • C.mulStab).Nonempty ht₁ : (t ∩ b • C.mulStab).Nonempty hab : ¬(a * b) • C.mulStab ⊆ s * t hC : Disjoint C (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) hCne : C.Nonempty x : α hx : x • C ∪ x • (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) = C ∪ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) h : (x • C ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty y : α hy : y ∈ C hyne : ((x * y) • C.mulStab ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty ⊢ x • C ⊆ C
case inr.inr.intro.intro α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hs₁ : (s ∩ a • C.mulStab).Nonempty ht₁ : (t ∩ b • C.mulStab).Nonempty hab : ¬(a * b) • C.mulStab ⊆ s * t hC : Disjoint C (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) hCne : C.Nonempty x : α hx : x • C ∪ x • (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) = C ∪ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) h : (x • C ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty y : α hy : y ∈ C hyne : ((x * y) • C.mulStab ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty hxyCsubC : (x * y) • C.mulStab ⊆ x • C ⊢ x • C ⊆ C
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.mulStab_union
[84, 1]
[131, 73]
have hxysub : (x * y) • C.mulStab ⊆ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) := hxyC.left_le_of_le_sup_left (hxyCsubC.trans $ subset_union_left.trans hx.subset')
case inr.inr.intro.intro α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hs₁ : (s ∩ a • C.mulStab).Nonempty ht₁ : (t ∩ b • C.mulStab).Nonempty hab : ¬(a * b) • C.mulStab ⊆ s * t hC : Disjoint C (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) hCne : C.Nonempty x : α hx : x • C ∪ x • (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) = C ∪ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) h : (x • C ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty y : α hy : y ∈ C hyne : ((x * y) • C.mulStab ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty hxyCsubC : (x * y) • C.mulStab ⊆ x • C hxyC : Disjoint ((x * y) • C.mulStab) C ⊢ x • C ⊆ C
case inr.inr.intro.intro α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hs₁ : (s ∩ a • C.mulStab).Nonempty ht₁ : (t ∩ b • C.mulStab).Nonempty hab : ¬(a * b) • C.mulStab ⊆ s * t hC : Disjoint C (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) hCne : C.Nonempty x : α hx : x • C ∪ x • (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) = C ∪ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) h : (x • C ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty y : α hy : y ∈ C hyne : ((x * y) • C.mulStab ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty hxyCsubC : (x * y) • C.mulStab ⊆ x • C hxyC : Disjoint ((x * y) • C.mulStab) C hxysub : (x * y) • C.mulStab ⊆ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) ⊢ x • C ⊆ C
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.mulStab_union
[84, 1]
[131, 73]
suffices s ∩ a • C.mulStab * (t ∩ b • C.mulStab) ⊂ (a * b) • C.mulStab by have := (card_le_card hxysub).not_lt ((card_lt_card this).trans_eq ?_) cases this simp_rw [card_smul_finset]
case inr.inr.intro.intro α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hs₁ : (s ∩ a • C.mulStab).Nonempty ht₁ : (t ∩ b • C.mulStab).Nonempty hab : ¬(a * b) • C.mulStab ⊆ s * t hC : Disjoint C (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) hCne : C.Nonempty x : α hx : x • C ∪ x • (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) = C ∪ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) h : (x • C ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty y : α hy : y ∈ C hyne : ((x * y) • C.mulStab ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty hxyCsubC : (x * y) • C.mulStab ⊆ x • C hxyC : Disjoint ((x * y) • C.mulStab) C hxysub : (x * y) • C.mulStab ⊆ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) ⊢ x • C ⊆ C
case inr.inr.intro.intro α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hs₁ : (s ∩ a • C.mulStab).Nonempty ht₁ : (t ∩ b • C.mulStab).Nonempty hab : ¬(a * b) • C.mulStab ⊆ s * t hC : Disjoint C (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) hCne : C.Nonempty x : α hx : x • C ∪ x • (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) = C ∪ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) h : (x • C ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty y : α hy : y ∈ C hyne : ((x * y) • C.mulStab ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty hxyCsubC : (x * y) • C.mulStab ⊆ x • C hxyC : Disjoint ((x * y) • C.mulStab) C hxysub : (x * y) • C.mulStab ⊆ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) ⊢ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) ⊂ (a * b) • C.mulStab
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.mulStab_union
[84, 1]
[131, 73]
apply ssubset_of_subset_not_subset
case inr.inr.intro.intro α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hs₁ : (s ∩ a • C.mulStab).Nonempty ht₁ : (t ∩ b • C.mulStab).Nonempty hab : ¬(a * b) • C.mulStab ⊆ s * t hC : Disjoint C (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) hCne : C.Nonempty x : α hx : x • C ∪ x • (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) = C ∪ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) h : (x • C ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty y : α hy : y ∈ C hyne : ((x * y) • C.mulStab ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty hxyCsubC : (x * y) • C.mulStab ⊆ x • C hxyC : Disjoint ((x * y) • C.mulStab) C hxysub : (x * y) • C.mulStab ⊆ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) ⊢ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) ⊂ (a * b) • C.mulStab
case inr.inr.intro.intro.h₁ α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hs₁ : (s ∩ a • C.mulStab).Nonempty ht₁ : (t ∩ b • C.mulStab).Nonempty hab : ¬(a * b) • C.mulStab ⊆ s * t hC : Disjoint C (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) hCne : C.Nonempty x : α hx : x • C ∪ x • (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) = C ∪ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) h : (x • C ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty y : α hy : y ∈ C hyne : ((x * y) • C.mulStab ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty hxyCsubC : (x * y) • C.mulStab ⊆ x • C hxyC : Disjoint ((x * y) • C.mulStab) C hxysub : (x * y) • C.mulStab ⊆ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) ⊢ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) ⊆ (a * b) • C.mulStab case inr.inr.intro.intro.h₂ α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hs₁ : (s ∩ a • C.mulStab).Nonempty ht₁ : (t ∩ b • C.mulStab).Nonempty hab : ¬(a * b) • C.mulStab ⊆ s * t hC : Disjoint C (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) hCne : C.Nonempty x : α hx : x • C ∪ x • (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) = C ∪ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) h : (x • C ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty y : α hy : y ∈ C hyne : ((x * y) • C.mulStab ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty hxyCsubC : (x * y) • C.mulStab ⊆ x • C hxyC : Disjoint ((x * y) • C.mulStab) C hxysub : (x * y) • C.mulStab ⊆ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) ⊢ ¬(a * b) • C.mulStab ⊆ s ∩ a • C.mulStab * (t ∩ b • C.mulStab)
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.mulStab_union
[84, 1]
[131, 73]
simp [hs₁]
case inl α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' : Finset α a b : α hs₁ : (s ∩ a • ∅.mulStab).Nonempty ht₁ : (t ∩ b • ∅.mulStab).Nonempty hab : ¬(a * b) • ∅.mulStab ⊆ s * t hC : Disjoint ∅ (s ∩ a • ∅.mulStab * (t ∩ b • ∅.mulStab)) ⊢ (∅ ∪ s ∩ a • ∅.mulStab * (t ∩ b • ∅.mulStab)).mulStab = (s ∩ a • ∅.mulStab * (t ∩ b • ∅.mulStab)).mulStab
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.mulStab_union
[84, 1]
[131, 73]
rw [(mem_mulStab hCne).mp hxC] at hx
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hs₁ : (s ∩ a • C.mulStab).Nonempty ht₁ : (t ∩ b • C.mulStab).Nonempty hab : ¬(a * b) • C.mulStab ⊆ s * t hC : Disjoint C (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) hCne : C.Nonempty x : α hx : x • C ∪ x • (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) = C ∪ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) hxC : x ∈ C.mulStab ⊢ x ∈ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hs₁ : (s ∩ a • C.mulStab).Nonempty ht₁ : (t ∩ b • C.mulStab).Nonempty hab : ¬(a * b) • C.mulStab ⊆ s * t hC : Disjoint C (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) hCne : C.Nonempty x : α hx : C ∪ x • (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) = C ∪ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) hxC : x ∈ C.mulStab ⊢ x ∈ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.mulStab_union
[84, 1]
[131, 73]
rw [mem_mulStab_iff_subset_smul_finset (hs₁.mul ht₁)]
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hs₁ : (s ∩ a • C.mulStab).Nonempty ht₁ : (t ∩ b • C.mulStab).Nonempty hab : ¬(a * b) • C.mulStab ⊆ s * t hC : Disjoint C (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) hCne : C.Nonempty x : α hx : C ∪ x • (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) = C ∪ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) hxC : x ∈ C.mulStab ⊢ x ∈ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hs₁ : (s ∩ a • C.mulStab).Nonempty ht₁ : (t ∩ b • C.mulStab).Nonempty hab : ¬(a * b) • C.mulStab ⊆ s * t hC : Disjoint C (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) hCne : C.Nonempty x : α hx : C ∪ x • (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) = C ∪ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) hxC : x ∈ C.mulStab ⊢ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) ⊆ x • (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.mulStab_union
[84, 1]
[131, 73]
exact hC.symm.left_le_of_le_sup_left (le_sup_right.trans hx.ge)
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hs₁ : (s ∩ a • C.mulStab).Nonempty ht₁ : (t ∩ b • C.mulStab).Nonempty hab : ¬(a * b) • C.mulStab ⊆ s * t hC : Disjoint C (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) hCne : C.Nonempty x : α hx : C ∪ x • (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) = C ∪ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) hxC : x ∈ C.mulStab ⊢ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) ⊆ x • (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.mulStab_union
[84, 1]
[131, 73]
exact h.left_le_of_le_sup_right (le_sup_left.trans_eq hx)
case inr.inl α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hs₁ : (s ∩ a • C.mulStab).Nonempty ht₁ : (t ∩ b • C.mulStab).Nonempty hab : ¬(a * b) • C.mulStab ⊆ s * t hC : Disjoint C (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) hCne : C.Nonempty x : α hx : x • C ∪ x • (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) = C ∪ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) h : Disjoint (x • C) (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) ⊢ x • C ⊆ C
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.mulStab_union
[84, 1]
[131, 73]
have : (x • C.biUnion fun y => y • C.mulStab) = C.biUnion fun y => x • y • C.mulStab := biUnion_image
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hs₁ : (s ∩ a • C.mulStab).Nonempty ht₁ : (t ∩ b • C.mulStab).Nonempty hab : ¬(a * b) • C.mulStab ⊆ s * t hC : Disjoint C (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) hCne : C.Nonempty x : α hx : x • C ∪ x • (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) = C ∪ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) h : (x • C ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty ⊢ ((C.biUnion fun y => x • y • C.mulStab) ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hs₁ : (s ∩ a • C.mulStab).Nonempty ht₁ : (t ∩ b • C.mulStab).Nonempty hab : ¬(a * b) • C.mulStab ⊆ s * t hC : Disjoint C (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) hCne : C.Nonempty x : α hx : x • C ∪ x • (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) = C ∪ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) h : (x • C ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty this : (x • C.biUnion fun y => y • C.mulStab) = C.biUnion fun y => x • y • C.mulStab ⊢ ((C.biUnion fun y => x • y • C.mulStab) ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.mulStab_union
[84, 1]
[131, 73]
simpa [← this]
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hs₁ : (s ∩ a • C.mulStab).Nonempty ht₁ : (t ∩ b • C.mulStab).Nonempty hab : ¬(a * b) • C.mulStab ⊆ s * t hC : Disjoint C (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) hCne : C.Nonempty x : α hx : x • C ∪ x • (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) = C ∪ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) h : (x • C ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty this : (x • C.biUnion fun y => y • C.mulStab) = C.biUnion fun y => x • y • C.mulStab ⊢ ((C.biUnion fun y => x • y • C.mulStab) ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.mulStab_union
[84, 1]
[131, 73]
rw [← smul_eq_mul, smul_assoc, smul_finset_subset_smul_finset_iff]
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hs₁ : (s ∩ a • C.mulStab).Nonempty ht₁ : (t ∩ b • C.mulStab).Nonempty hab : ¬(a * b) • C.mulStab ⊆ s * t hC : Disjoint C (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) hCne : C.Nonempty x : α hx : x • C ∪ x • (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) = C ∪ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) h : (x • C ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty y : α hy : y ∈ C hyne : ((x * y) • C.mulStab ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty ⊢ (x * y) • C.mulStab ⊆ x • C
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hs₁ : (s ∩ a • C.mulStab).Nonempty ht₁ : (t ∩ b • C.mulStab).Nonempty hab : ¬(a * b) • C.mulStab ⊆ s * t hC : Disjoint C (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) hCne : C.Nonempty x : α hx : x • C ∪ x • (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) = C ∪ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) h : (x • C ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty y : α hy : y ∈ C hyne : ((x * y) • C.mulStab ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty ⊢ y • C.mulStab ⊆ C
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.mulStab_union
[84, 1]
[131, 73]
exact smul_finset_mulStab_subset hy
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hs₁ : (s ∩ a • C.mulStab).Nonempty ht₁ : (t ∩ b • C.mulStab).Nonempty hab : ¬(a * b) • C.mulStab ⊆ s * t hC : Disjoint C (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) hCne : C.Nonempty x : α hx : x • C ∪ x • (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) = C ∪ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) h : (x • C ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty y : α hy : y ∈ C hyne : ((x * y) • C.mulStab ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty ⊢ y • C.mulStab ⊆ C
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.mulStab_union
[84, 1]
[131, 73]
convert disjoint_smul_finset_mulStab_mul_mulStab fun hxyC => _
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hs₁ : (s ∩ a • C.mulStab).Nonempty ht₁ : (t ∩ b • C.mulStab).Nonempty hab : ¬(a * b) • C.mulStab ⊆ s * t hC : Disjoint C (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) hCne : C.Nonempty x : α hx : x • C ∪ x • (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) = C ∪ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) h : (x • C ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty y : α hy : y ∈ C hyne : ((x * y) • C.mulStab ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty hxyCsubC : (x * y) • C.mulStab ⊆ x • C ⊢ Disjoint ((x * y) • C.mulStab) C
case h.e'_5 α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hs₁ : (s ∩ a • C.mulStab).Nonempty ht₁ : (t ∩ b • C.mulStab).Nonempty hab : ¬(a * b) • C.mulStab ⊆ s * t hC : Disjoint C (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) hCne : C.Nonempty x : α hx : x • C ∪ x • (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) = C ∪ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) h : (x • C ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty y : α hy : y ∈ C hyne : ((x * y) • C.mulStab ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty hxyCsubC : (x * y) • C.mulStab ⊆ x • C ⊢ C = ?convert_5 * C.mulStab case convert_5 α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hs₁ : (s ∩ a • C.mulStab).Nonempty ht₁ : (t ∩ b • C.mulStab).Nonempty hab : ¬(a * b) • C.mulStab ⊆ s * t hC : Disjoint C (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) hCne : C.Nonempty x : α hx : x • C ∪ x • (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) = C ∪ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) h : (x • C ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty y : α hy : y ∈ C hyne : ((x * y) • C.mulStab ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty hxyCsubC : (x * y) • C.mulStab ⊆ x • C ⊢ Finset α case convert_7 α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hs₁ : (s ∩ a • C.mulStab).Nonempty ht₁ : (t ∩ b • C.mulStab).Nonempty hab : ¬(a * b) • C.mulStab ⊆ s * t hC : Disjoint C (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) hCne : C.Nonempty x : α hx : x • C ∪ x • (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) = C ∪ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) h : (x • C ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty y : α hy : y ∈ C hyne : ((x * y) • C.mulStab ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty hxyCsubC : (x * y) • C.mulStab ⊆ x • C hxyC : (x * y) • C.mulStab ⊆ ?convert_5 * C.mulStab ⊢ False
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.mulStab_union
[84, 1]
[131, 73]
rw [mul_mulStab] at hxyC
case convert_7 α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hs₁ : (s ∩ a • C.mulStab).Nonempty ht₁ : (t ∩ b • C.mulStab).Nonempty hab : ¬(a * b) • C.mulStab ⊆ s * t hC : Disjoint C (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) hCne : C.Nonempty x : α hx : x • C ∪ x • (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) = C ∪ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) h : (x • C ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty y : α hy : y ∈ C hyne : ((x * y) • C.mulStab ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty hxyCsubC : (x * y) • C.mulStab ⊆ x • C hxyC : (x * y) • C.mulStab ⊆ C * C.mulStab ⊢ False
case convert_7 α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hs₁ : (s ∩ a • C.mulStab).Nonempty ht₁ : (t ∩ b • C.mulStab).Nonempty hab : ¬(a * b) • C.mulStab ⊆ s * t hC : Disjoint C (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) hCne : C.Nonempty x : α hx : x • C ∪ x • (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) = C ∪ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) h : (x • C ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty y : α hy : y ∈ C hyne : ((x * y) • C.mulStab ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty hxyCsubC : (x * y) • C.mulStab ⊆ x • C hxyC : (x * y) • C.mulStab ⊆ C ⊢ False
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.mulStab_union
[84, 1]
[131, 73]
exact hyne.not_disjoint (hC.mono_left $ le_iff_subset.2 hxyC)
case convert_7 α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hs₁ : (s ∩ a • C.mulStab).Nonempty ht₁ : (t ∩ b • C.mulStab).Nonempty hab : ¬(a * b) • C.mulStab ⊆ s * t hC : Disjoint C (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) hCne : C.Nonempty x : α hx : x • C ∪ x • (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) = C ∪ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) h : (x • C ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty y : α hy : y ∈ C hyne : ((x * y) • C.mulStab ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty hxyCsubC : (x * y) • C.mulStab ⊆ x • C hxyC : (x * y) • C.mulStab ⊆ C ⊢ False
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.mulStab_union
[84, 1]
[131, 73]
exact C.mul_mulStab.symm
case h.e'_5 α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hs₁ : (s ∩ a • C.mulStab).Nonempty ht₁ : (t ∩ b • C.mulStab).Nonempty hab : ¬(a * b) • C.mulStab ⊆ s * t hC : Disjoint C (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) hCne : C.Nonempty x : α hx : x • C ∪ x • (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) = C ∪ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) h : (x • C ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty y : α hy : y ∈ C hyne : ((x * y) • C.mulStab ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty hxyCsubC : (x * y) • C.mulStab ⊆ x • C ⊢ C = ?convert_5 * C.mulStab
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.mulStab_union
[84, 1]
[131, 73]
have := (card_le_card hxysub).not_lt ((card_lt_card this).trans_eq ?_)
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hs₁ : (s ∩ a • C.mulStab).Nonempty ht₁ : (t ∩ b • C.mulStab).Nonempty hab : ¬(a * b) • C.mulStab ⊆ s * t hC : Disjoint C (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) hCne : C.Nonempty x : α hx : x • C ∪ x • (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) = C ∪ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) h : (x • C ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty y : α hy : y ∈ C hyne : ((x * y) • C.mulStab ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty hxyCsubC : (x * y) • C.mulStab ⊆ x • C hxyC : Disjoint ((x * y) • C.mulStab) C hxysub : (x * y) • C.mulStab ⊆ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) this : s ∩ a • C.mulStab * (t ∩ b • C.mulStab) ⊂ (a * b) • C.mulStab ⊢ x • C ⊆ C
case refine_2 α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hs₁ : (s ∩ a • C.mulStab).Nonempty ht₁ : (t ∩ b • C.mulStab).Nonempty hab : ¬(a * b) • C.mulStab ⊆ s * t hC : Disjoint C (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) hCne : C.Nonempty x : α hx : x • C ∪ x • (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) = C ∪ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) h : (x • C ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty y : α hy : y ∈ C hyne : ((x * y) • C.mulStab ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty hxyCsubC : (x * y) • C.mulStab ⊆ x • C hxyC : Disjoint ((x * y) • C.mulStab) C hxysub : (x * y) • C.mulStab ⊆ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) this✝ : s ∩ a • C.mulStab * (t ∩ b • C.mulStab) ⊂ (a * b) • C.mulStab this : False ⊢ x • C ⊆ C case refine_1 α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hs₁ : (s ∩ a • C.mulStab).Nonempty ht₁ : (t ∩ b • C.mulStab).Nonempty hab : ¬(a * b) • C.mulStab ⊆ s * t hC : Disjoint C (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) hCne : C.Nonempty x : α hx : x • C ∪ x • (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) = C ∪ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) h : (x • C ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty y : α hy : y ∈ C hyne : ((x * y) • C.mulStab ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty hxyCsubC : (x * y) • C.mulStab ⊆ x • C hxyC : Disjoint ((x * y) • C.mulStab) C hxysub : (x * y) • C.mulStab ⊆ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) this : s ∩ a • C.mulStab * (t ∩ b • C.mulStab) ⊂ (a * b) • C.mulStab ⊢ ((a * b) • C.mulStab).card = ((x * y) • C.mulStab).card
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.mulStab_union
[84, 1]
[131, 73]
cases this
case refine_2 α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hs₁ : (s ∩ a • C.mulStab).Nonempty ht₁ : (t ∩ b • C.mulStab).Nonempty hab : ¬(a * b) • C.mulStab ⊆ s * t hC : Disjoint C (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) hCne : C.Nonempty x : α hx : x • C ∪ x • (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) = C ∪ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) h : (x • C ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty y : α hy : y ∈ C hyne : ((x * y) • C.mulStab ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty hxyCsubC : (x * y) • C.mulStab ⊆ x • C hxyC : Disjoint ((x * y) • C.mulStab) C hxysub : (x * y) • C.mulStab ⊆ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) this✝ : s ∩ a • C.mulStab * (t ∩ b • C.mulStab) ⊂ (a * b) • C.mulStab this : False ⊢ x • C ⊆ C case refine_1 α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hs₁ : (s ∩ a • C.mulStab).Nonempty ht₁ : (t ∩ b • C.mulStab).Nonempty hab : ¬(a * b) • C.mulStab ⊆ s * t hC : Disjoint C (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) hCne : C.Nonempty x : α hx : x • C ∪ x • (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) = C ∪ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) h : (x • C ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty y : α hy : y ∈ C hyne : ((x * y) • C.mulStab ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty hxyCsubC : (x * y) • C.mulStab ⊆ x • C hxyC : Disjoint ((x * y) • C.mulStab) C hxysub : (x * y) • C.mulStab ⊆ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) this : s ∩ a • C.mulStab * (t ∩ b • C.mulStab) ⊂ (a * b) • C.mulStab ⊢ ((a * b) • C.mulStab).card = ((x * y) • C.mulStab).card
case refine_1 α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hs₁ : (s ∩ a • C.mulStab).Nonempty ht₁ : (t ∩ b • C.mulStab).Nonempty hab : ¬(a * b) • C.mulStab ⊆ s * t hC : Disjoint C (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) hCne : C.Nonempty x : α hx : x • C ∪ x • (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) = C ∪ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) h : (x • C ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty y : α hy : y ∈ C hyne : ((x * y) • C.mulStab ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty hxyCsubC : (x * y) • C.mulStab ⊆ x • C hxyC : Disjoint ((x * y) • C.mulStab) C hxysub : (x * y) • C.mulStab ⊆ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) this : s ∩ a • C.mulStab * (t ∩ b • C.mulStab) ⊂ (a * b) • C.mulStab ⊢ ((a * b) • C.mulStab).card = ((x * y) • C.mulStab).card
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.mulStab_union
[84, 1]
[131, 73]
simp_rw [card_smul_finset]
case refine_1 α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hs₁ : (s ∩ a • C.mulStab).Nonempty ht₁ : (t ∩ b • C.mulStab).Nonempty hab : ¬(a * b) • C.mulStab ⊆ s * t hC : Disjoint C (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) hCne : C.Nonempty x : α hx : x • C ∪ x • (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) = C ∪ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) h : (x • C ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty y : α hy : y ∈ C hyne : ((x * y) • C.mulStab ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty hxyCsubC : (x * y) • C.mulStab ⊆ x • C hxyC : Disjoint ((x * y) • C.mulStab) C hxysub : (x * y) • C.mulStab ⊆ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) this : s ∩ a • C.mulStab * (t ∩ b • C.mulStab) ⊂ (a * b) • C.mulStab ⊢ ((a * b) • C.mulStab).card = ((x * y) • C.mulStab).card
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.mulStab_union
[84, 1]
[131, 73]
refine' (mul_subset_mul inter_subset_right inter_subset_right).trans _
case inr.inr.intro.intro.h₁ α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hs₁ : (s ∩ a • C.mulStab).Nonempty ht₁ : (t ∩ b • C.mulStab).Nonempty hab : ¬(a * b) • C.mulStab ⊆ s * t hC : Disjoint C (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) hCne : C.Nonempty x : α hx : x • C ∪ x • (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) = C ∪ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) h : (x • C ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty y : α hy : y ∈ C hyne : ((x * y) • C.mulStab ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty hxyCsubC : (x * y) • C.mulStab ⊆ x • C hxyC : Disjoint ((x * y) • C.mulStab) C hxysub : (x * y) • C.mulStab ⊆ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) ⊢ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) ⊆ (a * b) • C.mulStab
case inr.inr.intro.intro.h₁ α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hs₁ : (s ∩ a • C.mulStab).Nonempty ht₁ : (t ∩ b • C.mulStab).Nonempty hab : ¬(a * b) • C.mulStab ⊆ s * t hC : Disjoint C (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) hCne : C.Nonempty x : α hx : x • C ∪ x • (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) = C ∪ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) h : (x • C ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty y : α hy : y ∈ C hyne : ((x * y) • C.mulStab ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty hxyCsubC : (x * y) • C.mulStab ⊆ x • C hxyC : Disjoint ((x * y) • C.mulStab) C hxysub : (x * y) • C.mulStab ⊆ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) ⊢ a • C.mulStab * b • C.mulStab ⊆ (a * b) • C.mulStab
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.mulStab_union
[84, 1]
[131, 73]
simp only [smul_mul_smul, mulStab_mul_mulStab, subset_refl]
case inr.inr.intro.intro.h₁ α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hs₁ : (s ∩ a • C.mulStab).Nonempty ht₁ : (t ∩ b • C.mulStab).Nonempty hab : ¬(a * b) • C.mulStab ⊆ s * t hC : Disjoint C (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) hCne : C.Nonempty x : α hx : x • C ∪ x • (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) = C ∪ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) h : (x • C ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty y : α hy : y ∈ C hyne : ((x * y) • C.mulStab ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty hxyCsubC : (x * y) • C.mulStab ⊆ x • C hxyC : Disjoint ((x * y) • C.mulStab) C hxysub : (x * y) • C.mulStab ⊆ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) ⊢ a • C.mulStab * b • C.mulStab ⊆ (a * b) • C.mulStab
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.mulStab_union
[84, 1]
[131, 73]
contrapose! hab
case inr.inr.intro.intro.h₂ α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hs₁ : (s ∩ a • C.mulStab).Nonempty ht₁ : (t ∩ b • C.mulStab).Nonempty hab : ¬(a * b) • C.mulStab ⊆ s * t hC : Disjoint C (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) hCne : C.Nonempty x : α hx : x • C ∪ x • (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) = C ∪ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) h : (x • C ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty y : α hy : y ∈ C hyne : ((x * y) • C.mulStab ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty hxyCsubC : (x * y) • C.mulStab ⊆ x • C hxyC : Disjoint ((x * y) • C.mulStab) C hxysub : (x * y) • C.mulStab ⊆ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) ⊢ ¬(a * b) • C.mulStab ⊆ s ∩ a • C.mulStab * (t ∩ b • C.mulStab)
case inr.inr.intro.intro.h₂ α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hs₁ : (s ∩ a • C.mulStab).Nonempty ht₁ : (t ∩ b • C.mulStab).Nonempty hC : Disjoint C (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) hCne : C.Nonempty x : α hx : x • C ∪ x • (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) = C ∪ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) h : (x • C ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty y : α hy : y ∈ C hyne : ((x * y) • C.mulStab ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty hxyCsubC : (x * y) • C.mulStab ⊆ x • C hxyC : Disjoint ((x * y) • C.mulStab) C hxysub : (x * y) • C.mulStab ⊆ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) hab : (a * b) • C.mulStab ⊆ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) ⊢ (a * b) • C.mulStab ⊆ s * t
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.mulStab_union
[84, 1]
[131, 73]
exact hab.trans (mul_subset_mul inter_subset_left inter_subset_left)
case inr.inr.intro.intro.h₂ α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hs₁ : (s ∩ a • C.mulStab).Nonempty ht₁ : (t ∩ b • C.mulStab).Nonempty hC : Disjoint C (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) hCne : C.Nonempty x : α hx : x • C ∪ x • (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)) = C ∪ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) h : (x • C ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty y : α hy : y ∈ C hyne : ((x * y) • C.mulStab ∩ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab))).Nonempty hxyCsubC : (x * y) • C.mulStab ⊆ x • C hxyC : Disjoint ((x * y) • C.mulStab) C hxysub : (x * y) • C.mulStab ⊆ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) hab : (a * b) • C.mulStab ⊆ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) ⊢ (a * b) • C.mulStab ⊆ s * t
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.mul_aux1
[133, 1]
[158, 69]
set H := C.mulStab
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α ih : (s' * (s' * t').mulStab).card + (t' * (s' * t').mulStab).card ≤ (s' * t').card + (s' * t').mulStab.card hconv : (s ∩ t).card + ((s ∪ t) * C.mulStab).card ≤ C.card + C.mulStab.card hnotconv : (C ∪ s' * t').card + (C ∪ s' * t').mulStab.card < (s ∩ t).card + ((s ∪ t) * (C ∪ s' * t').mulStab).card hCun : (C ∪ s' * t').mulStab = (s' * t').mulStab hsub : (s' * t').mulStab ⊆ C.mulStab hdisj : Disjoint C (s' * t') ⊢ ↑((s ∪ t) * C.mulStab).card - ↑((s ∪ t) * (s' * t').mulStab).card < ↑C.mulStab.card - ↑(s' * (s' * t').mulStab).card - ↑(t' * (s' * t').mulStab).card
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α ih : (s' * (s' * t').mulStab).card + (t' * (s' * t').mulStab).card ≤ (s' * t').card + (s' * t').mulStab.card hnotconv : (C ∪ s' * t').card + (C ∪ s' * t').mulStab.card < (s ∩ t).card + ((s ∪ t) * (C ∪ s' * t').mulStab).card hCun : (C ∪ s' * t').mulStab = (s' * t').mulStab hdisj : Disjoint C (s' * t') H : Finset α := C.mulStab hconv : (s ∩ t).card + ((s ∪ t) * H).card ≤ C.card + H.card hsub : (s' * t').mulStab ⊆ H ⊢ ↑((s ∪ t) * H).card - ↑((s ∪ t) * (s' * t').mulStab).card < ↑H.card - ↑(s' * (s' * t').mulStab).card - ↑(t' * (s' * t').mulStab).card
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.mul_aux1
[133, 1]
[158, 69]
set H' := (s' * t').mulStab
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α ih : (s' * (s' * t').mulStab).card + (t' * (s' * t').mulStab).card ≤ (s' * t').card + (s' * t').mulStab.card hnotconv : (C ∪ s' * t').card + (C ∪ s' * t').mulStab.card < (s ∩ t).card + ((s ∪ t) * (C ∪ s' * t').mulStab).card hCun : (C ∪ s' * t').mulStab = (s' * t').mulStab hdisj : Disjoint C (s' * t') H : Finset α := C.mulStab hconv : (s ∩ t).card + ((s ∪ t) * H).card ≤ C.card + H.card hsub : (s' * t').mulStab ⊆ H ⊢ ↑((s ∪ t) * H).card - ↑((s ∪ t) * (s' * t').mulStab).card < ↑H.card - ↑(s' * (s' * t').mulStab).card - ↑(t' * (s' * t').mulStab).card
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hnotconv : (C ∪ s' * t').card + (C ∪ s' * t').mulStab.card < (s ∩ t).card + ((s ∪ t) * (C ∪ s' * t').mulStab).card hdisj : Disjoint C (s' * t') H : Finset α := C.mulStab hconv : (s ∩ t).card + ((s ∪ t) * H).card ≤ C.card + H.card H' : Finset α := (s' * t').mulStab ih : (s' * H').card + (t' * H').card ≤ (s' * t').card + H'.card hCun : (C ∪ s' * t').mulStab = H' hsub : H' ⊆ H ⊢ ↑((s ∪ t) * H).card - ↑((s ∪ t) * H').card < ↑H.card - ↑(s' * H').card - ↑(t' * H').card
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.mul_aux1
[133, 1]
[158, 69]
set C' := C ∪ s' * t'
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hnotconv : (C ∪ s' * t').card + (C ∪ s' * t').mulStab.card < (s ∩ t).card + ((s ∪ t) * (C ∪ s' * t').mulStab).card hdisj : Disjoint C (s' * t') H : Finset α := C.mulStab hconv : (s ∩ t).card + ((s ∪ t) * H).card ≤ C.card + H.card H' : Finset α := (s' * t').mulStab ih : (s' * H').card + (t' * H').card ≤ (s' * t').card + H'.card hCun : (C ∪ s' * t').mulStab = H' hsub : H' ⊆ H ⊢ ↑((s ∪ t) * H).card - ↑((s ∪ t) * H').card < ↑H.card - ↑(s' * H').card - ↑(t' * H').card
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hdisj : Disjoint C (s' * t') H : Finset α := C.mulStab hconv : (s ∩ t).card + ((s ∪ t) * H).card ≤ C.card + H.card H' : Finset α := (s' * t').mulStab ih : (s' * H').card + (t' * H').card ≤ (s' * t').card + H'.card hsub : H' ⊆ H C' : Finset α := C ∪ s' * t' hnotconv : C'.card + C'.mulStab.card < (s ∩ t).card + ((s ∪ t) * C'.mulStab).card hCun : C'.mulStab = H' ⊢ ↑((s ∪ t) * H).card - ↑((s ∪ t) * H').card < ↑H.card - ↑(s' * H').card - ↑(t' * H').card
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.mul_aux1
[133, 1]
[158, 69]
zify at hconv hnotconv ih
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hdisj : Disjoint C (s' * t') H : Finset α := C.mulStab hconv : (s ∩ t).card + ((s ∪ t) * H).card ≤ C.card + H.card H' : Finset α := (s' * t').mulStab ih : (s' * H').card + (t' * H').card ≤ (s' * t').card + H'.card hsub : H' ⊆ H C' : Finset α := C ∪ s' * t' hnotconv : C'.card + C'.mulStab.card < (s ∩ t).card + ((s ∪ t) * C'.mulStab).card hCun : C'.mulStab = H' ⊢ ↑((s ∪ t) * H).card - ↑((s ∪ t) * H').card < ↑H.card - ↑(s' * H').card - ↑(t' * H').card
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hdisj : Disjoint C (s' * t') H : Finset α := C.mulStab H' : Finset α := (s' * t').mulStab hsub : H' ⊆ H C' : Finset α := C ∪ s' * t' hCun : C'.mulStab = H' hconv : ↑(s ∩ t).card + ↑((s ∪ t) * H).card ≤ ↑C.card + ↑H.card hnotconv : ↑C'.card + ↑C'.mulStab.card < ↑(s ∩ t).card + ↑((s ∪ t) * C'.mulStab).card ih : ↑(s' * H').card + ↑(t' * H').card ≤ ↑(s' * t').card + ↑H'.card ⊢ ↑((s ∪ t) * H).card - ↑((s ∪ t) * H').card < ↑H.card - ↑(s' * H').card - ↑(t' * H').card
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.mul_aux1
[133, 1]
[158, 69]
calc (((s ∪ t) * H).card - ((s ∪ t) * H').card : ℤ) < C.card + H.card - (s ∩ t).card - (C'.card + H'.card - (s ∩ t).card) := by rw [← hCun] linarith [hconv, hnotconv] _ = H.card - (s' * t').card - H'.card := by rw [card_union_of_disjoint hdisj, Int.ofNat_add] abel _ ≤ H.card - (s' * H').card - (t' * H').card := by linarith [ih]
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hdisj : Disjoint C (s' * t') H : Finset α := C.mulStab H' : Finset α := (s' * t').mulStab hsub : H' ⊆ H C' : Finset α := C ∪ s' * t' hCun : C'.mulStab = H' hconv : ↑(s ∩ t).card + ↑((s ∪ t) * H).card ≤ ↑C.card + ↑H.card hnotconv : ↑C'.card + ↑C'.mulStab.card < ↑(s ∩ t).card + ↑((s ∪ t) * C'.mulStab).card ih : ↑(s' * H').card + ↑(t' * H').card ≤ ↑(s' * t').card + ↑H'.card ⊢ ↑((s ∪ t) * H).card - ↑((s ∪ t) * H').card < ↑H.card - ↑(s' * H').card - ↑(t' * H').card
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.mul_aux1
[133, 1]
[158, 69]
rw [← hCun]
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hdisj : Disjoint C (s' * t') H : Finset α := C.mulStab H' : Finset α := (s' * t').mulStab hsub : H' ⊆ H C' : Finset α := C ∪ s' * t' hCun : C'.mulStab = H' hconv : ↑(s ∩ t).card + ↑((s ∪ t) * H).card ≤ ↑C.card + ↑H.card hnotconv : ↑C'.card + ↑C'.mulStab.card < ↑(s ∩ t).card + ↑((s ∪ t) * C'.mulStab).card ih : ↑(s' * H').card + ↑(t' * H').card ≤ ↑(s' * t').card + ↑H'.card ⊢ ↑((s ∪ t) * H).card - ↑((s ∪ t) * H').card < ↑C.card + ↑H.card - ↑(s ∩ t).card - (↑C'.card + ↑H'.card - ↑(s ∩ t).card)
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hdisj : Disjoint C (s' * t') H : Finset α := C.mulStab H' : Finset α := (s' * t').mulStab hsub : H' ⊆ H C' : Finset α := C ∪ s' * t' hCun : C'.mulStab = H' hconv : ↑(s ∩ t).card + ↑((s ∪ t) * H).card ≤ ↑C.card + ↑H.card hnotconv : ↑C'.card + ↑C'.mulStab.card < ↑(s ∩ t).card + ↑((s ∪ t) * C'.mulStab).card ih : ↑(s' * H').card + ↑(t' * H').card ≤ ↑(s' * t').card + ↑H'.card ⊢ ↑((s ∪ t) * H).card - ↑((s ∪ t) * C'.mulStab).card < ↑C.card + ↑H.card - ↑(s ∩ t).card - (↑C'.card + ↑C'.mulStab.card - ↑(s ∩ t).card)
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.mul_aux1
[133, 1]
[158, 69]
linarith [hconv, hnotconv]
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hdisj : Disjoint C (s' * t') H : Finset α := C.mulStab H' : Finset α := (s' * t').mulStab hsub : H' ⊆ H C' : Finset α := C ∪ s' * t' hCun : C'.mulStab = H' hconv : ↑(s ∩ t).card + ↑((s ∪ t) * H).card ≤ ↑C.card + ↑H.card hnotconv : ↑C'.card + ↑C'.mulStab.card < ↑(s ∩ t).card + ↑((s ∪ t) * C'.mulStab).card ih : ↑(s' * H').card + ↑(t' * H').card ≤ ↑(s' * t').card + ↑H'.card ⊢ ↑((s ∪ t) * H).card - ↑((s ∪ t) * C'.mulStab).card < ↑C.card + ↑H.card - ↑(s ∩ t).card - (↑C'.card + ↑C'.mulStab.card - ↑(s ∩ t).card)
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.mul_aux1
[133, 1]
[158, 69]
rw [card_union_of_disjoint hdisj, Int.ofNat_add]
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hdisj : Disjoint C (s' * t') H : Finset α := C.mulStab H' : Finset α := (s' * t').mulStab hsub : H' ⊆ H C' : Finset α := C ∪ s' * t' hCun : C'.mulStab = H' hconv : ↑(s ∩ t).card + ↑((s ∪ t) * H).card ≤ ↑C.card + ↑H.card hnotconv : ↑C'.card + ↑C'.mulStab.card < ↑(s ∩ t).card + ↑((s ∪ t) * C'.mulStab).card ih : ↑(s' * H').card + ↑(t' * H').card ≤ ↑(s' * t').card + ↑H'.card ⊢ ↑C.card + ↑H.card - ↑(s ∩ t).card - (↑C'.card + ↑H'.card - ↑(s ∩ t).card) = ↑H.card - ↑(s' * t').card - ↑H'.card
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hdisj : Disjoint C (s' * t') H : Finset α := C.mulStab H' : Finset α := (s' * t').mulStab hsub : H' ⊆ H C' : Finset α := C ∪ s' * t' hCun : C'.mulStab = H' hconv : ↑(s ∩ t).card + ↑((s ∪ t) * H).card ≤ ↑C.card + ↑H.card hnotconv : ↑C'.card + ↑C'.mulStab.card < ↑(s ∩ t).card + ↑((s ∪ t) * C'.mulStab).card ih : ↑(s' * H').card + ↑(t' * H').card ≤ ↑(s' * t').card + ↑H'.card ⊢ ↑C.card + ↑H.card - ↑(s ∩ t).card - (↑C.card + ↑(s' * t').card + ↑H'.card - ↑(s ∩ t).card) = ↑H.card - ↑(s' * t').card - ↑H'.card
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.mul_aux1
[133, 1]
[158, 69]
abel
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hdisj : Disjoint C (s' * t') H : Finset α := C.mulStab H' : Finset α := (s' * t').mulStab hsub : H' ⊆ H C' : Finset α := C ∪ s' * t' hCun : C'.mulStab = H' hconv : ↑(s ∩ t).card + ↑((s ∪ t) * H).card ≤ ↑C.card + ↑H.card hnotconv : ↑C'.card + ↑C'.mulStab.card < ↑(s ∩ t).card + ↑((s ∪ t) * C'.mulStab).card ih : ↑(s' * H').card + ↑(t' * H').card ≤ ↑(s' * t').card + ↑H'.card ⊢ ↑C.card + ↑H.card - ↑(s ∩ t).card - (↑C.card + ↑(s' * t').card + ↑H'.card - ↑(s ∩ t).card) = ↑H.card - ↑(s' * t').card - ↑H'.card
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.mul_aux1
[133, 1]
[158, 69]
linarith [ih]
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hdisj : Disjoint C (s' * t') H : Finset α := C.mulStab H' : Finset α := (s' * t').mulStab hsub : H' ⊆ H C' : Finset α := C ∪ s' * t' hCun : C'.mulStab = H' hconv : ↑(s ∩ t).card + ↑((s ∪ t) * H).card ≤ ↑C.card + ↑H.card hnotconv : ↑C'.card + ↑C'.mulStab.card < ↑(s ∩ t).card + ↑((s ∪ t) * C'.mulStab).card ih : ↑(s' * H').card + ↑(t' * H').card ≤ ↑(s' * t').card + ↑H'.card ⊢ ↑H.card - ↑(s' * t').card - ↑H'.card ≤ ↑H.card - ↑(s' * H').card - ↑(t' * H').card
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.disjoint_smul_mulStab
[160, 1]
[168, 29]
suffices Disjoint (a • s.mulStab) (s * s.mulStab) by simpa [mul_comm, disjoint_comm, mulStab_mul]
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hst : s ⊆ t has : ¬a • s.mulStab ⊆ t ⊢ Disjoint s (a • s.mulStab)
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hst : s ⊆ t has : ¬a • s.mulStab ⊆ t ⊢ Disjoint (a • s.mulStab) (s * s.mulStab)
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.disjoint_smul_mulStab
[160, 1]
[168, 29]
apply disjoint_smul_finset_mulStab_mul_mulStab
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hst : s ⊆ t has : ¬a • s.mulStab ⊆ t ⊢ Disjoint (a • s.mulStab) (s * s.mulStab)
case a α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hst : s ⊆ t has : ¬a • s.mulStab ⊆ t ⊢ ¬a • s.mulStab ⊆ s * s.mulStab
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.disjoint_smul_mulStab
[160, 1]
[168, 29]
rw [mul_comm, mulStab_mul]
case a α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hst : s ⊆ t has : ¬a • s.mulStab ⊆ t ⊢ ¬a • s.mulStab ⊆ s * s.mulStab
case a α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hst : s ⊆ t has : ¬a • s.mulStab ⊆ t ⊢ ¬a • s.mulStab ⊆ s
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.disjoint_smul_mulStab
[160, 1]
[168, 29]
contrapose! has
case a α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hst : s ⊆ t has : ¬a • s.mulStab ⊆ t ⊢ ¬a • s.mulStab ⊆ s
case a α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hst : s ⊆ t has : a • s.mulStab ⊆ s ⊢ a • s.mulStab ⊆ t
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.disjoint_smul_mulStab
[160, 1]
[168, 29]
exact subset_trans has hst
case a α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hst : s ⊆ t has : a • s.mulStab ⊆ s ⊢ a • s.mulStab ⊆ t
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.disjoint_smul_mulStab
[160, 1]
[168, 29]
simpa [mul_comm, disjoint_comm, mulStab_mul]
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s s' t t' C : Finset α a b : α hst : s ⊆ t has : ¬a • s.mulStab ⊆ t this : Disjoint (a • s.mulStab) (s * s.mulStab) ⊢ Disjoint s (a • s.mulStab)
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.disjoint_mul_sub_card_le
[170, 1]
[218, 55]
obtain rfl | hC := C.eq_empty_or_nonempty
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C✝ : Finset α a✝ b✝ a b : α s t C : Finset α has : a ∈ s hsC : Disjoint t (a • C.mulStab) hst : (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊆ C.mulStab ⊢ ↑C.mulStab.card - ↑(s ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab).card ≤ ↑((s ∪ t) * C.mulStab).card - ↑((s ∪ t) * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab).card
case inl α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C : Finset α a✝ b✝ a b : α s t : Finset α has : a ∈ s hsC : Disjoint t (a • ∅.mulStab) hst : (s ∩ a • ∅.mulStab * (t ∩ b • ∅.mulStab)).mulStab ⊆ ∅.mulStab ⊢ ↑∅.mulStab.card - ↑(s ∩ a • ∅.mulStab * (s ∩ a • ∅.mulStab * (t ∩ b • ∅.mulStab)).mulStab).card ≤ ↑((s ∪ t) * ∅.mulStab).card - ↑((s ∪ t) * (s ∩ a • ∅.mulStab * (t ∩ b • ∅.mulStab)).mulStab).card case inr α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C✝ : Finset α a✝ b✝ a b : α s t C : Finset α has : a ∈ s hsC : Disjoint t (a • C.mulStab) hst : (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊆ C.mulStab hC : C.Nonempty ⊢ ↑C.mulStab.card - ↑(s ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab).card ≤ ↑((s ∪ t) * C.mulStab).card - ↑((s ∪ t) * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab).card
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.disjoint_mul_sub_card_le
[170, 1]
[218, 55]
simp
case inl α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C : Finset α a✝ b✝ a b : α s t : Finset α has : a ∈ s hsC : Disjoint t (a • ∅.mulStab) hst : (s ∩ a • ∅.mulStab * (t ∩ b • ∅.mulStab)).mulStab ⊆ ∅.mulStab ⊢ ↑∅.mulStab.card - ↑(s ∩ a • ∅.mulStab * (s ∩ a • ∅.mulStab * (t ∩ b • ∅.mulStab)).mulStab).card ≤ ↑((s ∪ t) * ∅.mulStab).card - ↑((s ∪ t) * (s ∩ a • ∅.mulStab * (t ∩ b • ∅.mulStab)).mulStab).card
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.disjoint_mul_sub_card_le
[170, 1]
[218, 55]
rw [card_sdiff (subset_trans (mul_subset_mul_left hst) (subset_trans (mul_subset_mul_right inter_subset_right) _)), card_smul_finset, Int.ofNat_sub]
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C✝ : Finset α a✝ b✝ a b : α s t C : Finset α has : a ∈ s hsC : Disjoint t (a • C.mulStab) hst : (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊆ C.mulStab hC : C.Nonempty ⊢ ↑C.mulStab.card - ↑(s ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab).card = ↑(a • C.mulStab \ (s ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab)).card
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C✝ : Finset α a✝ b✝ a b : α s t C : Finset α has : a ∈ s hsC : Disjoint t (a • C.mulStab) hst : (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊆ C.mulStab hC : C.Nonempty ⊢ (s ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab).card ≤ C.mulStab.card α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C✝ : Finset α a✝ b✝ a b : α s t C : Finset α has : a ∈ s hsC : Disjoint t (a • C.mulStab) hst : (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊆ C.mulStab hC : C.Nonempty ⊢ a • C.mulStab * C.mulStab ⊆ a • C.mulStab
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.disjoint_mul_sub_card_le
[170, 1]
[218, 55]
apply le_trans (card_le_card (mul_subset_mul_left hst))
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C✝ : Finset α a✝ b✝ a b : α s t C : Finset α has : a ∈ s hsC : Disjoint t (a • C.mulStab) hst : (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊆ C.mulStab hC : C.Nonempty ⊢ (s ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab).card ≤ C.mulStab.card
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C✝ : Finset α a✝ b✝ a b : α s t C : Finset α has : a ∈ s hsC : Disjoint t (a • C.mulStab) hst : (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊆ C.mulStab hC : C.Nonempty ⊢ (s ∩ a • C.mulStab * C.mulStab).card ≤ C.mulStab.card
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.disjoint_mul_sub_card_le
[170, 1]
[218, 55]
apply le_trans (card_le_card inter_mul_subset) (le_of_le_of_eq (card_le_card inter_subset_right) _)
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C✝ : Finset α a✝ b✝ a b : α s t C : Finset α has : a ∈ s hsC : Disjoint t (a • C.mulStab) hst : (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊆ C.mulStab hC : C.Nonempty ⊢ (s ∩ a • C.mulStab * C.mulStab).card ≤ C.mulStab.card
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C✝ : Finset α a✝ b✝ a b : α s t C : Finset α has : a ∈ s hsC : Disjoint t (a • C.mulStab) hst : (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊆ C.mulStab hC : C.Nonempty ⊢ (a • C.mulStab * C.mulStab).card = C.mulStab.card
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.disjoint_mul_sub_card_le
[170, 1]
[218, 55]
rw [smul_mul_assoc, mulStab_mul_mulStab, card_smul_finset]
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C✝ : Finset α a✝ b✝ a b : α s t C : Finset α has : a ∈ s hsC : Disjoint t (a • C.mulStab) hst : (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊆ C.mulStab hC : C.Nonempty ⊢ (a • C.mulStab * C.mulStab).card = C.mulStab.card
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.disjoint_mul_sub_card_le
[170, 1]
[218, 55]
simp only [smul_mul_assoc, mulStab_mul_mulStab, Subset.rfl]
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C✝ : Finset α a✝ b✝ a b : α s t C : Finset α has : a ∈ s hsC : Disjoint t (a • C.mulStab) hst : (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊆ C.mulStab hC : C.Nonempty ⊢ a • C.mulStab * C.mulStab ⊆ a • C.mulStab
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.disjoint_mul_sub_card_le
[170, 1]
[218, 55]
rw [← Int.ofNat_sub (card_le_card (mul_subset_mul_left hst)), ← card_sdiff (mul_subset_mul_left hst)]
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C✝ : Finset α a✝ b✝ a b : α s t C : Finset α has : a ∈ s hsC : Disjoint t (a • C.mulStab) hst : (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊆ C.mulStab hC : C.Nonempty ⊢ ↑(a • C.mulStab \ (s ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab)).card ≤ ↑((s ∪ t) * C.mulStab).card - ↑((s ∪ t) * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab).card
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C✝ : Finset α a✝ b✝ a b : α s t C : Finset α has : a ∈ s hsC : Disjoint t (a • C.mulStab) hst : (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊆ C.mulStab hC : C.Nonempty ⊢ ↑(a • C.mulStab \ (s ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab)).card ≤ ↑(((s ∪ t) * C.mulStab) \ ((s ∪ t) * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab)).card
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.disjoint_mul_sub_card_le
[170, 1]
[218, 55]
norm_cast
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C✝ : Finset α a✝ b✝ a b : α s t C : Finset α has : a ∈ s hsC : Disjoint t (a • C.mulStab) hst : (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊆ C.mulStab hC : C.Nonempty ⊢ ↑(a • C.mulStab \ (s ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab)).card ≤ ↑(((s ∪ t) * C.mulStab) \ ((s ∪ t) * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab)).card
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C✝ : Finset α a✝ b✝ a b : α s t C : Finset α has : a ∈ s hsC : Disjoint t (a • C.mulStab) hst : (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊆ C.mulStab hC : C.Nonempty ⊢ (a • C.mulStab \ (s ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab)).card ≤ (((s ∪ t) * C.mulStab) \ ((s ∪ t) * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab)).card
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.disjoint_mul_sub_card_le
[170, 1]
[218, 55]
apply card_le_card
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C✝ : Finset α a✝ b✝ a b : α s t C : Finset α has : a ∈ s hsC : Disjoint t (a • C.mulStab) hst : (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊆ C.mulStab hC : C.Nonempty ⊢ (a • C.mulStab \ (s ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab)).card ≤ (((s ∪ t) * C.mulStab) \ ((s ∪ t) * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab)).card
case a α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C✝ : Finset α a✝ b✝ a b : α s t C : Finset α has : a ∈ s hsC : Disjoint t (a • C.mulStab) hst : (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊆ C.mulStab hC : C.Nonempty ⊢ a • C.mulStab \ (s ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab) ⊆ ((s ∪ t) * C.mulStab) \ ((s ∪ t) * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab)
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.disjoint_mul_sub_card_le
[170, 1]
[218, 55]
refine' fun x hx => mem_sdiff.mpr ⟨_, _⟩
case a α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C✝ : Finset α a✝ b✝ a b : α s t C : Finset α has : a ∈ s hsC : Disjoint t (a • C.mulStab) hst : (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊆ C.mulStab hC : C.Nonempty ⊢ a • C.mulStab \ (s ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab) ⊆ ((s ∪ t) * C.mulStab) \ ((s ∪ t) * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab)
case a.refine'_1 α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C✝ : Finset α a✝ b✝ a b : α s t C : Finset α has : a ∈ s hsC : Disjoint t (a • C.mulStab) hst : (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊆ C.mulStab hC : C.Nonempty x : α hx : x ∈ a • C.mulStab \ (s ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab) ⊢ x ∈ (s ∪ t) * C.mulStab case a.refine'_2 α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C✝ : Finset α a✝ b✝ a b : α s t C : Finset α has : a ∈ s hsC : Disjoint t (a • C.mulStab) hst : (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊆ C.mulStab hC : C.Nonempty x : α hx : x ∈ a • C.mulStab \ (s ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab) ⊢ x ∉ (s ∪ t) * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.disjoint_mul_sub_card_le
[170, 1]
[218, 55]
have hx' := (mem_sdiff.mp hx).2
case a.refine'_2 α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C✝ : Finset α a✝ b✝ a b : α s t C : Finset α has : a ∈ s hsC : Disjoint t (a • C.mulStab) hst : (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊆ C.mulStab hC : C.Nonempty x : α hx : x ∈ a • C.mulStab \ (s ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab) ⊢ x ∉ (s ∪ t) * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab
case a.refine'_2 α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C✝ : Finset α a✝ b✝ a b : α s t C : Finset α has : a ∈ s hsC : Disjoint t (a • C.mulStab) hst : (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊆ C.mulStab hC : C.Nonempty x : α hx : x ∈ a • C.mulStab \ (s ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab) hx' : x ∉ s ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊢ x ∉ (s ∪ t) * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.disjoint_mul_sub_card_le
[170, 1]
[218, 55]
contrapose! hx'
case a.refine'_2 α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C✝ : Finset α a✝ b✝ a b : α s t C : Finset α has : a ∈ s hsC : Disjoint t (a • C.mulStab) hst : (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊆ C.mulStab hC : C.Nonempty x : α hx : x ∈ a • C.mulStab \ (s ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab) hx' : x ∉ s ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊢ x ∉ (s ∪ t) * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab
case a.refine'_2 α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C✝ : Finset α a✝ b✝ a b : α s t C : Finset α has : a ∈ s hsC : Disjoint t (a • C.mulStab) hst : (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊆ C.mulStab hC : C.Nonempty x : α hx : x ∈ a • C.mulStab \ (s ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab) hx' : x ∈ (s ∪ t) * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊢ x ∈ s ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.disjoint_mul_sub_card_le
[170, 1]
[218, 55]
obtain ⟨y, hyst, d, hd, hxyd⟩ := mem_mul.mp hx'
case a.refine'_2 α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C✝ : Finset α a✝ b✝ a b : α s t C : Finset α has : a ∈ s hsC : Disjoint t (a • C.mulStab) hst : (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊆ C.mulStab hC : C.Nonempty x : α hx : x ∈ a • C.mulStab \ (s ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab) hx' : x ∈ (s ∪ t) * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊢ x ∈ s ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab
case a.refine'_2.intro.intro.intro.intro α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C✝ : Finset α a✝ b✝ a b : α s t C : Finset α has : a ∈ s hsC : Disjoint t (a • C.mulStab) hst : (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊆ C.mulStab hC : C.Nonempty x : α hx : x ∈ a • C.mulStab \ (s ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab) hx' : x ∈ (s ∪ t) * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab y : α hyst : y ∈ s ∪ t d : α hd : d ∈ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab hxyd : y * d = x ⊢ x ∈ s ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.disjoint_mul_sub_card_le
[170, 1]
[218, 55]
obtain ⟨c, hc, hcx⟩ := mem_smul_finset.mp (mem_sdiff.mp hx).1
case a.refine'_2.intro.intro.intro.intro α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C✝ : Finset α a✝ b✝ a b : α s t C : Finset α has : a ∈ s hsC : Disjoint t (a • C.mulStab) hst : (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊆ C.mulStab hC : C.Nonempty x : α hx : x ∈ a • C.mulStab \ (s ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab) hx' : x ∈ (s ∪ t) * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab y : α hyst : y ∈ s ∪ t d : α hd : d ∈ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab hxyd : y * d = x ⊢ x ∈ s ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab
case a.refine'_2.intro.intro.intro.intro.intro.intro α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C✝ : Finset α a✝ b✝ a b : α s t C : Finset α has : a ∈ s hsC : Disjoint t (a • C.mulStab) hst : (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊆ C.mulStab hC : C.Nonempty x : α hx : x ∈ a • C.mulStab \ (s ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab) hx' : x ∈ (s ∪ t) * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab y : α hyst : y ∈ s ∪ t d : α hd : d ∈ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab hxyd : y * d = x c : α hc : c ∈ C.mulStab hcx : a • c = x ⊢ x ∈ s ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.disjoint_mul_sub_card_le
[170, 1]
[218, 55]
rw [← hcx, ← eq_mul_inv_iff_mul_eq] at hxyd
case a.refine'_2.intro.intro.intro.intro.intro.intro α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C✝ : Finset α a✝ b✝ a b : α s t C : Finset α has : a ∈ s hsC : Disjoint t (a • C.mulStab) hst : (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊆ C.mulStab hC : C.Nonempty x : α hx : x ∈ a • C.mulStab \ (s ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab) hx' : x ∈ (s ∪ t) * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab y : α hyst : y ∈ s ∪ t d : α hd : d ∈ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab hxyd : y * d = x c : α hc : c ∈ C.mulStab hcx : a • c = x ⊢ x ∈ s ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab
case a.refine'_2.intro.intro.intro.intro.intro.intro α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C✝ : Finset α a✝ b✝ a b : α s t C : Finset α has : a ∈ s hsC : Disjoint t (a • C.mulStab) hst : (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊆ C.mulStab hC : C.Nonempty x : α hx : x ∈ a • C.mulStab \ (s ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab) hx' : x ∈ (s ∪ t) * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab y : α hyst : y ∈ s ∪ t d : α hd : d ∈ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab c : α hxyd : y = a • c * d⁻¹ hc : c ∈ C.mulStab hcx : a • c = x ⊢ x ∈ s ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.disjoint_mul_sub_card_le
[170, 1]
[218, 55]
have hyC : y ∈ a • C.mulStab := by rw [hxyd, smul_mul_assoc, smul_mem_smul_finset_iff, ← mulStab_mul_mulStab] apply mul_mem_mul hc ((mem_mulStab hC).mpr (inv_smul_eq_iff.mpr _)) exact Eq.symm ((mem_mulStab hC).mp (hst hd))
case a.refine'_2.intro.intro.intro.intro.intro.intro α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C✝ : Finset α a✝ b✝ a b : α s t C : Finset α has : a ∈ s hsC : Disjoint t (a • C.mulStab) hst : (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊆ C.mulStab hC : C.Nonempty x : α hx : x ∈ a • C.mulStab \ (s ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab) hx' : x ∈ (s ∪ t) * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab y : α hyst : y ∈ s ∪ t d : α hd : d ∈ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab c : α hxyd : y = a • c * d⁻¹ hc : c ∈ C.mulStab hcx : a • c = x ⊢ x ∈ s ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab
case a.refine'_2.intro.intro.intro.intro.intro.intro α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C✝ : Finset α a✝ b✝ a b : α s t C : Finset α has : a ∈ s hsC : Disjoint t (a • C.mulStab) hst : (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊆ C.mulStab hC : C.Nonempty x : α hx : x ∈ a • C.mulStab \ (s ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab) hx' : x ∈ (s ∪ t) * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab y : α hyst : y ∈ s ∪ t d : α hd : d ∈ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab c : α hxyd : y = a • c * d⁻¹ hc : c ∈ C.mulStab hcx : a • c = x hyC : y ∈ a • C.mulStab ⊢ x ∈ s ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.disjoint_mul_sub_card_le
[170, 1]
[218, 55]
replace hyst : y ∈ s := by apply or_iff_not_imp_right.mp (mem_union.mp hyst) contrapose! hsC exact not_disjoint_iff.mpr ⟨y, hsC, hyC⟩
case a.refine'_2.intro.intro.intro.intro.intro.intro α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C✝ : Finset α a✝ b✝ a b : α s t C : Finset α has : a ∈ s hsC : Disjoint t (a • C.mulStab) hst : (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊆ C.mulStab hC : C.Nonempty x : α hx : x ∈ a • C.mulStab \ (s ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab) hx' : x ∈ (s ∪ t) * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab y : α hyst : y ∈ s ∪ t d : α hd : d ∈ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab c : α hxyd : y = a • c * d⁻¹ hc : c ∈ C.mulStab hcx : a • c = x hyC : y ∈ a • C.mulStab ⊢ x ∈ s ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab
case a.refine'_2.intro.intro.intro.intro.intro.intro α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C✝ : Finset α a✝ b✝ a b : α s t C : Finset α has : a ∈ s hsC : Disjoint t (a • C.mulStab) hst : (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊆ C.mulStab hC : C.Nonempty x : α hx : x ∈ a • C.mulStab \ (s ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab) hx' : x ∈ (s ∪ t) * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab y d : α hd : d ∈ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab c : α hxyd : y = a • c * d⁻¹ hc : c ∈ C.mulStab hcx : a • c = x hyC : y ∈ a • C.mulStab hyst : y ∈ s ⊢ x ∈ s ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.disjoint_mul_sub_card_le
[170, 1]
[218, 55]
rw [eq_mul_inv_iff_mul_eq, hcx] at hxyd
case a.refine'_2.intro.intro.intro.intro.intro.intro α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C✝ : Finset α a✝ b✝ a b : α s t C : Finset α has : a ∈ s hsC : Disjoint t (a • C.mulStab) hst : (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊆ C.mulStab hC : C.Nonempty x : α hx : x ∈ a • C.mulStab \ (s ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab) hx' : x ∈ (s ∪ t) * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab y d : α hd : d ∈ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab c : α hxyd : y = a • c * d⁻¹ hc : c ∈ C.mulStab hcx : a • c = x hyC : y ∈ a • C.mulStab hyst : y ∈ s ⊢ x ∈ s ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab
case a.refine'_2.intro.intro.intro.intro.intro.intro α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C✝ : Finset α a✝ b✝ a b : α s t C : Finset α has : a ∈ s hsC : Disjoint t (a • C.mulStab) hst : (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊆ C.mulStab hC : C.Nonempty x : α hx : x ∈ a • C.mulStab \ (s ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab) hx' : x ∈ (s ∪ t) * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab y d : α hd : d ∈ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab c : α hxyd : y * d = x hc : c ∈ C.mulStab hcx : a • c = x hyC : y ∈ a • C.mulStab hyst : y ∈ s ⊢ x ∈ s ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.disjoint_mul_sub_card_le
[170, 1]
[218, 55]
rw [← hxyd]
case a.refine'_2.intro.intro.intro.intro.intro.intro α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C✝ : Finset α a✝ b✝ a b : α s t C : Finset α has : a ∈ s hsC : Disjoint t (a • C.mulStab) hst : (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊆ C.mulStab hC : C.Nonempty x : α hx : x ∈ a • C.mulStab \ (s ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab) hx' : x ∈ (s ∪ t) * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab y d : α hd : d ∈ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab c : α hxyd : y * d = x hc : c ∈ C.mulStab hcx : a • c = x hyC : y ∈ a • C.mulStab hyst : y ∈ s ⊢ x ∈ s ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab
case a.refine'_2.intro.intro.intro.intro.intro.intro α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C✝ : Finset α a✝ b✝ a b : α s t C : Finset α has : a ∈ s hsC : Disjoint t (a • C.mulStab) hst : (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊆ C.mulStab hC : C.Nonempty x : α hx : x ∈ a • C.mulStab \ (s ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab) hx' : x ∈ (s ∪ t) * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab y d : α hd : d ∈ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab c : α hxyd : y * d = x hc : c ∈ C.mulStab hcx : a • c = x hyC : y ∈ a • C.mulStab hyst : y ∈ s ⊢ y * d ∈ s ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.disjoint_mul_sub_card_le
[170, 1]
[218, 55]
exact mul_mem_mul (mem_inter.mpr ⟨hyst, hyC⟩) hd
case a.refine'_2.intro.intro.intro.intro.intro.intro α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C✝ : Finset α a✝ b✝ a b : α s t C : Finset α has : a ∈ s hsC : Disjoint t (a • C.mulStab) hst : (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊆ C.mulStab hC : C.Nonempty x : α hx : x ∈ a • C.mulStab \ (s ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab) hx' : x ∈ (s ∪ t) * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab y d : α hd : d ∈ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab c : α hxyd : y * d = x hc : c ∈ C.mulStab hcx : a • c = x hyC : y ∈ a • C.mulStab hyst : y ∈ s ⊢ y * d ∈ s ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.disjoint_mul_sub_card_le
[170, 1]
[218, 55]
apply smul_finset_subset_smul (mem_union_left t has) (mem_sdiff.mp hx).1
case a.refine'_1 α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C✝ : Finset α a✝ b✝ a b : α s t C : Finset α has : a ∈ s hsC : Disjoint t (a • C.mulStab) hst : (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊆ C.mulStab hC : C.Nonempty x : α hx : x ∈ a • C.mulStab \ (s ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab) ⊢ x ∈ (s ∪ t) * C.mulStab
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.disjoint_mul_sub_card_le
[170, 1]
[218, 55]
rw [hxyd, smul_mul_assoc, smul_mem_smul_finset_iff, ← mulStab_mul_mulStab]
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C✝ : Finset α a✝ b✝ a b : α s t C : Finset α has : a ∈ s hsC : Disjoint t (a • C.mulStab) hst : (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊆ C.mulStab hC : C.Nonempty x : α hx : x ∈ a • C.mulStab \ (s ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab) hx' : x ∈ (s ∪ t) * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab y : α hyst : y ∈ s ∪ t d : α hd : d ∈ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab c : α hxyd : y = a • c * d⁻¹ hc : c ∈ C.mulStab hcx : a • c = x ⊢ y ∈ a • C.mulStab
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C✝ : Finset α a✝ b✝ a b : α s t C : Finset α has : a ∈ s hsC : Disjoint t (a • C.mulStab) hst : (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊆ C.mulStab hC : C.Nonempty x : α hx : x ∈ a • C.mulStab \ (s ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab) hx' : x ∈ (s ∪ t) * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab y : α hyst : y ∈ s ∪ t d : α hd : d ∈ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab c : α hxyd : y = a • c * d⁻¹ hc : c ∈ C.mulStab hcx : a • c = x ⊢ c * d⁻¹ ∈ C.mulStab * C.mulStab
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.disjoint_mul_sub_card_le
[170, 1]
[218, 55]
apply mul_mem_mul hc ((mem_mulStab hC).mpr (inv_smul_eq_iff.mpr _))
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C✝ : Finset α a✝ b✝ a b : α s t C : Finset α has : a ∈ s hsC : Disjoint t (a • C.mulStab) hst : (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊆ C.mulStab hC : C.Nonempty x : α hx : x ∈ a • C.mulStab \ (s ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab) hx' : x ∈ (s ∪ t) * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab y : α hyst : y ∈ s ∪ t d : α hd : d ∈ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab c : α hxyd : y = a • c * d⁻¹ hc : c ∈ C.mulStab hcx : a • c = x ⊢ c * d⁻¹ ∈ C.mulStab * C.mulStab
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C✝ : Finset α a✝ b✝ a b : α s t C : Finset α has : a ∈ s hsC : Disjoint t (a • C.mulStab) hst : (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊆ C.mulStab hC : C.Nonempty x : α hx : x ∈ a • C.mulStab \ (s ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab) hx' : x ∈ (s ∪ t) * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab y : α hyst : y ∈ s ∪ t d : α hd : d ∈ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab c : α hxyd : y = a • c * d⁻¹ hc : c ∈ C.mulStab hcx : a • c = x ⊢ C = d • C
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.disjoint_mul_sub_card_le
[170, 1]
[218, 55]
exact Eq.symm ((mem_mulStab hC).mp (hst hd))
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C✝ : Finset α a✝ b✝ a b : α s t C : Finset α has : a ∈ s hsC : Disjoint t (a • C.mulStab) hst : (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊆ C.mulStab hC : C.Nonempty x : α hx : x ∈ a • C.mulStab \ (s ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab) hx' : x ∈ (s ∪ t) * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab y : α hyst : y ∈ s ∪ t d : α hd : d ∈ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab c : α hxyd : y = a • c * d⁻¹ hc : c ∈ C.mulStab hcx : a • c = x ⊢ C = d • C
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.disjoint_mul_sub_card_le
[170, 1]
[218, 55]
apply or_iff_not_imp_right.mp (mem_union.mp hyst)
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C✝ : Finset α a✝ b✝ a b : α s t C : Finset α has : a ∈ s hsC : Disjoint t (a • C.mulStab) hst : (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊆ C.mulStab hC : C.Nonempty x : α hx : x ∈ a • C.mulStab \ (s ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab) hx' : x ∈ (s ∪ t) * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab y : α hyst : y ∈ s ∪ t d : α hd : d ∈ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab c : α hxyd : y = a • c * d⁻¹ hc : c ∈ C.mulStab hcx : a • c = x hyC : y ∈ a • C.mulStab ⊢ y ∈ s
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C✝ : Finset α a✝ b✝ a b : α s t C : Finset α has : a ∈ s hsC : Disjoint t (a • C.mulStab) hst : (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊆ C.mulStab hC : C.Nonempty x : α hx : x ∈ a • C.mulStab \ (s ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab) hx' : x ∈ (s ∪ t) * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab y : α hyst : y ∈ s ∪ t d : α hd : d ∈ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab c : α hxyd : y = a • c * d⁻¹ hc : c ∈ C.mulStab hcx : a • c = x hyC : y ∈ a • C.mulStab ⊢ y ∉ t
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.disjoint_mul_sub_card_le
[170, 1]
[218, 55]
contrapose! hsC
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C✝ : Finset α a✝ b✝ a b : α s t C : Finset α has : a ∈ s hsC : Disjoint t (a • C.mulStab) hst : (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊆ C.mulStab hC : C.Nonempty x : α hx : x ∈ a • C.mulStab \ (s ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab) hx' : x ∈ (s ∪ t) * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab y : α hyst : y ∈ s ∪ t d : α hd : d ∈ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab c : α hxyd : y = a • c * d⁻¹ hc : c ∈ C.mulStab hcx : a • c = x hyC : y ∈ a • C.mulStab ⊢ y ∉ t
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C✝ : Finset α a✝ b✝ a b : α s t C : Finset α has : a ∈ s hst : (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊆ C.mulStab hC : C.Nonempty x : α hx : x ∈ a • C.mulStab \ (s ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab) hx' : x ∈ (s ∪ t) * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab y : α hyst : y ∈ s ∪ t d : α hd : d ∈ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab c : α hxyd : y = a • c * d⁻¹ hc : c ∈ C.mulStab hcx : a • c = x hyC : y ∈ a • C.mulStab hsC : y ∈ t ⊢ ¬Disjoint t (a • C.mulStab)
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.disjoint_mul_sub_card_le
[170, 1]
[218, 55]
exact not_disjoint_iff.mpr ⟨y, hsC, hyC⟩
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C✝ : Finset α a✝ b✝ a b : α s t C : Finset α has : a ∈ s hst : (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊆ C.mulStab hC : C.Nonempty x : α hx : x ∈ a • C.mulStab \ (s ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab) hx' : x ∈ (s ∪ t) * (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab y : α hyst : y ∈ s ∪ t d : α hd : d ∈ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab c : α hxyd : y = a • c * d⁻¹ hc : c ∈ C.mulStab hcx : a • c = x hyC : y ∈ a • C.mulStab hsC : y ∈ t ⊢ ¬Disjoint t (a • C.mulStab)
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.inter_mul_sub_card_le
[220, 1]
[267, 55]
obtain rfl | hC := C.eq_empty_or_nonempty
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C✝ : Finset α a✝ b a : α s t C : Finset α has : a ∈ s hst : (s ∩ a • C.mulStab * (t ∩ a • C.mulStab)).mulStab ⊆ C.mulStab ⊢ ↑C.mulStab.card - ↑(s ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ a • C.mulStab)).mulStab).card - ↑(t ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ a • C.mulStab)).mulStab).card ≤ ↑((s ∪ t) * C.mulStab).card - ↑((s ∪ t) * (s ∩ a • C.mulStab * (t ∩ a • C.mulStab)).mulStab).card
case inl α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C : Finset α a✝ b a : α s t : Finset α has : a ∈ s hst : (s ∩ a • ∅.mulStab * (t ∩ a • ∅.mulStab)).mulStab ⊆ ∅.mulStab ⊢ ↑∅.mulStab.card - ↑(s ∩ a • ∅.mulStab * (s ∩ a • ∅.mulStab * (t ∩ a • ∅.mulStab)).mulStab).card - ↑(t ∩ a • ∅.mulStab * (s ∩ a • ∅.mulStab * (t ∩ a • ∅.mulStab)).mulStab).card ≤ ↑((s ∪ t) * ∅.mulStab).card - ↑((s ∪ t) * (s ∩ a • ∅.mulStab * (t ∩ a • ∅.mulStab)).mulStab).card case inr α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C✝ : Finset α a✝ b a : α s t C : Finset α has : a ∈ s hst : (s ∩ a • C.mulStab * (t ∩ a • C.mulStab)).mulStab ⊆ C.mulStab hC : C.Nonempty ⊢ ↑C.mulStab.card - ↑(s ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ a • C.mulStab)).mulStab).card - ↑(t ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ a • C.mulStab)).mulStab).card ≤ ↑((s ∪ t) * C.mulStab).card - ↑((s ∪ t) * (s ∩ a • C.mulStab * (t ∩ a • C.mulStab)).mulStab).card
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.inter_mul_sub_card_le
[220, 1]
[267, 55]
simp
case inl α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C : Finset α a✝ b a : α s t : Finset α has : a ∈ s hst : (s ∩ a • ∅.mulStab * (t ∩ a • ∅.mulStab)).mulStab ⊆ ∅.mulStab ⊢ ↑∅.mulStab.card - ↑(s ∩ a • ∅.mulStab * (s ∩ a • ∅.mulStab * (t ∩ a • ∅.mulStab)).mulStab).card - ↑(t ∩ a • ∅.mulStab * (s ∩ a • ∅.mulStab * (t ∩ a • ∅.mulStab)).mulStab).card ≤ ↑((s ∪ t) * ∅.mulStab).card - ↑((s ∪ t) * (s ∩ a • ∅.mulStab * (t ∩ a • ∅.mulStab)).mulStab).card
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.inter_mul_sub_card_le
[220, 1]
[267, 55]
rw [card_sdiff, Int.ofNat_sub (card_le_card _), card_smul_finset]
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C✝ : Finset α a✝ b a : α s t C : Finset α has : a ∈ s hst : (s ∩ a • C.mulStab * (t ∩ a • C.mulStab)).mulStab ⊆ C.mulStab hC : C.Nonempty ⊢ ↑C.mulStab.card - ↑(s ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ a • C.mulStab)).mulStab).card - ↑(t ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ a • C.mulStab)).mulStab).card ≤ ↑(a • C.mulStab \ ((s ∩ a • C.mulStab ∪ t ∩ a • C.mulStab) * (s ∩ a • C.mulStab * (t ∩ a • C.mulStab)).mulStab)).card
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C✝ : Finset α a✝ b a : α s t C : Finset α has : a ∈ s hst : (s ∩ a • C.mulStab * (t ∩ a • C.mulStab)).mulStab ⊆ C.mulStab hC : C.Nonempty ⊢ ↑C.mulStab.card - ↑(s ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ a • C.mulStab)).mulStab).card - ↑(t ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ a • C.mulStab)).mulStab).card ≤ ↑C.mulStab.card - ↑((s ∩ a • C.mulStab ∪ t ∩ a • C.mulStab) * (s ∩ a • C.mulStab * (t ∩ a • C.mulStab)).mulStab).card α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C✝ : Finset α a✝ b a : α s t C : Finset α has : a ∈ s hst : (s ∩ a • C.mulStab * (t ∩ a • C.mulStab)).mulStab ⊆ C.mulStab hC : C.Nonempty ⊢ (s ∩ a • C.mulStab ∪ t ∩ a • C.mulStab) * (s ∩ a • C.mulStab * (t ∩ a • C.mulStab)).mulStab ⊆ a • C.mulStab α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C✝ : Finset α a✝ b a : α s t C : Finset α has : a ∈ s hst : (s ∩ a • C.mulStab * (t ∩ a • C.mulStab)).mulStab ⊆ C.mulStab hC : C.Nonempty ⊢ (s ∩ a • C.mulStab ∪ t ∩ a • C.mulStab) * (s ∩ a • C.mulStab * (t ∩ a • C.mulStab)).mulStab ⊆ a • C.mulStab
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.inter_mul_sub_card_le
[220, 1]
[267, 55]
all_goals apply subset_trans (mul_subset_mul_left hst) rw [← union_inter_distrib_right] refine' subset_trans (mul_subset_mul_right inter_subset_right) _ simp only [smul_mul_assoc, mulStab_mul_mulStab, Subset.rfl]
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C✝ : Finset α a✝ b a : α s t C : Finset α has : a ∈ s hst : (s ∩ a • C.mulStab * (t ∩ a • C.mulStab)).mulStab ⊆ C.mulStab hC : C.Nonempty ⊢ (s ∩ a • C.mulStab ∪ t ∩ a • C.mulStab) * (s ∩ a • C.mulStab * (t ∩ a • C.mulStab)).mulStab ⊆ a • C.mulStab α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C✝ : Finset α a✝ b a : α s t C : Finset α has : a ∈ s hst : (s ∩ a • C.mulStab * (t ∩ a • C.mulStab)).mulStab ⊆ C.mulStab hC : C.Nonempty ⊢ (s ∩ a • C.mulStab ∪ t ∩ a • C.mulStab) * (s ∩ a • C.mulStab * (t ∩ a • C.mulStab)).mulStab ⊆ a • C.mulStab
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.inter_mul_sub_card_le
[220, 1]
[267, 55]
rw [union_mul, le_sub_iff_add_le]
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C✝ : Finset α a✝ b a : α s t C : Finset α has : a ∈ s hst : (s ∩ a • C.mulStab * (t ∩ a • C.mulStab)).mulStab ⊆ C.mulStab hC : C.Nonempty ⊢ ↑C.mulStab.card - ↑(s ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ a • C.mulStab)).mulStab).card - ↑(t ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ a • C.mulStab)).mulStab).card ≤ ↑C.mulStab.card - ↑((s ∩ a • C.mulStab ∪ t ∩ a • C.mulStab) * (s ∩ a • C.mulStab * (t ∩ a • C.mulStab)).mulStab).card
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C✝ : Finset α a✝ b a : α s t C : Finset α has : a ∈ s hst : (s ∩ a • C.mulStab * (t ∩ a • C.mulStab)).mulStab ⊆ C.mulStab hC : C.Nonempty ⊢ ↑C.mulStab.card - ↑(s ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ a • C.mulStab)).mulStab).card - ↑(t ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ a • C.mulStab)).mulStab).card + ↑(s ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ a • C.mulStab)).mulStab ∪ t ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ a • C.mulStab)).mulStab).card ≤ ↑C.mulStab.card
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.inter_mul_sub_card_le
[220, 1]
[267, 55]
apply le_trans (add_le_add_left (Int.ofNat_le.mpr $ card_union_le _ _) _)
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C✝ : Finset α a✝ b a : α s t C : Finset α has : a ∈ s hst : (s ∩ a • C.mulStab * (t ∩ a • C.mulStab)).mulStab ⊆ C.mulStab hC : C.Nonempty ⊢ ↑C.mulStab.card - ↑(s ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ a • C.mulStab)).mulStab).card - ↑(t ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ a • C.mulStab)).mulStab).card + ↑(s ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ a • C.mulStab)).mulStab ∪ t ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ a • C.mulStab)).mulStab).card ≤ ↑C.mulStab.card
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C✝ : Finset α a✝ b a : α s t C : Finset α has : a ∈ s hst : (s ∩ a • C.mulStab * (t ∩ a • C.mulStab)).mulStab ⊆ C.mulStab hC : C.Nonempty ⊢ ↑C.mulStab.card - ↑(s ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ a • C.mulStab)).mulStab).card - ↑(t ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ a • C.mulStab)).mulStab).card + ↑((s ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ a • C.mulStab)).mulStab).card + (t ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ a • C.mulStab)).mulStab).card) ≤ ↑C.mulStab.card
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.inter_mul_sub_card_le
[220, 1]
[267, 55]
norm_num
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C✝ : Finset α a✝ b a : α s t C : Finset α has : a ∈ s hst : (s ∩ a • C.mulStab * (t ∩ a • C.mulStab)).mulStab ⊆ C.mulStab hC : C.Nonempty ⊢ ↑C.mulStab.card - ↑(s ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ a • C.mulStab)).mulStab).card - ↑(t ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ a • C.mulStab)).mulStab).card + ↑((s ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ a • C.mulStab)).mulStab).card + (t ∩ a • C.mulStab * (s ∩ a • C.mulStab * (t ∩ a • C.mulStab)).mulStab).card) ≤ ↑C.mulStab.card
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.inter_mul_sub_card_le
[220, 1]
[267, 55]
apply subset_trans (mul_subset_mul_left hst)
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C✝ : Finset α a✝ b a : α s t C : Finset α has : a ∈ s hst : (s ∩ a • C.mulStab * (t ∩ a • C.mulStab)).mulStab ⊆ C.mulStab hC : C.Nonempty ⊢ (s ∩ a • C.mulStab ∪ t ∩ a • C.mulStab) * (s ∩ a • C.mulStab * (t ∩ a • C.mulStab)).mulStab ⊆ a • C.mulStab
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C✝ : Finset α a✝ b a : α s t C : Finset α has : a ∈ s hst : (s ∩ a • C.mulStab * (t ∩ a • C.mulStab)).mulStab ⊆ C.mulStab hC : C.Nonempty ⊢ (s ∩ a • C.mulStab ∪ t ∩ a • C.mulStab) * C.mulStab ⊆ a • C.mulStab
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.inter_mul_sub_card_le
[220, 1]
[267, 55]
rw [← union_inter_distrib_right]
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C✝ : Finset α a✝ b a : α s t C : Finset α has : a ∈ s hst : (s ∩ a • C.mulStab * (t ∩ a • C.mulStab)).mulStab ⊆ C.mulStab hC : C.Nonempty ⊢ (s ∩ a • C.mulStab ∪ t ∩ a • C.mulStab) * C.mulStab ⊆ a • C.mulStab
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C✝ : Finset α a✝ b a : α s t C : Finset α has : a ∈ s hst : (s ∩ a • C.mulStab * (t ∩ a • C.mulStab)).mulStab ⊆ C.mulStab hC : C.Nonempty ⊢ (s ∪ t) ∩ a • C.mulStab * C.mulStab ⊆ a • C.mulStab
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.inter_mul_sub_card_le
[220, 1]
[267, 55]
refine' subset_trans (mul_subset_mul_right inter_subset_right) _
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C✝ : Finset α a✝ b a : α s t C : Finset α has : a ∈ s hst : (s ∩ a • C.mulStab * (t ∩ a • C.mulStab)).mulStab ⊆ C.mulStab hC : C.Nonempty ⊢ (s ∪ t) ∩ a • C.mulStab * C.mulStab ⊆ a • C.mulStab
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C✝ : Finset α a✝ b a : α s t C : Finset α has : a ∈ s hst : (s ∩ a • C.mulStab * (t ∩ a • C.mulStab)).mulStab ⊆ C.mulStab hC : C.Nonempty ⊢ a • C.mulStab * C.mulStab ⊆ a • C.mulStab
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.inter_mul_sub_card_le
[220, 1]
[267, 55]
simp only [smul_mul_assoc, mulStab_mul_mulStab, Subset.rfl]
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C✝ : Finset α a✝ b a : α s t C : Finset α has : a ∈ s hst : (s ∩ a • C.mulStab * (t ∩ a • C.mulStab)).mulStab ⊆ C.mulStab hC : C.Nonempty ⊢ a • C.mulStab * C.mulStab ⊆ a • C.mulStab
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.inter_mul_sub_card_le
[220, 1]
[267, 55]
rw [← Int.ofNat_sub (card_le_card (mul_subset_mul_left hst)), ← card_sdiff (mul_subset_mul_left hst)]
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C✝ : Finset α a✝ b a : α s t C : Finset α has : a ∈ s hst : (s ∩ a • C.mulStab * (t ∩ a • C.mulStab)).mulStab ⊆ C.mulStab hC : C.Nonempty ⊢ ↑(a • C.mulStab \ ((s ∩ a • C.mulStab ∪ t ∩ a • C.mulStab) * (s ∩ a • C.mulStab * (t ∩ a • C.mulStab)).mulStab)).card ≤ ↑((s ∪ t) * C.mulStab).card - ↑((s ∪ t) * (s ∩ a • C.mulStab * (t ∩ a • C.mulStab)).mulStab).card
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C✝ : Finset α a✝ b a : α s t C : Finset α has : a ∈ s hst : (s ∩ a • C.mulStab * (t ∩ a • C.mulStab)).mulStab ⊆ C.mulStab hC : C.Nonempty ⊢ ↑(a • C.mulStab \ ((s ∩ a • C.mulStab ∪ t ∩ a • C.mulStab) * (s ∩ a • C.mulStab * (t ∩ a • C.mulStab)).mulStab)).card ≤ ↑(((s ∪ t) * C.mulStab) \ ((s ∪ t) * (s ∩ a • C.mulStab * (t ∩ a • C.mulStab)).mulStab)).card
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.inter_mul_sub_card_le
[220, 1]
[267, 55]
norm_cast
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C✝ : Finset α a✝ b a : α s t C : Finset α has : a ∈ s hst : (s ∩ a • C.mulStab * (t ∩ a • C.mulStab)).mulStab ⊆ C.mulStab hC : C.Nonempty ⊢ ↑(a • C.mulStab \ ((s ∩ a • C.mulStab ∪ t ∩ a • C.mulStab) * (s ∩ a • C.mulStab * (t ∩ a • C.mulStab)).mulStab)).card ≤ ↑(((s ∪ t) * C.mulStab) \ ((s ∪ t) * (s ∩ a • C.mulStab * (t ∩ a • C.mulStab)).mulStab)).card
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C✝ : Finset α a✝ b a : α s t C : Finset α has : a ∈ s hst : (s ∩ a • C.mulStab * (t ∩ a • C.mulStab)).mulStab ⊆ C.mulStab hC : C.Nonempty ⊢ (a • C.mulStab \ ((s ∩ a • C.mulStab ∪ t ∩ a • C.mulStab) * (s ∩ a • C.mulStab * (t ∩ a • C.mulStab)).mulStab)).card ≤ (((s ∪ t) * C.mulStab) \ ((s ∪ t) * (s ∩ a • C.mulStab * (t ∩ a • C.mulStab)).mulStab)).card
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Kneser/Kneser.lean
Finset.inter_mul_sub_card_le
[220, 1]
[267, 55]
apply card_le_card
α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C✝ : Finset α a✝ b a : α s t C : Finset α has : a ∈ s hst : (s ∩ a • C.mulStab * (t ∩ a • C.mulStab)).mulStab ⊆ C.mulStab hC : C.Nonempty ⊢ (a • C.mulStab \ ((s ∩ a • C.mulStab ∪ t ∩ a • C.mulStab) * (s ∩ a • C.mulStab * (t ∩ a • C.mulStab)).mulStab)).card ≤ (((s ∪ t) * C.mulStab) \ ((s ∪ t) * (s ∩ a • C.mulStab * (t ∩ a • C.mulStab)).mulStab)).card
case a α : Type u_1 inst✝¹ : CommGroup α inst✝ : DecidableEq α s✝ s' t✝ t' C✝ : Finset α a✝ b a : α s t C : Finset α has : a ∈ s hst : (s ∩ a • C.mulStab * (t ∩ a • C.mulStab)).mulStab ⊆ C.mulStab hC : C.Nonempty ⊢ a • C.mulStab \ ((s ∩ a • C.mulStab ∪ t ∩ a • C.mulStab) * (s ∩ a • C.mulStab * (t ∩ a • C.mulStab)).mulStab) ⊆ ((s ∪ t) * C.mulStab) \ ((s ∪ t) * (s ∩ a • C.mulStab * (t ∩ a • C.mulStab)).mulStab)