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/Basic.lean | Geometry.SimplicialComplex.combiInteriors_cover | [56, 1] | [66, 56] | rw [simplex_combiInteriors_cover] | case 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 y : E
s✝ t : Finset E
A : Set (Finset E)
m n : ℕ
s : Finset E
hs : s ∈ K
⊢ (convexHull 𝕜) ↑s ⊆ ⋃ i ∈ K, combiInterior 𝕜 i | case 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 y : E
s✝ t : Finset E
A : Set (Finset E)
m n : ℕ
s : Finset E
hs : s ∈ K
⊢ ⋃ t, ⋃ (_ : t ⊆ s), combiInterior 𝕜 t ⊆ ⋃ i ∈ K, combiInterior 𝕜 i |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Basic.lean | Geometry.SimplicialComplex.combiInteriors_cover | [56, 1] | [66, 56] | refine' Set.iUnion₂_mono' fun t hts => _ | case 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 y : E
s✝ t : Finset E
A : Set (Finset E)
m n : ℕ
s : Finset E
hs : s ∈ K
⊢ ⋃ t, ⋃ (_ : t ⊆ s), combiInterior 𝕜 t ⊆ ⋃ i ∈ K, combiInterior 𝕜 i | case 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 y : E
s✝ t✝ : Finset E
A : Set (Finset E)
m n : ℕ
s : Finset E
hs : s ∈ K
t : Finset E
hts : t ⊆ s
⊢ ∃ i', ∃ (_ : i' ∈ K), combiInterior 𝕜 t ⊆ combiInterior 𝕜 i' |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Basic.lean | Geometry.SimplicialComplex.combiInteriors_cover | [56, 1] | [66, 56] | obtain rfl | ht := t.eq_empty_or_nonempty | case 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 y : E
s✝ t✝ : Finset E
A : Set (Finset E)
m n : ℕ
s : Finset E
hs : s ∈ K
t : Finset E
hts : t ⊆ s
⊢ ∃ i', ∃ (_ : i' ∈ K), combiInterior 𝕜 t ⊆ combiInterior 𝕜 i' | case refine'_2.inl
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x y : E
s✝ t : Finset E
A : Set (Finset E)
m n : ℕ
s : Finset E
hs : s ∈ K
hts : ∅ ⊆ s
⊢ ∃ i', ∃ (_ : i' ∈ K), combiInterior 𝕜 ∅ ⊆ combiInterior 𝕜 i'
case refine'_2.inr
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x y : E
s✝ t✝ : Finset E
A : Set (Finset E)
m n : ℕ
s : Finset E
hs : s ∈ K
t : Finset E
hts : t ⊆ s
ht : t.Nonempty
⊢ ∃ i', ∃ (_ : i' ∈ K), combiInterior 𝕜 t ⊆ combiInterior 𝕜 i' |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Basic.lean | Geometry.SimplicialComplex.combiInteriors_cover | [56, 1] | [66, 56] | exact combiInterior_subset_convexHull | case 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 y : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
x✝¹ : Finset E
x✝ : x✝¹ ∈ K
⊢ combiInterior 𝕜 x✝¹ ⊆ (convexHull 𝕜) ↑x✝¹ | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Basic.lean | Geometry.SimplicialComplex.combiInteriors_cover | [56, 1] | [66, 56] | refine' ⟨s, hs, _⟩ | case refine'_2.inl
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x y : E
s✝ t : Finset E
A : Set (Finset E)
m n : ℕ
s : Finset E
hs : s ∈ K
hts : ∅ ⊆ s
⊢ ∃ i', ∃ (_ : i' ∈ K), combiInterior 𝕜 ∅ ⊆ combiInterior 𝕜 i' | case refine'_2.inl
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x y : E
s✝ t : Finset E
A : Set (Finset E)
m n : ℕ
s : Finset E
hs : s ∈ K
hts : ∅ ⊆ s
⊢ combiInterior 𝕜 ∅ ⊆ combiInterior 𝕜 s |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Basic.lean | Geometry.SimplicialComplex.combiInteriors_cover | [56, 1] | [66, 56] | rw [combiInterior_empty] | case refine'_2.inl
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x y : E
s✝ t : Finset E
A : Set (Finset E)
m n : ℕ
s : Finset E
hs : s ∈ K
hts : ∅ ⊆ s
⊢ combiInterior 𝕜 ∅ ⊆ combiInterior 𝕜 s | case refine'_2.inl
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x y : E
s✝ t : Finset E
A : Set (Finset E)
m n : ℕ
s : Finset E
hs : s ∈ K
hts : ∅ ⊆ s
⊢ ∅ ⊆ combiInterior 𝕜 s |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Basic.lean | Geometry.SimplicialComplex.combiInteriors_cover | [56, 1] | [66, 56] | exact Set.empty_subset _ | case refine'_2.inl
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x y : E
s✝ t : Finset E
A : Set (Finset E)
m n : ℕ
s : Finset E
hs : s ∈ K
hts : ∅ ⊆ s
⊢ ∅ ⊆ combiInterior 𝕜 s | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Basic.lean | Geometry.SimplicialComplex.combiInteriors_cover | [56, 1] | [66, 56] | exact ⟨t, K.down_closed' hs hts ht, Set.Subset.rfl⟩ | case refine'_2.inr
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x y : E
s✝ t✝ : Finset E
A : Set (Finset E)
m n : ℕ
s : Finset E
hs : s ∈ K
t : Finset E
hts : t ⊆ s
ht : t.Nonempty
⊢ ∃ i', ∃ (_ : i' ∈ K), combiInterior 𝕜 t ⊆ combiInterior 𝕜 i' | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Basic.lean | Geometry.SimplicialComplex.combiInteriors_partition | [68, 1] | [73, 78] | rw [← combiInteriors_cover] at hx | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x y : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
hx : x ∈ K.space
⊢ ∃! s, s ∈ K ∧ x ∈ combiInterior 𝕜 s | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x y : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
hx : x ∈ ⋃ s ∈ K, combiInterior 𝕜 s
⊢ ∃! s, s ∈ K ∧ x ∈ combiInterior 𝕜 s |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Basic.lean | Geometry.SimplicialComplex.combiInteriors_partition | [68, 1] | [73, 78] | obtain ⟨s, hs, hxs⟩ := Set.mem_iUnion₂.1 hx | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x y : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
hx : x ∈ ⋃ s ∈ K, combiInterior 𝕜 s
⊢ ∃! s, s ∈ K ∧ x ∈ combiInterior 𝕜 s | case 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 y : E
s✝ t : Finset E
A : Set (Finset E)
m n : ℕ
hx : x ∈ ⋃ s ∈ K, combiInterior 𝕜 s
s : Finset E
hs : s ∈ K
hxs : x ∈ combiInterior 𝕜 s
⊢ ∃! s, s ∈ K ∧ x ∈ combiInterior 𝕜 s |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Basic.lean | Geometry.SimplicialComplex.combiInteriors_partition | [68, 1] | [73, 78] | exact ⟨s, ⟨⟨hs, hxs⟩, fun t ⟨ht, hxt⟩ => disjoint_interiors ht hs hxt hxs⟩⟩ | case 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 y : E
s✝ t : Finset E
A : Set (Finset E)
m n : ℕ
hx : x ∈ ⋃ s ∈ K, combiInterior 𝕜 s
s : Finset E
hs : s ∈ K
hxs : x ∈ combiInterior 𝕜 s
⊢ ∃! s, s ∈ K ∧ x ∈ combiInterior 𝕜 s | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Basic.lean | Geometry.SimplicialComplex.mem_convexHull_iff | [75, 1] | [77, 38] | simp [simplex_combiInteriors_cover] | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x y : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
⊢ x ∈ (convexHull 𝕜) ↑s ↔ ∃ t ⊆ s, x ∈ combiInterior 𝕜 t | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Basic.lean | Geometry.SimplicialComplex.mem_combiFrontier_iff' | [79, 1] | [87, 26] | rw [mem_combiFrontier_iff] | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x y : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
⊢ x ∈ combiFrontier 𝕜 s ↔ ∃ t ⊂ s, x ∈ combiInterior 𝕜 t | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x y : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
⊢ (∃ t ⊂ s, x ∈ (convexHull 𝕜) ↑t) ↔ ∃ t ⊂ s, x ∈ combiInterior 𝕜 t |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Basic.lean | Geometry.SimplicialComplex.mem_combiFrontier_iff' | [79, 1] | [87, 26] | constructor | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x y : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
⊢ (∃ t ⊂ s, x ∈ (convexHull 𝕜) ↑t) ↔ ∃ t ⊂ s, x ∈ combiInterior 𝕜 t | 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 y : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
⊢ (∃ t ⊂ s, x ∈ (convexHull 𝕜) ↑t) → ∃ t ⊂ s, x ∈ combiInterior 𝕜 t
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 y : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
⊢ (∃ t ⊂ s, x ∈ combiInterior 𝕜 t) → ∃ t ⊂ s, x ∈ (convexHull 𝕜) ↑t |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Basic.lean | Geometry.SimplicialComplex.mem_combiFrontier_iff' | [79, 1] | [87, 26] | rintro ⟨t, hts, hxt⟩ | 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 y : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
⊢ (∃ t ⊂ s, x ∈ (convexHull 𝕜) ↑t) → ∃ t ⊂ s, x ∈ combiInterior 𝕜 t | case mp.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 y : E
s t✝ : Finset E
A : Set (Finset E)
m n : ℕ
t : Finset E
hts : t ⊂ s
hxt : x ∈ (convexHull 𝕜) ↑t
⊢ ∃ t ⊂ s, x ∈ combiInterior 𝕜 t |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Basic.lean | Geometry.SimplicialComplex.mem_combiFrontier_iff' | [79, 1] | [87, 26] | sorry | case mp.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 y : E
s t✝ : Finset E
A : Set (Finset E)
m n : ℕ
t : Finset E
hts : t ⊂ s
hxt : x ∈ (convexHull 𝕜) ↑t
⊢ ∃ t ⊂ s, x ∈ combiInterior 𝕜 t | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Basic.lean | Geometry.SimplicialComplex.mem_combiFrontier_iff' | [79, 1] | [87, 26] | rintro ⟨t, hts, hxt⟩ | 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 y : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
⊢ (∃ t ⊂ s, x ∈ combiInterior 𝕜 t) → ∃ t ⊂ s, x ∈ (convexHull 𝕜) ↑t | case mpr.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 y : E
s t✝ : Finset E
A : Set (Finset E)
m n : ℕ
t : Finset E
hts : t ⊂ s
hxt : x ∈ combiInterior 𝕜 t
⊢ ∃ t ⊂ s, x ∈ (convexHull 𝕜) ↑t |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Basic.lean | Geometry.SimplicialComplex.mem_combiFrontier_iff' | [79, 1] | [87, 26] | exact ⟨t, hts, hxt.1⟩ | case mpr.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 y : E
s t✝ : Finset E
A : Set (Finset E)
m n : ℕ
t : Finset E
hts : t ⊂ s
hxt : x ∈ combiInterior 𝕜 t
⊢ ∃ t ⊂ s, x ∈ (convexHull 𝕜) ↑t | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Basic.lean | Geometry.SimplicialComplex.subset_of_combiInterior_inter_convexHull_nonempty | [89, 1] | [96, 37] | obtain ⟨x, hxs, hxt⟩ := hst | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x y : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
hs : s ∈ K
ht : t ∈ K
hst : (combiInterior 𝕜 s ∩ (convexHull 𝕜) ↑t).Nonempty
⊢ s ⊆ t | case 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✝ y : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
hs : s ∈ K
ht : t ∈ K
x : E
hxs : x ∈ combiInterior 𝕜 s
hxt : x ∈ (convexHull 𝕜) ↑t
⊢ s ⊆ t |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Basic.lean | Geometry.SimplicialComplex.subset_of_combiInterior_inter_convexHull_nonempty | [89, 1] | [96, 37] | obtain ⟨u, hut, hxu⟩ := mem_convexHull_iff.1 hxt | case 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✝ y : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
hs : s ∈ K
ht : t ∈ K
x : E
hxs : x ∈ combiInterior 𝕜 s
hxt : x ∈ (convexHull 𝕜) ↑t
⊢ s ⊆ t | case 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✝ y : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
hs : s ∈ K
ht : t ∈ K
x : E
hxs : x ∈ combiInterior 𝕜 s
hxt : x ∈ (convexHull 𝕜) ↑t
u : Finset E
hut : u ⊆ t
hxu : x ∈ combiInterior 𝕜 u
⊢ s ⊆ t |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Basic.lean | Geometry.SimplicialComplex.subset_of_combiInterior_inter_convexHull_nonempty | [89, 1] | [96, 37] | rw [disjoint_interiors hs (K.down_closed' ht hut <| nonempty_of_ne_empty _) hxs hxu] | case 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✝ y : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
hs : s ∈ K
ht : t ∈ K
x : E
hxs : x ∈ combiInterior 𝕜 s
hxt : x ∈ (convexHull 𝕜) ↑t
u : Finset E
hut : u ⊆ t
hxu : x ∈ combiInterior 𝕜 u
⊢ s ⊆ t | case 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✝ y : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
hs : s ∈ K
ht : t ∈ K
x : E
hxs : x ∈ combiInterior 𝕜 s
hxt : x ∈ (convexHull 𝕜) ↑t
u : Finset E
hut : u ⊆ t
hxu : x ∈ combiInterior 𝕜 u
⊢ u ⊆ t
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x✝ y : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
hs : s ∈ K
ht : t ∈ K
x : E
hxs : x ∈ combiInterior 𝕜 s
hxt : x ∈ (convexHull 𝕜) ↑t
u : Finset E
hut : u ⊆ t
hxu : x ∈ combiInterior 𝕜 u
⊢ u ≠ ∅ |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Basic.lean | Geometry.SimplicialComplex.subset_of_combiInterior_inter_convexHull_nonempty | [89, 1] | [96, 37] | exact hut | case 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✝ y : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
hs : s ∈ K
ht : t ∈ K
x : E
hxs : x ∈ combiInterior 𝕜 s
hxt : x ∈ (convexHull 𝕜) ↑t
u : Finset E
hut : u ⊆ t
hxu : x ∈ combiInterior 𝕜 u
⊢ u ⊆ t
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x✝ y : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
hs : s ∈ K
ht : t ∈ K
x : E
hxs : x ∈ combiInterior 𝕜 s
hxt : x ∈ (convexHull 𝕜) ↑t
u : Finset E
hut : u ⊆ t
hxu : x ∈ combiInterior 𝕜 u
⊢ u ≠ ∅ | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x✝ y : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
hs : s ∈ K
ht : t ∈ K
x : E
hxs : x ∈ combiInterior 𝕜 s
hxt : x ∈ (convexHull 𝕜) ↑t
u : Finset E
hut : u ⊆ t
hxu : x ∈ combiInterior 𝕜 u
⊢ u ≠ ∅ |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Basic.lean | Geometry.SimplicialComplex.subset_of_combiInterior_inter_convexHull_nonempty | [89, 1] | [96, 37] | rintro rfl | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x✝ y : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
hs : s ∈ K
ht : t ∈ K
x : E
hxs : x ∈ combiInterior 𝕜 s
hxt : x ∈ (convexHull 𝕜) ↑t
u : Finset E
hut : u ⊆ t
hxu : x ∈ combiInterior 𝕜 u
⊢ u ≠ ∅ | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x✝ y : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
hs : s ∈ K
ht : t ∈ K
x : E
hxs : x ∈ combiInterior 𝕜 s
hxt : x ∈ (convexHull 𝕜) ↑t
hut : ∅ ⊆ t
hxu : x ∈ combiInterior 𝕜 ∅
⊢ False |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Basic.lean | Geometry.SimplicialComplex.subset_of_combiInterior_inter_convexHull_nonempty | [89, 1] | [96, 37] | rwa [combiInterior_empty] at hxu | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x✝ y : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
hs : s ∈ K
ht : t ∈ K
x : E
hxs : x ∈ combiInterior 𝕜 s
hxt : x ∈ (convexHull 𝕜) ↑t
hut : ∅ ⊆ t
hxu : x ∈ combiInterior 𝕜 ∅
⊢ False | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Basic.lean | Geometry.SimplicialComplex.cells_subset_facets | [106, 1] | [112, 11] | rintro s ⟨hs, hscard⟩ | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : LinearOrderedField 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K : SimplicialComplex 𝕜 E
x y : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : FiniteDimensional 𝕜 E
⊢ K.cells ⊆ K.facets | case intro
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : LinearOrderedField 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K : SimplicialComplex 𝕜 E
x y : E
s✝ t : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : FiniteDimensional 𝕜 E
s : Finset E
hs : s ∈ K
hscard : s.card = FiniteDimensional.finrank 𝕜 E + 1
⊢ s ∈ K.facets |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Basic.lean | Geometry.SimplicialComplex.cells_subset_facets | [106, 1] | [112, 11] | by_contra h | case intro
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : LinearOrderedField 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K : SimplicialComplex 𝕜 E
x y : E
s✝ t : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : FiniteDimensional 𝕜 E
s : Finset E
hs : s ∈ K
hscard : s.card = FiniteDimensional.finrank 𝕜 E + 1
⊢ s ∈ K.facets | case intro
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : LinearOrderedField 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K : SimplicialComplex 𝕜 E
x y : E
s✝ t : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : FiniteDimensional 𝕜 E
s : Finset E
hs : s ∈ K
hscard : s.card = FiniteDimensional.finrank 𝕜 E + 1
h : s ∉ K.facets
⊢ False |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Basic.lean | Geometry.SimplicialComplex.cells_subset_facets | [106, 1] | [112, 11] | obtain ⟨t, ht, hst⟩ := (not_facet_iff_subface hs).mp h | case intro
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : LinearOrderedField 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K : SimplicialComplex 𝕜 E
x y : E
s✝ t : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : FiniteDimensional 𝕜 E
s : Finset E
hs : s ∈ K
hscard : s.card = FiniteDimensional.finrank 𝕜 E + 1
h : s ∉ K.facets
⊢ False | case intro.intro.intro
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : LinearOrderedField 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K : SimplicialComplex 𝕜 E
x y : E
s✝ t✝ : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : FiniteDimensional 𝕜 E
s : Finset E
hs : s ∈ K
hscard : s.card = FiniteDimensional.finrank 𝕜 E + 1
h : s ∉ K.facets
t : Finset E
ht : t ∈ K.faces
hst : s ⊂ t
⊢ False |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Basic.lean | Geometry.SimplicialComplex.cells_subset_facets | [106, 1] | [112, 11] | have := card_lt_card hst | case intro.intro.intro
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : LinearOrderedField 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K : SimplicialComplex 𝕜 E
x y : E
s✝ t✝ : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : FiniteDimensional 𝕜 E
s : Finset E
hs : s ∈ K
hscard : s.card = FiniteDimensional.finrank 𝕜 E + 1
h : s ∉ K.facets
t : Finset E
ht : t ∈ K.faces
hst : s ⊂ t
⊢ False | case intro.intro.intro
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : LinearOrderedField 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K : SimplicialComplex 𝕜 E
x y : E
s✝ t✝ : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : FiniteDimensional 𝕜 E
s : Finset E
hs : s ∈ K
hscard : s.card = FiniteDimensional.finrank 𝕜 E + 1
h : s ∉ K.facets
t : Finset E
ht : t ∈ K.faces
hst : s ⊂ t
this : s.card < t.card
⊢ False |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Basic.lean | Geometry.SimplicialComplex.cells_subset_facets | [106, 1] | [112, 11] | have := face_dimension_le_space_dimension ht | case intro.intro.intro
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : LinearOrderedField 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K : SimplicialComplex 𝕜 E
x y : E
s✝ t✝ : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : FiniteDimensional 𝕜 E
s : Finset E
hs : s ∈ K
hscard : s.card = FiniteDimensional.finrank 𝕜 E + 1
h : s ∉ K.facets
t : Finset E
ht : t ∈ K.faces
hst : s ⊂ t
this : s.card < t.card
⊢ False | case intro.intro.intro
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : LinearOrderedField 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K : SimplicialComplex 𝕜 E
x y : E
s✝ t✝ : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : FiniteDimensional 𝕜 E
s : Finset E
hs : s ∈ K
hscard : s.card = FiniteDimensional.finrank 𝕜 E + 1
h : s ∉ K.facets
t : Finset E
ht : t ∈ K.faces
hst : s ⊂ t
this✝ : s.card < t.card
this : t.card ≤ FiniteDimensional.finrank 𝕜 E + 1
⊢ False |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Basic.lean | Geometry.SimplicialComplex.cells_subset_facets | [106, 1] | [112, 11] | linarith | case intro.intro.intro
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : LinearOrderedField 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K : SimplicialComplex 𝕜 E
x y : E
s✝ t✝ : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : FiniteDimensional 𝕜 E
s : Finset E
hs : s ∈ K
hscard : s.card = FiniteDimensional.finrank 𝕜 E + 1
h : s ∉ K.facets
t : Finset E
ht : t ∈ K.faces
hst : s ⊂ t
this✝ : s.card < t.card
this : t.card ≤ FiniteDimensional.finrank 𝕜 E + 1
⊢ False | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Basic.lean | Geometry.SimplicialComplex.simplex_combiInteriors_split_interiors | [114, 1] | [120, 8] | classical
let K := SimplicialComplex.ofSimplex ht
let F := t.powerset.filter fun v : Finset E => (s : Set E) ⊆ convexHull 𝕜 ↑v
sorry | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
K : SimplicialComplex 𝕜 E
x y : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
ht : AffineIndependent 𝕜 Subtype.val
hst : (convexHull 𝕜) ↑s ⊆ (convexHull 𝕜) ↑t
⊢ ∃ u ⊆ t, combiInterior 𝕜 s ⊆ combiInterior 𝕜 u | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Basic.lean | Geometry.SimplicialComplex.simplex_combiInteriors_split_interiors | [114, 1] | [120, 8] | let K := SimplicialComplex.ofSimplex ht | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
K : SimplicialComplex 𝕜 E
x y : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
ht : AffineIndependent 𝕜 Subtype.val
hst : (convexHull 𝕜) ↑s ⊆ (convexHull 𝕜) ↑t
⊢ ∃ u ⊆ t, combiInterior 𝕜 s ⊆ combiInterior 𝕜 u | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
K✝ : SimplicialComplex 𝕜 E
x y : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
ht : AffineIndependent 𝕜 Subtype.val
hst : (convexHull 𝕜) ↑s ⊆ (convexHull 𝕜) ↑t
K : SimplicialComplex 𝕜 E := ofSimplex ht
⊢ ∃ u ⊆ t, combiInterior 𝕜 s ⊆ combiInterior 𝕜 u |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Basic.lean | Geometry.SimplicialComplex.simplex_combiInteriors_split_interiors | [114, 1] | [120, 8] | let F := t.powerset.filter fun v : Finset E => (s : Set E) ⊆ convexHull 𝕜 ↑v | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
K✝ : SimplicialComplex 𝕜 E
x y : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
ht : AffineIndependent 𝕜 Subtype.val
hst : (convexHull 𝕜) ↑s ⊆ (convexHull 𝕜) ↑t
K : SimplicialComplex 𝕜 E := ofSimplex ht
⊢ ∃ u ⊆ t, combiInterior 𝕜 s ⊆ combiInterior 𝕜 u | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
K✝ : SimplicialComplex 𝕜 E
x y : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
ht : AffineIndependent 𝕜 Subtype.val
hst : (convexHull 𝕜) ↑s ⊆ (convexHull 𝕜) ↑t
K : SimplicialComplex 𝕜 E := ofSimplex ht
F : Finset (Finset E) := filter (fun v => ↑s ⊆ (convexHull 𝕜) ↑v) t.powerset
⊢ ∃ u ⊆ t, combiInterior 𝕜 s ⊆ combiInterior 𝕜 u |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Basic.lean | Geometry.SimplicialComplex.simplex_combiInteriors_split_interiors | [114, 1] | [120, 8] | sorry | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
K✝ : SimplicialComplex 𝕜 E
x y : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
ht : AffineIndependent 𝕜 Subtype.val
hst : (convexHull 𝕜) ↑s ⊆ (convexHull 𝕜) ↑t
K : SimplicialComplex 𝕜 E := ofSimplex ht
F : Finset (Finset E) := filter (fun v => ↑s ⊆ (convexHull 𝕜) ↑v) t.powerset
⊢ ∃ u ⊆ t, combiInterior 𝕜 s ⊆ combiInterior 𝕜 u | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Basic.lean | Geometry.SimplicialComplex.simplex_combiInteriors_split_interiors_nonempty | [186, 1] | [188, 80] | sorry | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
K : SimplicialComplex 𝕜 E
x y : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
hs : s.Nonempty
ht : AffineIndependent 𝕜 Subtype.val
hst : (convexHull 𝕜) ↑s ⊆ (convexHull 𝕜) ↑t
⊢ ∃ u ⊆ t, u.Nonempty ∧ combiInterior 𝕜 s ⊆ combiInterior 𝕜 u | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Impact.lean | Finset.mulImpact_empty | [29, 1] | [30, 86] | simp [mulImpact] | α : Type u_1
β : Type u_2
inst✝² : DecidableEq α
inst✝¹ : DecidableEq β
inst✝ : Mul α
n✝ n : ℕ
⊢ ∅.mulImpact n = 0 | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Impact.lean | Finset.mulImpact_singleton | [37, 1] | [41, 55] | simp only [mulImpact, singleton_mul', card_smul_finset] | α : Type u_1
β : Type u_2
inst✝³ : DecidableEq α
inst✝² : DecidableEq β
inst✝¹ : Group α
n✝ : ℕ
inst✝ : Infinite α
a : α
n : ℕ
⊢ {a}.mulImpact n = n | α : Type u_1
β : Type u_2
inst✝³ : DecidableEq α
inst✝² : DecidableEq β
inst✝¹ : Group α
n✝ : ℕ
inst✝ : Infinite α
a : α
n : ℕ
⊢ ⨅ t, (↑t).card = n |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Impact.lean | Finset.mulImpact_singleton | [37, 1] | [41, 55] | haveI : Nonempty {t : Finset α // t.card = n} := nonempty_subtype.2 (exists_card_eq _) | α : Type u_1
β : Type u_2
inst✝³ : DecidableEq α
inst✝² : DecidableEq β
inst✝¹ : Group α
n✝ : ℕ
inst✝ : Infinite α
a : α
n : ℕ
⊢ ⨅ t, (↑t).card = n | α : Type u_1
β : Type u_2
inst✝³ : DecidableEq α
inst✝² : DecidableEq β
inst✝¹ : Group α
n✝ : ℕ
inst✝ : Infinite α
a : α
n : ℕ
this : Nonempty { t // t.card = n }
⊢ ⨅ t, (↑t).card = n |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Impact.lean | Finset.mulImpact_singleton | [37, 1] | [41, 55] | exact Eq.trans (iInf_congr Subtype.prop) ciInf_const | α : Type u_1
β : Type u_2
inst✝³ : DecidableEq α
inst✝² : DecidableEq β
inst✝¹ : Group α
n✝ : ℕ
inst✝ : Infinite α
a : α
n : ℕ
this : Nonempty { t // t.card = n }
⊢ ⨅ t, (↑t).card = n | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Impact.lean | Finset.mulImpact_map_of_infinite | [56, 1] | [66, 10] | haveI : Infinite β := sorry | α : Type u_1
β : Type u_2
inst✝⁴ : DecidableEq α
inst✝³ : DecidableEq β
inst✝² : CommGroup α
inst✝¹ : CommGroup β
n : ℕ
inst✝ : Infinite α
s : Finset α
f : α →* β
hf : Injective ⇑f
⊢ (map { toFun := ⇑f, inj' := hf } s).mulImpact n = s.mulImpact n | α : Type u_1
β : Type u_2
inst✝⁴ : DecidableEq α
inst✝³ : DecidableEq β
inst✝² : CommGroup α
inst✝¹ : CommGroup β
n : ℕ
inst✝ : Infinite α
s : Finset α
f : α →* β
hf : Injective ⇑f
this : Infinite β
⊢ (map { toFun := ⇑f, inj' := hf } s).mulImpact n = s.mulImpact n |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Impact.lean | Finset.mulImpact_map_of_infinite | [56, 1] | [66, 10] | haveI : Nonempty {t : Finset α // t.card = n} := nonempty_subtype.2 (exists_card_eq _) | α : Type u_1
β : Type u_2
inst✝⁴ : DecidableEq α
inst✝³ : DecidableEq β
inst✝² : CommGroup α
inst✝¹ : CommGroup β
n : ℕ
inst✝ : Infinite α
s : Finset α
f : α →* β
hf : Injective ⇑f
this : Infinite β
⊢ (map { toFun := ⇑f, inj' := hf } s).mulImpact n = s.mulImpact n | α : Type u_1
β : Type u_2
inst✝⁴ : DecidableEq α
inst✝³ : DecidableEq β
inst✝² : CommGroup α
inst✝¹ : CommGroup β
n : ℕ
inst✝ : Infinite α
s : Finset α
f : α →* β
hf : Injective ⇑f
this✝ : Infinite β
this : Nonempty { t // t.card = n }
⊢ (map { toFun := ⇑f, inj' := hf } s).mulImpact n = s.mulImpact n |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Impact.lean | Finset.mulImpact_map_of_infinite | [56, 1] | [66, 10] | haveI : Nonempty {t : Finset β // t.card = n} := nonempty_subtype.2 (exists_card_eq _) | α : Type u_1
β : Type u_2
inst✝⁴ : DecidableEq α
inst✝³ : DecidableEq β
inst✝² : CommGroup α
inst✝¹ : CommGroup β
n : ℕ
inst✝ : Infinite α
s : Finset α
f : α →* β
hf : Injective ⇑f
this✝ : Infinite β
this : Nonempty { t // t.card = n }
⊢ (map { toFun := ⇑f, inj' := hf } s).mulImpact n = s.mulImpact n | α : Type u_1
β : Type u_2
inst✝⁴ : DecidableEq α
inst✝³ : DecidableEq β
inst✝² : CommGroup α
inst✝¹ : CommGroup β
n : ℕ
inst✝ : Infinite α
s : Finset α
f : α →* β
hf : Injective ⇑f
this✝¹ : Infinite β
this✝ : Nonempty { t // t.card = n }
this : Nonempty { t // t.card = n }
⊢ (map { toFun := ⇑f, inj' := hf } s).mulImpact n = s.mulImpact n |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Impact.lean | Finset.mulImpact_map_of_infinite | [56, 1] | [66, 10] | refine' le_antisymm _ _ | α : Type u_1
β : Type u_2
inst✝⁴ : DecidableEq α
inst✝³ : DecidableEq β
inst✝² : CommGroup α
inst✝¹ : CommGroup β
n : ℕ
inst✝ : Infinite α
s : Finset α
f : α →* β
hf : Injective ⇑f
this✝¹ : Infinite β
this✝ : Nonempty { t // t.card = n }
this : Nonempty { t // t.card = n }
⊢ (map { toFun := ⇑f, inj' := hf } s).mulImpact n = s.mulImpact n | case refine'_1
α : Type u_1
β : Type u_2
inst✝⁴ : DecidableEq α
inst✝³ : DecidableEq β
inst✝² : CommGroup α
inst✝¹ : CommGroup β
n : ℕ
inst✝ : Infinite α
s : Finset α
f : α →* β
hf : Injective ⇑f
this✝¹ : Infinite β
this✝ : Nonempty { t // t.card = n }
this : Nonempty { t // t.card = n }
⊢ (map { toFun := ⇑f, inj' := hf } s).mulImpact n ≤ s.mulImpact n
case refine'_2
α : Type u_1
β : Type u_2
inst✝⁴ : DecidableEq α
inst✝³ : DecidableEq β
inst✝² : CommGroup α
inst✝¹ : CommGroup β
n : ℕ
inst✝ : Infinite α
s : Finset α
f : α →* β
hf : Injective ⇑f
this✝¹ : Infinite β
this✝ : Nonempty { t // t.card = n }
this : Nonempty { t // t.card = n }
⊢ s.mulImpact n ≤ (map { toFun := ⇑f, inj' := hf } s).mulImpact n |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Impact.lean | Finset.mulImpact_map_of_infinite | [56, 1] | [66, 10] | refine' le_ciInf fun t => _ | case refine'_1
α : Type u_1
β : Type u_2
inst✝⁴ : DecidableEq α
inst✝³ : DecidableEq β
inst✝² : CommGroup α
inst✝¹ : CommGroup β
n : ℕ
inst✝ : Infinite α
s : Finset α
f : α →* β
hf : Injective ⇑f
this✝¹ : Infinite β
this✝ : Nonempty { t // t.card = n }
this : Nonempty { t // t.card = n }
⊢ (map { toFun := ⇑f, inj' := hf } s).mulImpact n ≤ s.mulImpact n | case refine'_1
α : Type u_1
β : Type u_2
inst✝⁴ : DecidableEq α
inst✝³ : DecidableEq β
inst✝² : CommGroup α
inst✝¹ : CommGroup β
n : ℕ
inst✝ : Infinite α
s : Finset α
f : α →* β
hf : Injective ⇑f
this✝¹ : Infinite β
this✝ : Nonempty { t // t.card = n }
this : Nonempty { t // t.card = n }
t : { t // t.card = n }
⊢ (map { toFun := ⇑f, inj' := hf } s).mulImpact n ≤ (s * ↑t).card |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Impact.lean | Finset.mulImpact_map_of_infinite | [56, 1] | [66, 10] | sorry | case refine'_1
α : Type u_1
β : Type u_2
inst✝⁴ : DecidableEq α
inst✝³ : DecidableEq β
inst✝² : CommGroup α
inst✝¹ : CommGroup β
n : ℕ
inst✝ : Infinite α
s : Finset α
f : α →* β
hf : Injective ⇑f
this✝¹ : Infinite β
this✝ : Nonempty { t // t.card = n }
this : Nonempty { t // t.card = n }
t : { t // t.card = n }
⊢ (map { toFun := ⇑f, inj' := hf } s).mulImpact n ≤ (s * ↑t).card | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Impact.lean | Finset.mulImpact_map_of_infinite | [56, 1] | [66, 10] | refine' le_ciInf fun t => _ | case refine'_2
α : Type u_1
β : Type u_2
inst✝⁴ : DecidableEq α
inst✝³ : DecidableEq β
inst✝² : CommGroup α
inst✝¹ : CommGroup β
n : ℕ
inst✝ : Infinite α
s : Finset α
f : α →* β
hf : Injective ⇑f
this✝¹ : Infinite β
this✝ : Nonempty { t // t.card = n }
this : Nonempty { t // t.card = n }
⊢ s.mulImpact n ≤ (map { toFun := ⇑f, inj' := hf } s).mulImpact n | case refine'_2
α : Type u_1
β : Type u_2
inst✝⁴ : DecidableEq α
inst✝³ : DecidableEq β
inst✝² : CommGroup α
inst✝¹ : CommGroup β
n : ℕ
inst✝ : Infinite α
s : Finset α
f : α →* β
hf : Injective ⇑f
this✝¹ : Infinite β
this✝ : Nonempty { t // t.card = n }
this : Nonempty { t // t.card = n }
t : { t // t.card = n }
⊢ s.mulImpact n ≤ (map { toFun := ⇑f, inj' := hf } s * ↑t).card |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Impact.lean | Finset.mulImpact_map_of_infinite | [56, 1] | [66, 10] | sorry | case refine'_2
α : Type u_1
β : Type u_2
inst✝⁴ : DecidableEq α
inst✝³ : DecidableEq β
inst✝² : CommGroup α
inst✝¹ : CommGroup β
n : ℕ
inst✝ : Infinite α
s : Finset α
f : α →* β
hf : Injective ⇑f
this✝¹ : Infinite β
this✝ : Nonempty { t // t.card = n }
this : Nonempty { t // t.card = n }
t : { t // t.card = n }
⊢ s.mulImpact n ≤ (map { toFun := ⇑f, inj' := hf } s * ↑t).card | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Analysis/Convex/Exposed.lean | IsExposed.span_lt | [25, 1] | [28, 8] | apply (affineSpan_mono _ hst.subset).lt_of_ne | E : Type u_1
inst✝¹ : NormedAddCommGroup E
inst✝ : NormedSpace ℝ E
x : E
s t C : Set E
X : Finset E
l : E →L[ℝ] ℝ
hst : IsExposed ℝ s t
hts : ¬s ⊆ t
⊢ affineSpan ℝ t < affineSpan ℝ s | E : Type u_1
inst✝¹ : NormedAddCommGroup E
inst✝ : NormedSpace ℝ E
x : E
s t C : Set E
X : Finset E
l : E →L[ℝ] ℝ
hst : IsExposed ℝ s t
hts : ¬s ⊆ t
⊢ affineSpan ℝ t ≠ affineSpan ℝ s |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Analysis/Convex/Exposed.lean | IsExposed.span_lt | [25, 1] | [28, 8] | rintro h | E : Type u_1
inst✝¹ : NormedAddCommGroup E
inst✝ : NormedSpace ℝ E
x : E
s t C : Set E
X : Finset E
l : E →L[ℝ] ℝ
hst : IsExposed ℝ s t
hts : ¬s ⊆ t
⊢ affineSpan ℝ t ≠ affineSpan ℝ s | E : Type u_1
inst✝¹ : NormedAddCommGroup E
inst✝ : NormedSpace ℝ E
x : E
s t C : Set E
X : Finset E
l : E →L[ℝ] ℝ
hst : IsExposed ℝ s t
hts : ¬s ⊆ t
h : affineSpan ℝ t = affineSpan ℝ s
⊢ False |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Analysis/Convex/Exposed.lean | IsExposed.span_lt | [25, 1] | [28, 8] | sorry | E : Type u_1
inst✝¹ : NormedAddCommGroup E
inst✝ : NormedSpace ℝ E
x : E
s t C : Set E
X : Finset E
l : E →L[ℝ] ℝ
hst : IsExposed ℝ s t
hts : ¬s ⊆ t
h : affineSpan ℝ t = affineSpan ℝ s
⊢ False | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Analysis/Convex/Exposed.lean | mem_exposed_set_iff_mem_frontier | [37, 1] | [51, 16] | use fun ⟨t, hst, hts, hxt⟩ => ⟨hst.subset hxt, hst.subset_frontier hts hxt⟩ | E : Type u_1
inst✝¹ : NormedAddCommGroup E
inst✝ : NormedSpace ℝ E
x : E
s t C : Set E
X : Finset E
l : E →L[ℝ] ℝ
hs₁ : Convex ℝ s
hs₂ : (interior s).Nonempty
⊢ (∃ t, IsExposed ℝ s t ∧ ¬s ⊆ t ∧ x ∈ t) ↔ x ∈ s ∧ x ∈ frontier s | case mpr
E : Type u_1
inst✝¹ : NormedAddCommGroup E
inst✝ : NormedSpace ℝ E
x : E
s t C : Set E
X : Finset E
l : E →L[ℝ] ℝ
hs₁ : Convex ℝ s
hs₂ : (interior s).Nonempty
⊢ x ∈ s ∧ x ∈ frontier s → ∃ t, IsExposed ℝ s t ∧ ¬s ⊆ t ∧ x ∈ t |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Analysis/Convex/Exposed.lean | mem_exposed_set_iff_mem_frontier | [37, 1] | [51, 16] | rintro ⟨hxA, hxfA⟩ | case mpr
E : Type u_1
inst✝¹ : NormedAddCommGroup E
inst✝ : NormedSpace ℝ E
x : E
s t C : Set E
X : Finset E
l : E →L[ℝ] ℝ
hs₁ : Convex ℝ s
hs₂ : (interior s).Nonempty
⊢ x ∈ s ∧ x ∈ frontier s → ∃ t, IsExposed ℝ s t ∧ ¬s ⊆ t ∧ x ∈ t | case mpr.intro
E : Type u_1
inst✝¹ : NormedAddCommGroup E
inst✝ : NormedSpace ℝ E
x : E
s t C : Set E
X : Finset E
l : E →L[ℝ] ℝ
hs₁ : Convex ℝ s
hs₂ : (interior s).Nonempty
hxA : x ∈ s
hxfA : x ∈ frontier s
⊢ ∃ t, IsExposed ℝ s t ∧ ¬s ⊆ t ∧ x ∈ t |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Analysis/Convex/Exposed.lean | mem_exposed_set_iff_mem_frontier | [37, 1] | [51, 16] | obtain ⟨y, hyA⟩ := id hs₂ | case mpr.intro
E : Type u_1
inst✝¹ : NormedAddCommGroup E
inst✝ : NormedSpace ℝ E
x : E
s t C : Set E
X : Finset E
l : E →L[ℝ] ℝ
hs₁ : Convex ℝ s
hs₂ : (interior s).Nonempty
hxA : x ∈ s
hxfA : x ∈ frontier s
⊢ ∃ t, IsExposed ℝ s t ∧ ¬s ⊆ t ∧ x ∈ t | case mpr.intro.intro
E : Type u_1
inst✝¹ : NormedAddCommGroup E
inst✝ : NormedSpace ℝ E
x : E
s t C : Set E
X : Finset E
l : E →L[ℝ] ℝ
hs₁ : Convex ℝ s
hs₂ : (interior s).Nonempty
hxA : x ∈ s
hxfA : x ∈ frontier s
y : E
hyA : y ∈ interior s
⊢ ∃ t, IsExposed ℝ s t ∧ ¬s ⊆ t ∧ x ∈ t |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Analysis/Convex/Exposed.lean | mem_exposed_set_iff_mem_frontier | [37, 1] | [51, 16] | obtain ⟨l, hl⟩ := geometric_hahn_banach_open_point (Convex.interior hs₁) isOpen_interior hxfA.2 | case mpr.intro.intro
E : Type u_1
inst✝¹ : NormedAddCommGroup E
inst✝ : NormedSpace ℝ E
x : E
s t C : Set E
X : Finset E
l : E →L[ℝ] ℝ
hs₁ : Convex ℝ s
hs₂ : (interior s).Nonempty
hxA : x ∈ s
hxfA : x ∈ frontier s
y : E
hyA : y ∈ interior s
⊢ ∃ t, IsExposed ℝ s t ∧ ¬s ⊆ t ∧ x ∈ t | case mpr.intro.intro.intro
E : Type u_1
inst✝¹ : NormedAddCommGroup E
inst✝ : NormedSpace ℝ E
x : E
s t C : Set E
X : Finset E
l✝ : E →L[ℝ] ℝ
hs₁ : Convex ℝ s
hs₂ : (interior s).Nonempty
hxA : x ∈ s
hxfA : x ∈ frontier s
y : E
hyA : y ∈ interior s
l : E →L[ℝ] ℝ
hl : ∀ a ∈ interior s, l a < l x
⊢ ∃ t, IsExposed ℝ s t ∧ ¬s ⊆ t ∧ x ∈ t |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Analysis/Convex/Exposed.lean | mem_exposed_set_iff_mem_frontier | [37, 1] | [51, 16] | refine'
⟨{x ∈ s | ∀ y ∈ s, l y ≤ l x}, fun _ => ⟨l, rfl⟩, fun h =>
not_le.2 (hl y hyA) ((h (interior_subset hyA)).2 x hxA), hxA, fun z hzA => _⟩ | case mpr.intro.intro.intro
E : Type u_1
inst✝¹ : NormedAddCommGroup E
inst✝ : NormedSpace ℝ E
x : E
s t C : Set E
X : Finset E
l✝ : E →L[ℝ] ℝ
hs₁ : Convex ℝ s
hs₂ : (interior s).Nonempty
hxA : x ∈ s
hxfA : x ∈ frontier s
y : E
hyA : y ∈ interior s
l : E →L[ℝ] ℝ
hl : ∀ a ∈ interior s, l a < l x
⊢ ∃ t, IsExposed ℝ s t ∧ ¬s ⊆ t ∧ x ∈ t | case mpr.intro.intro.intro
E : Type u_1
inst✝¹ : NormedAddCommGroup E
inst✝ : NormedSpace ℝ E
x : E
s t C : Set E
X : Finset E
l✝ : E →L[ℝ] ℝ
hs₁ : Convex ℝ s
hs₂ : (interior s).Nonempty
hxA : x ∈ s
hxfA : x ∈ frontier s
y : E
hyA : y ∈ interior s
l : E →L[ℝ] ℝ
hl : ∀ a ∈ interior s, l a < l x
z : E
hzA : z ∈ s
⊢ l z ≤ l x |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Analysis/Convex/Exposed.lean | mem_exposed_set_iff_mem_frontier | [37, 1] | [51, 16] | suffices h : l '' closure (interior s) ⊆ closure (Iio (l x)) by
rw [closure_Iio, ← closure_eq_closure_interior hs₁ hs₂] at h
exact h ⟨z, subset_closure hzA, rfl⟩ | case mpr.intro.intro.intro
E : Type u_1
inst✝¹ : NormedAddCommGroup E
inst✝ : NormedSpace ℝ E
x : E
s t C : Set E
X : Finset E
l✝ : E →L[ℝ] ℝ
hs₁ : Convex ℝ s
hs₂ : (interior s).Nonempty
hxA : x ∈ s
hxfA : x ∈ frontier s
y : E
hyA : y ∈ interior s
l : E →L[ℝ] ℝ
hl : ∀ a ∈ interior s, l a < l x
z : E
hzA : z ∈ s
⊢ l z ≤ l x | case mpr.intro.intro.intro
E : Type u_1
inst✝¹ : NormedAddCommGroup E
inst✝ : NormedSpace ℝ E
x : E
s t C : Set E
X : Finset E
l✝ : E →L[ℝ] ℝ
hs₁ : Convex ℝ s
hs₂ : (interior s).Nonempty
hxA : x ∈ s
hxfA : x ∈ frontier s
y : E
hyA : y ∈ interior s
l : E →L[ℝ] ℝ
hl : ∀ a ∈ interior s, l a < l x
z : E
hzA : z ∈ s
⊢ ⇑l '' closure (interior s) ⊆ closure (Iio (l x)) |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Analysis/Convex/Exposed.lean | mem_exposed_set_iff_mem_frontier | [37, 1] | [51, 16] | refine' (image_closure_subset_closure_image l.continuous).trans $ closure_mono _ | case mpr.intro.intro.intro
E : Type u_1
inst✝¹ : NormedAddCommGroup E
inst✝ : NormedSpace ℝ E
x : E
s t C : Set E
X : Finset E
l✝ : E →L[ℝ] ℝ
hs₁ : Convex ℝ s
hs₂ : (interior s).Nonempty
hxA : x ∈ s
hxfA : x ∈ frontier s
y : E
hyA : y ∈ interior s
l : E →L[ℝ] ℝ
hl : ∀ a ∈ interior s, l a < l x
z : E
hzA : z ∈ s
⊢ ⇑l '' closure (interior s) ⊆ closure (Iio (l x)) | case mpr.intro.intro.intro
E : Type u_1
inst✝¹ : NormedAddCommGroup E
inst✝ : NormedSpace ℝ E
x : E
s t C : Set E
X : Finset E
l✝ : E →L[ℝ] ℝ
hs₁ : Convex ℝ s
hs₂ : (interior s).Nonempty
hxA : x ∈ s
hxfA : x ∈ frontier s
y : E
hyA : y ∈ interior s
l : E →L[ℝ] ℝ
hl : ∀ a ∈ interior s, l a < l x
z : E
hzA : z ∈ s
⊢ ⇑l '' interior s ⊆ Iio (l x) |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Analysis/Convex/Exposed.lean | mem_exposed_set_iff_mem_frontier | [37, 1] | [51, 16] | rintro _ ⟨w, hw, rfl⟩ | case mpr.intro.intro.intro
E : Type u_1
inst✝¹ : NormedAddCommGroup E
inst✝ : NormedSpace ℝ E
x : E
s t C : Set E
X : Finset E
l✝ : E →L[ℝ] ℝ
hs₁ : Convex ℝ s
hs₂ : (interior s).Nonempty
hxA : x ∈ s
hxfA : x ∈ frontier s
y : E
hyA : y ∈ interior s
l : E →L[ℝ] ℝ
hl : ∀ a ∈ interior s, l a < l x
z : E
hzA : z ∈ s
⊢ ⇑l '' interior s ⊆ Iio (l x) | case mpr.intro.intro.intro.intro.intro
E : Type u_1
inst✝¹ : NormedAddCommGroup E
inst✝ : NormedSpace ℝ E
x : E
s t C : Set E
X : Finset E
l✝ : E →L[ℝ] ℝ
hs₁ : Convex ℝ s
hs₂ : (interior s).Nonempty
hxA : x ∈ s
hxfA : x ∈ frontier s
y : E
hyA : y ∈ interior s
l : E →L[ℝ] ℝ
hl : ∀ a ∈ interior s, l a < l x
z : E
hzA : z ∈ s
w : E
hw : w ∈ interior s
⊢ l w ∈ Iio (l x) |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Analysis/Convex/Exposed.lean | mem_exposed_set_iff_mem_frontier | [37, 1] | [51, 16] | exact hl w hw | case mpr.intro.intro.intro.intro.intro
E : Type u_1
inst✝¹ : NormedAddCommGroup E
inst✝ : NormedSpace ℝ E
x : E
s t C : Set E
X : Finset E
l✝ : E →L[ℝ] ℝ
hs₁ : Convex ℝ s
hs₂ : (interior s).Nonempty
hxA : x ∈ s
hxfA : x ∈ frontier s
y : E
hyA : y ∈ interior s
l : E →L[ℝ] ℝ
hl : ∀ a ∈ interior s, l a < l x
z : E
hzA : z ∈ s
w : E
hw : w ∈ interior s
⊢ l w ∈ Iio (l x) | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Analysis/Convex/Exposed.lean | mem_exposed_set_iff_mem_frontier | [37, 1] | [51, 16] | rw [closure_Iio, ← closure_eq_closure_interior hs₁ hs₂] at h | E : Type u_1
inst✝¹ : NormedAddCommGroup E
inst✝ : NormedSpace ℝ E
x : E
s t C : Set E
X : Finset E
l✝ : E →L[ℝ] ℝ
hs₁ : Convex ℝ s
hs₂ : (interior s).Nonempty
hxA : x ∈ s
hxfA : x ∈ frontier s
y : E
hyA : y ∈ interior s
l : E →L[ℝ] ℝ
hl : ∀ a ∈ interior s, l a < l x
z : E
hzA : z ∈ s
h : ⇑l '' closure (interior s) ⊆ closure (Iio (l x))
⊢ l z ≤ l x | E : Type u_1
inst✝¹ : NormedAddCommGroup E
inst✝ : NormedSpace ℝ E
x : E
s t C : Set E
X : Finset E
l✝ : E →L[ℝ] ℝ
hs₁ : Convex ℝ s
hs₂ : (interior s).Nonempty
hxA : x ∈ s
hxfA : x ∈ frontier s
y : E
hyA : y ∈ interior s
l : E →L[ℝ] ℝ
hl : ∀ a ∈ interior s, l a < l x
z : E
hzA : z ∈ s
h : ⇑l '' closure s ⊆ Iic (l x)
⊢ l z ≤ l x |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Analysis/Convex/Exposed.lean | mem_exposed_set_iff_mem_frontier | [37, 1] | [51, 16] | exact h ⟨z, subset_closure hzA, rfl⟩ | E : Type u_1
inst✝¹ : NormedAddCommGroup E
inst✝ : NormedSpace ℝ E
x : E
s t C : Set E
X : Finset E
l✝ : E →L[ℝ] ℝ
hs₁ : Convex ℝ s
hs₂ : (interior s).Nonempty
hxA : x ∈ s
hxfA : x ∈ frontier s
y : E
hyA : y ∈ interior s
l : E →L[ℝ] ℝ
hl : ∀ a ∈ interior s, l a < l x
z : E
hzA : z ∈ s
h : ⇑l '' closure s ⊆ Iic (l x)
⊢ l z ≤ l x | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Analysis/Convex/Exposed.lean | mem_extreme_set_iff_mem_frontier | [53, 1] | [58, 37] | use fun ⟨t, hst, hts, hxt⟩ => ⟨hst.1 hxt, hst.subset_frontier hts hxt⟩ | E : Type u_1
inst✝¹ : NormedAddCommGroup E
inst✝ : NormedSpace ℝ E
x : E
s t C : Set E
X : Finset E
l : E →L[ℝ] ℝ
hs₁ : Convex ℝ s
hs₂ : (interior s).Nonempty
⊢ (∃ t, IsExtreme ℝ s t ∧ ¬s ⊆ t ∧ x ∈ t) ↔ x ∈ s ∧ x ∈ frontier s | case mpr
E : Type u_1
inst✝¹ : NormedAddCommGroup E
inst✝ : NormedSpace ℝ E
x : E
s t C : Set E
X : Finset E
l : E →L[ℝ] ℝ
hs₁ : Convex ℝ s
hs₂ : (interior s).Nonempty
⊢ x ∈ s ∧ x ∈ frontier s → ∃ t, IsExtreme ℝ s t ∧ ¬s ⊆ t ∧ x ∈ t |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Analysis/Convex/Exposed.lean | mem_extreme_set_iff_mem_frontier | [53, 1] | [58, 37] | rintro h | case mpr
E : Type u_1
inst✝¹ : NormedAddCommGroup E
inst✝ : NormedSpace ℝ E
x : E
s t C : Set E
X : Finset E
l : E →L[ℝ] ℝ
hs₁ : Convex ℝ s
hs₂ : (interior s).Nonempty
⊢ x ∈ s ∧ x ∈ frontier s → ∃ t, IsExtreme ℝ s t ∧ ¬s ⊆ t ∧ x ∈ t | case mpr
E : Type u_1
inst✝¹ : NormedAddCommGroup E
inst✝ : NormedSpace ℝ E
x : E
s t C : Set E
X : Finset E
l : E →L[ℝ] ℝ
hs₁ : Convex ℝ s
hs₂ : (interior s).Nonempty
h : x ∈ s ∧ x ∈ frontier s
⊢ ∃ t, IsExtreme ℝ s t ∧ ¬s ⊆ t ∧ x ∈ t |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Analysis/Convex/Exposed.lean | mem_extreme_set_iff_mem_frontier | [53, 1] | [58, 37] | obtain ⟨t, hst, hts, hxt⟩ := (mem_exposed_set_iff_mem_frontier hs₁ hs₂).2 h | case mpr
E : Type u_1
inst✝¹ : NormedAddCommGroup E
inst✝ : NormedSpace ℝ E
x : E
s t C : Set E
X : Finset E
l : E →L[ℝ] ℝ
hs₁ : Convex ℝ s
hs₂ : (interior s).Nonempty
h : x ∈ s ∧ x ∈ frontier s
⊢ ∃ t, IsExtreme ℝ s t ∧ ¬s ⊆ t ∧ x ∈ t | case mpr.intro.intro.intro
E : Type u_1
inst✝¹ : NormedAddCommGroup E
inst✝ : NormedSpace ℝ E
x : E
s t✝ C : Set E
X : Finset E
l : E →L[ℝ] ℝ
hs₁ : Convex ℝ s
hs₂ : (interior s).Nonempty
h : x ∈ s ∧ x ∈ frontier s
t : Set E
hst : IsExposed ℝ s t
hts : ¬s ⊆ t
hxt : x ∈ t
⊢ ∃ t, IsExtreme ℝ s t ∧ ¬s ⊆ t ∧ x ∈ t |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Analysis/Convex/Exposed.lean | mem_extreme_set_iff_mem_frontier | [53, 1] | [58, 37] | exact ⟨t, hst.isExtreme, hts, hxt⟩ | case mpr.intro.intro.intro
E : Type u_1
inst✝¹ : NormedAddCommGroup E
inst✝ : NormedSpace ℝ E
x : E
s t✝ C : Set E
X : Finset E
l : E →L[ℝ] ℝ
hs₁ : Convex ℝ s
hs₂ : (interior s).Nonempty
h : x ∈ s ∧ x ∈ frontier s
t : Set E
hst : IsExposed ℝ s t
hts : ¬s ⊆ t
hxt : x ∈ t
⊢ ∃ t, IsExtreme ℝ s t ∧ ¬s ⊆ t ∧ x ∈ t | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Analysis/Convex/Exposed.lean | extremePoints_subset_closure_exposedPoints | [65, 1] | [66, 64] | sorry | E : Type u_1
inst✝¹ : NormedAddCommGroup E
inst✝ : NormedSpace ℝ E
x : E
s t C : Set E
X : Finset E
l : E →L[ℝ] ℝ
hs₁ : Convex ℝ s
hs₂ : IsClosed s
⊢ extremePoints ℝ s ⊆ closure (exposedPoints ℝ 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 |
Subsets and Splits
No community queries yet
The top public SQL queries from the community will appear here once available.