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/SimplicialComplex/Finite.lean | Geometry.SimplicialComplex.locallyFinite_iff_mem_finitely_many_faces | [58, 1] | [82, 88] | unfold LocallyFinite | case mp
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : OrderedRing 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x t✝ : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : DecidableEq E
⊢ K.LocallyFinite → ∀ (x : E), {s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}.Finite | case mp
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : OrderedRing 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x t✝ : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : DecidableEq E
⊢ (∀ ⦃s : Finset E⦄, s ∈ K.faces → s.Nonempty → K.LocallyFiniteAt s) →
∀ (x : E), {s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}.Finite |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Finite.lean | Geometry.SimplicialComplex.locallyFinite_iff_mem_finitely_many_faces | [58, 1] | [82, 88] | contrapose! | case mp
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : OrderedRing 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x t✝ : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : DecidableEq E
⊢ (∀ ⦃s : Finset E⦄, s ∈ K.faces → s.Nonempty → K.LocallyFiniteAt s) →
∀ (x : E), {s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}.Finite | case mp
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : OrderedRing 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x t✝ : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : DecidableEq E
⊢ (∃ x, ¬{s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}.Finite) → ∃ s ∈ K.faces, s.Nonempty ∧ ¬K.LocallyFiniteAt s |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Finite.lean | Geometry.SimplicialComplex.locallyFinite_iff_mem_finitely_many_faces | [58, 1] | [82, 88] | rintro ⟨x, hx⟩ | case mp
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : OrderedRing 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x t✝ : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : DecidableEq E
⊢ (∃ x, ¬{s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}.Finite) → ∃ s ∈ K.faces, s.Nonempty ∧ ¬K.LocallyFiniteAt s | case mp.intro
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : OrderedRing 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x✝ t✝ : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : DecidableEq E
x : E
hx : ¬{s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}.Finite
⊢ ∃ s ∈ K.faces, s.Nonempty ∧ ¬K.LocallyFiniteAt s |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Finite.lean | Geometry.SimplicialComplex.locallyFinite_iff_mem_finitely_many_faces | [58, 1] | [82, 88] | by_cases hxspace : x ∈ K.space | case mp.intro
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : OrderedRing 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x✝ t✝ : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : DecidableEq E
x : E
hx : ¬{s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}.Finite
⊢ ∃ s ∈ K.faces, s.Nonempty ∧ ¬K.LocallyFiniteAt s | case pos
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : OrderedRing 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x✝ t✝ : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : DecidableEq E
x : E
hx : ¬{s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}.Finite
hxspace : x ∈ K.space
⊢ ∃ s ∈ K.faces, s.Nonempty ∧ ¬K.LocallyFiniteAt s
case neg
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : OrderedRing 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x✝ t✝ : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : DecidableEq E
x : E
hx : ¬{s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}.Finite
hxspace : x ∉ K.space
⊢ ∃ s ∈ K.faces, s.Nonempty ∧ ¬K.LocallyFiniteAt s |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Finite.lean | Geometry.SimplicialComplex.locallyFinite_iff_mem_finitely_many_faces | [58, 1] | [82, 88] | obtain ⟨s, ⟨hX, hXhull, hXbound⟩, hXunique⟩ := combiInteriors_partition hxspace | case pos
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : OrderedRing 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x✝ t✝ : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : DecidableEq E
x : E
hx : ¬{s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}.Finite
hxspace : x ∈ K.space
⊢ ∃ s ∈ K.faces, s.Nonempty ∧ ¬K.LocallyFiniteAt s | case pos.intro.intro.intro.intro
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : OrderedRing 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x✝ t✝ : E
s✝ t : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : DecidableEq E
x : E
hx : ¬{s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}.Finite
hxspace : x ∈ K.space
s : Finset E
hXunique : ∀ (y : Finset E), (fun s => s ∈ K ∧ x ∈ combiInterior 𝕜 s) y → y = s
hX : s ∈ K
hXhull : x ∈ (convexHull 𝕜) ↑s
hXbound : x ∉ combiFrontier 𝕜 s
⊢ ∃ s ∈ K.faces, s.Nonempty ∧ ¬K.LocallyFiniteAt s |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Finite.lean | Geometry.SimplicialComplex.locallyFinite_iff_mem_finitely_many_faces | [58, 1] | [82, 88] | simp at hXunique | case pos.intro.intro.intro.intro
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : OrderedRing 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x✝ t✝ : E
s✝ t : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : DecidableEq E
x : E
hx : ¬{s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}.Finite
hxspace : x ∈ K.space
s : Finset E
hXunique : ∀ (y : Finset E), (fun s => s ∈ K ∧ x ∈ combiInterior 𝕜 s) y → y = s
hX : s ∈ K
hXhull : x ∈ (convexHull 𝕜) ↑s
hXbound : x ∉ combiFrontier 𝕜 s
⊢ ∃ s ∈ K.faces, s.Nonempty ∧ ¬K.LocallyFiniteAt s | case pos.intro.intro.intro.intro
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : OrderedRing 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x✝ t✝ : E
s✝ t : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : DecidableEq E
x : E
hx : ¬{s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}.Finite
hxspace : x ∈ K.space
s : Finset E
hX : s ∈ K
hXhull : x ∈ (convexHull 𝕜) ↑s
hXbound : x ∉ combiFrontier 𝕜 s
hXunique : ∀ y ∈ K, x ∈ combiInterior 𝕜 y → y = s
⊢ ∃ s ∈ K.faces, s.Nonempty ∧ ¬K.LocallyFiniteAt s |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Finite.lean | Geometry.SimplicialComplex.locallyFinite_iff_mem_finitely_many_faces | [58, 1] | [82, 88] | refine'
⟨s, hX, Finset.nonempty_of_ne_empty _, fun hXlocallyfinite =>
hx <| hXlocallyfinite.subset fun t hY => ⟨hY.1, _⟩⟩ | case pos.intro.intro.intro.intro
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : OrderedRing 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x✝ t✝ : E
s✝ t : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : DecidableEq E
x : E
hx : ¬{s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}.Finite
hxspace : x ∈ K.space
s : Finset E
hX : s ∈ K
hXhull : x ∈ (convexHull 𝕜) ↑s
hXbound : x ∉ combiFrontier 𝕜 s
hXunique : ∀ y ∈ K, x ∈ combiInterior 𝕜 y → y = s
⊢ ∃ s ∈ K.faces, s.Nonempty ∧ ¬K.LocallyFiniteAt s | case pos.intro.intro.intro.intro.refine'_1
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : OrderedRing 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x✝ t✝ : E
s✝ t : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : DecidableEq E
x : E
hx : ¬{s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}.Finite
hxspace : x ∈ K.space
s : Finset E
hX : s ∈ K
hXhull : x ∈ (convexHull 𝕜) ↑s
hXbound : x ∉ combiFrontier 𝕜 s
hXunique : ∀ y ∈ K, x ∈ combiInterior 𝕜 y → y = s
⊢ s ≠ ∅
case pos.intro.intro.intro.intro.refine'_2
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : OrderedRing 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x✝ t✝¹ : E
s✝ t✝ : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : DecidableEq E
x : E
hx : ¬{s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}.Finite
hxspace : x ∈ K.space
s : Finset E
hX : s ∈ K
hXhull : x ∈ (convexHull 𝕜) ↑s
hXbound : x ∉ combiFrontier 𝕜 s
hXunique : ∀ y ∈ K, x ∈ combiInterior 𝕜 y → y = s
hXlocallyfinite : K.LocallyFiniteAt s
t : Finset E
hY : t ∈ {s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}
⊢ s ⊆ t |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Finite.lean | Geometry.SimplicialComplex.locallyFinite_iff_mem_finitely_many_faces | [58, 1] | [82, 88] | have hXYhull := K.inter_subset_convexHull hX hY.1 ⟨hXhull, hY.2⟩ | case pos.intro.intro.intro.intro.refine'_2
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : OrderedRing 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x✝ t✝¹ : E
s✝ t✝ : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : DecidableEq E
x : E
hx : ¬{s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}.Finite
hxspace : x ∈ K.space
s : Finset E
hX : s ∈ K
hXhull : x ∈ (convexHull 𝕜) ↑s
hXbound : x ∉ combiFrontier 𝕜 s
hXunique : ∀ y ∈ K, x ∈ combiInterior 𝕜 y → y = s
hXlocallyfinite : K.LocallyFiniteAt s
t : Finset E
hY : t ∈ {s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}
⊢ s ⊆ t | case pos.intro.intro.intro.intro.refine'_2
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : OrderedRing 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x✝ t✝¹ : E
s✝ t✝ : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : DecidableEq E
x : E
hx : ¬{s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}.Finite
hxspace : x ∈ K.space
s : Finset E
hX : s ∈ K
hXhull : x ∈ (convexHull 𝕜) ↑s
hXbound : x ∉ combiFrontier 𝕜 s
hXunique : ∀ y ∈ K, x ∈ combiInterior 𝕜 y → y = s
hXlocallyfinite : K.LocallyFiniteAt s
t : Finset E
hY : t ∈ {s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}
hXYhull : x ∈ (convexHull 𝕜) (↑s ∩ ↑t)
⊢ s ⊆ t |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Finite.lean | Geometry.SimplicialComplex.locallyFinite_iff_mem_finitely_many_faces | [58, 1] | [82, 88] | rw [← Finset.coe_inter] at hXYhull | case pos.intro.intro.intro.intro.refine'_2
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : OrderedRing 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x✝ t✝¹ : E
s✝ t✝ : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : DecidableEq E
x : E
hx : ¬{s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}.Finite
hxspace : x ∈ K.space
s : Finset E
hX : s ∈ K
hXhull : x ∈ (convexHull 𝕜) ↑s
hXbound : x ∉ combiFrontier 𝕜 s
hXunique : ∀ y ∈ K, x ∈ combiInterior 𝕜 y → y = s
hXlocallyfinite : K.LocallyFiniteAt s
t : Finset E
hY : t ∈ {s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}
hXYhull : x ∈ (convexHull 𝕜) (↑s ∩ ↑t)
⊢ s ⊆ t | case pos.intro.intro.intro.intro.refine'_2
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : OrderedRing 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x✝ t✝¹ : E
s✝ t✝ : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : DecidableEq E
x : E
hx : ¬{s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}.Finite
hxspace : x ∈ K.space
s : Finset E
hX : s ∈ K
hXhull : x ∈ (convexHull 𝕜) ↑s
hXbound : x ∉ combiFrontier 𝕜 s
hXunique : ∀ y ∈ K, x ∈ combiInterior 𝕜 y → y = s
hXlocallyfinite : K.LocallyFiniteAt s
t : Finset E
hY : t ∈ {s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}
hXYhull : x ∈ (convexHull 𝕜) ↑(s ∩ t)
⊢ s ⊆ t |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Finite.lean | Geometry.SimplicialComplex.locallyFinite_iff_mem_finitely_many_faces | [58, 1] | [82, 88] | by_contra hXY | case pos.intro.intro.intro.intro.refine'_2
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : OrderedRing 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x✝ t✝¹ : E
s✝ t✝ : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : DecidableEq E
x : E
hx : ¬{s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}.Finite
hxspace : x ∈ K.space
s : Finset E
hX : s ∈ K
hXhull : x ∈ (convexHull 𝕜) ↑s
hXbound : x ∉ combiFrontier 𝕜 s
hXunique : ∀ y ∈ K, x ∈ combiInterior 𝕜 y → y = s
hXlocallyfinite : K.LocallyFiniteAt s
t : Finset E
hY : t ∈ {s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}
hXYhull : x ∈ (convexHull 𝕜) ↑(s ∩ t)
⊢ s ⊆ t | case pos.intro.intro.intro.intro.refine'_2
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : OrderedRing 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x✝ t✝¹ : E
s✝ t✝ : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : DecidableEq E
x : E
hx : ¬{s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}.Finite
hxspace : x ∈ K.space
s : Finset E
hX : s ∈ K
hXhull : x ∈ (convexHull 𝕜) ↑s
hXbound : x ∉ combiFrontier 𝕜 s
hXunique : ∀ y ∈ K, x ∈ combiInterior 𝕜 y → y = s
hXlocallyfinite : K.LocallyFiniteAt s
t : Finset E
hY : t ∈ {s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}
hXYhull : x ∈ (convexHull 𝕜) ↑(s ∩ t)
hXY : ¬s ⊆ t
⊢ False |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Finite.lean | Geometry.SimplicialComplex.locallyFinite_iff_mem_finitely_many_faces | [58, 1] | [82, 88] | exact hXbound (mem_combiFrontier_iff.2 ⟨s ∩ t, ⟨Finset.inter_subset_left,
fun hXXY => hXY (Finset.subset_inter_iff.1 hXXY).2⟩, hXYhull⟩) | case pos.intro.intro.intro.intro.refine'_2
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : OrderedRing 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x✝ t✝¹ : E
s✝ t✝ : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : DecidableEq E
x : E
hx : ¬{s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}.Finite
hxspace : x ∈ K.space
s : Finset E
hX : s ∈ K
hXhull : x ∈ (convexHull 𝕜) ↑s
hXbound : x ∉ combiFrontier 𝕜 s
hXunique : ∀ y ∈ K, x ∈ combiInterior 𝕜 y → y = s
hXlocallyfinite : K.LocallyFiniteAt s
t : Finset E
hY : t ∈ {s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}
hXYhull : x ∈ (convexHull 𝕜) ↑(s ∩ t)
hXY : ¬s ⊆ t
⊢ False | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Finite.lean | Geometry.SimplicialComplex.locallyFinite_iff_mem_finitely_many_faces | [58, 1] | [82, 88] | rintro rfl | case pos.intro.intro.intro.intro.refine'_1
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : OrderedRing 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x✝ t✝ : E
s✝ t : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : DecidableEq E
x : E
hx : ¬{s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}.Finite
hxspace : x ∈ K.space
s : Finset E
hX : s ∈ K
hXhull : x ∈ (convexHull 𝕜) ↑s
hXbound : x ∉ combiFrontier 𝕜 s
hXunique : ∀ y ∈ K, x ∈ combiInterior 𝕜 y → y = s
⊢ s ≠ ∅ | case pos.intro.intro.intro.intro.refine'_1
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : OrderedRing 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x✝ t✝ : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : DecidableEq E
x : E
hx : ¬{s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}.Finite
hxspace : x ∈ K.space
hX : ∅ ∈ K
hXhull : x ∈ (convexHull 𝕜) ↑∅
hXbound : x ∉ combiFrontier 𝕜 ∅
hXunique : ∀ y ∈ K, x ∈ combiInterior 𝕜 y → y = ∅
⊢ False |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Finite.lean | Geometry.SimplicialComplex.locallyFinite_iff_mem_finitely_many_faces | [58, 1] | [82, 88] | simp at hXhull | case pos.intro.intro.intro.intro.refine'_1
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : OrderedRing 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x✝ t✝ : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : DecidableEq E
x : E
hx : ¬{s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}.Finite
hxspace : x ∈ K.space
hX : ∅ ∈ K
hXhull : x ∈ (convexHull 𝕜) ↑∅
hXbound : x ∉ combiFrontier 𝕜 ∅
hXunique : ∀ y ∈ K, x ∈ combiInterior 𝕜 y → y = ∅
⊢ False | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Finite.lean | Geometry.SimplicialComplex.locallyFinite_iff_mem_finitely_many_faces | [58, 1] | [82, 88] | refine (hx ?_).elim | case neg
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : OrderedRing 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x✝ t✝ : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : DecidableEq E
x : E
hx : ¬{s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}.Finite
hxspace : x ∉ K.space
⊢ ∃ s ∈ K.faces, s.Nonempty ∧ ¬K.LocallyFiniteAt s | case neg
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : OrderedRing 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x✝ t✝ : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : DecidableEq E
x : E
hx : ¬{s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}.Finite
hxspace : x ∉ K.space
⊢ {s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}.Finite |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Finite.lean | Geometry.SimplicialComplex.locallyFinite_iff_mem_finitely_many_faces | [58, 1] | [82, 88] | convert finite_empty | case neg
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : OrderedRing 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x✝ t✝ : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : DecidableEq E
x : E
hx : ¬{s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}.Finite
hxspace : x ∉ K.space
⊢ {s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}.Finite | case h.e'_2
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : OrderedRing 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x✝ t✝ : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : DecidableEq E
x : E
hx : ¬{s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}.Finite
hxspace : x ∉ K.space
⊢ {s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s} = ∅ |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Finite.lean | Geometry.SimplicialComplex.locallyFinite_iff_mem_finitely_many_faces | [58, 1] | [82, 88] | exact eq_empty_of_forall_not_mem fun s hX => hxspace <| mem_biUnion hX.1 hX.2 | case h.e'_2
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : OrderedRing 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x✝ t✝ : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : DecidableEq E
x : E
hx : ¬{s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}.Finite
hxspace : x ∉ K.space
⊢ {s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s} = ∅ | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Finite.lean | Geometry.SimplicialComplex.locallyFinite_iff_mem_finitely_many_faces | [58, 1] | [82, 88] | rintro hS s - ⟨x, hx⟩ | case mpr
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : OrderedRing 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x t✝ : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : DecidableEq E
⊢ (∀ (x : E), {s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}.Finite) → K.LocallyFinite | case mpr.intro
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : OrderedRing 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x✝ t✝ : E
s✝ t : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : DecidableEq E
hS : ∀ (x : E), {s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}.Finite
s : Finset E
x : E
hx : x ∈ s
⊢ K.LocallyFiniteAt s |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Finite.lean | Geometry.SimplicialComplex.locallyFinite_iff_mem_finitely_many_faces | [58, 1] | [82, 88] | exact (hS x).subset fun t => And.imp_right fun ht => subset_convexHull _ _ <| ht hx | case mpr.intro
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : OrderedRing 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x✝ t✝ : E
s✝ t : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : DecidableEq E
hS : ∀ (x : E), {s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}.Finite
s : Finset E
x : E
hx : x ∈ s
⊢ K.LocallyFiniteAt s | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Kneser/Kneser.lean | Finset.mulStab_mul_ssubset_mulStab | [36, 1] | [82, 79] | have hCne : C.Nonempty := by
contrapose! hab
simp only [not_nonempty_iff_eq_empty] at hab
simp only [hab, mulStab_empty, smul_finset_empty, empty_subset] | α : 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
⊢ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊂ C.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
hCne : C.Nonempty
⊢ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊂ C.mulStab |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Kneser/Kneser.lean | Finset.mulStab_mul_ssubset_mulStab | [36, 1] | [82, 79] | obtain ⟨x, hx⟩ := hs₁ | α : 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
hCne : C.Nonempty
⊢ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊂ C.mulStab | case intro
α : Type u_1
inst✝¹ : CommGroup α
inst✝ : DecidableEq α
s s' t t' C : Finset α
a b : α
ht₁ : (t ∩ b • C.mulStab).Nonempty
hab : ¬(a * b) • C.mulStab ⊆ s * t
hCne : C.Nonempty
x : α
hx : x ∈ s ∩ a • C.mulStab
⊢ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊂ C.mulStab |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Kneser/Kneser.lean | Finset.mulStab_mul_ssubset_mulStab | [36, 1] | [82, 79] | obtain ⟨y, hy⟩ := ht₁ | case intro
α : Type u_1
inst✝¹ : CommGroup α
inst✝ : DecidableEq α
s s' t t' C : Finset α
a b : α
ht₁ : (t ∩ b • C.mulStab).Nonempty
hab : ¬(a * b) • C.mulStab ⊆ s * t
hCne : C.Nonempty
x : α
hx : x ∈ s ∩ a • C.mulStab
⊢ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊂ C.mulStab | case intro.intro
α : 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
⊢ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊂ C.mulStab |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Kneser/Kneser.lean | Finset.mulStab_mul_ssubset_mulStab | [36, 1] | [82, 79] | obtain ⟨c, hc, hac⟩ := mem_smul_finset.mp (mem_of_mem_inter_right hx) | case intro.intro
α : 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
⊢ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊂ C.mulStab | case intro.intro.intro.intro
α : 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
⊢ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊂ C.mulStab |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Kneser/Kneser.lean | Finset.mulStab_mul_ssubset_mulStab | [36, 1] | [82, 79] | obtain ⟨d, hd, had⟩ := mem_smul_finset.mp (mem_of_mem_inter_right hy) | case intro.intro.intro.intro
α : 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
⊢ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊂ C.mulStab | case intro.intro.intro.intro.intro.intro
α : 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
⊢ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊂ C.mulStab |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Kneser/Kneser.lean | Finset.mulStab_mul_ssubset_mulStab | [36, 1] | [82, 79] | have hsubset : (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊆ C.mulStab := by
have hxymem : x * y ∈ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) := mul_mem_mul hx hy
apply subset_trans (mulStab_subset_div_right hxymem)
have : s ∩ a • C.mulStab * (t ∩ b • C.mulStab) ⊆ (x * y) • C.mulStab := by
apply subset_trans (mul_subset_mul inter_subset_right inter_subset_right)
rw [smul_mul_smul]
rw [← hac, ← had, smul_mul_smul, smul_assoc]
apply smul_finset_subset_smul_finset
rw [← smul_smul]
rw [mul_subset_iff]
intro x hx y hy
rw [smul_mulStab hd, smul_mulStab hc, mem_mulStab hCne, ← smul_smul,
(mem_mulStab hCne).mp hy, (mem_mulStab hCne).mp hx]
apply subset_trans (div_subset_div_right this) _
have hsing : (x * y) • C.mulStab = {x * y} * C.mulStab := by rw [singleton_mul]; rfl
simp_rw [hsing, singleton_mul, div_singleton, image_image, div_eq_mul_inv, mul_comm, comp,
mul_inv_cancel_right, image_id', subset_refl] | case intro.intro.intro.intro.intro.intro
α : 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
⊢ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊂ C.mulStab | case intro.intro.intro.intro.intro.intro
α : 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
⊢ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊂ C.mulStab |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Kneser/Kneser.lean | Finset.mulStab_mul_ssubset_mulStab | [36, 1] | [82, 79] | have : (a * b) • C.mulStab = (a * c * (b * d)) • C.mulStab := by
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] | case intro.intro.intro.intro.intro.intro
α : 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
⊢ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊂ C.mulStab | case intro.intro.intro.intro.intro.intro
α : 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)).mulStab ⊂ C.mulStab |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Kneser/Kneser.lean | Finset.mulStab_mul_ssubset_mulStab | [36, 1] | [82, 79] | have hsub : s ∩ a • C.mulStab * (t ∩ b • C.mulStab) ⊆ (a * b) • C.mulStab := by
apply subset_trans (mul_subset_mul inter_subset_right inter_subset_right)
simp only [smul_mul_smul, mulStab_mul_mulStab, subset_refl] | case intro.intro.intro.intro.intro.intro
α : 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)).mulStab ⊂ C.mulStab | case intro.intro.intro.intro.intro.intro
α : 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
hsub : s ∩ a • C.mulStab * (t ∩ b • C.mulStab) ⊆ (a * b) • C.mulStab
⊢ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊂ C.mulStab |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Kneser/Kneser.lean | Finset.mulStab_mul_ssubset_mulStab | [36, 1] | [82, 79] | have hxy : x * y ∈ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) := mul_mem_mul hx hy | case intro.intro.intro.intro.intro.intro
α : 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
hsub : s ∩ a • C.mulStab * (t ∩ b • C.mulStab) ⊆ (a * b) • C.mulStab
⊢ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊂ C.mulStab | case intro.intro.intro.intro.intro.intro
α : 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
hsub : s ∩ a • C.mulStab * (t ∩ b • C.mulStab) ⊆ (a * b) • C.mulStab
hxy : x * y ∈ s ∩ a • C.mulStab * (t ∩ b • C.mulStab)
⊢ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊂ C.mulStab |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Kneser/Kneser.lean | Finset.mulStab_mul_ssubset_mulStab | [36, 1] | [82, 79] | rw [this] at hsub | case intro.intro.intro.intro.intro.intro
α : 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
hsub : s ∩ a • C.mulStab * (t ∩ b • C.mulStab) ⊆ (a * b) • C.mulStab
hxy : x * y ∈ s ∩ a • C.mulStab * (t ∩ b • C.mulStab)
⊢ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊂ C.mulStab | case intro.intro.intro.intro.intro.intro
α : 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
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)
⊢ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊂ C.mulStab |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Kneser/Kneser.lean | Finset.mulStab_mul_ssubset_mulStab | [36, 1] | [82, 79] | rw [this] at hab | case intro.intro.intro.intro.intro.intro
α : 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
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)
⊢ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊂ C.mulStab | case intro.intro.intro.intro.intro.intro
α : 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)
⊢ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊂ C.mulStab |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Kneser/Kneser.lean | Finset.mulStab_mul_ssubset_mulStab | [36, 1] | [82, 79] | obtain ⟨z, hz, hzst⟩ := not_subset.1 hab | case intro.intro.intro.intro.intro.intro
α : 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)
⊢ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊂ C.mulStab | case intro.intro.intro.intro.intro.intro.intro.intro
α : 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
⊢ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊂ C.mulStab |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Kneser/Kneser.lean | Finset.mulStab_mul_ssubset_mulStab | [36, 1] | [82, 79] | obtain ⟨w, hw, hwz⟩ := mem_smul_finset.mp hz | case intro.intro.intro.intro.intro.intro.intro.intro
α : 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
⊢ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊂ C.mulStab | case intro.intro.intro.intro.intro.intro.intro.intro.intro.intro
α : 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
⊢ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊂ C.mulStab |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Kneser/Kneser.lean | Finset.mulStab_mul_ssubset_mulStab | [36, 1] | [82, 79] | refine' (Finset.ssubset_iff_of_subset hsubset).mpr ⟨w, hw, _⟩ | case intro.intro.intro.intro.intro.intro.intro.intro.intro.intro
α : 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
⊢ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊂ C.mulStab | case intro.intro.intro.intro.intro.intro.intro.intro.intro.intro
α : 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
⊢ w ∉ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Kneser/Kneser.lean | Finset.mulStab_mul_ssubset_mulStab | [36, 1] | [82, 79] | rw [mem_mulStab' ⟨x * y, hxy⟩] | case intro.intro.intro.intro.intro.intro.intro.intro.intro.intro
α : 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
⊢ w ∉ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab | case intro.intro.intro.intro.intro.intro.intro.intro.intro.intro
α : 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
⊢ ¬∀ ⦃b_1 : α⦄, b_1 ∈ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) → w • b_1 ∈ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Kneser/Kneser.lean | Finset.mulStab_mul_ssubset_mulStab | [36, 1] | [82, 79] | push_neg | case intro.intro.intro.intro.intro.intro.intro.intro.intro.intro
α : 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
⊢ ¬∀ ⦃b_1 : α⦄, b_1 ∈ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) → w • b_1 ∈ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) | case intro.intro.intro.intro.intro.intro.intro.intro.intro.intro
α : 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
⊢ ∃ b_1 ∈ s ∩ a • C.mulStab * (t ∩ b • C.mulStab), w • b_1 ∉ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Kneser/Kneser.lean | Finset.mulStab_mul_ssubset_mulStab | [36, 1] | [82, 79] | refine' ⟨a * c * (b * d), by convert hxy, _⟩ | case intro.intro.intro.intro.intro.intro.intro.intro.intro.intro
α : 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
⊢ ∃ b_1 ∈ s ∩ a • C.mulStab * (t ∩ b • C.mulStab), w • b_1 ∉ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) | case intro.intro.intro.intro.intro.intro.intro.intro.intro.intro
α : 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
⊢ w • (a * c * (b * d)) ∉ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Kneser/Kneser.lean | Finset.mulStab_mul_ssubset_mulStab | [36, 1] | [82, 79] | rw [smul_eq_mul, mul_comm, ← smul_eq_mul, hwz] | case intro.intro.intro.intro.intro.intro.intro.intro.intro.intro
α : 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
⊢ w • (a * c * (b * d)) ∉ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) | case intro.intro.intro.intro.intro.intro.intro.intro.intro.intro
α : 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
⊢ z ∉ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Kneser/Kneser.lean | Finset.mulStab_mul_ssubset_mulStab | [36, 1] | [82, 79] | exact not_mem_mono (mul_subset_mul inter_subset_left inter_subset_left) hzst | case intro.intro.intro.intro.intro.intro.intro.intro.intro.intro
α : 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
⊢ z ∉ s ∩ a • C.mulStab * (t ∩ 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] | contrapose! hab | α : 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
⊢ C.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 : ¬C.Nonempty
⊢ (a * b) • C.mulStab ⊆ s * t |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Kneser/Kneser.lean | Finset.mulStab_mul_ssubset_mulStab | [36, 1] | [82, 79] | simp only [not_nonempty_iff_eq_empty] at hab | α : 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 : ¬C.Nonempty
⊢ (a * b) • C.mulStab ⊆ s * t | α : 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 : C = ∅
⊢ (a * b) • C.mulStab ⊆ s * t |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Kneser/Kneser.lean | Finset.mulStab_mul_ssubset_mulStab | [36, 1] | [82, 79] | simp only [hab, mulStab_empty, smul_finset_empty, empty_subset] | α : 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 : C = ∅
⊢ (a * b) • C.mulStab ⊆ s * t | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Kneser/Kneser.lean | Finset.mulStab_mul_ssubset_mulStab | [36, 1] | [82, 79] | have hxymem : x * y ∈ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) := mul_mem_mul hx hy | α : 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
⊢ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊆ 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)
⊢ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊆ C.mulStab |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Kneser/Kneser.lean | Finset.mulStab_mul_ssubset_mulStab | [36, 1] | [82, 79] | apply subset_trans (mulStab_subset_div_right hxymem) | α : 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)
⊢ (s ∩ a • C.mulStab * (t ∩ b • C.mulStab)).mulStab ⊆ 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)
⊢ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) / {x * y} ⊆ C.mulStab |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Kneser/Kneser.lean | Finset.mulStab_mul_ssubset_mulStab | [36, 1] | [82, 79] | have : s ∩ a • C.mulStab * (t ∩ b • C.mulStab) ⊆ (x * y) • C.mulStab := by
apply subset_trans (mul_subset_mul inter_subset_right inter_subset_right)
rw [smul_mul_smul]
rw [← hac, ← had, smul_mul_smul, smul_assoc]
apply smul_finset_subset_smul_finset
rw [← smul_smul]
rw [mul_subset_iff]
intro x hx y hy
rw [smul_mulStab hd, smul_mulStab hc, mem_mulStab hCne, ← smul_smul,
(mem_mulStab hCne).mp hy, (mem_mulStab hCne).mp hx] | α : 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)
⊢ s ∩ a • C.mulStab * (t ∩ b • 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
⊢ s ∩ a • C.mulStab * (t ∩ b • C.mulStab) / {x * y} ⊆ C.mulStab |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Kneser/Kneser.lean | Finset.mulStab_mul_ssubset_mulStab | [36, 1] | [82, 79] | apply subset_trans (div_subset_div_right this) _ | α : 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
⊢ s ∩ a • C.mulStab * (t ∩ b • 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 / {x * y} ⊆ C.mulStab |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Kneser/Kneser.lean | Finset.mulStab_mul_ssubset_mulStab | [36, 1] | [82, 79] | have hsing : (x * y) • C.mulStab = {x * y} * C.mulStab := by rw [singleton_mul]; 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 / {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
hsing : (x * y) • C.mulStab = {x * y} * C.mulStab
⊢ (x * y) • C.mulStab / {x * y} ⊆ C.mulStab |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Kneser/Kneser.lean | Finset.mulStab_mul_ssubset_mulStab | [36, 1] | [82, 79] | simp_rw [hsing, singleton_mul, div_singleton, image_image, div_eq_mul_inv, mul_comm, comp,
mul_inv_cancel_right, image_id', 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
hxymem : x * y ∈ s ∩ a • C.mulStab * (t ∩ b • C.mulStab)
this : s ∩ a • C.mulStab * (t ∩ b • C.mulStab) ⊆ (x * y) • C.mulStab
hsing : (x * y) • C.mulStab = {x * y} * C.mulStab
⊢ (x * y) • C.mulStab / {x * y} ⊆ 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
hxymem : x * y ∈ s ∩ a • C.mulStab * (t ∩ b • C.mulStab)
⊢ s ∩ a • C.mulStab * (t ∩ b • 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)
⊢ a • C.mulStab * b • C.mulStab ⊆ (x * y) • C.mulStab |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Kneser/Kneser.lean | Finset.mulStab_mul_ssubset_mulStab | [36, 1] | [82, 79] | rw [smul_mul_smul] | α : 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)
⊢ a • C.mulStab * b • 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)
⊢ (a * b) • (C.mulStab * C.mulStab) ⊆ (x * y) • C.mulStab |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Kneser/Kneser.lean | Finset.mulStab_mul_ssubset_mulStab | [36, 1] | [82, 79] | rw [← hac, ← had, smul_mul_smul, smul_assoc] | α : 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)
⊢ (a * b) • (C.mulStab * 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)
⊢ (a * b) • (C.mulStab * C.mulStab) ⊆ (a * b) • (c * d) • C.mulStab |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Kneser/Kneser.lean | Finset.mulStab_mul_ssubset_mulStab | [36, 1] | [82, 79] | apply smul_finset_subset_smul_finset | α : 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)
⊢ (a * b) • (C.mulStab * C.mulStab) ⊆ (a * b) • (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)
⊢ C.mulStab * C.mulStab ⊆ (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_smul] | 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)
⊢ C.mulStab * C.mulStab ⊆ (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)
⊢ C.mulStab * C.mulStab ⊆ 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 [mul_subset_iff] | 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)
⊢ C.mulStab * C.mulStab ⊆ 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 ∈ C.mulStab, ∀ 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] | 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) |
Subsets and Splits
No community queries yet
The top public SQL queries from the community will appear here once available.