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/Simplex.lean | combiFrontier_eq | [90, 1] | [135, 14] | simp only [and_imp, exists_prop, exists_imp] | case h.mpr
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x✝ x : E
⊢ (∃ w, ∃ (_ : ∀ y ∈ s, 0 ≤ w y) (_ : ∑ y ∈ s, w y = 1) (_ : ∃ y ∈ s, w y = 0), s.centerMass w id = x) →
∃ i, ∃ (_ : i ⊂ s), x ∈ (convexHull 𝕜) ↑i | case h.mpr
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x✝ x : E
⊢ ∀ (x_1 : E → 𝕜),
(∀ y ∈ s, 0 ≤ x_1 y) →
∑ y ∈ s, x_1 y = 1 → ∀ x_2 ∈ s, x_1 x_2 = 0 → s.centerMass x_1 id = x → ∃ i ⊂ s, x ∈ (convexHull 𝕜) ↑i |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | combiFrontier_eq | [90, 1] | [135, 14] | intro w hw₁ hw₂ y hy₁ hy₂ hy₃ | case h.mpr
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x✝ x : E
⊢ ∀ (x_1 : E → 𝕜),
(∀ y ∈ s, 0 ≤ x_1 y) →
∑ y ∈ s, x_1 y = 1 → ∀ x_2 ∈ s, x_1 x_2 = 0 → s.centerMass x_1 id = x → ∃ i ⊂ s, x ∈ (convexHull 𝕜) ↑i | case h.mpr
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x✝ x : E
w : E → 𝕜
hw₁ : ∀ y ∈ s, 0 ≤ w y
hw₂ : ∑ y ∈ s, w y = 1
y : E
hy₁ : y ∈ s
hy₂ : w y = 0
hy₃ : s.centerMass w id = x
⊢ ∃ i ⊂ s, x ∈ (convexHull 𝕜) ↑i |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | combiFrontier_eq | [90, 1] | [135, 14] | refine' ⟨s.erase y, Finset.erase_ssubset hy₁, _⟩ | case h.mpr
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x✝ x : E
w : E → 𝕜
hw₁ : ∀ y ∈ s, 0 ≤ w y
hw₂ : ∑ y ∈ s, w y = 1
y : E
hy₁ : y ∈ s
hy₂ : w y = 0
hy₃ : s.centerMass w id = x
⊢ ∃ i ⊂ s, x ∈ (convexHull 𝕜) ↑i | case h.mpr
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x✝ x : E
w : E → 𝕜
hw₁ : ∀ y ∈ s, 0 ≤ w y
hw₂ : ∑ y ∈ s, w y = 1
y : E
hy₁ : y ∈ s
hy₂ : w y = 0
hy₃ : s.centerMass w id = x
⊢ x ∈ (convexHull 𝕜) ↑(s.erase y) |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | combiFrontier_eq | [90, 1] | [135, 14] | rw [Finset.convexHull_eq, Set.mem_setOf_eq] | case h.mpr
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x✝ x : E
w : E → 𝕜
hw₁ : ∀ y ∈ s, 0 ≤ w y
hw₂ : ∑ y ∈ s, w y = 1
y : E
hy₁ : y ∈ s
hy₂ : w y = 0
hy₃ : s.centerMass w id = x
⊢ x ∈ (convexHull 𝕜) ↑(s.erase y) | case h.mpr
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x✝ x : E
w : E → 𝕜
hw₁ : ∀ y ∈ s, 0 ≤ w y
hw₂ : ∑ y ∈ s, w y = 1
y : E
hy₁ : y ∈ s
hy₂ : w y = 0
hy₃ : s.centerMass w id = x
⊢ ∃ w, (∀ y_1 ∈ s.erase y, 0 ≤ w y_1) ∧ ∑ y ∈ s.erase y, w y = 1 ∧ (s.erase y).centerMass w id = x |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | combiFrontier_eq | [90, 1] | [135, 14] | refine' ⟨w, fun z hz => hw₁ z (s.erase_subset _ hz), _, _⟩ | case h.mpr
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x✝ x : E
w : E → 𝕜
hw₁ : ∀ y ∈ s, 0 ≤ w y
hw₂ : ∑ y ∈ s, w y = 1
y : E
hy₁ : y ∈ s
hy₂ : w y = 0
hy₃ : s.centerMass w id = x
⊢ ∃ w, (∀ y_1 ∈ s.erase y, 0 ≤ w y_1) ∧ ∑ y ∈ s.erase y, w y = 1 ∧ (s.erase y).centerMass w id = x | case h.mpr.refine'_1
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x✝ x : E
w : E → 𝕜
hw₁ : ∀ y ∈ s, 0 ≤ w y
hw₂ : ∑ y ∈ s, w y = 1
y : E
hy₁ : y ∈ s
hy₂ : w y = 0
hy₃ : s.centerMass w id = x
⊢ ∑ y ∈ s.erase y, w y = 1
case h.mpr.refine'_2
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x✝ x : E
w : E → 𝕜
hw₁ : ∀ y ∈ s, 0 ≤ w y
hw₂ : ∑ y ∈ s, w y = 1
y : E
hy₁ : y ∈ s
hy₂ : w y = 0
hy₃ : s.centerMass w id = x
⊢ (s.erase y).centerMass w id = x |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | combiFrontier_eq | [90, 1] | [135, 14] | rw [Finset.sum_erase _ hy₂] | case h.mpr.refine'_1
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x✝ x : E
w : E → 𝕜
hw₁ : ∀ y ∈ s, 0 ≤ w y
hw₂ : ∑ y ∈ s, w y = 1
y : E
hy₁ : y ∈ s
hy₂ : w y = 0
hy₃ : s.centerMass w id = x
⊢ ∑ y ∈ s.erase y, w y = 1
case h.mpr.refine'_2
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x✝ x : E
w : E → 𝕜
hw₁ : ∀ y ∈ s, 0 ≤ w y
hw₂ : ∑ y ∈ s, w y = 1
y : E
hy₁ : y ∈ s
hy₂ : w y = 0
hy₃ : s.centerMass w id = x
⊢ (s.erase y).centerMass w id = x | case h.mpr.refine'_1
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x✝ x : E
w : E → 𝕜
hw₁ : ∀ y ∈ s, 0 ≤ w y
hw₂ : ∑ y ∈ s, w y = 1
y : E
hy₁ : y ∈ s
hy₂ : w y = 0
hy₃ : s.centerMass w id = x
⊢ ∑ x ∈ s, w x = 1
case h.mpr.refine'_2
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x✝ x : E
w : E → 𝕜
hw₁ : ∀ y ∈ s, 0 ≤ w y
hw₂ : ∑ y ∈ s, w y = 1
y : E
hy₁ : y ∈ s
hy₂ : w y = 0
hy₃ : s.centerMass w id = x
⊢ (s.erase y).centerMass w id = x |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | combiFrontier_eq | [90, 1] | [135, 14] | apply hw₂ | case h.mpr.refine'_1
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x✝ x : E
w : E → 𝕜
hw₁ : ∀ y ∈ s, 0 ≤ w y
hw₂ : ∑ y ∈ s, w y = 1
y : E
hy₁ : y ∈ s
hy₂ : w y = 0
hy₃ : s.centerMass w id = x
⊢ ∑ x ∈ s, w x = 1
case h.mpr.refine'_2
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x✝ x : E
w : E → 𝕜
hw₁ : ∀ y ∈ s, 0 ≤ w y
hw₂ : ∑ y ∈ s, w y = 1
y : E
hy₁ : y ∈ s
hy₂ : w y = 0
hy₃ : s.centerMass w id = x
⊢ (s.erase y).centerMass w id = x | case h.mpr.refine'_2
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x✝ x : E
w : E → 𝕜
hw₁ : ∀ y ∈ s, 0 ≤ w y
hw₂ : ∑ y ∈ s, w y = 1
y : E
hy₁ : y ∈ s
hy₂ : w y = 0
hy₃ : s.centerMass w id = x
⊢ (s.erase y).centerMass w id = x |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | combiFrontier_eq | [90, 1] | [135, 14] | rwa [Finset.centerMass_subset _ (s.erase_subset _)] | case h.mpr.refine'_2
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x✝ x : E
w : E → 𝕜
hw₁ : ∀ y ∈ s, 0 ≤ w y
hw₂ : ∑ y ∈ s, w y = 1
y : E
hy₁ : y ∈ s
hy₂ : w y = 0
hy₃ : s.centerMass w id = x
⊢ (s.erase y).centerMass w id = x | case h.mpr.refine'_2
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x✝ x : E
w : E → 𝕜
hw₁ : ∀ y ∈ s, 0 ≤ w y
hw₂ : ∑ y ∈ s, w y = 1
y : E
hy₁ : y ∈ s
hy₂ : w y = 0
hy₃ : s.centerMass w id = x
⊢ ∀ i ∈ s, i ∉ s.erase y → w i = 0 |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | combiFrontier_eq | [90, 1] | [135, 14] | intro i hi₁ hi₂ | case h.mpr.refine'_2
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x✝ x : E
w : E → 𝕜
hw₁ : ∀ y ∈ s, 0 ≤ w y
hw₂ : ∑ y ∈ s, w y = 1
y : E
hy₁ : y ∈ s
hy₂ : w y = 0
hy₃ : s.centerMass w id = x
⊢ ∀ i ∈ s, i ∉ s.erase y → w i = 0 | case h.mpr.refine'_2
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x✝ x : E
w : E → 𝕜
hw₁ : ∀ y ∈ s, 0 ≤ w y
hw₂ : ∑ y ∈ s, w y = 1
y : E
hy₁ : y ∈ s
hy₂ : w y = 0
hy₃ : s.centerMass w id = x
i : E
hi₁ : i ∈ s
hi₂ : i ∉ s.erase y
⊢ w i = 0 |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | combiFrontier_eq | [90, 1] | [135, 14] | simp only [hi₁, and_true_iff, Classical.not_not, Finset.mem_erase] at hi₂ | case h.mpr.refine'_2
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x✝ x : E
w : E → 𝕜
hw₁ : ∀ y ∈ s, 0 ≤ w y
hw₂ : ∑ y ∈ s, w y = 1
y : E
hy₁ : y ∈ s
hy₂ : w y = 0
hy₃ : s.centerMass w id = x
i : E
hi₁ : i ∈ s
hi₂ : i ∉ s.erase y
⊢ w i = 0 | case h.mpr.refine'_2
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x✝ x : E
w : E → 𝕜
hw₁ : ∀ y ∈ s, 0 ≤ w y
hw₂ : ∑ y ∈ s, w y = 1
y : E
hy₁ : y ∈ s
hy₂ : w y = 0
hy₃ : s.centerMass w id = x
i : E
hi₁ : i ∈ s
hi₂ : i = y
⊢ w i = 0 |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | combiFrontier_eq | [90, 1] | [135, 14] | subst hi₂ | case h.mpr.refine'_2
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x✝ x : E
w : E → 𝕜
hw₁ : ∀ y ∈ s, 0 ≤ w y
hw₂ : ∑ y ∈ s, w y = 1
y : E
hy₁ : y ∈ s
hy₂ : w y = 0
hy₃ : s.centerMass w id = x
i : E
hi₁ : i ∈ s
hi₂ : i = y
⊢ w i = 0 | case h.mpr.refine'_2
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x✝ x : E
w : E → 𝕜
hw₁ : ∀ y ∈ s, 0 ≤ w y
hw₂ : ∑ y ∈ s, w y = 1
hy₃ : s.centerMass w id = x
i : E
hi₁ hy₁ : i ∈ s
hy₂ : w i = 0
⊢ w i = 0 |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | combiFrontier_eq | [90, 1] | [135, 14] | apply hy₂ | case h.mpr.refine'_2
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x✝ x : E
w : E → 𝕜
hw₁ : ∀ y ∈ s, 0 ≤ w y
hw₂ : ∑ y ∈ s, w y = 1
hy₃ : s.centerMass w id = x
i : E
hi₁ hy₁ : i ∈ s
hy₂ : w i = 0
⊢ w i = 0 | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | combiInterior_subset_positive_weighings | [137, 1] | [146, 76] | rw [combiInterior, Finset.convexHull_eq, combiFrontier_eq] | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x : E
⊢ combiInterior 𝕜 s ⊆ {x | ∃ w, ∃ (_ : ∀ y ∈ s, 0 < w y) (_ : ∑ y ∈ s, w y = 1), s.centerMass w id = x} | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x : E
⊢ {x | ∃ w, (∀ y ∈ s, 0 ≤ w y) ∧ ∑ y ∈ s, w y = 1 ∧ s.centerMass w id = x} \
{x | ∃ w, ∃ (_ : ∀ y ∈ s, 0 ≤ w y) (_ : ∑ y ∈ s, w y = 1) (_ : ∃ y ∈ s, w y = 0), s.centerMass w id = x} ⊆
{x | ∃ w, ∃ (_ : ∀ y ∈ s, 0 < w y) (_ : ∑ y ∈ s, w y = 1), s.centerMass w id = x} |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | combiInterior_subset_positive_weighings | [137, 1] | [146, 76] | rintro x | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x : E
⊢ {x | ∃ w, (∀ y ∈ s, 0 ≤ w y) ∧ ∑ y ∈ s, w y = 1 ∧ s.centerMass w id = x} \
{x | ∃ w, ∃ (_ : ∀ y ∈ s, 0 ≤ w y) (_ : ∑ y ∈ s, w y = 1) (_ : ∃ y ∈ s, w y = 0), s.centerMass w id = x} ⊆
{x | ∃ w, ∃ (_ : ∀ y ∈ s, 0 < w y) (_ : ∑ y ∈ s, w y = 1), s.centerMass w id = x} | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x✝ x : E
⊢ x ∈
{x | ∃ w, (∀ y ∈ s, 0 ≤ w y) ∧ ∑ y ∈ s, w y = 1 ∧ s.centerMass w id = x} \
{x | ∃ w, ∃ (_ : ∀ y ∈ s, 0 ≤ w y) (_ : ∑ y ∈ s, w y = 1) (_ : ∃ y ∈ s, w y = 0), s.centerMass w id = x} →
x ∈ {x | ∃ w, ∃ (_ : ∀ y ∈ s, 0 < w y) (_ : ∑ y ∈ s, w y = 1), s.centerMass w id = x} |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | combiInterior_subset_positive_weighings | [137, 1] | [146, 76] | simp only [not_exists, and_imp, not_and, mem_setOf_eq, mem_diff, exists_imp] | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x✝ x : E
⊢ x ∈
{x | ∃ w, (∀ y ∈ s, 0 ≤ w y) ∧ ∑ y ∈ s, w y = 1 ∧ s.centerMass w id = x} \
{x | ∃ w, ∃ (_ : ∀ y ∈ s, 0 ≤ w y) (_ : ∑ y ∈ s, w y = 1) (_ : ∃ y ∈ s, w y = 0), s.centerMass w id = x} →
x ∈ {x | ∃ w, ∃ (_ : ∀ y ∈ s, 0 < w y) (_ : ∑ y ∈ s, w y = 1), s.centerMass w id = x} | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x✝ x : E
⊢ ∀ (x_1 : E → 𝕜),
(∀ y ∈ s, 0 ≤ x_1 y) →
∑ y ∈ s, x_1 y = 1 →
s.centerMass x_1 id = x →
(∀ (x_2 : E → 𝕜),
(∀ y ∈ s, 0 ≤ x_2 y) → ∑ y ∈ s, x_2 y = 1 → ∀ x_5 ∈ s, x_2 x_5 = 0 → ¬s.centerMass x_2 id = x) →
∃ w, ∃ (_ : ∀ y ∈ s, 0 < w y) (_ : ∑ y ∈ s, w y = 1), s.centerMass w id = x |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | combiInterior_subset_positive_weighings | [137, 1] | [146, 76] | rintro w hw₁ hw₂ hw₃ q | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x✝ x : E
⊢ ∀ (x_1 : E → 𝕜),
(∀ y ∈ s, 0 ≤ x_1 y) →
∑ y ∈ s, x_1 y = 1 →
s.centerMass x_1 id = x →
(∀ (x_2 : E → 𝕜),
(∀ y ∈ s, 0 ≤ x_2 y) → ∑ y ∈ s, x_2 y = 1 → ∀ x_5 ∈ s, x_2 x_5 = 0 → ¬s.centerMass x_2 id = x) →
∃ w, ∃ (_ : ∀ y ∈ s, 0 < w y) (_ : ∑ y ∈ s, w y = 1), s.centerMass w id = x | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x✝ x : E
w : E → 𝕜
hw₁ : ∀ y ∈ s, 0 ≤ w y
hw₂ : ∑ y ∈ s, w y = 1
hw₃ : s.centerMass w id = x
q : ∀ (x_1 : E → 𝕜), (∀ y ∈ s, 0 ≤ x_1 y) → ∑ y ∈ s, x_1 y = 1 → ∀ x_4 ∈ s, x_1 x_4 = 0 → ¬s.centerMass x_1 id = x
⊢ ∃ w, ∃ (_ : ∀ y ∈ s, 0 < w y) (_ : ∑ y ∈ s, w y = 1), s.centerMass w id = x |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | combiInterior_subset_positive_weighings | [137, 1] | [146, 76] | refine' ⟨w, fun y hy => _, hw₂, hw₃⟩ | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x✝ x : E
w : E → 𝕜
hw₁ : ∀ y ∈ s, 0 ≤ w y
hw₂ : ∑ y ∈ s, w y = 1
hw₃ : s.centerMass w id = x
q : ∀ (x_1 : E → 𝕜), (∀ y ∈ s, 0 ≤ x_1 y) → ∑ y ∈ s, x_1 y = 1 → ∀ x_4 ∈ s, x_1 x_4 = 0 → ¬s.centerMass x_1 id = x
⊢ ∃ w, ∃ (_ : ∀ y ∈ s, 0 < w y) (_ : ∑ y ∈ s, w y = 1), s.centerMass w id = x | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x✝ x : E
w : E → 𝕜
hw₁ : ∀ y ∈ s, 0 ≤ w y
hw₂ : ∑ y ∈ s, w y = 1
hw₃ : s.centerMass w id = x
q : ∀ (x_1 : E → 𝕜), (∀ y ∈ s, 0 ≤ x_1 y) → ∑ y ∈ s, x_1 y = 1 → ∀ x_4 ∈ s, x_1 x_4 = 0 → ¬s.centerMass x_1 id = x
y : E
hy : y ∈ s
⊢ 0 < w y |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | combiInterior_subset_positive_weighings | [137, 1] | [146, 76] | exact lt_of_le_of_ne (hw₁ _ hy) (Ne.symm fun t => q w hw₁ hw₂ y hy t hw₃) | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x✝ x : E
w : E → 𝕜
hw₁ : ∀ y ∈ s, 0 ≤ w y
hw₂ : ∑ y ∈ s, w y = 1
hw₃ : s.centerMass w id = x
q : ∀ (x_1 : E → 𝕜), (∀ y ∈ s, 0 ≤ x_1 y) → ∑ y ∈ s, x_1 y = 1 → ∀ x_4 ∈ s, x_1 x_4 = 0 → ¬s.centerMass x_1 id = x
y : E
hy : y ∈ s
⊢ 0 < w y | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | combiInterior_eq | [148, 1] | [159, 66] | refine' combiInterior_subset_positive_weighings.antisymm fun x => _ | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x : E
hs : AffineIndependent 𝕜 Subtype.val
⊢ combiInterior 𝕜 s = {x | ∃ w, ∃ (_ : ∀ y ∈ s, 0 < w y) (_ : ∑ y ∈ s, w y = 1), s.centerMass w id = x} | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x✝ : E
hs : AffineIndependent 𝕜 Subtype.val
x : E
⊢ x ∈ {x | ∃ w, ∃ (_ : ∀ y ∈ s, 0 < w y) (_ : ∑ y ∈ s, w y = 1), s.centerMass w id = x} → x ∈ combiInterior 𝕜 s |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | combiInterior_eq | [148, 1] | [159, 66] | rw [combiInterior, Finset.convexHull_eq, combiFrontier_eq] | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x✝ : E
hs : AffineIndependent 𝕜 Subtype.val
x : E
⊢ x ∈ {x | ∃ w, ∃ (_ : ∀ y ∈ s, 0 < w y) (_ : ∑ y ∈ s, w y = 1), s.centerMass w id = x} → x ∈ combiInterior 𝕜 s | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x✝ : E
hs : AffineIndependent 𝕜 Subtype.val
x : E
⊢ x ∈ {x | ∃ w, ∃ (_ : ∀ y ∈ s, 0 < w y) (_ : ∑ y ∈ s, w y = 1), s.centerMass w id = x} →
x ∈
{x | ∃ w, (∀ y ∈ s, 0 ≤ w y) ∧ ∑ y ∈ s, w y = 1 ∧ s.centerMass w id = x} \
{x | ∃ w, ∃ (_ : ∀ y ∈ s, 0 ≤ w y) (_ : ∑ y ∈ s, w y = 1) (_ : ∃ y ∈ s, w y = 0), s.centerMass w id = x} |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | combiInterior_eq | [148, 1] | [159, 66] | simp only [not_exists, and_imp, not_and, mem_setOf_eq, mem_diff, exists_imp] | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x✝ : E
hs : AffineIndependent 𝕜 Subtype.val
x : E
⊢ x ∈ {x | ∃ w, ∃ (_ : ∀ y ∈ s, 0 < w y) (_ : ∑ y ∈ s, w y = 1), s.centerMass w id = x} →
x ∈
{x | ∃ w, (∀ y ∈ s, 0 ≤ w y) ∧ ∑ y ∈ s, w y = 1 ∧ s.centerMass w id = x} \
{x | ∃ w, ∃ (_ : ∀ y ∈ s, 0 ≤ w y) (_ : ∑ y ∈ s, w y = 1) (_ : ∃ y ∈ s, w y = 0), s.centerMass w id = x} | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x✝ : E
hs : AffineIndependent 𝕜 Subtype.val
x : E
⊢ ∀ (x_1 : E → 𝕜),
(∀ y ∈ s, 0 < x_1 y) →
∑ y ∈ s, x_1 y = 1 →
s.centerMass x_1 id = x →
(∃ w, (∀ y ∈ s, 0 ≤ w y) ∧ ∑ y ∈ s, w y = 1 ∧ s.centerMass w id = x) ∧
∀ (x_4 : E → 𝕜),
(∀ y ∈ s, 0 ≤ x_4 y) → ∑ y ∈ s, x_4 y = 1 → ∀ x_7 ∈ s, x_4 x_7 = 0 → ¬s.centerMass x_4 id = x |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | combiInterior_eq | [148, 1] | [159, 66] | intro w hw₀ hw₁ hw₂ | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x✝ : E
hs : AffineIndependent 𝕜 Subtype.val
x : E
⊢ ∀ (x_1 : E → 𝕜),
(∀ y ∈ s, 0 < x_1 y) →
∑ y ∈ s, x_1 y = 1 →
s.centerMass x_1 id = x →
(∃ w, (∀ y ∈ s, 0 ≤ w y) ∧ ∑ y ∈ s, w y = 1 ∧ s.centerMass w id = x) ∧
∀ (x_4 : E → 𝕜),
(∀ y ∈ s, 0 ≤ x_4 y) → ∑ y ∈ s, x_4 y = 1 → ∀ x_7 ∈ s, x_4 x_7 = 0 → ¬s.centerMass x_4 id = x | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x✝ : E
hs : AffineIndependent 𝕜 Subtype.val
x : E
w : E → 𝕜
hw₀ : ∀ y ∈ s, 0 < w y
hw₁ : ∑ y ∈ s, w y = 1
hw₂ : s.centerMass w id = x
⊢ (∃ w, (∀ y ∈ s, 0 ≤ w y) ∧ ∑ y ∈ s, w y = 1 ∧ s.centerMass w id = x) ∧
∀ (x_1 : E → 𝕜), (∀ y ∈ s, 0 ≤ x_1 y) → ∑ y ∈ s, x_1 y = 1 → ∀ x_4 ∈ s, x_1 x_4 = 0 → ¬s.centerMass x_1 id = x |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | combiInterior_eq | [148, 1] | [159, 66] | refine' ⟨⟨w, fun y hy => (hw₀ y hy).le, hw₁, hw₂⟩, fun v hv₀ hv₁ y hy hvy hv₂ => (hw₀ y hy).ne' _⟩ | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x✝ : E
hs : AffineIndependent 𝕜 Subtype.val
x : E
w : E → 𝕜
hw₀ : ∀ y ∈ s, 0 < w y
hw₁ : ∑ y ∈ s, w y = 1
hw₂ : s.centerMass w id = x
⊢ (∃ w, (∀ y ∈ s, 0 ≤ w y) ∧ ∑ y ∈ s, w y = 1 ∧ s.centerMass w id = x) ∧
∀ (x_1 : E → 𝕜), (∀ y ∈ s, 0 ≤ x_1 y) → ∑ y ∈ s, x_1 y = 1 → ∀ x_4 ∈ s, x_1 x_4 = 0 → ¬s.centerMass x_1 id = x | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x✝ : E
hs : AffineIndependent 𝕜 Subtype.val
x : E
w : E → 𝕜
hw₀ : ∀ y ∈ s, 0 < w y
hw₁ : ∑ y ∈ s, w y = 1
hw₂ : s.centerMass w id = x
v : E → 𝕜
hv₀ : ∀ y ∈ s, 0 ≤ v y
hv₁ : ∑ y ∈ s, v y = 1
y : E
hy : y ∈ s
hvy : v y = 0
hv₂ : s.centerMass v id = x
⊢ w y = 0 |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | combiInterior_eq | [148, 1] | [159, 66] | rw [← hv₂] at hw₂ | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x✝ : E
hs : AffineIndependent 𝕜 Subtype.val
x : E
w : E → 𝕜
hw₀ : ∀ y ∈ s, 0 < w y
hw₁ : ∑ y ∈ s, w y = 1
hw₂ : s.centerMass w id = x
v : E → 𝕜
hv₀ : ∀ y ∈ s, 0 ≤ v y
hv₁ : ∑ y ∈ s, v y = 1
y : E
hy : y ∈ s
hvy : v y = 0
hv₂ : s.centerMass v id = x
⊢ w y = 0 | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x✝ : E
hs : AffineIndependent 𝕜 Subtype.val
x : E
w : E → 𝕜
hw₀ : ∀ y ∈ s, 0 < w y
hw₁ : ∑ y ∈ s, w y = 1
v : E → 𝕜
hw₂ : s.centerMass w id = s.centerMass v id
hv₀ : ∀ y ∈ s, 0 ≤ v y
hv₁ : ∑ y ∈ s, v y = 1
y : E
hy : y ∈ s
hvy : v y = 0
hv₂ : s.centerMass v id = x
⊢ w y = 0 |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | combiInterior_eq | [148, 1] | [159, 66] | rw [Finset.centerMass_eq_of_sum_1 _ _ hv₁, Finset.centerMass_eq_of_sum_1 _ _ hw₁] at hw₂ | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x✝ : E
hs : AffineIndependent 𝕜 Subtype.val
x : E
w : E → 𝕜
hw₀ : ∀ y ∈ s, 0 < w y
hw₁ : ∑ y ∈ s, w y = 1
v : E → 𝕜
hw₂ : s.centerMass w id = s.centerMass v id
hv₀ : ∀ y ∈ s, 0 ≤ v y
hv₁ : ∑ y ∈ s, v y = 1
y : E
hy : y ∈ s
hvy : v y = 0
hv₂ : s.centerMass v id = x
⊢ w y = 0 | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x✝ : E
hs : AffineIndependent 𝕜 Subtype.val
x : E
w : E → 𝕜
hw₀ : ∀ y ∈ s, 0 < w y
hw₁ : ∑ y ∈ s, w y = 1
v : E → 𝕜
hw₂ : ∑ i ∈ s, w i • id i = ∑ i ∈ s, v i • id i
hv₀ : ∀ y ∈ s, 0 ≤ v y
hv₁ : ∑ y ∈ s, v y = 1
y : E
hy : y ∈ s
hvy : v y = 0
hv₂ : s.centerMass v id = x
⊢ w y = 0 |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | combiInterior_eq | [148, 1] | [159, 66] | rw [← hvy] | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x✝ : E
hs : AffineIndependent 𝕜 Subtype.val
x : E
w : E → 𝕜
hw₀ : ∀ y ∈ s, 0 < w y
hw₁ : ∑ y ∈ s, w y = 1
v : E → 𝕜
hw₂ : ∑ i ∈ s, w i • id i = ∑ i ∈ s, v i • id i
hv₀ : ∀ y ∈ s, 0 ≤ v y
hv₁ : ∑ y ∈ s, v y = 1
y : E
hy : y ∈ s
hvy : v y = 0
hv₂ : s.centerMass v id = x
⊢ w y = 0 | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x✝ : E
hs : AffineIndependent 𝕜 Subtype.val
x : E
w : E → 𝕜
hw₀ : ∀ y ∈ s, 0 < w y
hw₁ : ∑ y ∈ s, w y = 1
v : E → 𝕜
hw₂ : ∑ i ∈ s, w i • id i = ∑ i ∈ s, v i • id i
hv₀ : ∀ y ∈ s, 0 ≤ v y
hv₁ : ∑ y ∈ s, v y = 1
y : E
hy : y ∈ s
hvy : v y = 0
hv₂ : s.centerMass v id = x
⊢ w y = v y |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | combiInterior_eq | [148, 1] | [159, 66] | exact hs.eq_of_sum_eq_sum_subtype (hw₁.trans hv₁.symm) hw₂ _ hy | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x✝ : E
hs : AffineIndependent 𝕜 Subtype.val
x : E
w : E → 𝕜
hw₀ : ∀ y ∈ s, 0 < w y
hw₁ : ∑ y ∈ s, w y = 1
v : E → 𝕜
hw₂ : ∑ i ∈ s, w i • id i = ∑ i ∈ s, v i • id i
hv₀ : ∀ y ∈ s, 0 ≤ v y
hv₁ : ∑ y ∈ s, v y = 1
y : E
hy : y ∈ s
hvy : v y = 0
hv₂ : s.centerMass v id = x
⊢ w y = v y | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | centroid_mem_combiInterior | [161, 1] | [168, 27] | rw [Finset.centroid_def] | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x : E
hs : AffineIndependent 𝕜 Subtype.val
hs' : s.Nonempty
⊢ Finset.centroid 𝕜 s id ∈ combiInterior 𝕜 s | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x : E
hs : AffineIndependent 𝕜 Subtype.val
hs' : s.Nonempty
⊢ (Finset.affineCombination 𝕜 s id) (Finset.centroidWeights 𝕜 s) ∈ combiInterior 𝕜 s |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | centroid_mem_combiInterior | [161, 1] | [168, 27] | have hsweights := s.sum_centroidWeights_eq_one_of_nonempty 𝕜 hs' | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x : E
hs : AffineIndependent 𝕜 Subtype.val
hs' : s.Nonempty
⊢ (Finset.affineCombination 𝕜 s id) (Finset.centroidWeights 𝕜 s) ∈ combiInterior 𝕜 s | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x : E
hs : AffineIndependent 𝕜 Subtype.val
hs' : s.Nonempty
hsweights : ∑ i ∈ s, Finset.centroidWeights 𝕜 s i = 1
⊢ (Finset.affineCombination 𝕜 s id) (Finset.centroidWeights 𝕜 s) ∈ combiInterior 𝕜 s |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | centroid_mem_combiInterior | [161, 1] | [168, 27] | rw [affineCombination_eq_centerMass hsweights] | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x : E
hs : AffineIndependent 𝕜 Subtype.val
hs' : s.Nonempty
hsweights : ∑ i ∈ s, Finset.centroidWeights 𝕜 s i = 1
⊢ (Finset.affineCombination 𝕜 s id) (Finset.centroidWeights 𝕜 s) ∈ combiInterior 𝕜 s | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x : E
hs : AffineIndependent 𝕜 Subtype.val
hs' : s.Nonempty
hsweights : ∑ i ∈ s, Finset.centroidWeights 𝕜 s i = 1
⊢ s.centerMass (fun i => Finset.centroidWeights 𝕜 s i) id ∈ combiInterior 𝕜 s |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | centroid_mem_combiInterior | [161, 1] | [168, 27] | rw [combiInterior_eq hs] | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x : E
hs : AffineIndependent 𝕜 Subtype.val
hs' : s.Nonempty
hsweights : ∑ i ∈ s, Finset.centroidWeights 𝕜 s i = 1
⊢ s.centerMass (fun i => Finset.centroidWeights 𝕜 s i) id ∈ combiInterior 𝕜 s | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x : E
hs : AffineIndependent 𝕜 Subtype.val
hs' : s.Nonempty
hsweights : ∑ i ∈ s, Finset.centroidWeights 𝕜 s i = 1
⊢ s.centerMass (fun i => Finset.centroidWeights 𝕜 s i) id ∈
{x | ∃ w, ∃ (_ : ∀ y ∈ s, 0 < w y) (_ : ∑ y ∈ s, w y = 1), s.centerMass w id = x} |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | centroid_mem_combiInterior | [161, 1] | [168, 27] | refine' ⟨_, fun y _ => _, hsweights, rfl⟩ | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x : E
hs : AffineIndependent 𝕜 Subtype.val
hs' : s.Nonempty
hsweights : ∑ i ∈ s, Finset.centroidWeights 𝕜 s i = 1
⊢ s.centerMass (fun i => Finset.centroidWeights 𝕜 s i) id ∈
{x | ∃ w, ∃ (_ : ∀ y ∈ s, 0 < w y) (_ : ∑ y ∈ s, w y = 1), s.centerMass w id = x} | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x : E
hs : AffineIndependent 𝕜 Subtype.val
hs' : s.Nonempty
hsweights : ∑ i ∈ s, Finset.centroidWeights 𝕜 s i = 1
y : E
x✝ : y ∈ s
⊢ 0 < Finset.centroidWeights 𝕜 s y |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | centroid_mem_combiInterior | [161, 1] | [168, 27] | simpa using hs'.card_pos | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x : E
hs : AffineIndependent 𝕜 Subtype.val
hs' : s.Nonempty
hsweights : ∑ i ∈ s, Finset.centroidWeights 𝕜 s i = 1
y : E
x✝ : y ∈ s
⊢ 0 < Finset.centroidWeights 𝕜 s y | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | convex_combiInterior | [179, 1] | [187, 55] | simp_rw [convex_iff_forall_pos, combiInterior_eq hs] | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x : E
hs : AffineIndependent 𝕜 Subtype.val
⊢ Convex 𝕜 (combiInterior 𝕜 s) | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x : E
hs : AffineIndependent 𝕜 Subtype.val
⊢ ∀ ⦃x : E⦄,
x ∈ {x | ∃ w, ∃ (_ : ∀ y ∈ s, 0 < w y) (_ : ∑ y ∈ s, w y = 1), s.centerMass w id = x} →
∀ ⦃y : E⦄,
y ∈ {x | ∃ w, ∃ (_ : ∀ y ∈ s, 0 < w y) (_ : ∑ y ∈ s, w y = 1), s.centerMass w id = x} →
∀ ⦃a b : 𝕜⦄,
0 < a →
0 < b →
a + b = 1 →
a • x + b • y ∈ {x | ∃ w, ∃ (_ : ∀ y ∈ s, 0 < w y) (_ : ∑ y ∈ s, w y = 1), s.centerMass w id = x} |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | convex_combiInterior | [179, 1] | [187, 55] | rintro x ⟨v, hv₀, hv₁, rfl⟩ y ⟨w, hw₀, hw₁, rfl⟩ a b ha hb h | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x : E
hs : AffineIndependent 𝕜 Subtype.val
⊢ ∀ ⦃x : E⦄,
x ∈ {x | ∃ w, ∃ (_ : ∀ y ∈ s, 0 < w y) (_ : ∑ y ∈ s, w y = 1), s.centerMass w id = x} →
∀ ⦃y : E⦄,
y ∈ {x | ∃ w, ∃ (_ : ∀ y ∈ s, 0 < w y) (_ : ∑ y ∈ s, w y = 1), s.centerMass w id = x} →
∀ ⦃a b : 𝕜⦄,
0 < a →
0 < b →
a + b = 1 →
a • x + b • y ∈ {x | ∃ w, ∃ (_ : ∀ y ∈ s, 0 < w y) (_ : ∑ y ∈ s, w y = 1), s.centerMass w id = x} | case intro.intro.intro.intro.intro.intro
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x : E
hs : AffineIndependent 𝕜 Subtype.val
v : E → 𝕜
hv₀ : ∀ y ∈ s, 0 < v y
hv₁ : ∑ y ∈ s, v y = 1
w : E → 𝕜
hw₀ : ∀ y ∈ s, 0 < w y
hw₁ : ∑ y ∈ s, w y = 1
a b : 𝕜
ha : 0 < a
hb : 0 < b
h : a + b = 1
⊢ a • s.centerMass v id + b • s.centerMass w id ∈
{x | ∃ w, ∃ (_ : ∀ y ∈ s, 0 < w y) (_ : ∑ y ∈ s, w y = 1), s.centerMass w id = x} |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | convex_combiInterior | [179, 1] | [187, 55] | refine' ⟨fun x => a * v x + b * w x, fun x hx => _, _, _⟩ | case intro.intro.intro.intro.intro.intro
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x : E
hs : AffineIndependent 𝕜 Subtype.val
v : E → 𝕜
hv₀ : ∀ y ∈ s, 0 < v y
hv₁ : ∑ y ∈ s, v y = 1
w : E → 𝕜
hw₀ : ∀ y ∈ s, 0 < w y
hw₁ : ∑ y ∈ s, w y = 1
a b : 𝕜
ha : 0 < a
hb : 0 < b
h : a + b = 1
⊢ a • s.centerMass v id + b • s.centerMass w id ∈
{x | ∃ w, ∃ (_ : ∀ y ∈ s, 0 < w y) (_ : ∑ y ∈ s, w y = 1), s.centerMass w id = x} | case intro.intro.intro.intro.intro.intro.refine'_1
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x✝ : E
hs : AffineIndependent 𝕜 Subtype.val
v : E → 𝕜
hv₀ : ∀ y ∈ s, 0 < v y
hv₁ : ∑ y ∈ s, v y = 1
w : E → 𝕜
hw₀ : ∀ y ∈ s, 0 < w y
hw₁ : ∑ y ∈ s, w y = 1
a b : 𝕜
ha : 0 < a
hb : 0 < b
h : a + b = 1
x : E
hx : x ∈ s
⊢ 0 < (fun x => a * v x + b * w x) x
case intro.intro.intro.intro.intro.intro.refine'_2
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x : E
hs : AffineIndependent 𝕜 Subtype.val
v : E → 𝕜
hv₀ : ∀ y ∈ s, 0 < v y
hv₁ : ∑ y ∈ s, v y = 1
w : E → 𝕜
hw₀ : ∀ y ∈ s, 0 < w y
hw₁ : ∑ y ∈ s, w y = 1
a b : 𝕜
ha : 0 < a
hb : 0 < b
h : a + b = 1
⊢ ∑ y ∈ s, (fun x => a * v x + b * w x) y = 1
case intro.intro.intro.intro.intro.intro.refine'_3
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x : E
hs : AffineIndependent 𝕜 Subtype.val
v : E → 𝕜
hv₀ : ∀ y ∈ s, 0 < v y
hv₁ : ∑ y ∈ s, v y = 1
w : E → 𝕜
hw₀ : ∀ y ∈ s, 0 < w y
hw₁ : ∑ y ∈ s, w y = 1
a b : 𝕜
ha : 0 < a
hb : 0 < b
h : a + b = 1
⊢ s.centerMass (fun x => a * v x + b * w x) id = a • s.centerMass v id + b • s.centerMass w id |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | convex_combiInterior | [179, 1] | [187, 55] | rw [Finset.centerMass_segment _ _ _ _ hv₁ hw₁ _ _ h] | case intro.intro.intro.intro.intro.intro.refine'_3
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x : E
hs : AffineIndependent 𝕜 Subtype.val
v : E → 𝕜
hv₀ : ∀ y ∈ s, 0 < v y
hv₁ : ∑ y ∈ s, v y = 1
w : E → 𝕜
hw₀ : ∀ y ∈ s, 0 < w y
hw₁ : ∑ y ∈ s, w y = 1
a b : 𝕜
ha : 0 < a
hb : 0 < b
h : a + b = 1
⊢ s.centerMass (fun x => a * v x + b * w x) id = a • s.centerMass v id + b • s.centerMass w id | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | convex_combiInterior | [179, 1] | [187, 55] | exact add_pos (mul_pos ha <| hv₀ x hx) (mul_pos hb <| hw₀ x hx) | case intro.intro.intro.intro.intro.intro.refine'_1
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x✝ : E
hs : AffineIndependent 𝕜 Subtype.val
v : E → 𝕜
hv₀ : ∀ y ∈ s, 0 < v y
hv₁ : ∑ y ∈ s, v y = 1
w : E → 𝕜
hw₀ : ∀ y ∈ s, 0 < w y
hw₁ : ∑ y ∈ s, w y = 1
a b : 𝕜
ha : 0 < a
hb : 0 < b
h : a + b = 1
x : E
hx : x ∈ s
⊢ 0 < (fun x => a * v x + b * w x) x | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | convex_combiInterior | [179, 1] | [187, 55] | rw [Finset.sum_add_distrib, ← Finset.mul_sum, ← Finset.mul_sum, hv₁, hw₁] | case intro.intro.intro.intro.intro.intro.refine'_2
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x : E
hs : AffineIndependent 𝕜 Subtype.val
v : E → 𝕜
hv₀ : ∀ y ∈ s, 0 < v y
hv₁ : ∑ y ∈ s, v y = 1
w : E → 𝕜
hw₀ : ∀ y ∈ s, 0 < w y
hw₁ : ∑ y ∈ s, w y = 1
a b : 𝕜
ha : 0 < a
hb : 0 < b
h : a + b = 1
⊢ ∑ y ∈ s, (fun x => a * v x + b * w x) y = 1 | case intro.intro.intro.intro.intro.intro.refine'_2
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x : E
hs : AffineIndependent 𝕜 Subtype.val
v : E → 𝕜
hv₀ : ∀ y ∈ s, 0 < v y
hv₁ : ∑ y ∈ s, v y = 1
w : E → 𝕜
hw₀ : ∀ y ∈ s, 0 < w y
hw₁ : ∑ y ∈ s, w y = 1
a b : 𝕜
ha : 0 < a
hb : 0 < b
h : a + b = 1
⊢ a * 1 + b * 1 = 1 |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | convex_combiInterior | [179, 1] | [187, 55] | simp [h] | case intro.intro.intro.intro.intro.intro.refine'_2
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x : E
hs : AffineIndependent 𝕜 Subtype.val
v : E → 𝕜
hv₀ : ∀ y ∈ s, 0 < v y
hv₁ : ∑ y ∈ s, v y = 1
w : E → 𝕜
hw₀ : ∀ y ∈ s, 0 < w y
hw₁ : ∑ y ∈ s, w y = 1
a b : 𝕜
ha : 0 < a
hb : 0 < b
h : a + b = 1
⊢ a * 1 + b * 1 = 1 | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | isClosed_combiFrontier | [199, 1] | [204, 7] | refine' Set.Finite.isClosed_biUnion _ fun t _ => t.isClosed_convexHull | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝⁵ : TopologicalSpace E
inst✝⁴ : AddCommGroup E
inst✝³ : Module ℝ E
inst✝² : TopologicalAddGroup E
inst✝¹ : ContinuousSMul ℝ E
inst✝ : T2Space E
s t : Finset E
⊢ IsClosed (combiFrontier ℝ s) | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝⁵ : TopologicalSpace E
inst✝⁴ : AddCommGroup E
inst✝³ : Module ℝ E
inst✝² : TopologicalAddGroup E
inst✝¹ : ContinuousSMul ℝ E
inst✝ : T2Space E
s t : Finset E
⊢ Set.Finite fun t => t ⊆ s ∧ ¬s ⊆ t |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | isClosed_combiFrontier | [199, 1] | [204, 7] | suffices Set.Finite {t | t ⊆ s} by exact this.subset fun i h => h.1 | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝⁵ : TopologicalSpace E
inst✝⁴ : AddCommGroup E
inst✝³ : Module ℝ E
inst✝² : TopologicalAddGroup E
inst✝¹ : ContinuousSMul ℝ E
inst✝ : T2Space E
s t : Finset E
⊢ Set.Finite fun t => t ⊆ s ∧ ¬s ⊆ t | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝⁵ : TopologicalSpace E
inst✝⁴ : AddCommGroup E
inst✝³ : Module ℝ E
inst✝² : TopologicalAddGroup E
inst✝¹ : ContinuousSMul ℝ E
inst✝ : T2Space E
s t : Finset E
⊢ {t | t ⊆ s}.Finite |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | isClosed_combiFrontier | [199, 1] | [204, 7] | convert s.powerset.finite_toSet using 1 | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝⁵ : TopologicalSpace E
inst✝⁴ : AddCommGroup E
inst✝³ : Module ℝ E
inst✝² : TopologicalAddGroup E
inst✝¹ : ContinuousSMul ℝ E
inst✝ : T2Space E
s t : Finset E
⊢ {t | t ⊆ s}.Finite | case h.e'_2
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝⁵ : TopologicalSpace E
inst✝⁴ : AddCommGroup E
inst✝³ : Module ℝ E
inst✝² : TopologicalAddGroup E
inst✝¹ : ContinuousSMul ℝ E
inst✝ : T2Space E
s t : Finset E
⊢ {t | t ⊆ s} = ↑s.powerset |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | isClosed_combiFrontier | [199, 1] | [204, 7] | ext | case h.e'_2
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝⁵ : TopologicalSpace E
inst✝⁴ : AddCommGroup E
inst✝³ : Module ℝ E
inst✝² : TopologicalAddGroup E
inst✝¹ : ContinuousSMul ℝ E
inst✝ : T2Space E
s t : Finset E
⊢ {t | t ⊆ s} = ↑s.powerset | case h.e'_2.h
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝⁵ : TopologicalSpace E
inst✝⁴ : AddCommGroup E
inst✝³ : Module ℝ E
inst✝² : TopologicalAddGroup E
inst✝¹ : ContinuousSMul ℝ E
inst✝ : T2Space E
s t x✝ : Finset E
⊢ x✝ ∈ {t | t ⊆ s} ↔ x✝ ∈ ↑s.powerset |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | isClosed_combiFrontier | [199, 1] | [204, 7] | simp | case h.e'_2.h
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝⁵ : TopologicalSpace E
inst✝⁴ : AddCommGroup E
inst✝³ : Module ℝ E
inst✝² : TopologicalAddGroup E
inst✝¹ : ContinuousSMul ℝ E
inst✝ : T2Space E
s t x✝ : Finset E
⊢ x✝ ∈ {t | t ⊆ s} ↔ x✝ ∈ ↑s.powerset | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | isClosed_combiFrontier | [199, 1] | [204, 7] | exact this.subset fun i h => h.1 | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝⁵ : TopologicalSpace E
inst✝⁴ : AddCommGroup E
inst✝³ : Module ℝ E
inst✝² : TopologicalAddGroup E
inst✝¹ : ContinuousSMul ℝ E
inst✝ : T2Space E
s t : Finset E
this : {t | t ⊆ s}.Finite
⊢ Set.Finite fun t => t ⊆ s ∧ ¬s ⊆ t | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | interiors_agree_of_full_dimensional | [206, 1] | [211, 8] | unfold combiInterior | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝⁶ : TopologicalSpace E
inst✝⁵ : AddCommGroup E
inst✝⁴ : Module ℝ E
inst✝³ : TopologicalAddGroup E
inst✝² : ContinuousSMul ℝ E
inst✝¹ : T2Space E
s t : Finset E
inst✝ : FiniteDimensional ℝ E
hs : AffineIndependent ℝ Subtype.val
hscard : s.card = FiniteDimensional.finrank ℝ E + 1
⊢ combiInterior ℝ s = interior ((convexHull ℝ) ↑s) | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝⁶ : TopologicalSpace E
inst✝⁵ : AddCommGroup E
inst✝⁴ : Module ℝ E
inst✝³ : TopologicalAddGroup E
inst✝² : ContinuousSMul ℝ E
inst✝¹ : T2Space E
s t : Finset E
inst✝ : FiniteDimensional ℝ E
hs : AffineIndependent ℝ Subtype.val
hscard : s.card = FiniteDimensional.finrank ℝ E + 1
⊢ (convexHull ℝ) ↑s \ combiFrontier ℝ s = interior ((convexHull ℝ) ↑s) |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | interiors_agree_of_full_dimensional | [206, 1] | [211, 8] | sorry | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝⁶ : TopologicalSpace E
inst✝⁵ : AddCommGroup E
inst✝⁴ : Module ℝ E
inst✝³ : TopologicalAddGroup E
inst✝² : ContinuousSMul ℝ E
inst✝¹ : T2Space E
s t : Finset E
inst✝ : FiniteDimensional ℝ E
hs : AffineIndependent ℝ Subtype.val
hscard : s.card = FiniteDimensional.finrank ℝ E + 1
⊢ (convexHull ℝ) ↑s \ combiFrontier ℝ s = interior ((convexHull ℝ) ↑s) | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | frontiers_agree_of_full_dimensional | [213, 1] | [227, 10] | ext x | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝⁶ : TopologicalSpace E
inst✝⁵ : AddCommGroup E
inst✝⁴ : Module ℝ E
inst✝³ : TopologicalAddGroup E
inst✝² : ContinuousSMul ℝ E
inst✝¹ : T2Space E
s t : Finset E
inst✝ : FiniteDimensional ℝ E
hscard : s.card = FiniteDimensional.finrank ℝ E + 1
⊢ combiFrontier ℝ s = frontier ((convexHull ℝ) ↑s) | case h
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝⁶ : TopologicalSpace E
inst✝⁵ : AddCommGroup E
inst✝⁴ : Module ℝ E
inst✝³ : TopologicalAddGroup E
inst✝² : ContinuousSMul ℝ E
inst✝¹ : T2Space E
s t : Finset E
inst✝ : FiniteDimensional ℝ E
hscard : s.card = FiniteDimensional.finrank ℝ E + 1
x : E
⊢ x ∈ combiFrontier ℝ s ↔ x ∈ frontier ((convexHull ℝ) ↑s) |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | frontiers_agree_of_full_dimensional | [213, 1] | [227, 10] | constructor | case h
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝⁶ : TopologicalSpace E
inst✝⁵ : AddCommGroup E
inst✝⁴ : Module ℝ E
inst✝³ : TopologicalAddGroup E
inst✝² : ContinuousSMul ℝ E
inst✝¹ : T2Space E
s t : Finset E
inst✝ : FiniteDimensional ℝ E
hscard : s.card = FiniteDimensional.finrank ℝ E + 1
x : E
⊢ x ∈ combiFrontier ℝ s ↔ x ∈ frontier ((convexHull ℝ) ↑s) | case h.mp
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝⁶ : TopologicalSpace E
inst✝⁵ : AddCommGroup E
inst✝⁴ : Module ℝ E
inst✝³ : TopologicalAddGroup E
inst✝² : ContinuousSMul ℝ E
inst✝¹ : T2Space E
s t : Finset E
inst✝ : FiniteDimensional ℝ E
hscard : s.card = FiniteDimensional.finrank ℝ E + 1
x : E
⊢ x ∈ combiFrontier ℝ s → x ∈ frontier ((convexHull ℝ) ↑s)
case h.mpr
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝⁶ : TopologicalSpace E
inst✝⁵ : AddCommGroup E
inst✝⁴ : Module ℝ E
inst✝³ : TopologicalAddGroup E
inst✝² : ContinuousSMul ℝ E
inst✝¹ : T2Space E
s t : Finset E
inst✝ : FiniteDimensional ℝ E
hscard : s.card = FiniteDimensional.finrank ℝ E + 1
x : E
⊢ x ∈ frontier ((convexHull ℝ) ↑s) → x ∈ combiFrontier ℝ s |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | frontiers_agree_of_full_dimensional | [213, 1] | [227, 10] | unfold combiFrontier | case h.mp
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝⁶ : TopologicalSpace E
inst✝⁵ : AddCommGroup E
inst✝⁴ : Module ℝ E
inst✝³ : TopologicalAddGroup E
inst✝² : ContinuousSMul ℝ E
inst✝¹ : T2Space E
s t : Finset E
inst✝ : FiniteDimensional ℝ E
hscard : s.card = FiniteDimensional.finrank ℝ E + 1
x : E
⊢ x ∈ combiFrontier ℝ s → x ∈ frontier ((convexHull ℝ) ↑s) | case h.mp
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝⁶ : TopologicalSpace E
inst✝⁵ : AddCommGroup E
inst✝⁴ : Module ℝ E
inst✝³ : TopologicalAddGroup E
inst✝² : ContinuousSMul ℝ E
inst✝¹ : T2Space E
s t : Finset E
inst✝ : FiniteDimensional ℝ E
hscard : s.card = FiniteDimensional.finrank ℝ E + 1
x : E
⊢ x ∈ ⋃ t, ⋃ (_ : t ⊂ s), (convexHull ℝ) ↑t → x ∈ frontier ((convexHull ℝ) ↑s) |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | frontiers_agree_of_full_dimensional | [213, 1] | [227, 10] | simp_rw [Set.mem_iUnion] | case h.mp
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝⁶ : TopologicalSpace E
inst✝⁵ : AddCommGroup E
inst✝⁴ : Module ℝ E
inst✝³ : TopologicalAddGroup E
inst✝² : ContinuousSMul ℝ E
inst✝¹ : T2Space E
s t : Finset E
inst✝ : FiniteDimensional ℝ E
hscard : s.card = FiniteDimensional.finrank ℝ E + 1
x : E
⊢ x ∈ ⋃ t, ⋃ (_ : t ⊂ s), (convexHull ℝ) ↑t → x ∈ frontier ((convexHull ℝ) ↑s) | case h.mp
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝⁶ : TopologicalSpace E
inst✝⁵ : AddCommGroup E
inst✝⁴ : Module ℝ E
inst✝³ : TopologicalAddGroup E
inst✝² : ContinuousSMul ℝ E
inst✝¹ : T2Space E
s t : Finset E
inst✝ : FiniteDimensional ℝ E
hscard : s.card = FiniteDimensional.finrank ℝ E + 1
x : E
⊢ (∃ i, ∃ (_ : i ⊂ s), x ∈ (convexHull ℝ) ↑i) → x ∈ frontier ((convexHull ℝ) ↑s) |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | frontiers_agree_of_full_dimensional | [213, 1] | [227, 10] | rintro ⟨t, hts, hx⟩ | case h.mp
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝⁶ : TopologicalSpace E
inst✝⁵ : AddCommGroup E
inst✝⁴ : Module ℝ E
inst✝³ : TopologicalAddGroup E
inst✝² : ContinuousSMul ℝ E
inst✝¹ : T2Space E
s t : Finset E
inst✝ : FiniteDimensional ℝ E
hscard : s.card = FiniteDimensional.finrank ℝ E + 1
x : E
⊢ (∃ i, ∃ (_ : i ⊂ s), x ∈ (convexHull ℝ) ↑i) → x ∈ frontier ((convexHull ℝ) ↑s) | case h.mp.intro.intro
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝⁶ : TopologicalSpace E
inst✝⁵ : AddCommGroup E
inst✝⁴ : Module ℝ E
inst✝³ : TopologicalAddGroup E
inst✝² : ContinuousSMul ℝ E
inst✝¹ : T2Space E
s t✝ : Finset E
inst✝ : FiniteDimensional ℝ E
hscard : s.card = FiniteDimensional.finrank ℝ E + 1
x : E
t : Finset E
hts : t ⊂ s
hx : x ∈ (convexHull ℝ) ↑t
⊢ x ∈ frontier ((convexHull ℝ) ↑s) |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | frontiers_agree_of_full_dimensional | [213, 1] | [227, 10] | constructor | case h.mp.intro.intro
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝⁶ : TopologicalSpace E
inst✝⁵ : AddCommGroup E
inst✝⁴ : Module ℝ E
inst✝³ : TopologicalAddGroup E
inst✝² : ContinuousSMul ℝ E
inst✝¹ : T2Space E
s t✝ : Finset E
inst✝ : FiniteDimensional ℝ E
hscard : s.card = FiniteDimensional.finrank ℝ E + 1
x : E
t : Finset E
hts : t ⊂ s
hx : x ∈ (convexHull ℝ) ↑t
⊢ x ∈ frontier ((convexHull ℝ) ↑s) | case h.mp.intro.intro.left
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝⁶ : TopologicalSpace E
inst✝⁵ : AddCommGroup E
inst✝⁴ : Module ℝ E
inst✝³ : TopologicalAddGroup E
inst✝² : ContinuousSMul ℝ E
inst✝¹ : T2Space E
s t✝ : Finset E
inst✝ : FiniteDimensional ℝ E
hscard : s.card = FiniteDimensional.finrank ℝ E + 1
x : E
t : Finset E
hts : t ⊂ s
hx : x ∈ (convexHull ℝ) ↑t
⊢ x ∈ closure ((convexHull ℝ) ↑s)
case h.mp.intro.intro.right
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝⁶ : TopologicalSpace E
inst✝⁵ : AddCommGroup E
inst✝⁴ : Module ℝ E
inst✝³ : TopologicalAddGroup E
inst✝² : ContinuousSMul ℝ E
inst✝¹ : T2Space E
s t✝ : Finset E
inst✝ : FiniteDimensional ℝ E
hscard : s.card = FiniteDimensional.finrank ℝ E + 1
x : E
t : Finset E
hts : t ⊂ s
hx : x ∈ (convexHull ℝ) ↑t
⊢ x ∉ interior ((convexHull ℝ) ↑s) |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | frontiers_agree_of_full_dimensional | [213, 1] | [227, 10] | exact subset_closure (convexHull_mono hts.1 hx) | case h.mp.intro.intro.left
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝⁶ : TopologicalSpace E
inst✝⁵ : AddCommGroup E
inst✝⁴ : Module ℝ E
inst✝³ : TopologicalAddGroup E
inst✝² : ContinuousSMul ℝ E
inst✝¹ : T2Space E
s t✝ : Finset E
inst✝ : FiniteDimensional ℝ E
hscard : s.card = FiniteDimensional.finrank ℝ E + 1
x : E
t : Finset E
hts : t ⊂ s
hx : x ∈ (convexHull ℝ) ↑t
⊢ x ∈ closure ((convexHull ℝ) ↑s) | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | frontiers_agree_of_full_dimensional | [213, 1] | [227, 10] | rintro h | case h.mp.intro.intro.right
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝⁶ : TopologicalSpace E
inst✝⁵ : AddCommGroup E
inst✝⁴ : Module ℝ E
inst✝³ : TopologicalAddGroup E
inst✝² : ContinuousSMul ℝ E
inst✝¹ : T2Space E
s t✝ : Finset E
inst✝ : FiniteDimensional ℝ E
hscard : s.card = FiniteDimensional.finrank ℝ E + 1
x : E
t : Finset E
hts : t ⊂ s
hx : x ∈ (convexHull ℝ) ↑t
⊢ x ∉ interior ((convexHull ℝ) ↑s) | case h.mp.intro.intro.right
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝⁶ : TopologicalSpace E
inst✝⁵ : AddCommGroup E
inst✝⁴ : Module ℝ E
inst✝³ : TopologicalAddGroup E
inst✝² : ContinuousSMul ℝ E
inst✝¹ : T2Space E
s t✝ : Finset E
inst✝ : FiniteDimensional ℝ E
hscard : s.card = FiniteDimensional.finrank ℝ E + 1
x : E
t : Finset E
hts : t ⊂ s
hx : x ∈ (convexHull ℝ) ↑t
h : x ∈ interior ((convexHull ℝ) ↑s)
⊢ False |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | frontiers_agree_of_full_dimensional | [213, 1] | [227, 10] | sorry | case h.mp.intro.intro.right
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝⁶ : TopologicalSpace E
inst✝⁵ : AddCommGroup E
inst✝⁴ : Module ℝ E
inst✝³ : TopologicalAddGroup E
inst✝² : ContinuousSMul ℝ E
inst✝¹ : T2Space E
s t✝ : Finset E
inst✝ : FiniteDimensional ℝ E
hscard : s.card = FiniteDimensional.finrank ℝ E + 1
x : E
t : Finset E
hts : t ⊂ s
hx : x ∈ (convexHull ℝ) ↑t
h : x ∈ interior ((convexHull ℝ) ↑s)
⊢ False | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | frontiers_agree_of_full_dimensional | [213, 1] | [227, 10] | rintro ⟨h, g⟩ | case h.mpr
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝⁶ : TopologicalSpace E
inst✝⁵ : AddCommGroup E
inst✝⁴ : Module ℝ E
inst✝³ : TopologicalAddGroup E
inst✝² : ContinuousSMul ℝ E
inst✝¹ : T2Space E
s t : Finset E
inst✝ : FiniteDimensional ℝ E
hscard : s.card = FiniteDimensional.finrank ℝ E + 1
x : E
⊢ x ∈ frontier ((convexHull ℝ) ↑s) → x ∈ combiFrontier ℝ s | case h.mpr.intro
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝⁶ : TopologicalSpace E
inst✝⁵ : AddCommGroup E
inst✝⁴ : Module ℝ E
inst✝³ : TopologicalAddGroup E
inst✝² : ContinuousSMul ℝ E
inst✝¹ : T2Space E
s t : Finset E
inst✝ : FiniteDimensional ℝ E
hscard : s.card = FiniteDimensional.finrank ℝ E + 1
x : E
h : x ∈ closure ((convexHull ℝ) ↑s)
g : x ∉ interior ((convexHull ℝ) ↑s)
⊢ x ∈ combiFrontier ℝ s |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | frontiers_agree_of_full_dimensional | [213, 1] | [227, 10] | sorry | case h.mpr.intro
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝⁶ : TopologicalSpace E
inst✝⁵ : AddCommGroup E
inst✝⁴ : Module ℝ E
inst✝³ : TopologicalAddGroup E
inst✝² : ContinuousSMul ℝ E
inst✝¹ : T2Space E
s t : Finset E
inst✝ : FiniteDimensional ℝ E
hscard : s.card = FiniteDimensional.finrank ℝ E + 1
x : E
h : x ∈ closure ((convexHull ℝ) ↑s)
g : x ∉ interior ((convexHull ℝ) ↑s)
⊢ x ∈ combiFrontier ℝ s | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | subset_closure_combiInterior | [234, 1] | [288, 39] | rintro x (hx : x ∈ s) | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
⊢ ↑s ⊆ closure (combiInterior ℝ s) | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
⊢ x ∈ closure (combiInterior ℝ s) |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | subset_closure_combiInterior | [234, 1] | [288, 39] | apply seqClosure_subset_closure | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
⊢ x ∈ closure (combiInterior ℝ s) | case a
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
⊢ x ∈ seqClosure (combiInterior ℝ s) |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | subset_closure_combiInterior | [234, 1] | [288, 39] | have hsnonempty : s.Nonempty := ⟨x, hx⟩ | case a
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
⊢ x ∈ seqClosure (combiInterior ℝ s) | case a
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
hsnonempty : s.Nonempty
⊢ x ∈ seqClosure (combiInterior ℝ s) |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | subset_closure_combiInterior | [234, 1] | [288, 39] | have centroid_weights : ∑ i : E in s, Finset.centroidWeights ℝ s i = 1 := by
apply Finset.sum_centroidWeights_eq_one_of_nonempty ℝ _ hsnonempty | case a
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
hsnonempty : s.Nonempty
⊢ x ∈ seqClosure (combiInterior ℝ s) | case a
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
hsnonempty : s.Nonempty
centroid_weights : ∑ i ∈ s, Finset.centroidWeights ℝ s i = 1
⊢ x ∈ seqClosure (combiInterior ℝ s) |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | subset_closure_combiInterior | [234, 1] | [288, 39] | refine' ⟨fun n => _, fun n => _, _⟩ | case a
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
hsnonempty : s.Nonempty
centroid_weights : ∑ i ∈ s, Finset.centroidWeights ℝ s i = 1
⊢ x ∈ seqClosure (combiInterior ℝ s) | case a.refine'_1
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
hsnonempty : s.Nonempty
centroid_weights : ∑ i ∈ s, Finset.centroidWeights ℝ s i = 1
n : ℕ
⊢ E
case a.refine'_2
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
hsnonempty : s.Nonempty
centroid_weights : ∑ i ∈ s, Finset.centroidWeights ℝ s i = 1
n : ℕ
⊢ (fun n => ?m.106180 n) n ∈ combiInterior ℝ s
case a.refine'_3
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
hsnonempty : s.Nonempty
centroid_weights : ∑ i ∈ s, Finset.centroidWeights ℝ s i = 1
⊢ Filter.Tendsto (fun n => ?m.106180 n) Filter.atTop (nhds x) |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | subset_closure_combiInterior | [234, 1] | [288, 39] | apply Finset.sum_centroidWeights_eq_one_of_nonempty ℝ _ hsnonempty | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
hsnonempty : s.Nonempty
⊢ ∑ i ∈ s, Finset.centroidWeights ℝ s i = 1 | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | subset_closure_combiInterior | [234, 1] | [288, 39] | apply ((n : ℝ) + 2)⁻¹ • s.centroid ℝ id + (1 - ((n : ℝ) + 2)⁻¹) • x | case a.refine'_1
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
hsnonempty : s.Nonempty
centroid_weights : ∑ i ∈ s, Finset.centroidWeights ℝ s i = 1
n : ℕ
⊢ E | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | subset_closure_combiInterior | [234, 1] | [288, 39] | rw [Finset.centroid_def] | case a.refine'_2
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
hsnonempty : s.Nonempty
centroid_weights : ∑ i ∈ s, Finset.centroidWeights ℝ s i = 1
n : ℕ
⊢ (fun n => (↑n + 2)⁻¹ • Finset.centroid ℝ s id + (1 - (↑n + 2)⁻¹) • x) n ∈ combiInterior ℝ s | case a.refine'_2
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
hsnonempty : s.Nonempty
centroid_weights : ∑ i ∈ s, Finset.centroidWeights ℝ s i = 1
n : ℕ
⊢ (fun n => (↑n + 2)⁻¹ • (Finset.affineCombination ℝ s id) (Finset.centroidWeights ℝ s) + (1 - (↑n + 2)⁻¹) • x) n ∈
combiInterior ℝ s |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | subset_closure_combiInterior | [234, 1] | [288, 39] | rw [affineCombination_eq_centerMass _] | case a.refine'_2
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
hsnonempty : s.Nonempty
centroid_weights : ∑ i ∈ s, Finset.centroidWeights ℝ s i = 1
n : ℕ
⊢ (fun n => (↑n + 2)⁻¹ • (Finset.affineCombination ℝ s id) (Finset.centroidWeights ℝ s) + (1 - (↑n + 2)⁻¹) • x) n ∈
combiInterior ℝ s | case a.refine'_2
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
hsnonempty : s.Nonempty
centroid_weights : ∑ i ∈ s, Finset.centroidWeights ℝ s i = 1
n : ℕ
⊢ (fun n => (↑n + 2)⁻¹ • s.centerMass (Finset.centroidWeights ℝ s) id + (1 - (↑n + 2)⁻¹) • x) n ∈ combiInterior ℝ s
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
hsnonempty : s.Nonempty
centroid_weights : ∑ i ∈ s, Finset.centroidWeights ℝ s i = 1
n : ℕ
⊢ ∑ i ∈ s, Finset.centroidWeights ℝ s i = 1 |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | subset_closure_combiInterior | [234, 1] | [288, 39] | apply Finset.sum_centroidWeights_eq_one_of_nonempty ℝ _ hsnonempty | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
hsnonempty : s.Nonempty
centroid_weights : ∑ i ∈ s, Finset.centroidWeights ℝ s i = 1
n : ℕ
⊢ ∑ i ∈ s, Finset.centroidWeights ℝ s i = 1 | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | subset_closure_combiInterior | [234, 1] | [288, 39] | rw [← id_def x] | case a.refine'_2
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
hsnonempty : s.Nonempty
centroid_weights : ∑ i ∈ s, Finset.centroidWeights ℝ s i = 1
n : ℕ
⊢ (fun n => (↑n + 2)⁻¹ • s.centerMass (Finset.centroidWeights ℝ s) id + (1 - (↑n + 2)⁻¹) • x) n ∈ combiInterior ℝ s | case a.refine'_2
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
hsnonempty : s.Nonempty
centroid_weights : ∑ i ∈ s, Finset.centroidWeights ℝ s i = 1
n : ℕ
⊢ (fun n => (↑n + 2)⁻¹ • s.centerMass (Finset.centroidWeights ℝ s) id + (1 - (↑n + 2)⁻¹) • id x) n ∈ combiInterior ℝ s |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | subset_closure_combiInterior | [234, 1] | [288, 39] | rw [← Finset.centerMass_ite_eq (R := ℝ) _ _ id hx] | case a.refine'_2
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
hsnonempty : s.Nonempty
centroid_weights : ∑ i ∈ s, Finset.centroidWeights ℝ s i = 1
n : ℕ
⊢ (fun n => (↑n + 2)⁻¹ • s.centerMass (Finset.centroidWeights ℝ s) id + (1 - (↑n + 2)⁻¹) • id x) n ∈ combiInterior ℝ s | case a.refine'_2
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
hsnonempty : s.Nonempty
centroid_weights : ∑ i ∈ s, Finset.centroidWeights ℝ s i = 1
n : ℕ
⊢ (fun n =>
(↑n + 2)⁻¹ • s.centerMass (Finset.centroidWeights ℝ s) id +
(1 - (↑n + 2)⁻¹) • s.centerMass (fun j => if x = j then 1 else 0) id)
n ∈
combiInterior ℝ s |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | subset_closure_combiInterior | [234, 1] | [288, 39] | simp only | case a.refine'_2
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
hsnonempty : s.Nonempty
centroid_weights : ∑ i ∈ s, Finset.centroidWeights ℝ s i = 1
n : ℕ
⊢ (fun n =>
(↑n + 2)⁻¹ • s.centerMass (Finset.centroidWeights ℝ s) id +
(1 - (↑n + 2)⁻¹) • s.centerMass (fun j => if x = j then 1 else 0) id)
n ∈
combiInterior ℝ s | case a.refine'_2
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
hsnonempty : s.Nonempty
centroid_weights : ∑ i ∈ s, Finset.centroidWeights ℝ s i = 1
n : ℕ
⊢ (↑n + 2)⁻¹ • s.centerMass (Finset.centroidWeights ℝ s) id +
(1 - (↑n + 2)⁻¹) • s.centerMass (fun j => if x = j then 1 else 0) id ∈
combiInterior ℝ s |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | subset_closure_combiInterior | [234, 1] | [288, 39] | rw [Finset.centerMass_segment] | case a.refine'_2
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
hsnonempty : s.Nonempty
centroid_weights : ∑ i ∈ s, Finset.centroidWeights ℝ s i = 1
n : ℕ
⊢ (↑n + 2)⁻¹ • s.centerMass (Finset.centroidWeights ℝ s) id +
(1 - (↑n + 2)⁻¹) • s.centerMass (fun j => if x = j then 1 else 0) id ∈
combiInterior ℝ s | case a.refine'_2
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
hsnonempty : s.Nonempty
centroid_weights : ∑ i ∈ s, Finset.centroidWeights ℝ s i = 1
n : ℕ
⊢ s.centerMass (fun i => (↑n + 2)⁻¹ * Finset.centroidWeights ℝ s i + (1 - (↑n + 2)⁻¹) * if x = i then 1 else 0) id ∈
combiInterior ℝ s
case a.refine'_2.hw₁
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
hsnonempty : s.Nonempty
centroid_weights : ∑ i ∈ s, Finset.centroidWeights ℝ s i = 1
n : ℕ
⊢ ∑ i ∈ s, Finset.centroidWeights ℝ s i = 1
case a.refine'_2.hw₂
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
hsnonempty : s.Nonempty
centroid_weights : ∑ i ∈ s, Finset.centroidWeights ℝ s i = 1
n : ℕ
⊢ (∑ i ∈ s, if x = i then 1 else 0) = 1
case a.refine'_2.hab
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
hsnonempty : s.Nonempty
centroid_weights : ∑ i ∈ s, Finset.centroidWeights ℝ s i = 1
n : ℕ
⊢ (↑n + 2)⁻¹ + (1 - (↑n + 2)⁻¹) = 1 |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | subset_closure_combiInterior | [234, 1] | [288, 39] | rw [combiInterior_eq hs] | case a.refine'_2
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
hsnonempty : s.Nonempty
centroid_weights : ∑ i ∈ s, Finset.centroidWeights ℝ s i = 1
n : ℕ
⊢ s.centerMass (fun i => (↑n + 2)⁻¹ * Finset.centroidWeights ℝ s i + (1 - (↑n + 2)⁻¹) * if x = i then 1 else 0) id ∈
combiInterior ℝ s | case a.refine'_2
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
hsnonempty : s.Nonempty
centroid_weights : ∑ i ∈ s, Finset.centroidWeights ℝ s i = 1
n : ℕ
⊢ s.centerMass (fun i => (↑n + 2)⁻¹ * Finset.centroidWeights ℝ s i + (1 - (↑n + 2)⁻¹) * if x = i then 1 else 0) id ∈
{x | ∃ w, ∃ (_ : ∀ y ∈ s, 0 < w y) (_ : ∑ y ∈ s, w y = 1), s.centerMass w id = x} |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | subset_closure_combiInterior | [234, 1] | [288, 39] | refine' ⟨_, _, _, rfl⟩ | case a.refine'_2
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
hsnonempty : s.Nonempty
centroid_weights : ∑ i ∈ s, Finset.centroidWeights ℝ s i = 1
n : ℕ
⊢ s.centerMass (fun i => (↑n + 2)⁻¹ * Finset.centroidWeights ℝ s i + (1 - (↑n + 2)⁻¹) * if x = i then 1 else 0) id ∈
{x | ∃ w, ∃ (_ : ∀ y ∈ s, 0 < w y) (_ : ∑ y ∈ s, w y = 1), s.centerMass w id = x} | case a.refine'_2.refine'_1
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
hsnonempty : s.Nonempty
centroid_weights : ∑ i ∈ s, Finset.centroidWeights ℝ s i = 1
n : ℕ
⊢ ∀ y ∈ s, 0 < (↑n + 2)⁻¹ * Finset.centroidWeights ℝ s y + (1 - (↑n + 2)⁻¹) * if x = y then 1 else 0
case a.refine'_2.refine'_2
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
hsnonempty : s.Nonempty
centroid_weights : ∑ i ∈ s, Finset.centroidWeights ℝ s i = 1
n : ℕ
⊢ ∑ y ∈ s, ((↑n + 2)⁻¹ * Finset.centroidWeights ℝ s y + (1 - (↑n + 2)⁻¹) * if x = y then 1 else 0) = 1 |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | subset_closure_combiInterior | [234, 1] | [288, 39] | sorry | case a.refine'_2.refine'_2
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
hsnonempty : s.Nonempty
centroid_weights : ∑ i ∈ s, Finset.centroidWeights ℝ s i = 1
n : ℕ
⊢ ∑ y ∈ s, ((↑n + 2)⁻¹ * Finset.centroidWeights ℝ s y + (1 - (↑n + 2)⁻¹) * if x = y then 1 else 0) = 1 | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | subset_closure_combiInterior | [234, 1] | [288, 39] | simp only [mul_boole, Finset.centroidWeights_apply] | case a.refine'_2.refine'_1
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
hsnonempty : s.Nonempty
centroid_weights : ∑ i ∈ s, Finset.centroidWeights ℝ s i = 1
n : ℕ
⊢ ∀ y ∈ s, 0 < (↑n + 2)⁻¹ * Finset.centroidWeights ℝ s y + (1 - (↑n + 2)⁻¹) * if x = y then 1 else 0 | case a.refine'_2.refine'_1
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
hsnonempty : s.Nonempty
centroid_weights : ∑ i ∈ s, Finset.centroidWeights ℝ s i = 1
n : ℕ
⊢ ∀ y ∈ s, 0 < (↑n + 2)⁻¹ * (↑s.card)⁻¹ + if x = y then 1 - (↑n + 2)⁻¹ else 0 |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | subset_closure_combiInterior | [234, 1] | [288, 39] | intro y hy | case a.refine'_2.refine'_1
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
hsnonempty : s.Nonempty
centroid_weights : ∑ i ∈ s, Finset.centroidWeights ℝ s i = 1
n : ℕ
⊢ ∀ y ∈ s, 0 < (↑n + 2)⁻¹ * (↑s.card)⁻¹ + if x = y then 1 - (↑n + 2)⁻¹ else 0 | case a.refine'_2.refine'_1
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
hsnonempty : s.Nonempty
centroid_weights : ∑ i ∈ s, Finset.centroidWeights ℝ s i = 1
n : ℕ
y : E
hy : y ∈ s
⊢ 0 < (↑n + 2)⁻¹ * (↑s.card)⁻¹ + if x = y then 1 - (↑n + 2)⁻¹ else 0 |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | subset_closure_combiInterior | [234, 1] | [288, 39] | apply add_pos_of_pos_of_nonneg | case a.refine'_2.refine'_1
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
hsnonempty : s.Nonempty
centroid_weights : ∑ i ∈ s, Finset.centroidWeights ℝ s i = 1
n : ℕ
y : E
hy : y ∈ s
⊢ 0 < (↑n + 2)⁻¹ * (↑s.card)⁻¹ + if x = y then 1 - (↑n + 2)⁻¹ else 0 | case a.refine'_2.refine'_1.ha
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
hsnonempty : s.Nonempty
centroid_weights : ∑ i ∈ s, Finset.centroidWeights ℝ s i = 1
n : ℕ
y : E
hy : y ∈ s
⊢ 0 < (↑n + 2)⁻¹ * (↑s.card)⁻¹
case a.refine'_2.refine'_1.hb
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
hsnonempty : s.Nonempty
centroid_weights : ∑ i ∈ s, Finset.centroidWeights ℝ s i = 1
n : ℕ
y : E
hy : y ∈ s
⊢ 0 ≤ if x = y then 1 - (↑n + 2)⁻¹ else 0 |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | subset_closure_combiInterior | [234, 1] | [288, 39] | apply mul_pos | case a.refine'_2.refine'_1.ha
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
hsnonempty : s.Nonempty
centroid_weights : ∑ i ∈ s, Finset.centroidWeights ℝ s i = 1
n : ℕ
y : E
hy : y ∈ s
⊢ 0 < (↑n + 2)⁻¹ * (↑s.card)⁻¹ | case a.refine'_2.refine'_1.ha.ha
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
hsnonempty : s.Nonempty
centroid_weights : ∑ i ∈ s, Finset.centroidWeights ℝ s i = 1
n : ℕ
y : E
hy : y ∈ s
⊢ 0 < (↑n + 2)⁻¹
case a.refine'_2.refine'_1.ha.hb
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
hsnonempty : s.Nonempty
centroid_weights : ∑ i ∈ s, Finset.centroidWeights ℝ s i = 1
n : ℕ
y : E
hy : y ∈ s
⊢ 0 < (↑s.card)⁻¹ |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | subset_closure_combiInterior | [234, 1] | [288, 39] | rw [inv_pos] | case a.refine'_2.refine'_1.ha.ha
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
hsnonempty : s.Nonempty
centroid_weights : ∑ i ∈ s, Finset.centroidWeights ℝ s i = 1
n : ℕ
y : E
hy : y ∈ s
⊢ 0 < (↑n + 2)⁻¹ | case a.refine'_2.refine'_1.ha.ha
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
hsnonempty : s.Nonempty
centroid_weights : ∑ i ∈ s, Finset.centroidWeights ℝ s i = 1
n : ℕ
y : E
hy : y ∈ s
⊢ 0 < ↑n + 2 |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | subset_closure_combiInterior | [234, 1] | [288, 39] | norm_cast | case a.refine'_2.refine'_1.ha.ha
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
hsnonempty : s.Nonempty
centroid_weights : ∑ i ∈ s, Finset.centroidWeights ℝ s i = 1
n : ℕ
y : E
hy : y ∈ s
⊢ 0 < ↑n + 2 | case a.refine'_2.refine'_1.ha.ha
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
hsnonempty : s.Nonempty
centroid_weights : ∑ i ∈ s, Finset.centroidWeights ℝ s i = 1
n : ℕ
y : E
hy : y ∈ s
⊢ 0 < n + 2 |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | subset_closure_combiInterior | [234, 1] | [288, 39] | simp | case a.refine'_2.refine'_1.ha.ha
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
hsnonempty : s.Nonempty
centroid_weights : ∑ i ∈ s, Finset.centroidWeights ℝ s i = 1
n : ℕ
y : E
hy : y ∈ s
⊢ 0 < n + 2 | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | subset_closure_combiInterior | [234, 1] | [288, 39] | rw [inv_pos] | case a.refine'_2.refine'_1.ha.hb
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
hsnonempty : s.Nonempty
centroid_weights : ∑ i ∈ s, Finset.centroidWeights ℝ s i = 1
n : ℕ
y : E
hy : y ∈ s
⊢ 0 < (↑s.card)⁻¹ | case a.refine'_2.refine'_1.ha.hb
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
hsnonempty : s.Nonempty
centroid_weights : ∑ i ∈ s, Finset.centroidWeights ℝ s i = 1
n : ℕ
y : E
hy : y ∈ s
⊢ 0 < ↑s.card |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | subset_closure_combiInterior | [234, 1] | [288, 39] | norm_cast | case a.refine'_2.refine'_1.ha.hb
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
hsnonempty : s.Nonempty
centroid_weights : ∑ i ∈ s, Finset.centroidWeights ℝ s i = 1
n : ℕ
y : E
hy : y ∈ s
⊢ 0 < ↑s.card | case a.refine'_2.refine'_1.ha.hb
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
hsnonempty : s.Nonempty
centroid_weights : ∑ i ∈ s, Finset.centroidWeights ℝ s i = 1
n : ℕ
y : E
hy : y ∈ s
⊢ 0 < s.card |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | subset_closure_combiInterior | [234, 1] | [288, 39] | rwa [Finset.card_pos] | case a.refine'_2.refine'_1.ha.hb
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
hsnonempty : s.Nonempty
centroid_weights : ∑ i ∈ s, Finset.centroidWeights ℝ s i = 1
n : ℕ
y : E
hy : y ∈ s
⊢ 0 < s.card | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | subset_closure_combiInterior | [234, 1] | [288, 39] | split_ifs | case a.refine'_2.refine'_1.hb
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
hsnonempty : s.Nonempty
centroid_weights : ∑ i ∈ s, Finset.centroidWeights ℝ s i = 1
n : ℕ
y : E
hy : y ∈ s
⊢ 0 ≤ if x = y then 1 - (↑n + 2)⁻¹ else 0 | case pos
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
hsnonempty : s.Nonempty
centroid_weights : ∑ i ∈ s, Finset.centroidWeights ℝ s i = 1
n : ℕ
y : E
hy : y ∈ s
h✝ : x = y
⊢ 0 ≤ 1 - (↑n + 2)⁻¹
case neg
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
hsnonempty : s.Nonempty
centroid_weights : ∑ i ∈ s, Finset.centroidWeights ℝ s i = 1
n : ℕ
y : E
hy : y ∈ s
h✝ : ¬x = y
⊢ 0 ≤ 0 |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | subset_closure_combiInterior | [234, 1] | [288, 39] | rw [sub_nonneg] | case pos
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
hsnonempty : s.Nonempty
centroid_weights : ∑ i ∈ s, Finset.centroidWeights ℝ s i = 1
n : ℕ
y : E
hy : y ∈ s
h✝ : x = y
⊢ 0 ≤ 1 - (↑n + 2)⁻¹ | case pos
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
hsnonempty : s.Nonempty
centroid_weights : ∑ i ∈ s, Finset.centroidWeights ℝ s i = 1
n : ℕ
y : E
hy : y ∈ s
h✝ : x = y
⊢ (↑n + 2)⁻¹ ≤ 1 |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | subset_closure_combiInterior | [234, 1] | [288, 39] | apply inv_le_one | case pos
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
hsnonempty : s.Nonempty
centroid_weights : ∑ i ∈ s, Finset.centroidWeights ℝ s i = 1
n : ℕ
y : E
hy : y ∈ s
h✝ : x = y
⊢ (↑n + 2)⁻¹ ≤ 1 | case pos.ha
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
hsnonempty : s.Nonempty
centroid_weights : ∑ i ∈ s, Finset.centroidWeights ℝ s i = 1
n : ℕ
y : E
hy : y ∈ s
h✝ : x = y
⊢ 1 ≤ ↑n + 2 |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | subset_closure_combiInterior | [234, 1] | [288, 39] | norm_cast | case pos.ha
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
hsnonempty : s.Nonempty
centroid_weights : ∑ i ∈ s, Finset.centroidWeights ℝ s i = 1
n : ℕ
y : E
hy : y ∈ s
h✝ : x = y
⊢ 1 ≤ ↑n + 2 | case pos.ha
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
hsnonempty : s.Nonempty
centroid_weights : ∑ i ∈ s, Finset.centroidWeights ℝ s i = 1
n : ℕ
y : E
hy : y ∈ s
h✝ : x = y
⊢ 1 ≤ n + 2 |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | subset_closure_combiInterior | [234, 1] | [288, 39] | apply Nat.succ_pos | case pos.ha
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
hsnonempty : s.Nonempty
centroid_weights : ∑ i ∈ s, Finset.centroidWeights ℝ s i = 1
n : ℕ
y : E
hy : y ∈ s
h✝ : x = y
⊢ 1 ≤ n + 2 | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | subset_closure_combiInterior | [234, 1] | [288, 39] | rfl | case neg
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
hsnonempty : s.Nonempty
centroid_weights : ∑ i ∈ s, Finset.centroidWeights ℝ s i = 1
n : ℕ
y : E
hy : y ∈ s
h✝ : ¬x = y
⊢ 0 ≤ 0 | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | subset_closure_combiInterior | [234, 1] | [288, 39] | apply centroid_weights | case a.refine'_2.hw₁
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
hsnonempty : s.Nonempty
centroid_weights : ∑ i ∈ s, Finset.centroidWeights ℝ s i = 1
n : ℕ
⊢ ∑ i ∈ s, Finset.centroidWeights ℝ s i = 1 | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | subset_closure_combiInterior | [234, 1] | [288, 39] | simp [Finset.sum_boole, Finset.filter_eq, hx] | case a.refine'_2.hw₂
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
hsnonempty : s.Nonempty
centroid_weights : ∑ i ∈ s, Finset.centroidWeights ℝ s i = 1
n : ℕ
⊢ (∑ i ∈ s, if x = i then 1 else 0) = 1 | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | subset_closure_combiInterior | [234, 1] | [288, 39] | simp only [add_sub_cancel] | case a.refine'_2.hab
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
hsnonempty : s.Nonempty
centroid_weights : ∑ i ∈ s, Finset.centroidWeights ℝ s i = 1
n : ℕ
⊢ (↑n + 2)⁻¹ + (1 - (↑n + 2)⁻¹) = 1 | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | subset_closure_combiInterior | [234, 1] | [288, 39] | rw [tendsto_iff_norm_sub_tendsto_zero] | case a.refine'_3
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
hsnonempty : s.Nonempty
centroid_weights : ∑ i ∈ s, Finset.centroidWeights ℝ s i = 1
⊢ Filter.Tendsto (fun n => (↑n + 2)⁻¹ • Finset.centroid ℝ s id + (1 - (↑n + 2)⁻¹) • x) Filter.atTop (nhds x) | case a.refine'_3
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
hsnonempty : s.Nonempty
centroid_weights : ∑ i ∈ s, Finset.centroidWeights ℝ s i = 1
⊢ Filter.Tendsto (fun e => ‖(↑e + 2)⁻¹ • Finset.centroid ℝ s id + (1 - (↑e + 2)⁻¹) • x - x‖) Filter.atTop (nhds 0) |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | subset_closure_combiInterior | [234, 1] | [288, 39] | convert_to Filter.Tendsto (fun e : ℕ => ((e : ℝ) + 2)⁻¹ * ‖s.centroid ℝ id - x‖) Filter.atTop _ | case a.refine'_3
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
hsnonempty : s.Nonempty
centroid_weights : ∑ i ∈ s, Finset.centroidWeights ℝ s i = 1
⊢ Filter.Tendsto (fun e => ‖(↑e + 2)⁻¹ • Finset.centroid ℝ s id + (1 - (↑e + 2)⁻¹) • x - x‖) Filter.atTop (nhds 0) | case h.e'_3
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
hsnonempty : s.Nonempty
centroid_weights : ∑ i ∈ s, Finset.centroidWeights ℝ s i = 1
⊢ (fun e => ‖(↑e + 2)⁻¹ • Finset.centroid ℝ s id + (1 - (↑e + 2)⁻¹) • x - x‖) = fun e =>
(↑e + 2)⁻¹ * ‖Finset.centroid ℝ s id - x‖
case a.refine'_3.convert_2
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
hsnonempty : s.Nonempty
centroid_weights : ∑ i ∈ s, Finset.centroidWeights ℝ s i = 1
⊢ Filter.Tendsto (fun e => (↑e + 2)⁻¹ * ‖Finset.centroid ℝ s id - x‖) Filter.atTop (nhds 0) |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | subset_closure_combiInterior | [234, 1] | [288, 39] | suffices Filter.Tendsto (fun e : ℕ => (↑(e + 2) : ℝ)⁻¹) Filter.atTop (nhds 0) by
simpa using this.mul_const _ | case a.refine'_3.convert_2
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
hsnonempty : s.Nonempty
centroid_weights : ∑ i ∈ s, Finset.centroidWeights ℝ s i = 1
⊢ Filter.Tendsto (fun e => (↑e + 2)⁻¹ * ‖Finset.centroid ℝ s id - x‖) Filter.atTop (nhds 0) | case a.refine'_3.convert_2
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
hsnonempty : s.Nonempty
centroid_weights : ∑ i ∈ s, Finset.centroidWeights ℝ s i = 1
⊢ Filter.Tendsto (fun e => (↑(e + 2))⁻¹) Filter.atTop (nhds 0) |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | subset_closure_combiInterior | [234, 1] | [288, 39] | refine' tendsto_inv_atTop_zero.comp _ | case a.refine'_3.convert_2
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
hsnonempty : s.Nonempty
centroid_weights : ∑ i ∈ s, Finset.centroidWeights ℝ s i = 1
⊢ Filter.Tendsto (fun e => (↑(e + 2))⁻¹) Filter.atTop (nhds 0) | case a.refine'_3.convert_2
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
hsnonempty : s.Nonempty
centroid_weights : ∑ i ∈ s, Finset.centroidWeights ℝ s i = 1
⊢ Filter.Tendsto (fun e => ↑(e + 2)) Filter.atTop Filter.atTop |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | subset_closure_combiInterior | [234, 1] | [288, 39] | rw [tendsto_natCast_atTop_iff] | case a.refine'_3.convert_2
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
hsnonempty : s.Nonempty
centroid_weights : ∑ i ∈ s, Finset.centroidWeights ℝ s i = 1
⊢ Filter.Tendsto (fun e => ↑(e + 2)) Filter.atTop Filter.atTop | case a.refine'_3.convert_2
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝¹ : SeminormedAddCommGroup E
inst✝ : NormedSpace ℝ E
s t : Finset E
hs : AffineIndependent ℝ Subtype.val
x : E
hx : x ∈ s
hsnonempty : s.Nonempty
centroid_weights : ∑ i ∈ s, Finset.centroidWeights ℝ s i = 1
⊢ Filter.Tendsto (fun e => e + 2) Filter.atTop Filter.atTop |
Subsets and Splits
No community queries yet
The top public SQL queries from the community will appear here once available.