url
stringclasses 147
values | commit
stringclasses 147
values | file_path
stringlengths 7
101
| full_name
stringlengths 1
94
| start
stringlengths 6
10
| end
stringlengths 6
11
| tactic
stringlengths 1
11.2k
| state_before
stringlengths 3
2.09M
| state_after
stringlengths 6
2.09M
|
---|---|---|---|---|---|---|---|---|
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Data/Finset/PosDiffs.lean | Finset.card_posDiffs_self_le | [73, 1] | [81, 10] | rfl | case refine'_2
α : Type u_1
inst✝ : DecidableEq α
𝒜 ℬ : Finset (Finset α)
h𝒜✝ : (↑{∅}).OrdConnected
⊢ ({∅} \₊ {∅}).card ≤ {∅}.card | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Data/Finset/PosDiffs.lean | Finset.card_posDiffs_self_le | [73, 1] | [81, 10] | rintro a 𝒜 h𝒜₀ h𝒜₁ h𝒜 | case refine'_3
α : Type u_1
inst✝ : DecidableEq α
𝒜 ℬ : Finset (Finset α)
⊢ ∀ (a : α) ⦃𝒜 : Finset (Finset α)⦄,
((↑(nonMemberSubfamily a 𝒜)).OrdConnected →
(nonMemberSubfamily a 𝒜 \₊ nonMemberSubfamily a 𝒜).card ≤ (nonMemberSubfamily a 𝒜).card) →
((↑(memberSubfamily a 𝒜)).OrdConnected →
(memberSubfamily a 𝒜 \₊ memberSubfamily a 𝒜).card ≤ (memberSubfamily a 𝒜).card) →
(↑𝒜).OrdConnected → (𝒜 \₊ 𝒜).card ≤ 𝒜.card | case refine'_3
α : Type u_1
inst✝ : DecidableEq α
𝒜✝ ℬ : Finset (Finset α)
a : α
𝒜 : Finset (Finset α)
h𝒜₀ :
(↑(nonMemberSubfamily a 𝒜)).OrdConnected →
(nonMemberSubfamily a 𝒜 \₊ nonMemberSubfamily a 𝒜).card ≤ (nonMemberSubfamily a 𝒜).card
h𝒜₁ :
(↑(memberSubfamily a 𝒜)).OrdConnected → (memberSubfamily a 𝒜 \₊ memberSubfamily a 𝒜).card ≤ (memberSubfamily a 𝒜).card
h𝒜 : (↑𝒜).OrdConnected
⊢ (𝒜 \₊ 𝒜).card ≤ 𝒜.card |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Data/Finset/PosDiffs.lean | Finset.card_posDiffs_self_le | [73, 1] | [81, 10] | sorry | case refine'_3
α : Type u_1
inst✝ : DecidableEq α
𝒜✝ ℬ : Finset (Finset α)
a : α
𝒜 : Finset (Finset α)
h𝒜₀ :
(↑(nonMemberSubfamily a 𝒜)).OrdConnected →
(nonMemberSubfamily a 𝒜 \₊ nonMemberSubfamily a 𝒜).card ≤ (nonMemberSubfamily a 𝒜).card
h𝒜₁ :
(↑(memberSubfamily a 𝒜)).OrdConnected → (memberSubfamily a 𝒜 \₊ memberSubfamily a 𝒜).card ≤ (memberSubfamily a 𝒜).card
h𝒜 : (↑𝒜).OrdConnected
⊢ (𝒜 \₊ 𝒜).card ≤ 𝒜.card | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Data/Finset/PosDiffs.lean | Finset.le_card_upper_inter_lower | [83, 1] | [91, 48] | refine' (card_le_card _).trans (card_posDiffs_self_le _) | α : Type u_1
inst✝ : DecidableEq α
𝒜 ℬ : Finset (Finset α)
h𝒜 : IsLowerSet ↑𝒜
hℬ : IsUpperSet ↑ℬ
⊢ (𝒜 \₊ ℬ).card ≤ (𝒜 ∩ ℬ).card | case refine'_1
α : Type u_1
inst✝ : DecidableEq α
𝒜 ℬ : Finset (Finset α)
h𝒜 : IsLowerSet ↑𝒜
hℬ : IsUpperSet ↑ℬ
⊢ 𝒜 \₊ ℬ ⊆ 𝒜 ∩ ℬ \₊ (𝒜 ∩ ℬ)
case refine'_2
α : Type u_1
inst✝ : DecidableEq α
𝒜 ℬ : Finset (Finset α)
h𝒜 : IsLowerSet ↑𝒜
hℬ : IsUpperSet ↑ℬ
⊢ (↑(𝒜 ∩ ℬ)).OrdConnected |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Data/Finset/PosDiffs.lean | Finset.le_card_upper_inter_lower | [83, 1] | [91, 48] | simp_rw [subset_iff, mem_posDiffs, mem_inter] | case refine'_1
α : Type u_1
inst✝ : DecidableEq α
𝒜 ℬ : Finset (Finset α)
h𝒜 : IsLowerSet ↑𝒜
hℬ : IsUpperSet ↑ℬ
⊢ 𝒜 \₊ ℬ ⊆ 𝒜 ∩ ℬ \₊ (𝒜 ∩ ℬ) | case refine'_1
α : Type u_1
inst✝ : DecidableEq α
𝒜 ℬ : Finset (Finset α)
h𝒜 : IsLowerSet ↑𝒜
hℬ : IsUpperSet ↑ℬ
⊢ ∀ ⦃x : Finset α⦄,
(∃ b ∈ 𝒜, ∃ c ∈ ℬ, c ≤ b ∧ b \ c = x) → ∃ b, (b ∈ 𝒜 ∧ b ∈ ℬ) ∧ ∃ c, (c ∈ 𝒜 ∧ c ∈ ℬ) ∧ c ≤ b ∧ b \ c = x |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Data/Finset/PosDiffs.lean | Finset.le_card_upper_inter_lower | [83, 1] | [91, 48] | rintro _ ⟨s, hs, t, ht, hts, rfl⟩ | case refine'_1
α : Type u_1
inst✝ : DecidableEq α
𝒜 ℬ : Finset (Finset α)
h𝒜 : IsLowerSet ↑𝒜
hℬ : IsUpperSet ↑ℬ
⊢ ∀ ⦃x : Finset α⦄,
(∃ b ∈ 𝒜, ∃ c ∈ ℬ, c ≤ b ∧ b \ c = x) → ∃ b, (b ∈ 𝒜 ∧ b ∈ ℬ) ∧ ∃ c, (c ∈ 𝒜 ∧ c ∈ ℬ) ∧ c ≤ b ∧ b \ c = x | case refine'_1.intro.intro.intro.intro.intro
α : Type u_1
inst✝ : DecidableEq α
𝒜 ℬ : Finset (Finset α)
h𝒜 : IsLowerSet ↑𝒜
hℬ : IsUpperSet ↑ℬ
s : Finset α
hs : s ∈ 𝒜
t : Finset α
ht : t ∈ ℬ
hts : t ≤ s
⊢ ∃ b, (b ∈ 𝒜 ∧ b ∈ ℬ) ∧ ∃ c, (c ∈ 𝒜 ∧ c ∈ ℬ) ∧ c ≤ b ∧ b \ c = s \ t |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Data/Finset/PosDiffs.lean | Finset.le_card_upper_inter_lower | [83, 1] | [91, 48] | exact ⟨s, ⟨hs, hℬ hts ht⟩, t, ⟨h𝒜 hts hs, ht⟩, hts, rfl⟩ | case refine'_1.intro.intro.intro.intro.intro
α : Type u_1
inst✝ : DecidableEq α
𝒜 ℬ : Finset (Finset α)
h𝒜 : IsLowerSet ↑𝒜
hℬ : IsUpperSet ↑ℬ
s : Finset α
hs : s ∈ 𝒜
t : Finset α
ht : t ∈ ℬ
hts : t ≤ s
⊢ ∃ b, (b ∈ 𝒜 ∧ b ∈ ℬ) ∧ ∃ c, (c ∈ 𝒜 ∧ c ∈ ℬ) ∧ c ≤ b ∧ b \ c = s \ t | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Data/Finset/PosDiffs.lean | Finset.le_card_upper_inter_lower | [83, 1] | [91, 48] | rw [coe_inter] | case refine'_2
α : Type u_1
inst✝ : DecidableEq α
𝒜 ℬ : Finset (Finset α)
h𝒜 : IsLowerSet ↑𝒜
hℬ : IsUpperSet ↑ℬ
⊢ (↑(𝒜 ∩ ℬ)).OrdConnected | case refine'_2
α : Type u_1
inst✝ : DecidableEq α
𝒜 ℬ : Finset (Finset α)
h𝒜 : IsLowerSet ↑𝒜
hℬ : IsUpperSet ↑ℬ
⊢ (↑𝒜 ∩ ↑ℬ).OrdConnected |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Data/Finset/PosDiffs.lean | Finset.le_card_upper_inter_lower | [83, 1] | [91, 48] | exact h𝒜.ordConnected.inter hℬ.ordConnected | case refine'_2
α : Type u_1
inst✝ : DecidableEq α
𝒜 ℬ : Finset (Finset α)
h𝒜 : IsLowerSet ↑𝒜
hℬ : IsUpperSet ↑ℬ
⊢ (↑𝒜 ∩ ↑ℬ).OrdConnected | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Data/Finset/PosDiffs.lean | Finset.mem_posSub | [111, 1] | [112, 96] | simp_rw [posSub, mem_image, mem_filter, mem_product, Prod.exists, and_assoc, exists_and_left] | α : Type u_1
inst✝³ : Sub α
inst✝² : Preorder α
inst✝¹ : DecidableRel fun x x_1 => x ≤ x_1
inst✝ : DecidableEq α
s t : Finset α
a : α
⊢ a ∈ s -₊ t ↔ ∃ b ∈ s, ∃ c ∈ t, c ≤ b ∧ b - c = a | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Data/Finset/PosDiffs.lean | Finset.posSub_subset_sub | [114, 1] | [115, 79] | rw [mem_posSub, mem_sub] | α : Type u_1
inst✝³ : Sub α
inst✝² : Preorder α
inst✝¹ : DecidableRel fun x x_1 => x ≤ x_1
inst✝ : DecidableEq α
s t : Finset α
a x : α
⊢ x ∈ s -₊ t → x ∈ s - t | α : Type u_1
inst✝³ : Sub α
inst✝² : Preorder α
inst✝¹ : DecidableRel fun x x_1 => x ≤ x_1
inst✝ : DecidableEq α
s t : Finset α
a x : α
⊢ (∃ b ∈ s, ∃ c ∈ t, c ≤ b ∧ b - c = x) → ∃ b ∈ s, ∃ c ∈ t, b - c = x |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Data/Finset/PosDiffs.lean | Finset.posSub_subset_sub | [114, 1] | [115, 79] | exact fun ⟨b, hb, c, hc, _, h⟩ ↦ ⟨b, hb, c, hc, h⟩ | α : Type u_1
inst✝³ : Sub α
inst✝² : Preorder α
inst✝¹ : DecidableRel fun x x_1 => x ≤ x_1
inst✝ : DecidableEq α
s t : Finset α
a x : α
⊢ (∃ b ∈ s, ∃ c ∈ t, c ≤ b ∧ b - c = x) → ∃ b ∈ s, ∃ c ∈ t, b - c = x | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Basic.lean | Geometry.SimplicialComplex.disjoint_interiors | [33, 1] | [44, 55] | classical
by_contra h
have hst : s ∩ t ⊂ s := by
use inter_subset_left
intro H
exact hxt.2 $ Set.mem_biUnion ⟨H.trans inter_subset_right,
fun H2 => h $ (H.trans inter_subset_right).antisymm H2⟩ hxs.1
refine' hxs.2 (Set.mem_biUnion hst _)
push_cast
exact K.inter_subset_convexHull hs ht ⟨hxs.1, hxt.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 : ℕ
hs : s ∈ K
ht : t ∈ K
hxs : x ∈ combiInterior 𝕜 s
hxt : x ∈ combiInterior 𝕜 t
⊢ s = t | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Basic.lean | Geometry.SimplicialComplex.disjoint_interiors | [33, 1] | [44, 55] | by_contra h | 𝕜 : 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
hxs : x ∈ combiInterior 𝕜 s
hxt : x ∈ combiInterior 𝕜 t
⊢ s = 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
hxs : x ∈ combiInterior 𝕜 s
hxt : x ∈ combiInterior 𝕜 t
h : ¬s = t
⊢ False |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Basic.lean | Geometry.SimplicialComplex.disjoint_interiors | [33, 1] | [44, 55] | have hst : s ∩ t ⊂ s := by
use inter_subset_left
intro H
exact hxt.2 $ Set.mem_biUnion ⟨H.trans inter_subset_right,
fun H2 => h $ (H.trans inter_subset_right).antisymm H2⟩ hxs.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 : ℕ
hs : s ∈ K
ht : t ∈ K
hxs : x ∈ combiInterior 𝕜 s
hxt : x ∈ combiInterior 𝕜 t
h : ¬s = t
⊢ False | 𝕜 : 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
hxs : x ∈ combiInterior 𝕜 s
hxt : x ∈ combiInterior 𝕜 t
h : ¬s = t
hst : s ∩ t ⊂ s
⊢ False |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Basic.lean | Geometry.SimplicialComplex.disjoint_interiors | [33, 1] | [44, 55] | refine' hxs.2 (Set.mem_biUnion 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
hxs : x ∈ combiInterior 𝕜 s
hxt : x ∈ combiInterior 𝕜 t
h : ¬s = t
hst : s ∩ t ⊂ s
⊢ False | 𝕜 : 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
hxs : x ∈ combiInterior 𝕜 s
hxt : x ∈ combiInterior 𝕜 t
h : ¬s = t
hst : s ∩ t ⊂ s
⊢ x ∈ (convexHull 𝕜) ↑(s ∩ t) |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Basic.lean | Geometry.SimplicialComplex.disjoint_interiors | [33, 1] | [44, 55] | push_cast | 𝕜 : 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
hxs : x ∈ combiInterior 𝕜 s
hxt : x ∈ combiInterior 𝕜 t
h : ¬s = t
hst : s ∩ t ⊂ s
⊢ x ∈ (convexHull 𝕜) ↑(s ∩ 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
hxs : x ∈ combiInterior 𝕜 s
hxt : x ∈ combiInterior 𝕜 t
h : ¬s = t
hst : s ∩ t ⊂ s
⊢ x ∈ (convexHull 𝕜) (↑s ∩ ↑t) |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Basic.lean | Geometry.SimplicialComplex.disjoint_interiors | [33, 1] | [44, 55] | exact K.inter_subset_convexHull hs ht ⟨hxs.1, hxt.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 : ℕ
hs : s ∈ K
ht : t ∈ K
hxs : x ∈ combiInterior 𝕜 s
hxt : x ∈ combiInterior 𝕜 t
h : ¬s = t
hst : s ∩ t ⊂ s
⊢ x ∈ (convexHull 𝕜) (↑s ∩ ↑t) | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Basic.lean | Geometry.SimplicialComplex.disjoint_interiors | [33, 1] | [44, 55] | use inter_subset_left | 𝕜 : 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
hxs : x ∈ combiInterior 𝕜 s
hxt : x ∈ combiInterior 𝕜 t
h : ¬s = t
⊢ s ∩ t ⊂ s | case right
𝕜 : 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
hxs : x ∈ combiInterior 𝕜 s
hxt : x ∈ combiInterior 𝕜 t
h : ¬s = t
⊢ ¬s ⊆ s ∩ t |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Basic.lean | Geometry.SimplicialComplex.disjoint_interiors | [33, 1] | [44, 55] | intro H | case right
𝕜 : 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
hxs : x ∈ combiInterior 𝕜 s
hxt : x ∈ combiInterior 𝕜 t
h : ¬s = t
⊢ ¬s ⊆ s ∩ t | case right
𝕜 : 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
hxs : x ∈ combiInterior 𝕜 s
hxt : x ∈ combiInterior 𝕜 t
h : ¬s = t
H : s ⊆ s ∩ t
⊢ False |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Basic.lean | Geometry.SimplicialComplex.disjoint_interiors | [33, 1] | [44, 55] | exact hxt.2 $ Set.mem_biUnion ⟨H.trans inter_subset_right,
fun H2 => h $ (H.trans inter_subset_right).antisymm H2⟩ hxs.1 | case right
𝕜 : 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
hxs : x ∈ combiInterior 𝕜 s
hxt : x ∈ combiInterior 𝕜 t
h : ¬s = t
H : s ⊆ s ∩ t
⊢ False | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Basic.lean | Geometry.SimplicialComplex.eq_singleton_of_singleton_mem_combiInterior | [50, 1] | [54, 28] | apply disjoint_interiors hs hx hxs | 𝕜 : 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
hs : s ∈ K
hxs : x ∈ combiInterior 𝕜 s
⊢ s = {x} | 𝕜 : 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
hs : s ∈ K
hxs : x ∈ combiInterior 𝕜 s
⊢ x ∈ combiInterior 𝕜 {x} |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Basic.lean | Geometry.SimplicialComplex.eq_singleton_of_singleton_mem_combiInterior | [50, 1] | [54, 28] | rw [combiInterior_singleton] | 𝕜 : 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
hs : s ∈ K
hxs : x ∈ combiInterior 𝕜 s
⊢ x ∈ combiInterior 𝕜 {x} | 𝕜 : 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
hs : s ∈ K
hxs : x ∈ combiInterior 𝕜 s
⊢ x ∈ {x} |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Basic.lean | Geometry.SimplicialComplex.eq_singleton_of_singleton_mem_combiInterior | [50, 1] | [54, 28] | exact Set.mem_singleton x | 𝕜 : 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
hs : s ∈ K
hxs : x ∈ combiInterior 𝕜 s
⊢ x ∈ {x} | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Basic.lean | Geometry.SimplicialComplex.combiInteriors_cover | [56, 1] | [66, 56] | unfold space | 𝕜 : 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 ∈ K, combiInterior 𝕜 s = K.space | 𝕜 : 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 ∈ K, combiInterior 𝕜 s = ⋃ s ∈ K.faces, (convexHull 𝕜) ↑s |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Basic.lean | Geometry.SimplicialComplex.combiInteriors_cover | [56, 1] | [66, 56] | refine' (Set.iUnion₂_mono fun _ _ => _).antisymm (Set.iUnion₂_subset fun s hs => _) | 𝕜 : 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 ∈ K, combiInterior 𝕜 s = ⋃ s ∈ K.faces, (convexHull 𝕜) ↑s | 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✝¹
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 |
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/SimplicialComplex/Skeleton.lean | Geometry.SimplicialComplex.skeleton_nonempty_iff | [32, 1] | [38, 20] | refine' ⟨Set.Nonempty.mono skeleton_le, _⟩ | 𝕜 : Type u_1
E : Type u_2
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
m n k : ℕ
K : SimplicialComplex 𝕜 E
s t : Finset E
A : Set (Finset E)
⊢ (K.skeleton k).faces.Nonempty ↔ K.faces.Nonempty | 𝕜 : Type u_1
E : Type u_2
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
m n k : ℕ
K : SimplicialComplex 𝕜 E
s t : Finset E
A : Set (Finset E)
⊢ K.faces.Nonempty → (K.skeleton k).faces.Nonempty |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Skeleton.lean | Geometry.SimplicialComplex.skeleton_nonempty_iff | [32, 1] | [38, 20] | rintro ⟨s, hs⟩ | 𝕜 : Type u_1
E : Type u_2
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
m n k : ℕ
K : SimplicialComplex 𝕜 E
s t : Finset E
A : Set (Finset E)
⊢ K.faces.Nonempty → (K.skeleton k).faces.Nonempty | case intro
𝕜 : Type u_1
E : Type u_2
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
m n k : ℕ
K : SimplicialComplex 𝕜 E
s✝ t : Finset E
A : Set (Finset E)
s : Finset E
hs : s ∈ K.faces
⊢ (K.skeleton k).faces.Nonempty |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Skeleton.lean | Geometry.SimplicialComplex.skeleton_nonempty_iff | [32, 1] | [38, 20] | obtain ⟨x, hx⟩ := K.nonempty hs | case intro
𝕜 : Type u_1
E : Type u_2
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
m n k : ℕ
K : SimplicialComplex 𝕜 E
s✝ t : Finset E
A : Set (Finset E)
s : Finset E
hs : s ∈ K.faces
⊢ (K.skeleton k).faces.Nonempty | case intro.intro
𝕜 : Type u_1
E : Type u_2
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
m n k : ℕ
K : SimplicialComplex 𝕜 E
s✝ t : Finset E
A : Set (Finset E)
s : Finset E
hs : s ∈ K.faces
x : E
hx : x ∈ s
⊢ (K.skeleton k).faces.Nonempty |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Skeleton.lean | Geometry.SimplicialComplex.skeleton_nonempty_iff | [32, 1] | [38, 20] | refine' ⟨{x}, K.down_closed' hs (singleton_subset_iff.2 hx) <| singleton_nonempty _, _⟩ | case intro.intro
𝕜 : Type u_1
E : Type u_2
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
m n k : ℕ
K : SimplicialComplex 𝕜 E
s✝ t : Finset E
A : Set (Finset E)
s : Finset E
hs : s ∈ K.faces
x : E
hx : x ∈ s
⊢ (K.skeleton k).faces.Nonempty | case intro.intro
𝕜 : Type u_1
E : Type u_2
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
m n k : ℕ
K : SimplicialComplex 𝕜 E
s✝ t : Finset E
A : Set (Finset E)
s : Finset E
hs : s ∈ K.faces
x : E
hx : x ∈ s
⊢ {x}.card ≤ k + 1 |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Skeleton.lean | Geometry.SimplicialComplex.skeleton_nonempty_iff | [32, 1] | [38, 20] | rw [card_singleton] | case intro.intro
𝕜 : Type u_1
E : Type u_2
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
m n k : ℕ
K : SimplicialComplex 𝕜 E
s✝ t : Finset E
A : Set (Finset E)
s : Finset E
hs : s ∈ K.faces
x : E
hx : x ∈ s
⊢ {x}.card ≤ k + 1 | case intro.intro
𝕜 : Type u_1
E : Type u_2
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
m n k : ℕ
K : SimplicialComplex 𝕜 E
s✝ t : Finset E
A : Set (Finset E)
s : Finset E
hs : s ∈ K.faces
x : E
hx : x ∈ s
⊢ 1 ≤ k + 1 |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Skeleton.lean | Geometry.SimplicialComplex.skeleton_nonempty_iff | [32, 1] | [38, 20] | exact le_add_self | case intro.intro
𝕜 : Type u_1
E : Type u_2
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
m n k : ℕ
K : SimplicialComplex 𝕜 E
s✝ t : Finset E
A : Set (Finset E)
s : Finset E
hs : s ∈ K.faces
x : E
hx : x ∈ s
⊢ 1 ≤ k + 1 | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Skeleton.lean | Geometry.SimplicialComplex.Pure.skeleton_of_le | [40, 1] | [44, 34] | refine' ⟨fun s hs => hs.2, _⟩ | 𝕜 : Type u_1
E : Type u_2
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
m n k : ℕ
K : SimplicialComplex 𝕜 E
s t : Finset E
A : Set (Finset E)
hK : K.Pure n
h : k ≤ n
⊢ (K.skeleton k).Pure k | 𝕜 : Type u_1
E : Type u_2
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
m n k : ℕ
K : SimplicialComplex 𝕜 E
s t : Finset E
A : Set (Finset E)
hK : K.Pure n
h : k ≤ n
⊢ Set.Sized (k + 1) (K.skeleton k).facets |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Skeleton.lean | Geometry.SimplicialComplex.Pure.skeleton_of_le | [40, 1] | [44, 34] | rintro s ⟨⟨hs, hscard⟩, hsmax⟩ | 𝕜 : Type u_1
E : Type u_2
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
m n k : ℕ
K : SimplicialComplex 𝕜 E
s t : Finset E
A : Set (Finset E)
hK : K.Pure n
h : k ≤ n
⊢ Set.Sized (k + 1) (K.skeleton k).facets | case intro.intro
𝕜 : Type u_1
E : Type u_2
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
m n k : ℕ
K : SimplicialComplex 𝕜 E
s✝ t : Finset E
A : Set (Finset E)
hK : K.Pure n
h : k ≤ n
s : Finset E
hsmax : ∀ ⦃t : Finset E⦄, t ∈ (K.skeleton k).faces → s ⊆ t → s = t
hs : s ∈ K
hscard : s.card ≤ k + 1
⊢ s.card = k + 1 |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Skeleton.lean | Geometry.SimplicialComplex.Pure.skeleton_of_le | [40, 1] | [44, 34] | obtain ⟨t, ht, hst, htcard⟩ := hK.exists_face_of_card_le (add_le_add_right h 1) hs hscard | case intro.intro
𝕜 : Type u_1
E : Type u_2
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
m n k : ℕ
K : SimplicialComplex 𝕜 E
s✝ t : Finset E
A : Set (Finset E)
hK : K.Pure n
h : k ≤ n
s : Finset E
hsmax : ∀ ⦃t : Finset E⦄, t ∈ (K.skeleton k).faces → s ⊆ t → s = t
hs : s ∈ K
hscard : s.card ≤ k + 1
⊢ s.card = k + 1 | case intro.intro.intro.intro.intro
𝕜 : Type u_1
E : Type u_2
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
m n k : ℕ
K : SimplicialComplex 𝕜 E
s✝ t✝ : Finset E
A : Set (Finset E)
hK : K.Pure n
h : k ≤ n
s : Finset E
hsmax : ∀ ⦃t : Finset E⦄, t ∈ (K.skeleton k).faces → s ⊆ t → s = t
hs : s ∈ K
hscard : s.card ≤ k + 1
t : Finset E
ht : t ∈ K
hst : s ⊆ t
htcard : t.card = k + 1
⊢ s.card = k + 1 |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Skeleton.lean | Geometry.SimplicialComplex.Pure.skeleton_of_le | [40, 1] | [44, 34] | rwa [hsmax ⟨ht, htcard.le⟩ hst] | case intro.intro.intro.intro.intro
𝕜 : Type u_1
E : Type u_2
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
m n k : ℕ
K : SimplicialComplex 𝕜 E
s✝ t✝ : Finset E
A : Set (Finset E)
hK : K.Pure n
h : k ≤ n
s : Finset E
hsmax : ∀ ⦃t : Finset E⦄, t ∈ (K.skeleton k).faces → s ⊆ t → s = t
hs : s ∈ K
hscard : s.card ≤ k + 1
t : Finset E
ht : t ∈ K
hst : s ⊆ t
htcard : t.card = k + 1
⊢ s.card = k + 1 | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Skeleton.lean | Geometry.SimplicialComplex.Pure.skeleton | [53, 1] | [61, 18] | obtain hn | hn := le_total k n | 𝕜 : Type u_1
E : Type u_2
inst✝³ : LinearOrderedField 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
inst✝ : FiniteDimensional 𝕜 E
m n k : ℕ
K : SimplicialComplex 𝕜 E
s t : Finset E
A : Set (Finset E)
hK : K.Pure n
⊢ (K.skeleton k).Pure (min k n) | case inl
𝕜 : Type u_1
E : Type u_2
inst✝³ : LinearOrderedField 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
inst✝ : FiniteDimensional 𝕜 E
m n k : ℕ
K : SimplicialComplex 𝕜 E
s t : Finset E
A : Set (Finset E)
hK : K.Pure n
hn : k ≤ n
⊢ (K.skeleton k).Pure (min k n)
case inr
𝕜 : Type u_1
E : Type u_2
inst✝³ : LinearOrderedField 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
inst✝ : FiniteDimensional 𝕜 E
m n k : ℕ
K : SimplicialComplex 𝕜 E
s t : Finset E
A : Set (Finset E)
hK : K.Pure n
hn : n ≤ k
⊢ (K.skeleton k).Pure (min k n) |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Skeleton.lean | Geometry.SimplicialComplex.Pure.skeleton | [53, 1] | [61, 18] | rw [min_eq_left hn] | case inl
𝕜 : Type u_1
E : Type u_2
inst✝³ : LinearOrderedField 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
inst✝ : FiniteDimensional 𝕜 E
m n k : ℕ
K : SimplicialComplex 𝕜 E
s t : Finset E
A : Set (Finset E)
hK : K.Pure n
hn : k ≤ n
⊢ (K.skeleton k).Pure (min k n) | case inl
𝕜 : Type u_1
E : Type u_2
inst✝³ : LinearOrderedField 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
inst✝ : FiniteDimensional 𝕜 E
m n k : ℕ
K : SimplicialComplex 𝕜 E
s t : Finset E
A : Set (Finset E)
hK : K.Pure n
hn : k ≤ n
⊢ (K.skeleton k).Pure k |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Skeleton.lean | Geometry.SimplicialComplex.Pure.skeleton | [53, 1] | [61, 18] | exact hK.skeleton_of_le hn | case inl
𝕜 : Type u_1
E : Type u_2
inst✝³ : LinearOrderedField 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
inst✝ : FiniteDimensional 𝕜 E
m n k : ℕ
K : SimplicialComplex 𝕜 E
s t : Finset E
A : Set (Finset E)
hK : K.Pure n
hn : k ≤ n
⊢ (K.skeleton k).Pure k | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Skeleton.lean | Geometry.SimplicialComplex.Pure.skeleton | [53, 1] | [61, 18] | rw [min_eq_right hn] | case inr
𝕜 : Type u_1
E : Type u_2
inst✝³ : LinearOrderedField 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
inst✝ : FiniteDimensional 𝕜 E
m n k : ℕ
K : SimplicialComplex 𝕜 E
s t : Finset E
A : Set (Finset E)
hK : K.Pure n
hn : n ≤ k
⊢ (K.skeleton k).Pure (min k n) | case inr
𝕜 : Type u_1
E : Type u_2
inst✝³ : LinearOrderedField 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
inst✝ : FiniteDimensional 𝕜 E
m n k : ℕ
K : SimplicialComplex 𝕜 E
s t : Finset E
A : Set (Finset E)
hK : K.Pure n
hn : n ≤ k
⊢ (K.skeleton k).Pure n |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Skeleton.lean | Geometry.SimplicialComplex.Pure.skeleton | [53, 1] | [61, 18] | refine' ⟨fun s hs => hK.1 <| skeleton_le hs, fun s hs => _⟩ | case inr
𝕜 : Type u_1
E : Type u_2
inst✝³ : LinearOrderedField 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
inst✝ : FiniteDimensional 𝕜 E
m n k : ℕ
K : SimplicialComplex 𝕜 E
s t : Finset E
A : Set (Finset E)
hK : K.Pure n
hn : n ≤ k
⊢ (K.skeleton k).Pure n | case inr
𝕜 : Type u_1
E : Type u_2
inst✝³ : LinearOrderedField 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
inst✝ : FiniteDimensional 𝕜 E
m n k : ℕ
K : SimplicialComplex 𝕜 E
s✝ t : Finset E
A : Set (Finset E)
hK : K.Pure n
hn : n ≤ k
s : Finset E
hs : s ∈ (K.skeleton k).facets
⊢ s.card = n + 1 |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Skeleton.lean | Geometry.SimplicialComplex.Pure.skeleton | [53, 1] | [61, 18] | obtain ⟨t, ht, hst⟩ := subfacet (skeleton_le hs.1) | case inr
𝕜 : Type u_1
E : Type u_2
inst✝³ : LinearOrderedField 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
inst✝ : FiniteDimensional 𝕜 E
m n k : ℕ
K : SimplicialComplex 𝕜 E
s✝ t : Finset E
A : Set (Finset E)
hK : K.Pure n
hn : n ≤ k
s : Finset E
hs : s ∈ (K.skeleton k).facets
⊢ s.card = n + 1 | case inr.intro.intro
𝕜 : Type u_1
E : Type u_2
inst✝³ : LinearOrderedField 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
inst✝ : FiniteDimensional 𝕜 E
m n k : ℕ
K : SimplicialComplex 𝕜 E
s✝ t✝ : Finset E
A : Set (Finset E)
hK : K.Pure n
hn : n ≤ k
s : Finset E
hs : s ∈ (K.skeleton k).facets
t : Finset E
ht : t ∈ K.facets
hst : s ⊆ t
⊢ s.card = n + 1 |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Skeleton.lean | Geometry.SimplicialComplex.Pure.skeleton | [53, 1] | [61, 18] | rw [hs.2 ⟨facets_subset ht, (hK.2 ht).le.trans (add_le_add_right hn _)⟩ hst] | case inr.intro.intro
𝕜 : Type u_1
E : Type u_2
inst✝³ : LinearOrderedField 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
inst✝ : FiniteDimensional 𝕜 E
m n k : ℕ
K : SimplicialComplex 𝕜 E
s✝ t✝ : Finset E
A : Set (Finset E)
hK : K.Pure n
hn : n ≤ k
s : Finset E
hs : s ∈ (K.skeleton k).facets
t : Finset E
ht : t ∈ K.facets
hst : s ⊆ t
⊢ s.card = n + 1 | case inr.intro.intro
𝕜 : Type u_1
E : Type u_2
inst✝³ : LinearOrderedField 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
inst✝ : FiniteDimensional 𝕜 E
m n k : ℕ
K : SimplicialComplex 𝕜 E
s✝ t✝ : Finset E
A : Set (Finset E)
hK : K.Pure n
hn : n ≤ k
s : Finset E
hs : s ∈ (K.skeleton k).facets
t : Finset E
ht : t ∈ K.facets
hst : s ⊆ t
⊢ t.card = n + 1 |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Skeleton.lean | Geometry.SimplicialComplex.Pure.skeleton | [53, 1] | [61, 18] | exact hK.2 ht | case inr.intro.intro
𝕜 : Type u_1
E : Type u_2
inst✝³ : LinearOrderedField 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
inst✝ : FiniteDimensional 𝕜 E
m n k : ℕ
K : SimplicialComplex 𝕜 E
s✝ t✝ : Finset E
A : Set (Finset E)
hK : K.Pure n
hn : n ≤ k
s : Finset E
hs : s ∈ (K.skeleton k).facets
t : Finset E
ht : t ∈ K.facets
hst : s ⊆ t
⊢ t.card = n + 1 | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Data/List/Basic.lean | List.getLast_filter | [6, 1] | [18, 42] | rw [List.getLast_singleton'] at h' | α✝ : Type u_1
l l' l₀ l₁ l₂ : List α✝
a✝ b : α✝
m n : ℕ
α : Type u_2
p : α → Bool
a : α
h : filter p [a] ≠ []
h' : p ([a].getLast ⋯) = true
⊢ (filter p [a]).getLast h = [a].getLast ⋯ | α✝ : Type u_1
l l' l₀ l₁ l₂ : List α✝
a✝ b : α✝
m n : ℕ
α : Type u_2
p : α → Bool
a : α
h : filter p [a] ≠ []
h' : p a = true
⊢ (filter p [a]).getLast h = [a].getLast ⋯ |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Data/List/Basic.lean | List.getLast_filter | [6, 1] | [18, 42] | simp [List.filter_cons, h'] | α✝ : Type u_1
l l' l₀ l₁ l₂ : List α✝
a✝ b : α✝
m n : ℕ
α : Type u_2
p : α → Bool
a : α
h : filter p [a] ≠ []
h' : p a = true
⊢ (filter p [a]).getLast h = [a].getLast ⋯ | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Data/List/Basic.lean | List.getLast_filter | [6, 1] | [18, 42] | rw [List.getLast_cons_cons] at h' ⊢ | α✝ : Type u_1
l l' l₀ l₁ l₂ : List α✝
a✝ b✝ : α✝
m n : ℕ
α : Type u_2
p : α → Bool
a b : α
as : List α
h : filter p (a :: b :: as) ≠ []
h' : p ((a :: b :: as).getLast ⋯) = true
⊢ (filter p (a :: b :: as)).getLast h = (a :: b :: as).getLast ⋯ | α✝ : Type u_1
l l' l₀ l₁ l₂ : List α✝
a✝ b✝ : α✝
m n : ℕ
α : Type u_2
p : α → Bool
a b : α
as : List α
h : filter p (a :: b :: as) ≠ []
h' : p ((b :: as).getLast ⋯) = true
⊢ (filter p (a :: b :: as)).getLast h = (b :: as).getLast ⋯ |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Data/List/Basic.lean | List.getLast_filter | [6, 1] | [18, 42] | simp only [List.filter_cons (x := a)] at h ⊢ | α✝ : Type u_1
l l' l₀ l₁ l₂ : List α✝
a✝ b✝ : α✝
m n : ℕ
α : Type u_2
p : α → Bool
a b : α
as : List α
h : filter p (a :: b :: as) ≠ []
h' : p ((b :: as).getLast ⋯) = true
⊢ (filter p (a :: b :: as)).getLast h = (b :: as).getLast ⋯ | α✝ : Type u_1
l l' l₀ l₁ l₂ : List α✝
a✝ b✝ : α✝
m n : ℕ
α : Type u_2
p : α → Bool
a b : α
as : List α
h✝ : filter p (a :: b :: as) ≠ []
h' : p ((b :: as).getLast ⋯) = true
h : (if p a = true then a :: filter p (b :: as) else filter p (b :: as)) ≠ []
⊢ (if p a = true then a :: filter p (b :: as) else filter p (b :: as)).getLast ⋯ = (b :: as).getLast ⋯ |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Data/List/Basic.lean | List.getLast_filter | [6, 1] | [18, 42] | obtain ha | ha := Bool.eq_false_or_eq_true (p a) | α✝ : Type u_1
l l' l₀ l₁ l₂ : List α✝
a✝ b✝ : α✝
m n : ℕ
α : Type u_2
p : α → Bool
a b : α
as : List α
h✝ : filter p (a :: b :: as) ≠ []
h' : p ((b :: as).getLast ⋯) = true
h : (if p a = true then a :: filter p (b :: as) else filter p (b :: as)) ≠ []
⊢ (if p a = true then a :: filter p (b :: as) else filter p (b :: as)).getLast ⋯ = (b :: as).getLast ⋯ | case inl
α✝ : Type u_1
l l' l₀ l₁ l₂ : List α✝
a✝ b✝ : α✝
m n : ℕ
α : Type u_2
p : α → Bool
a b : α
as : List α
h✝ : filter p (a :: b :: as) ≠ []
h' : p ((b :: as).getLast ⋯) = true
h : (if p a = true then a :: filter p (b :: as) else filter p (b :: as)) ≠ []
ha : p a = true
⊢ (if p a = true then a :: filter p (b :: as) else filter p (b :: as)).getLast ⋯ = (b :: as).getLast ⋯
case inr
α✝ : Type u_1
l l' l₀ l₁ l₂ : List α✝
a✝ b✝ : α✝
m n : ℕ
α : Type u_2
p : α → Bool
a b : α
as : List α
h✝ : filter p (a :: b :: as) ≠ []
h' : p ((b :: as).getLast ⋯) = true
h : (if p a = true then a :: filter p (b :: as) else filter p (b :: as)) ≠ []
ha : p a = false
⊢ (if p a = true then a :: filter p (b :: as) else filter p (b :: as)).getLast ⋯ = (b :: as).getLast ⋯ |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Data/List/Basic.lean | List.getLast_filter | [6, 1] | [18, 42] | simp only [ha, ite_true] | case inl
α✝ : Type u_1
l l' l₀ l₁ l₂ : List α✝
a✝ b✝ : α✝
m n : ℕ
α : Type u_2
p : α → Bool
a b : α
as : List α
h✝ : filter p (a :: b :: as) ≠ []
h' : p ((b :: as).getLast ⋯) = true
h : (if p a = true then a :: filter p (b :: as) else filter p (b :: as)) ≠ []
ha : p a = true
⊢ (if p a = true then a :: filter p (b :: as) else filter p (b :: as)).getLast ⋯ = (b :: as).getLast ⋯ | case inl
α✝ : Type u_1
l l' l₀ l₁ l₂ : List α✝
a✝ b✝ : α✝
m n : ℕ
α : Type u_2
p : α → Bool
a b : α
as : List α
h✝ : filter p (a :: b :: as) ≠ []
h' : p ((b :: as).getLast ⋯) = true
h : (if p a = true then a :: filter p (b :: as) else filter p (b :: as)) ≠ []
ha : p a = true
⊢ (a :: filter p (b :: as)).getLast ⋯ = (b :: as).getLast ⋯ |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Data/List/Basic.lean | List.getLast_filter | [6, 1] | [18, 42] | rw [getLast_cons, getLast_filter (b :: as) _ h'] | case inl
α✝ : Type u_1
l l' l₀ l₁ l₂ : List α✝
a✝ b✝ : α✝
m n : ℕ
α : Type u_2
p : α → Bool
a b : α
as : List α
h✝ : filter p (a :: b :: as) ≠ []
h' : p ((b :: as).getLast ⋯) = true
h : (if p a = true then a :: filter p (b :: as) else filter p (b :: as)) ≠ []
ha : p a = true
⊢ (a :: filter p (b :: as)).getLast ⋯ = (b :: as).getLast ⋯ | α✝ : Type u_1
l l' l₀ l₁ l₂ : List α✝
a✝ b✝ : α✝
m n : ℕ
α : Type u_2
p : α → Bool
a b : α
as : List α
h✝ : filter p (a :: b :: as) ≠ []
h' : p ((b :: as).getLast ⋯) = true
h : (if p a = true then a :: filter p (b :: as) else filter p (b :: as)) ≠ []
ha : p a = true
⊢ filter p (b :: as) ≠ [] |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Data/List/Basic.lean | List.getLast_filter | [6, 1] | [18, 42] | exact ne_nil_of_mem $ mem_filter.2 ⟨getLast_mem _, h'⟩ | α✝ : Type u_1
l l' l₀ l₁ l₂ : List α✝
a✝ b✝ : α✝
m n : ℕ
α : Type u_2
p : α → Bool
a b : α
as : List α
h✝ : filter p (a :: b :: as) ≠ []
h' : p ((b :: as).getLast ⋯) = true
h : (if p a = true then a :: filter p (b :: as) else filter p (b :: as)) ≠ []
ha : p a = true
⊢ filter p (b :: as) ≠ [] | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Data/List/Basic.lean | List.getLast_filter | [6, 1] | [18, 42] | simp only [ha, cond_false] at h ⊢ | case inr
α✝ : Type u_1
l l' l₀ l₁ l₂ : List α✝
a✝ b✝ : α✝
m n : ℕ
α : Type u_2
p : α → Bool
a b : α
as : List α
h✝ : filter p (a :: b :: as) ≠ []
h' : p ((b :: as).getLast ⋯) = true
h : (if p a = true then a :: filter p (b :: as) else filter p (b :: as)) ≠ []
ha : p a = false
⊢ (if p a = true then a :: filter p (b :: as) else filter p (b :: as)).getLast ⋯ = (b :: as).getLast ⋯ | case inr
α✝ : Type u_1
l l' l₀ l₁ l₂ : List α✝
a✝ b✝ : α✝
m n : ℕ
α : Type u_2
p : α → Bool
a b : α
as : List α
h✝ : filter p (a :: b :: as) ≠ []
h' : p ((b :: as).getLast ⋯) = true
ha : p a = false
h : (if False then a :: filter p (b :: as) else filter p (b :: as)) ≠ []
⊢ (if False then a :: filter p (b :: as) else filter p (b :: as)).getLast ⋯ = (b :: as).getLast ⋯ |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Data/List/Basic.lean | List.getLast_filter | [6, 1] | [18, 42] | exact getLast_filter (b :: as) h h' | case inr
α✝ : Type u_1
l l' l₀ l₁ l₂ : List α✝
a✝ b✝ : α✝
m n : ℕ
α : Type u_2
p : α → Bool
a b : α
as : List α
h✝ : filter p (a :: b :: as) ≠ []
h' : p ((b :: as).getLast ⋯) = true
ha : p a = false
h : (if False then a :: filter p (b :: as) else filter p (b :: as)) ≠ []
⊢ (if False then a :: filter p (b :: as) else filter p (b :: as)).getLast ⋯ = (b :: as).getLast ⋯ | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Data/List/Basic.lean | List.cons_sublist_cons_iff' | [20, 1] | [27, 30] | constructor | α : Type u_1
l l' l₀ l₁ l₂ : List α
a b : α
m n : ℕ
⊢ a :: l₁ <+ b :: l₂ ↔ a :: l₁ <+ l₂ ∨ a = b ∧ l₁ <+ l₂ | case mp
α : Type u_1
l l' l₀ l₁ l₂ : List α
a b : α
m n : ℕ
⊢ a :: l₁ <+ b :: l₂ → a :: l₁ <+ l₂ ∨ a = b ∧ l₁ <+ l₂
case mpr
α : Type u_1
l l' l₀ l₁ l₂ : List α
a b : α
m n : ℕ
⊢ a :: l₁ <+ l₂ ∨ a = b ∧ l₁ <+ l₂ → a :: l₁ <+ b :: l₂ |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Data/List/Basic.lean | List.cons_sublist_cons_iff' | [20, 1] | [27, 30] | rintro (_ | _) | case mp
α : Type u_1
l l' l₀ l₁ l₂ : List α
a b : α
m n : ℕ
⊢ a :: l₁ <+ b :: l₂ → a :: l₁ <+ l₂ ∨ a = b ∧ l₁ <+ l₂ | case mp.cons
α : Type u_1
l l' l₀ l₁ l₂ : List α
a b : α
m n : ℕ
a✝ : a :: l₁ <+ l₂
⊢ a :: l₁ <+ l₂ ∨ a = b ∧ l₁ <+ l₂
case mp.cons₂
α : Type u_1
l l' l₀ l₁ l₂ : List α
a : α
m n : ℕ
a✝ : l₁ <+ l₂
⊢ a :: l₁ <+ l₂ ∨ a = a ∧ l₁ <+ l₂ |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Data/List/Basic.lean | List.cons_sublist_cons_iff' | [20, 1] | [27, 30] | exact Or.inl ‹_› | case mp.cons
α : Type u_1
l l' l₀ l₁ l₂ : List α
a b : α
m n : ℕ
a✝ : a :: l₁ <+ l₂
⊢ a :: l₁ <+ l₂ ∨ a = b ∧ l₁ <+ l₂ | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Data/List/Basic.lean | List.cons_sublist_cons_iff' | [20, 1] | [27, 30] | exact Or.inr ⟨rfl, ‹_›⟩ | case mp.cons₂
α : Type u_1
l l' l₀ l₁ l₂ : List α
a : α
m n : ℕ
a✝ : l₁ <+ l₂
⊢ a :: l₁ <+ l₂ ∨ a = a ∧ l₁ <+ l₂ | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Data/List/Basic.lean | List.cons_sublist_cons_iff' | [20, 1] | [27, 30] | rintro (h | ⟨rfl, h⟩) | case mpr
α : Type u_1
l l' l₀ l₁ l₂ : List α
a b : α
m n : ℕ
⊢ a :: l₁ <+ l₂ ∨ a = b ∧ l₁ <+ l₂ → a :: l₁ <+ b :: l₂ | case mpr.inl
α : Type u_1
l l' l₀ l₁ l₂ : List α
a b : α
m n : ℕ
h : a :: l₁ <+ l₂
⊢ a :: l₁ <+ b :: l₂
case mpr.inr.intro
α : Type u_1
l l' l₀ l₁ l₂ : List α
a : α
m n : ℕ
h : l₁ <+ l₂
⊢ a :: l₁ <+ a :: l₂ |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Data/List/Basic.lean | List.cons_sublist_cons_iff' | [20, 1] | [27, 30] | exact sublist_cons_of_sublist _ h | case mpr.inl
α : Type u_1
l l' l₀ l₁ l₂ : List α
a b : α
m n : ℕ
h : a :: l₁ <+ l₂
⊢ a :: l₁ <+ b :: l₂ | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Data/List/Basic.lean | List.cons_sublist_cons_iff' | [20, 1] | [27, 30] | rwa [cons_sublist_cons] | case mpr.inr.intro
α : Type u_1
l l' l₀ l₁ l₂ : List α
a : α
m n : ℕ
h : l₁ <+ l₂
⊢ a :: l₁ <+ a :: l₂ | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Data/List/Basic.lean | List.subperm_nil | [33, 1] | [34, 77] | rintro rfl | α : Type u_1
l l' l₀ l₁ l₂ : List α
a b : α
m n : ℕ
⊢ l = [] → l <+~ [] | α : Type u_1
l' l₀ l₁ l₂ : List α
a b : α
m n : ℕ
⊢ [] <+~ [] |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Data/List/Basic.lean | List.subperm_nil | [33, 1] | [34, 77] | rfl | α : Type u_1
l' l₀ l₁ l₂ : List α
a b : α
m n : ℕ
⊢ [] <+~ [] | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Combinatorics/SimpleGraph/Maps.lean | SimpleGraph.spanningCoe_induce | [9, 1] | [10, 79] | ext | α : Type u_1
G : SimpleGraph α
s : Set α
⊢ (induce s G).spanningCoe = G.ind s | case Adj.h.h.a
α : Type u_1
G : SimpleGraph α
s : Set α
x✝¹ x✝ : α
⊢ (induce s G).spanningCoe.Adj x✝¹ x✝ ↔ (G.ind s).Adj x✝¹ x✝ |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Combinatorics/SimpleGraph/Maps.lean | SimpleGraph.spanningCoe_induce | [9, 1] | [10, 79] | simp [← and_assoc] | case Adj.h.h.a
α : Type u_1
G : SimpleGraph α
s : Set α
x✝¹ x✝ : α
⊢ (induce s G).spanningCoe.Adj x✝¹ x✝ ↔ (G.ind s).Adj x✝¹ x✝ | no goals |
Subsets and Splits
No community queries yet
The top public SQL queries from the community will appear here once available.