url
stringclasses 147
values | commit
stringclasses 147
values | file_path
stringlengths 7
101
| full_name
stringlengths 1
94
| start
stringlengths 6
10
| end
stringlengths 6
11
| tactic
stringlengths 1
11.2k
| state_before
stringlengths 3
2.09M
| state_after
stringlengths 6
2.09M
|
---|---|---|---|---|---|---|---|---|
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Kneser/KneserRuzsa.lean | Finset.le_card_mul_add_card_mulStab_mul | [204, 1] | [248, 67] | rwa [mem_inv_smul_finset_iff, smul_eq_mul, inv_mul_cancel_right] | α : Type u_1
inst✝¹ : CommGroup α
inst✝ : DecidableEq α
s t : Finset α
hs : s.Nonempty
ht : t.Nonempty
this✝ :
∀ (b : { x // x ∈ t }),
∃ n s' t', ↑b ∈ t' ∧ s ⊆ s' ∧ s' * t' ⊆ s * t ∧ s'.card + t'.card = s.card + t.card ∧ n = t'.card
s' t' : { x // x ∈ t } → Finset α
hbt' : ∀ (b : { x // x ∈ t }), ↑b ∈ t' b
hs' : ∀ (b : { x // x ∈ t }), s ⊆ s' b
hst' : ∀ (b : { x // x ∈ t }), s' b * t' b ⊆ s * t
hstcard : ∀ (b : { x // x ∈ t }), (s' b).card + (t' b).card = s.card + t.card
ht' : ∀ (b : { x // x ∈ t }), Nat.find ⋯ = (t' b).card
this : s * t = univ.sup fun b => s' b * t' b
b : { x // x ∈ t }
x✝ : b ∈ t.attach
c : α
hc : c ∈ s' b
⊢ ↑b ∈ (c * (↑b)⁻¹)⁻¹ • (s' b, t' b).1 | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Kneser/KneserRuzsa.lean | Finset.le_card_mul_add_card_mulStab_mul | [204, 1] | [248, 67] | refine' le_antisymm _ (Finset.sup_le_iff.2 fun _ _ => hst' _) | α : Type u_1
inst✝¹ : CommGroup α
inst✝ : DecidableEq α
s t : Finset α
hs : s.Nonempty
ht : t.Nonempty
this :
∀ (b : { x // x ∈ t }),
∃ n s' t', ↑b ∈ t' ∧ s ⊆ s' ∧ s' * t' ⊆ s * t ∧ s'.card + t'.card = s.card + t.card ∧ n = t'.card
s' t' : { x // x ∈ t } → Finset α
hbt' : ∀ (b : { x // x ∈ t }), ↑b ∈ t' b
hs' : ∀ (b : { x // x ∈ t }), s ⊆ s' b
hst' : ∀ (b : { x // x ∈ t }), s' b * t' b ⊆ s * t
hstcard : ∀ (b : { x // x ∈ t }), (s' b).card + (t' b).card = s.card + t.card
ht' : ∀ (b : { x // x ∈ t }), Nat.find ⋯ = (t' b).card
⊢ s * t = univ.sup fun b => s' b * t' b | α : Type u_1
inst✝¹ : CommGroup α
inst✝ : DecidableEq α
s t : Finset α
hs : s.Nonempty
ht : t.Nonempty
this :
∀ (b : { x // x ∈ t }),
∃ n s' t', ↑b ∈ t' ∧ s ⊆ s' ∧ s' * t' ⊆ s * t ∧ s'.card + t'.card = s.card + t.card ∧ n = t'.card
s' t' : { x // x ∈ t } → Finset α
hbt' : ∀ (b : { x // x ∈ t }), ↑b ∈ t' b
hs' : ∀ (b : { x // x ∈ t }), s ⊆ s' b
hst' : ∀ (b : { x // x ∈ t }), s' b * t' b ⊆ s * t
hstcard : ∀ (b : { x // x ∈ t }), (s' b).card + (t' b).card = s.card + t.card
ht' : ∀ (b : { x // x ∈ t }), Nat.find ⋯ = (t' b).card
⊢ s * t ≤ univ.sup fun b => s' b * t' b |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Kneser/KneserRuzsa.lean | Finset.le_card_mul_add_card_mulStab_mul | [204, 1] | [248, 67] | exact
mul_subset_iff_right.2 fun b hb =>
(smul_finset_subset_smul_finset $ hs' ⟨b, hb⟩).trans $
(op_smul_finset_subset_mul $ hbt' ⟨b, hb⟩).trans $
@le_sup _ _ _ _ _ (fun b => s' b * t' b) _ $ mem_univ _ | α : Type u_1
inst✝¹ : CommGroup α
inst✝ : DecidableEq α
s t : Finset α
hs : s.Nonempty
ht : t.Nonempty
this :
∀ (b : { x // x ∈ t }),
∃ n s' t', ↑b ∈ t' ∧ s ⊆ s' ∧ s' * t' ⊆ s * t ∧ s'.card + t'.card = s.card + t.card ∧ n = t'.card
s' t' : { x // x ∈ t } → Finset α
hbt' : ∀ (b : { x // x ∈ t }), ↑b ∈ t' b
hs' : ∀ (b : { x // x ∈ t }), s ⊆ s' b
hst' : ∀ (b : { x // x ∈ t }), s' b * t' b ⊆ s * t
hstcard : ∀ (b : { x // x ∈ t }), (s' b).card + (t' b).card = s.card + t.card
ht' : ∀ (b : { x // x ∈ t }), Nat.find ⋯ = (t' b).card
⊢ s * t ≤ univ.sup fun b => s' b * t' b | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Kneser/KneserRuzsa.lean | Finset.mul_kneser' | [250, 1] | [266, 43] | obtain rfl | hs := s.eq_empty_or_nonempty | α : Type u_1
inst✝¹ : CommGroup α
inst✝ : DecidableEq α
s✝ t✝ s t : Finset α
⊢ (s * (s * t).mulStab).card + (t * (s * t).mulStab).card ≤ (s * t).card + (s * t).mulStab.card | case inl
α : Type u_1
inst✝¹ : CommGroup α
inst✝ : DecidableEq α
s t✝ t : Finset α
⊢ (∅ * (∅ * t).mulStab).card + (t * (∅ * t).mulStab).card ≤ (∅ * t).card + (∅ * t).mulStab.card
case inr
α : Type u_1
inst✝¹ : CommGroup α
inst✝ : DecidableEq α
s✝ t✝ s t : Finset α
hs : s.Nonempty
⊢ (s * (s * t).mulStab).card + (t * (s * t).mulStab).card ≤ (s * t).card + (s * t).mulStab.card |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Kneser/KneserRuzsa.lean | Finset.mul_kneser' | [250, 1] | [266, 43] | obtain rfl | ht := t.eq_empty_or_nonempty | case inr
α : Type u_1
inst✝¹ : CommGroup α
inst✝ : DecidableEq α
s✝ t✝ s t : Finset α
hs : s.Nonempty
⊢ (s * (s * t).mulStab).card + (t * (s * t).mulStab).card ≤ (s * t).card + (s * t).mulStab.card | case inr.inl
α : Type u_1
inst✝¹ : CommGroup α
inst✝ : DecidableEq α
s✝ t s : Finset α
hs : s.Nonempty
⊢ (s * (s * ∅).mulStab).card + (∅ * (s * ∅).mulStab).card ≤ (s * ∅).card + (s * ∅).mulStab.card
case inr.inr
α : Type u_1
inst✝¹ : CommGroup α
inst✝ : DecidableEq α
s✝ t✝ s t : Finset α
hs : s.Nonempty
ht : t.Nonempty
⊢ (s * (s * t).mulStab).card + (t * (s * t).mulStab).card ≤ (s * t).card + (s * t).mulStab.card |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Kneser/KneserRuzsa.lean | Finset.mul_kneser' | [250, 1] | [266, 43] | refine'
(le_card_mul_add_card_mulStab_mul (hs.mul (hs.mul ht).mulStab) $
ht.mul (hs.mul ht).mulStab).trans_eq
_ | case inr.inr
α : Type u_1
inst✝¹ : CommGroup α
inst✝ : DecidableEq α
s✝ t✝ s t : Finset α
hs : s.Nonempty
ht : t.Nonempty
⊢ (s * (s * t).mulStab).card + (t * (s * t).mulStab).card ≤ (s * t).card + (s * t).mulStab.card | case inr.inr
α : Type u_1
inst✝¹ : CommGroup α
inst✝ : DecidableEq α
s✝ t✝ s t : Finset α
hs : s.Nonempty
ht : t.Nonempty
⊢ (s * (s * t).mulStab * (t * (s * t).mulStab)).card + (s * (s * t).mulStab * (t * (s * t).mulStab)).mulStab.card =
(s * t).card + (s * t).mulStab.card |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Kneser/KneserRuzsa.lean | Finset.mul_kneser' | [250, 1] | [266, 43] | rw [mul_mulStab_mul_mul_mul_mulStab_mul] | case inr.inr
α : Type u_1
inst✝¹ : CommGroup α
inst✝ : DecidableEq α
s✝ t✝ s t : Finset α
hs : s.Nonempty
ht : t.Nonempty
⊢ (s * (s * t).mulStab * (t * (s * t).mulStab)).card + (s * (s * t).mulStab * (t * (s * t).mulStab)).mulStab.card =
(s * t).card + (s * t).mulStab.card | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Kneser/KneserRuzsa.lean | Finset.mul_kneser' | [250, 1] | [266, 43] | simp | case inl
α : Type u_1
inst✝¹ : CommGroup α
inst✝ : DecidableEq α
s t✝ t : Finset α
⊢ (∅ * (∅ * t).mulStab).card + (t * (∅ * t).mulStab).card ≤ (∅ * t).card + (∅ * t).mulStab.card | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Kneser/KneserRuzsa.lean | Finset.mul_kneser' | [250, 1] | [266, 43] | simp | case inr.inl
α : Type u_1
inst✝¹ : CommGroup α
inst✝ : DecidableEq α
s✝ t s : Finset α
hs : s.Nonempty
⊢ (s * (s * ∅).mulStab).card + (∅ * (s * ∅).mulStab).card ≤ (s * ∅).card + (s * ∅).mulStab.card | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Finite.lean | Geometry.SimplicialComplex.LocallyFiniteAt.mono | [47, 1] | [50, 43] | apply hX.subset | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x t✝ : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
hX : K.LocallyFiniteAt s
hXY : s ⊆ t
⊢ K.LocallyFiniteAt 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 t✝ : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
hX : K.LocallyFiniteAt s
hXY : s ⊆ t
⊢ {t_1 | t_1 ∈ K.faces ∧ t ⊆ t_1} ⊆ {t | t ∈ K.faces ∧ s ⊆ t} |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Finite.lean | Geometry.SimplicialComplex.LocallyFiniteAt.mono | [47, 1] | [50, 43] | rintro 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 t✝ : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
hX : K.LocallyFiniteAt s
hXY : s ⊆ t
⊢ {t_1 | t_1 ∈ K.faces ∧ t ⊆ t_1} ⊆ {t | t ∈ K.faces ∧ s ⊆ t} | case intro
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x t✝ : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
hX : K.LocallyFiniteAt s
hXY : s ⊆ t
u : Finset E
left✝ : u ∈ K.faces
right✝ : t ⊆ u
⊢ u ∈ {t | t ∈ K.faces ∧ s ⊆ t} |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Finite.lean | Geometry.SimplicialComplex.LocallyFiniteAt.mono | [47, 1] | [50, 43] | exact ⟨‹u ∈ K.faces›, hXY.trans ‹t ⊆ u›⟩ | case intro
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x t✝ : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
hX : K.LocallyFiniteAt s
hXY : s ⊆ t
u : Finset E
left✝ : u ∈ K.faces
right✝ : t ⊆ u
⊢ u ∈ {t | t ∈ K.faces ∧ s ⊆ t} | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Finite.lean | Geometry.SimplicialComplex.locallyFinite_iff_mem_finitely_many_faces | [58, 1] | [82, 88] | 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 t✝ : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : DecidableEq E
⊢ K.LocallyFinite ↔ ∀ (x : E), {s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}.Finite | case mp
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : OrderedRing 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x t✝ : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : DecidableEq E
⊢ K.LocallyFinite → ∀ (x : E), {s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}.Finite
case mpr
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : OrderedRing 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x t✝ : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : DecidableEq E
⊢ (∀ (x : E), {s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}.Finite) → K.LocallyFinite |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Finite.lean | Geometry.SimplicialComplex.locallyFinite_iff_mem_finitely_many_faces | [58, 1] | [82, 88] | unfold LocallyFinite | case mp
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : OrderedRing 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x t✝ : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : DecidableEq E
⊢ K.LocallyFinite → ∀ (x : E), {s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}.Finite | case mp
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : OrderedRing 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x t✝ : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : DecidableEq E
⊢ (∀ ⦃s : Finset E⦄, s ∈ K.faces → s.Nonempty → K.LocallyFiniteAt s) →
∀ (x : E), {s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}.Finite |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Finite.lean | Geometry.SimplicialComplex.locallyFinite_iff_mem_finitely_many_faces | [58, 1] | [82, 88] | contrapose! | case mp
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : OrderedRing 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x t✝ : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : DecidableEq E
⊢ (∀ ⦃s : Finset E⦄, s ∈ K.faces → s.Nonempty → K.LocallyFiniteAt s) →
∀ (x : E), {s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}.Finite | case mp
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : OrderedRing 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x t✝ : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : DecidableEq E
⊢ (∃ x, ¬{s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}.Finite) → ∃ s ∈ K.faces, s.Nonempty ∧ ¬K.LocallyFiniteAt s |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Finite.lean | Geometry.SimplicialComplex.locallyFinite_iff_mem_finitely_many_faces | [58, 1] | [82, 88] | rintro ⟨x, hx⟩ | case mp
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : OrderedRing 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x t✝ : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : DecidableEq E
⊢ (∃ x, ¬{s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}.Finite) → ∃ s ∈ K.faces, s.Nonempty ∧ ¬K.LocallyFiniteAt s | case mp.intro
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : OrderedRing 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x✝ t✝ : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : DecidableEq E
x : E
hx : ¬{s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}.Finite
⊢ ∃ s ∈ K.faces, s.Nonempty ∧ ¬K.LocallyFiniteAt s |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Finite.lean | Geometry.SimplicialComplex.locallyFinite_iff_mem_finitely_many_faces | [58, 1] | [82, 88] | by_cases hxspace : x ∈ K.space | case mp.intro
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : OrderedRing 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x✝ t✝ : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : DecidableEq E
x : E
hx : ¬{s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}.Finite
⊢ ∃ s ∈ K.faces, s.Nonempty ∧ ¬K.LocallyFiniteAt s | case pos
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : OrderedRing 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x✝ t✝ : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : DecidableEq E
x : E
hx : ¬{s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}.Finite
hxspace : x ∈ K.space
⊢ ∃ s ∈ K.faces, s.Nonempty ∧ ¬K.LocallyFiniteAt s
case neg
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : OrderedRing 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x✝ t✝ : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : DecidableEq E
x : E
hx : ¬{s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}.Finite
hxspace : x ∉ K.space
⊢ ∃ s ∈ K.faces, s.Nonempty ∧ ¬K.LocallyFiniteAt s |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Finite.lean | Geometry.SimplicialComplex.locallyFinite_iff_mem_finitely_many_faces | [58, 1] | [82, 88] | obtain ⟨s, ⟨hX, hXhull, hXbound⟩, hXunique⟩ := combiInteriors_partition hxspace | case pos
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : OrderedRing 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x✝ t✝ : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : DecidableEq E
x : E
hx : ¬{s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}.Finite
hxspace : x ∈ K.space
⊢ ∃ s ∈ K.faces, s.Nonempty ∧ ¬K.LocallyFiniteAt s | case pos.intro.intro.intro.intro
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : OrderedRing 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x✝ t✝ : E
s✝ t : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : DecidableEq E
x : E
hx : ¬{s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}.Finite
hxspace : x ∈ K.space
s : Finset E
hXunique : ∀ (y : Finset E), (fun s => s ∈ K ∧ x ∈ combiInterior 𝕜 s) y → y = s
hX : s ∈ K
hXhull : x ∈ (convexHull 𝕜) ↑s
hXbound : x ∉ combiFrontier 𝕜 s
⊢ ∃ s ∈ K.faces, s.Nonempty ∧ ¬K.LocallyFiniteAt s |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Finite.lean | Geometry.SimplicialComplex.locallyFinite_iff_mem_finitely_many_faces | [58, 1] | [82, 88] | simp at hXunique | case pos.intro.intro.intro.intro
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : OrderedRing 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x✝ t✝ : E
s✝ t : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : DecidableEq E
x : E
hx : ¬{s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}.Finite
hxspace : x ∈ K.space
s : Finset E
hXunique : ∀ (y : Finset E), (fun s => s ∈ K ∧ x ∈ combiInterior 𝕜 s) y → y = s
hX : s ∈ K
hXhull : x ∈ (convexHull 𝕜) ↑s
hXbound : x ∉ combiFrontier 𝕜 s
⊢ ∃ s ∈ K.faces, s.Nonempty ∧ ¬K.LocallyFiniteAt s | case pos.intro.intro.intro.intro
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : OrderedRing 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x✝ t✝ : E
s✝ t : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : DecidableEq E
x : E
hx : ¬{s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}.Finite
hxspace : x ∈ K.space
s : Finset E
hX : s ∈ K
hXhull : x ∈ (convexHull 𝕜) ↑s
hXbound : x ∉ combiFrontier 𝕜 s
hXunique : ∀ y ∈ K, x ∈ combiInterior 𝕜 y → y = s
⊢ ∃ s ∈ K.faces, s.Nonempty ∧ ¬K.LocallyFiniteAt s |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Finite.lean | Geometry.SimplicialComplex.locallyFinite_iff_mem_finitely_many_faces | [58, 1] | [82, 88] | refine'
⟨s, hX, Finset.nonempty_of_ne_empty _, fun hXlocallyfinite =>
hx <| hXlocallyfinite.subset fun t hY => ⟨hY.1, _⟩⟩ | case pos.intro.intro.intro.intro
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : OrderedRing 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x✝ t✝ : E
s✝ t : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : DecidableEq E
x : E
hx : ¬{s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}.Finite
hxspace : x ∈ K.space
s : Finset E
hX : s ∈ K
hXhull : x ∈ (convexHull 𝕜) ↑s
hXbound : x ∉ combiFrontier 𝕜 s
hXunique : ∀ y ∈ K, x ∈ combiInterior 𝕜 y → y = s
⊢ ∃ s ∈ K.faces, s.Nonempty ∧ ¬K.LocallyFiniteAt s | case pos.intro.intro.intro.intro.refine'_1
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : OrderedRing 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x✝ t✝ : E
s✝ t : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : DecidableEq E
x : E
hx : ¬{s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}.Finite
hxspace : x ∈ K.space
s : Finset E
hX : s ∈ K
hXhull : x ∈ (convexHull 𝕜) ↑s
hXbound : x ∉ combiFrontier 𝕜 s
hXunique : ∀ y ∈ K, x ∈ combiInterior 𝕜 y → y = s
⊢ s ≠ ∅
case pos.intro.intro.intro.intro.refine'_2
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : OrderedRing 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x✝ t✝¹ : E
s✝ t✝ : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : DecidableEq E
x : E
hx : ¬{s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}.Finite
hxspace : x ∈ K.space
s : Finset E
hX : s ∈ K
hXhull : x ∈ (convexHull 𝕜) ↑s
hXbound : x ∉ combiFrontier 𝕜 s
hXunique : ∀ y ∈ K, x ∈ combiInterior 𝕜 y → y = s
hXlocallyfinite : K.LocallyFiniteAt s
t : Finset E
hY : t ∈ {s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}
⊢ s ⊆ t |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Finite.lean | Geometry.SimplicialComplex.locallyFinite_iff_mem_finitely_many_faces | [58, 1] | [82, 88] | have hXYhull := K.inter_subset_convexHull hX hY.1 ⟨hXhull, hY.2⟩ | case pos.intro.intro.intro.intro.refine'_2
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : OrderedRing 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x✝ t✝¹ : E
s✝ t✝ : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : DecidableEq E
x : E
hx : ¬{s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}.Finite
hxspace : x ∈ K.space
s : Finset E
hX : s ∈ K
hXhull : x ∈ (convexHull 𝕜) ↑s
hXbound : x ∉ combiFrontier 𝕜 s
hXunique : ∀ y ∈ K, x ∈ combiInterior 𝕜 y → y = s
hXlocallyfinite : K.LocallyFiniteAt s
t : Finset E
hY : t ∈ {s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}
⊢ s ⊆ t | case pos.intro.intro.intro.intro.refine'_2
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : OrderedRing 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x✝ t✝¹ : E
s✝ t✝ : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : DecidableEq E
x : E
hx : ¬{s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}.Finite
hxspace : x ∈ K.space
s : Finset E
hX : s ∈ K
hXhull : x ∈ (convexHull 𝕜) ↑s
hXbound : x ∉ combiFrontier 𝕜 s
hXunique : ∀ y ∈ K, x ∈ combiInterior 𝕜 y → y = s
hXlocallyfinite : K.LocallyFiniteAt s
t : Finset E
hY : t ∈ {s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}
hXYhull : x ∈ (convexHull 𝕜) (↑s ∩ ↑t)
⊢ s ⊆ t |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Finite.lean | Geometry.SimplicialComplex.locallyFinite_iff_mem_finitely_many_faces | [58, 1] | [82, 88] | rw [← Finset.coe_inter] at hXYhull | case pos.intro.intro.intro.intro.refine'_2
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : OrderedRing 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x✝ t✝¹ : E
s✝ t✝ : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : DecidableEq E
x : E
hx : ¬{s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}.Finite
hxspace : x ∈ K.space
s : Finset E
hX : s ∈ K
hXhull : x ∈ (convexHull 𝕜) ↑s
hXbound : x ∉ combiFrontier 𝕜 s
hXunique : ∀ y ∈ K, x ∈ combiInterior 𝕜 y → y = s
hXlocallyfinite : K.LocallyFiniteAt s
t : Finset E
hY : t ∈ {s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}
hXYhull : x ∈ (convexHull 𝕜) (↑s ∩ ↑t)
⊢ s ⊆ t | case pos.intro.intro.intro.intro.refine'_2
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : OrderedRing 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x✝ t✝¹ : E
s✝ t✝ : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : DecidableEq E
x : E
hx : ¬{s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}.Finite
hxspace : x ∈ K.space
s : Finset E
hX : s ∈ K
hXhull : x ∈ (convexHull 𝕜) ↑s
hXbound : x ∉ combiFrontier 𝕜 s
hXunique : ∀ y ∈ K, x ∈ combiInterior 𝕜 y → y = s
hXlocallyfinite : K.LocallyFiniteAt s
t : Finset E
hY : t ∈ {s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}
hXYhull : x ∈ (convexHull 𝕜) ↑(s ∩ t)
⊢ s ⊆ t |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Finite.lean | Geometry.SimplicialComplex.locallyFinite_iff_mem_finitely_many_faces | [58, 1] | [82, 88] | by_contra hXY | case pos.intro.intro.intro.intro.refine'_2
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : OrderedRing 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x✝ t✝¹ : E
s✝ t✝ : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : DecidableEq E
x : E
hx : ¬{s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}.Finite
hxspace : x ∈ K.space
s : Finset E
hX : s ∈ K
hXhull : x ∈ (convexHull 𝕜) ↑s
hXbound : x ∉ combiFrontier 𝕜 s
hXunique : ∀ y ∈ K, x ∈ combiInterior 𝕜 y → y = s
hXlocallyfinite : K.LocallyFiniteAt s
t : Finset E
hY : t ∈ {s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}
hXYhull : x ∈ (convexHull 𝕜) ↑(s ∩ t)
⊢ s ⊆ t | case pos.intro.intro.intro.intro.refine'_2
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : OrderedRing 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x✝ t✝¹ : E
s✝ t✝ : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : DecidableEq E
x : E
hx : ¬{s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}.Finite
hxspace : x ∈ K.space
s : Finset E
hX : s ∈ K
hXhull : x ∈ (convexHull 𝕜) ↑s
hXbound : x ∉ combiFrontier 𝕜 s
hXunique : ∀ y ∈ K, x ∈ combiInterior 𝕜 y → y = s
hXlocallyfinite : K.LocallyFiniteAt s
t : Finset E
hY : t ∈ {s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}
hXYhull : x ∈ (convexHull 𝕜) ↑(s ∩ t)
hXY : ¬s ⊆ t
⊢ False |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Finite.lean | Geometry.SimplicialComplex.locallyFinite_iff_mem_finitely_many_faces | [58, 1] | [82, 88] | exact hXbound (mem_combiFrontier_iff.2 ⟨s ∩ t, ⟨Finset.inter_subset_left,
fun hXXY => hXY (Finset.subset_inter_iff.1 hXXY).2⟩, hXYhull⟩) | case pos.intro.intro.intro.intro.refine'_2
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : OrderedRing 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x✝ t✝¹ : E
s✝ t✝ : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : DecidableEq E
x : E
hx : ¬{s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}.Finite
hxspace : x ∈ K.space
s : Finset E
hX : s ∈ K
hXhull : x ∈ (convexHull 𝕜) ↑s
hXbound : x ∉ combiFrontier 𝕜 s
hXunique : ∀ y ∈ K, x ∈ combiInterior 𝕜 y → y = s
hXlocallyfinite : K.LocallyFiniteAt s
t : Finset E
hY : t ∈ {s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}
hXYhull : x ∈ (convexHull 𝕜) ↑(s ∩ t)
hXY : ¬s ⊆ t
⊢ False | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Finite.lean | Geometry.SimplicialComplex.locallyFinite_iff_mem_finitely_many_faces | [58, 1] | [82, 88] | rintro rfl | case pos.intro.intro.intro.intro.refine'_1
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : OrderedRing 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x✝ t✝ : E
s✝ t : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : DecidableEq E
x : E
hx : ¬{s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}.Finite
hxspace : x ∈ K.space
s : Finset E
hX : s ∈ K
hXhull : x ∈ (convexHull 𝕜) ↑s
hXbound : x ∉ combiFrontier 𝕜 s
hXunique : ∀ y ∈ K, x ∈ combiInterior 𝕜 y → y = s
⊢ s ≠ ∅ | case pos.intro.intro.intro.intro.refine'_1
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : OrderedRing 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x✝ t✝ : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : DecidableEq E
x : E
hx : ¬{s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}.Finite
hxspace : x ∈ K.space
hX : ∅ ∈ K
hXhull : x ∈ (convexHull 𝕜) ↑∅
hXbound : x ∉ combiFrontier 𝕜 ∅
hXunique : ∀ y ∈ K, x ∈ combiInterior 𝕜 y → y = ∅
⊢ False |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Finite.lean | Geometry.SimplicialComplex.locallyFinite_iff_mem_finitely_many_faces | [58, 1] | [82, 88] | simp at hXhull | case pos.intro.intro.intro.intro.refine'_1
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : OrderedRing 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x✝ t✝ : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : DecidableEq E
x : E
hx : ¬{s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}.Finite
hxspace : x ∈ K.space
hX : ∅ ∈ K
hXhull : x ∈ (convexHull 𝕜) ↑∅
hXbound : x ∉ combiFrontier 𝕜 ∅
hXunique : ∀ y ∈ K, x ∈ combiInterior 𝕜 y → y = ∅
⊢ False | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Finite.lean | Geometry.SimplicialComplex.locallyFinite_iff_mem_finitely_many_faces | [58, 1] | [82, 88] | refine (hx ?_).elim | case neg
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : OrderedRing 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x✝ t✝ : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : DecidableEq E
x : E
hx : ¬{s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}.Finite
hxspace : x ∉ K.space
⊢ ∃ s ∈ K.faces, s.Nonempty ∧ ¬K.LocallyFiniteAt s | case neg
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : OrderedRing 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x✝ t✝ : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : DecidableEq E
x : E
hx : ¬{s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}.Finite
hxspace : x ∉ K.space
⊢ {s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}.Finite |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Finite.lean | Geometry.SimplicialComplex.locallyFinite_iff_mem_finitely_many_faces | [58, 1] | [82, 88] | convert finite_empty | case neg
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : OrderedRing 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x✝ t✝ : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : DecidableEq E
x : E
hx : ¬{s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}.Finite
hxspace : x ∉ K.space
⊢ {s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}.Finite | case h.e'_2
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : OrderedRing 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x✝ t✝ : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : DecidableEq E
x : E
hx : ¬{s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}.Finite
hxspace : x ∉ K.space
⊢ {s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s} = ∅ |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Finite.lean | Geometry.SimplicialComplex.locallyFinite_iff_mem_finitely_many_faces | [58, 1] | [82, 88] | exact eq_empty_of_forall_not_mem fun s hX => hxspace <| mem_biUnion hX.1 hX.2 | case h.e'_2
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : OrderedRing 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x✝ t✝ : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : DecidableEq E
x : E
hx : ¬{s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}.Finite
hxspace : x ∉ K.space
⊢ {s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s} = ∅ | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Finite.lean | Geometry.SimplicialComplex.locallyFinite_iff_mem_finitely_many_faces | [58, 1] | [82, 88] | rintro hS s - ⟨x, hx⟩ | case mpr
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : OrderedRing 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x t✝ : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : DecidableEq E
⊢ (∀ (x : E), {s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}.Finite) → K.LocallyFinite | case mpr.intro
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : OrderedRing 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x✝ t✝ : E
s✝ t : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : DecidableEq E
hS : ∀ (x : E), {s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}.Finite
s : Finset E
x : E
hx : x ∈ s
⊢ K.LocallyFiniteAt s |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Finite.lean | Geometry.SimplicialComplex.locallyFinite_iff_mem_finitely_many_faces | [58, 1] | [82, 88] | exact (hS x).subset fun t => And.imp_right fun ht => subset_convexHull _ _ <| ht hx | case mpr.intro
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : OrderedRing 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x✝ t✝ : E
s✝ t : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : DecidableEq E
hS : ∀ (x : E), {s | s ∈ K.faces ∧ x ∈ (convexHull 𝕜) ↑s}.Finite
s : Finset E
x : E
hx : x ∈ s
⊢ K.LocallyFiniteAt s | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/ExampleSheets/Graph/ES1.lean | GraphTheory.ES1.q4 | [67, 1] | [70, 8] | cases nonempty_fintype α | ι : Type u_1
α : Type u_2
β : Type u_3
γ : Type u_4
inst✝¹ : Finite α
inst✝ : Nontrivial α
G : SimpleGraph α
hG : G.Connected
⊢ ∃ a, (⊤.deleteVerts {a}).coe.Connected | case intro
ι : Type u_1
α : Type u_2
β : Type u_3
γ : Type u_4
inst✝¹ : Finite α
inst✝ : Nontrivial α
G : SimpleGraph α
hG : G.Connected
val✝ : Fintype α
⊢ ∃ a, (⊤.deleteVerts {a}).coe.Connected |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/ExampleSheets/Graph/ES1.lean | GraphTheory.ES1.q4 | [67, 1] | [70, 8] | sorry | case intro
ι : Type u_1
α : Type u_2
β : Type u_3
γ : Type u_4
inst✝¹ : Finite α
inst✝ : Nontrivial α
G : SimpleGraph α
hG : G.Connected
val✝ : Fintype α
⊢ ∃ a, (⊤.deleteVerts {a}).coe.Connected | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/ExampleSheets/Graph/ES1.lean | GraphTheory.ES1.q5 | [79, 1] | [83, 8] | cases isEmpty_or_nonempty α | ι : Type u_1
α : Type u_2
β : Type u_3
γ : Type u_4
inst✝² : Fintype α
inst✝¹ : DecidableEq α
G : SimpleGraph α
inst✝ : DecidableRel G.Adj
hG : G.IsAcyclic
⊢ G.edgeFinset.card ≤ card α - 1 | case inl
ι : Type u_1
α : Type u_2
β : Type u_3
γ : Type u_4
inst✝² : Fintype α
inst✝¹ : DecidableEq α
G : SimpleGraph α
inst✝ : DecidableRel G.Adj
hG : G.IsAcyclic
h✝ : IsEmpty α
⊢ G.edgeFinset.card ≤ card α - 1
case inr
ι : Type u_1
α : Type u_2
β : Type u_3
γ : Type u_4
inst✝² : Fintype α
inst✝¹ : DecidableEq α
G : SimpleGraph α
inst✝ : DecidableRel G.Adj
hG : G.IsAcyclic
h✝ : Nonempty α
⊢ G.edgeFinset.card ≤ card α - 1 |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/ExampleSheets/Graph/ES1.lean | GraphTheory.ES1.q5 | [79, 1] | [83, 8] | sorry | case inr
ι : Type u_1
α : Type u_2
β : Type u_3
γ : Type u_4
inst✝² : Fintype α
inst✝¹ : DecidableEq α
G : SimpleGraph α
inst✝ : DecidableRel G.Adj
hG : G.IsAcyclic
h✝ : Nonempty α
⊢ G.edgeFinset.card ≤ card α - 1 | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/ExampleSheets/Graph/ES1.lean | GraphTheory.ES1.q5 | [79, 1] | [83, 8] | simp | case inl
ι : Type u_1
α : Type u_2
β : Type u_3
γ : Type u_4
inst✝² : Fintype α
inst✝¹ : DecidableEq α
G : SimpleGraph α
inst✝ : DecidableRel G.Adj
hG : G.IsAcyclic
h✝ : IsEmpty α
⊢ G.edgeFinset.card ≤ card α - 1 | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Pure.lean | Geometry.SimplicialComplex.Pure.exists_facet | [36, 1] | [36, 89] | sorry | 𝕜 : Type u_1
E : Type u_2
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
a b n k : ℕ
K : SimplicialComplex 𝕜 E
s : Finset E
hK : K.Pure n
hs : s ∈ K
⊢ ∃ t ∈ K.facets, s ⊆ t | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Pure.lean | Geometry.SimplicialComplex.Pure.exists_face_of_card_le | [38, 1] | [44, 10] | by_cases H : s ∈ K.facets | 𝕜 : Type u_1
E : Type u_2
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
a b n k : ℕ
K : SimplicialComplex 𝕜 E
s : Finset E
hK : K.Pure n
h : k ≤ n + 1
hs : s ∈ K
hcard : s.card ≤ k
⊢ ∃ t ∈ K, s ⊆ t ∧ t.card = k | case pos
𝕜 : Type u_1
E : Type u_2
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
a b n k : ℕ
K : SimplicialComplex 𝕜 E
s : Finset E
hK : K.Pure n
h : k ≤ n + 1
hs : s ∈ K
hcard : s.card ≤ k
H : s ∈ K.facets
⊢ ∃ t ∈ K, s ⊆ t ∧ t.card = k
case neg
𝕜 : Type u_1
E : Type u_2
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
a b n k : ℕ
K : SimplicialComplex 𝕜 E
s : Finset E
hK : K.Pure n
h : k ≤ n + 1
hs : s ∈ K
hcard : s.card ≤ k
H : s ∉ K.facets
⊢ ∃ t ∈ K, s ⊆ t ∧ t.card = k |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Pure.lean | Geometry.SimplicialComplex.Pure.exists_face_of_card_le | [38, 1] | [44, 10] | exact ⟨s, hs, Subset.rfl, hcard.antisymm <| h.trans (hK.2 H).ge⟩ | case pos
𝕜 : Type u_1
E : Type u_2
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
a b n k : ℕ
K : SimplicialComplex 𝕜 E
s : Finset E
hK : K.Pure n
h : k ≤ n + 1
hs : s ∈ K
hcard : s.card ≤ k
H : s ∈ K.facets
⊢ ∃ t ∈ K, s ⊆ t ∧ t.card = k | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Pure.lean | Geometry.SimplicialComplex.Pure.exists_face_of_card_le | [38, 1] | [44, 10] | unfold facets at H | case neg
𝕜 : Type u_1
E : Type u_2
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
a b n k : ℕ
K : SimplicialComplex 𝕜 E
s : Finset E
hK : K.Pure n
h : k ≤ n + 1
hs : s ∈ K
hcard : s.card ≤ k
H : s ∉ K.facets
⊢ ∃ t ∈ K, s ⊆ t ∧ t.card = k | case neg
𝕜 : Type u_1
E : Type u_2
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
a b n k : ℕ
K : SimplicialComplex 𝕜 E
s : Finset E
hK : K.Pure n
h : k ≤ n + 1
hs : s ∈ K
hcard : s.card ≤ k
H : s ∉ {s | s ∈ K.faces ∧ ∀ ⦃t : Finset E⦄, t ∈ K.faces → s ⊆ t → s = t}
⊢ ∃ t ∈ K, s ⊆ t ∧ t.card = k |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Pure.lean | Geometry.SimplicialComplex.Pure.exists_face_of_card_le | [38, 1] | [44, 10] | simp at H | case neg
𝕜 : Type u_1
E : Type u_2
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
a b n k : ℕ
K : SimplicialComplex 𝕜 E
s : Finset E
hK : K.Pure n
h : k ≤ n + 1
hs : s ∈ K
hcard : s.card ≤ k
H : s ∉ {s | s ∈ K.faces ∧ ∀ ⦃t : Finset E⦄, t ∈ K.faces → s ⊆ t → s = t}
⊢ ∃ t ∈ K, s ⊆ t ∧ t.card = k | case neg
𝕜 : Type u_1
E : Type u_2
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
a b n k : ℕ
K : SimplicialComplex 𝕜 E
s : Finset E
hK : K.Pure n
h : k ≤ n + 1
hs : s ∈ K
hcard : s.card ≤ k
H : s ∈ K → ∃ x ∈ K, s ⊆ x ∧ ¬s = x
⊢ ∃ t ∈ K, s ⊆ t ∧ t.card = k |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Pure.lean | Geometry.SimplicialComplex.Pure.exists_face_of_card_le | [38, 1] | [44, 10] | sorry | case neg
𝕜 : Type u_1
E : Type u_2
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
a b n k : ℕ
K : SimplicialComplex 𝕜 E
s : Finset E
hK : K.Pure n
h : k ≤ n + 1
hs : s ∈ K
hcard : s.card ≤ k
H : s ∈ K → ∃ x ∈ K, s ⊆ x ∧ ¬s = x
⊢ ∃ t ∈ K, s ⊆ t ∧ t.card = k | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Pure.lean | Geometry.SimplicialComplex.pure_unique | [46, 1] | [49, 59] | obtain ⟨s, hs⟩ := hK | 𝕜 : Type u_1
E : Type u_2
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
a b n k : ℕ
K : SimplicialComplex 𝕜 E
s : Finset E
hK : K.faces.Nonempty
ha : K.Pure a
hb : K.Pure b
⊢ a = b | case intro
𝕜 : Type u_1
E : Type u_2
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
a b n k : ℕ
K : SimplicialComplex 𝕜 E
s✝ : Finset E
ha : K.Pure a
hb : K.Pure b
s : Finset E
hs : s ∈ K.faces
⊢ a = b |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Pure.lean | Geometry.SimplicialComplex.pure_unique | [46, 1] | [49, 59] | obtain ⟨t, ht, -⟩ := ha.exists_facet hs | case intro
𝕜 : Type u_1
E : Type u_2
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
a b n k : ℕ
K : SimplicialComplex 𝕜 E
s✝ : Finset E
ha : K.Pure a
hb : K.Pure b
s : Finset E
hs : s ∈ K.faces
⊢ a = b | case intro.intro.intro
𝕜 : Type u_1
E : Type u_2
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
a b n k : ℕ
K : SimplicialComplex 𝕜 E
s✝ : Finset E
ha : K.Pure a
hb : K.Pure b
s : Finset E
hs : s ∈ K.faces
t : Finset E
ht : t ∈ K.facets
⊢ a = b |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Pure.lean | Geometry.SimplicialComplex.pure_unique | [46, 1] | [49, 59] | exact add_right_cancel ((ha.2 ht).symm.trans <| hb.2 ht) | case intro.intro.intro
𝕜 : Type u_1
E : Type u_2
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
a b n k : ℕ
K : SimplicialComplex 𝕜 E
s✝ : Finset E
ha : K.Pure a
hb : K.Pure b
s : Finset E
hs : s ∈ K.faces
t : Finset E
ht : t ∈ K.facets
⊢ a = b | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Pure.lean | Geometry.SimplicialComplex.pure_iff | [55, 1] | [64, 22] | refine' ⟨fun hK s hs => _, fun hK => ⟨fun s hs => _, fun s hs => _⟩⟩ | 𝕜 : Type u_1
E : Type u_2
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
a b n k : ℕ
K : SimplicialComplex 𝕜 E
s : Finset E
⊢ K.Pure n ↔ ∀ ⦃s : Finset E⦄, s ∈ K → ∃ t ∈ K, t.card = n + 1 ∧ s ⊆ t | case refine'_1
𝕜 : Type u_1
E : Type u_2
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
a b n k : ℕ
K : SimplicialComplex 𝕜 E
s✝ : Finset E
hK : K.Pure n
s : Finset E
hs : s ∈ K
⊢ ∃ t ∈ K, t.card = n + 1 ∧ s ⊆ t
case refine'_2
𝕜 : Type u_1
E : Type u_2
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
a b n k : ℕ
K : SimplicialComplex 𝕜 E
s✝ : Finset E
hK : ∀ ⦃s : Finset E⦄, s ∈ K → ∃ t ∈ K, t.card = n + 1 ∧ s ⊆ t
s : Finset E
hs : s ∈ K
⊢ s.card ≤ n + 1
case refine'_3
𝕜 : Type u_1
E : Type u_2
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
a b n k : ℕ
K : SimplicialComplex 𝕜 E
s✝ : Finset E
hK : ∀ ⦃s : Finset E⦄, s ∈ K → ∃ t ∈ K, t.card = n + 1 ∧ s ⊆ t
s : Finset E
hs : s ∈ K.facets
⊢ s.card = n + 1 |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Pure.lean | Geometry.SimplicialComplex.pure_iff | [55, 1] | [64, 22] | obtain ⟨t, ht, hst⟩ := hK.exists_facet hs | case refine'_1
𝕜 : Type u_1
E : Type u_2
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
a b n k : ℕ
K : SimplicialComplex 𝕜 E
s✝ : Finset E
hK : K.Pure n
s : Finset E
hs : s ∈ K
⊢ ∃ t ∈ K, t.card = n + 1 ∧ s ⊆ t | case refine'_1.intro.intro
𝕜 : Type u_1
E : Type u_2
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
a b n k : ℕ
K : SimplicialComplex 𝕜 E
s✝ : Finset E
hK : K.Pure n
s : Finset E
hs : s ∈ K
t : Finset E
ht : t ∈ K.facets
hst : s ⊆ t
⊢ ∃ t ∈ K, t.card = n + 1 ∧ s ⊆ t |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Pure.lean | Geometry.SimplicialComplex.pure_iff | [55, 1] | [64, 22] | exact ⟨t, ht.1, hK.2 ht, hst⟩ | case refine'_1.intro.intro
𝕜 : Type u_1
E : Type u_2
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
a b n k : ℕ
K : SimplicialComplex 𝕜 E
s✝ : Finset E
hK : K.Pure n
s : Finset E
hs : s ∈ K
t : Finset E
ht : t ∈ K.facets
hst : s ⊆ t
⊢ ∃ t ∈ K, t.card = n + 1 ∧ s ⊆ t | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Pure.lean | Geometry.SimplicialComplex.pure_iff | [55, 1] | [64, 22] | obtain ⟨t, _, htcard, hst⟩ := hK hs | case refine'_2
𝕜 : Type u_1
E : Type u_2
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
a b n k : ℕ
K : SimplicialComplex 𝕜 E
s✝ : Finset E
hK : ∀ ⦃s : Finset E⦄, s ∈ K → ∃ t ∈ K, t.card = n + 1 ∧ s ⊆ t
s : Finset E
hs : s ∈ K
⊢ s.card ≤ n + 1 | case refine'_2.intro.intro.intro
𝕜 : Type u_1
E : Type u_2
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
a b n k : ℕ
K : SimplicialComplex 𝕜 E
s✝ : Finset E
hK : ∀ ⦃s : Finset E⦄, s ∈ K → ∃ t ∈ K, t.card = n + 1 ∧ s ⊆ t
s : Finset E
hs : s ∈ K
t : Finset E
left✝ : t ∈ K
htcard : t.card = n + 1
hst : s ⊆ t
⊢ s.card ≤ n + 1 |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Pure.lean | Geometry.SimplicialComplex.pure_iff | [55, 1] | [64, 22] | exact (Finset.card_le_card hst).trans_eq htcard | case refine'_2.intro.intro.intro
𝕜 : Type u_1
E : Type u_2
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
a b n k : ℕ
K : SimplicialComplex 𝕜 E
s✝ : Finset E
hK : ∀ ⦃s : Finset E⦄, s ∈ K → ∃ t ∈ K, t.card = n + 1 ∧ s ⊆ t
s : Finset E
hs : s ∈ K
t : Finset E
left✝ : t ∈ K
htcard : t.card = n + 1
hst : s ⊆ t
⊢ s.card ≤ n + 1 | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Pure.lean | Geometry.SimplicialComplex.pure_iff | [55, 1] | [64, 22] | obtain ⟨t, ht, htcard, hst⟩ := hK hs.1 | case refine'_3
𝕜 : Type u_1
E : Type u_2
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
a b n k : ℕ
K : SimplicialComplex 𝕜 E
s✝ : Finset E
hK : ∀ ⦃s : Finset E⦄, s ∈ K → ∃ t ∈ K, t.card = n + 1 ∧ s ⊆ t
s : Finset E
hs : s ∈ K.facets
⊢ s.card = n + 1 | case refine'_3.intro.intro.intro
𝕜 : Type u_1
E : Type u_2
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
a b n k : ℕ
K : SimplicialComplex 𝕜 E
s✝ : Finset E
hK : ∀ ⦃s : Finset E⦄, s ∈ K → ∃ t ∈ K, t.card = n + 1 ∧ s ⊆ t
s : Finset E
hs : s ∈ K.facets
t : Finset E
ht : t ∈ K
htcard : t.card = n + 1
hst : s ⊆ t
⊢ s.card = n + 1 |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Pure.lean | Geometry.SimplicialComplex.pure_iff | [55, 1] | [64, 22] | rwa [hs.2 ht hst] | case refine'_3.intro.intro.intro
𝕜 : Type u_1
E : Type u_2
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
a b n k : ℕ
K : SimplicialComplex 𝕜 E
s✝ : Finset E
hK : ∀ ⦃s : Finset E⦄, s ∈ K → ∃ t ∈ K, t.card = n + 1 ∧ s ⊆ t
s : Finset E
hs : s ∈ K.facets
t : Finset E
ht : t ∈ K
htcard : t.card = n + 1
hst : s ⊆ t
⊢ s.card = n + 1 | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Pure.lean | Geometry.SimplicialComplex.facets_mono | [66, 1] | [70, 23] | refine' fun s hs => ⟨h hs.1, fun t ht hst => Finset.eq_of_subset_of_card_le hst _⟩ | 𝕜 : Type u_1
E : Type u_2
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
a b n k : ℕ
K : SimplicialComplex 𝕜 E
s : Finset E
K₁ K₂ : SimplicialComplex 𝕜 E
h : K₁ ≤ K₂
hK₁ : K₁.Pure n
hK₂ : K₂.Pure n
⊢ K₁.facets ⊆ K₂.facets | 𝕜 : Type u_1
E : Type u_2
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
a b n k : ℕ
K : SimplicialComplex 𝕜 E
s✝ : Finset E
K₁ K₂ : SimplicialComplex 𝕜 E
h : K₁ ≤ K₂
hK₁ : K₁.Pure n
hK₂ : K₂.Pure n
s : Finset E
hs : s ∈ K₁.facets
t : Finset E
ht : t ∈ K₂.faces
hst : s ⊆ t
⊢ t.card ≤ s.card |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Pure.lean | Geometry.SimplicialComplex.facets_mono | [66, 1] | [70, 23] | rw [hK₁.2 hs] | 𝕜 : Type u_1
E : Type u_2
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
a b n k : ℕ
K : SimplicialComplex 𝕜 E
s✝ : Finset E
K₁ K₂ : SimplicialComplex 𝕜 E
h : K₁ ≤ K₂
hK₁ : K₁.Pure n
hK₂ : K₂.Pure n
s : Finset E
hs : s ∈ K₁.facets
t : Finset E
ht : t ∈ K₂.faces
hst : s ⊆ t
⊢ t.card ≤ s.card | 𝕜 : Type u_1
E : Type u_2
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
a b n k : ℕ
K : SimplicialComplex 𝕜 E
s✝ : Finset E
K₁ K₂ : SimplicialComplex 𝕜 E
h : K₁ ≤ K₂
hK₁ : K₁.Pure n
hK₂ : K₂.Pure n
s : Finset E
hs : s ∈ K₁.facets
t : Finset E
ht : t ∈ K₂.faces
hst : s ⊆ t
⊢ t.card ≤ n + 1 |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Pure.lean | Geometry.SimplicialComplex.facets_mono | [66, 1] | [70, 23] | exact hK₂.card_le ht | 𝕜 : Type u_1
E : Type u_2
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
a b n k : ℕ
K : SimplicialComplex 𝕜 E
s✝ : Finset E
K₁ K₂ : SimplicialComplex 𝕜 E
h : K₁ ≤ K₂
hK₁ : K₁.Pure n
hK₂ : K₂.Pure n
s : Finset E
hs : s ∈ K₁.facets
t : Finset E
ht : t ∈ K₂.faces
hst : s ⊆ t
⊢ t.card ≤ n + 1 | 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 |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | mem_combiFrontier_iff | [36, 1] | [37, 97] | simp [combiFrontier] | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x : E
⊢ x ∈ combiFrontier 𝕜 s ↔ ∃ t ⊂ s, x ∈ (convexHull 𝕜) ↑t | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | combiFrontier_empty | [44, 1] | [47, 42] | apply Set.eq_empty_of_subset_empty | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x : E
⊢ combiFrontier 𝕜 ∅ = ∅ | case a
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x : E
⊢ combiFrontier 𝕜 ∅ ⊆ ∅ |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | combiFrontier_empty | [44, 1] | [47, 42] | convert combiFrontier_subset_convexHull | case a
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x : E
⊢ combiFrontier 𝕜 ∅ ⊆ ∅ | case h.e'_4
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x : E
⊢ ∅ = (convexHull 𝕜) ↑∅ |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | combiFrontier_empty | [44, 1] | [47, 42] | rw [Finset.coe_empty, convexHull_empty] | case h.e'_4
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x : E
⊢ ∅ = (convexHull 𝕜) ↑∅ | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | combiInterior_empty | [49, 1] | [52, 42] | apply Set.eq_empty_of_subset_empty | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x : E
⊢ combiInterior 𝕜 ∅ = ∅ | case a
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x : E
⊢ combiInterior 𝕜 ∅ ⊆ ∅ |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | combiInterior_empty | [49, 1] | [52, 42] | convert combiInterior_subset_convexHull | case a
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x : E
⊢ combiInterior 𝕜 ∅ ⊆ ∅ | case h.e'_4
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x : E
⊢ ∅ = (convexHull 𝕜) ↑∅ |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | combiInterior_empty | [49, 1] | [52, 42] | rw [Finset.coe_empty, convexHull_empty] | case h.e'_4
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x : E
⊢ ∅ = (convexHull 𝕜) ↑∅ | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | combiFrontier_singleton | [54, 1] | [59, 14] | refine eq_empty_of_subset_empty fun y hy ↦ ?_ | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x : E
⊢ combiFrontier 𝕜 {x} = ∅ | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x y : E
hy : y ∈ combiFrontier 𝕜 {x}
⊢ y ∈ ∅ |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | combiFrontier_singleton | [54, 1] | [59, 14] | rw [mem_combiFrontier_iff] at hy | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x y : E
hy : y ∈ combiFrontier 𝕜 {x}
⊢ y ∈ ∅ | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x y : E
hy : ∃ t ⊂ {x}, y ∈ (convexHull 𝕜) ↑t
⊢ y ∈ ∅ |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | combiFrontier_singleton | [54, 1] | [59, 14] | obtain ⟨s, hs, hys⟩ := hy | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x y : E
hy : ∃ t ⊂ {x}, y ∈ (convexHull 𝕜) ↑t
⊢ y ∈ ∅ | case intro.intro
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s✝ t : Finset E
x y : E
s : Finset E
hs : s ⊂ {x}
hys : y ∈ (convexHull 𝕜) ↑s
⊢ y ∈ ∅ |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | combiFrontier_singleton | [54, 1] | [59, 14] | rw [Finset.eq_empty_of_ssubset_singleton hs] at hys | case intro.intro
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s✝ t : Finset E
x y : E
s : Finset E
hs : s ⊂ {x}
hys : y ∈ (convexHull 𝕜) ↑s
⊢ y ∈ ∅ | case intro.intro
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s✝ t : Finset E
x y : E
s : Finset E
hs : s ⊂ {x}
hys : y ∈ (convexHull 𝕜) ↑∅
⊢ y ∈ ∅ |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | combiFrontier_singleton | [54, 1] | [59, 14] | simp at hys | case intro.intro
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s✝ t : Finset E
x y : E
s : Finset E
hs : s ⊂ {x}
hys : y ∈ (convexHull 𝕜) ↑∅
⊢ y ∈ ∅ | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | combiInterior_singleton | [61, 1] | [64, 7] | unfold combiInterior | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x : E
⊢ combiInterior 𝕜 {x} = {x} | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x : E
⊢ (convexHull 𝕜) ↑{x} \ combiFrontier 𝕜 {x} = {x} |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | combiInterior_singleton | [61, 1] | [64, 7] | rw [combiFrontier_singleton] | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x : E
⊢ (convexHull 𝕜) ↑{x} \ combiFrontier 𝕜 {x} = {x} | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x : E
⊢ (convexHull 𝕜) ↑{x} \ ∅ = {x} |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | combiInterior_singleton | [61, 1] | [64, 7] | simp | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x : E
⊢ (convexHull 𝕜) ↑{x} \ ∅ = {x} | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | simplex_combiInteriors_cover | [70, 1] | [82, 75] | apply Subset.antisymm _ _ | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x : E
⊢ (convexHull 𝕜) ↑s = ⋃ t, ⋃ (_ : t ⊆ s), combiInterior 𝕜 t | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x : E
⊢ (convexHull 𝕜) ↑s ⊆ ⋃ t, ⋃ (_ : t ⊆ s), combiInterior 𝕜 t
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x : E
⊢ ⋃ t, ⋃ (_ : t ⊆ s), combiInterior 𝕜 t ⊆ (convexHull 𝕜) ↑s |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | simplex_combiInteriors_cover | [70, 1] | [82, 75] | refine s.strongInductionOn ?_ | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x : E
⊢ (convexHull 𝕜) ↑s ⊆ ⋃ t, ⋃ (_ : t ⊆ s), combiInterior 𝕜 t | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x : E
⊢ ∀ (s : Finset E),
(∀ t ⊂ s, (convexHull 𝕜) ↑t ⊆ ⋃ t_1, ⋃ (_ : t_1 ⊆ t), combiInterior 𝕜 t_1) →
(convexHull 𝕜) ↑s ⊆ ⋃ t, ⋃ (_ : t ⊆ s), combiInterior 𝕜 t |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | simplex_combiInteriors_cover | [70, 1] | [82, 75] | rintro s ih x hx | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x : E
⊢ ∀ (s : Finset E),
(∀ t ⊂ s, (convexHull 𝕜) ↑t ⊆ ⋃ t_1, ⋃ (_ : t_1 ⊆ t), combiInterior 𝕜 t_1) →
(convexHull 𝕜) ↑s ⊆ ⋃ t, ⋃ (_ : t ⊆ s), combiInterior 𝕜 t | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s✝ t : Finset E
x✝ : E
s : Finset E
ih : ∀ t ⊂ s, (convexHull 𝕜) ↑t ⊆ ⋃ t_1, ⋃ (_ : t_1 ⊆ t), combiInterior 𝕜 t_1
x : E
hx : x ∈ (convexHull 𝕜) ↑s
⊢ x ∈ ⋃ t, ⋃ (_ : t ⊆ s), combiInterior 𝕜 t |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | simplex_combiInteriors_cover | [70, 1] | [82, 75] | by_cases h : x ∈ combiFrontier 𝕜 s | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s✝ t : Finset E
x✝ : E
s : Finset E
ih : ∀ t ⊂ s, (convexHull 𝕜) ↑t ⊆ ⋃ t_1, ⋃ (_ : t_1 ⊆ t), combiInterior 𝕜 t_1
x : E
hx : x ∈ (convexHull 𝕜) ↑s
⊢ x ∈ ⋃ t, ⋃ (_ : t ⊆ s), combiInterior 𝕜 t | case pos
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s✝ t : Finset E
x✝ : E
s : Finset E
ih : ∀ t ⊂ s, (convexHull 𝕜) ↑t ⊆ ⋃ t_1, ⋃ (_ : t_1 ⊆ t), combiInterior 𝕜 t_1
x : E
hx : x ∈ (convexHull 𝕜) ↑s
h : x ∈ combiFrontier 𝕜 s
⊢ x ∈ ⋃ t, ⋃ (_ : t ⊆ s), combiInterior 𝕜 t
case neg
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s✝ t : Finset E
x✝ : E
s : Finset E
ih : ∀ t ⊂ s, (convexHull 𝕜) ↑t ⊆ ⋃ t_1, ⋃ (_ : t_1 ⊆ t), combiInterior 𝕜 t_1
x : E
hx : x ∈ (convexHull 𝕜) ↑s
h : x ∉ combiFrontier 𝕜 s
⊢ x ∈ ⋃ t, ⋃ (_ : t ⊆ s), combiInterior 𝕜 t |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | simplex_combiInteriors_cover | [70, 1] | [82, 75] | rw [mem_combiFrontier_iff] at h | case pos
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s✝ t : Finset E
x✝ : E
s : Finset E
ih : ∀ t ⊂ s, (convexHull 𝕜) ↑t ⊆ ⋃ t_1, ⋃ (_ : t_1 ⊆ t), combiInterior 𝕜 t_1
x : E
hx : x ∈ (convexHull 𝕜) ↑s
h : x ∈ combiFrontier 𝕜 s
⊢ x ∈ ⋃ t, ⋃ (_ : t ⊆ s), combiInterior 𝕜 t | case pos
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s✝ t : Finset E
x✝ : E
s : Finset E
ih : ∀ t ⊂ s, (convexHull 𝕜) ↑t ⊆ ⋃ t_1, ⋃ (_ : t_1 ⊆ t), combiInterior 𝕜 t_1
x : E
hx : x ∈ (convexHull 𝕜) ↑s
h : ∃ t ⊂ s, x ∈ (convexHull 𝕜) ↑t
⊢ x ∈ ⋃ t, ⋃ (_ : t ⊆ s), combiInterior 𝕜 t |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | simplex_combiInteriors_cover | [70, 1] | [82, 75] | obtain ⟨t, st, ht⟩ := h | case pos
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s✝ t : Finset E
x✝ : E
s : Finset E
ih : ∀ t ⊂ s, (convexHull 𝕜) ↑t ⊆ ⋃ t_1, ⋃ (_ : t_1 ⊆ t), combiInterior 𝕜 t_1
x : E
hx : x ∈ (convexHull 𝕜) ↑s
h : ∃ t ⊂ s, x ∈ (convexHull 𝕜) ↑t
⊢ x ∈ ⋃ t, ⋃ (_ : t ⊆ s), combiInterior 𝕜 t | case pos.intro.intro
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s✝ t✝ : Finset E
x✝ : E
s : Finset E
ih : ∀ t ⊂ s, (convexHull 𝕜) ↑t ⊆ ⋃ t_1, ⋃ (_ : t_1 ⊆ t), combiInterior 𝕜 t_1
x : E
hx : x ∈ (convexHull 𝕜) ↑s
t : Finset E
st : t ⊂ s
ht : x ∈ (convexHull 𝕜) ↑t
⊢ x ∈ ⋃ t, ⋃ (_ : t ⊆ s), combiInterior 𝕜 t |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | simplex_combiInteriors_cover | [70, 1] | [82, 75] | specialize ih _ st ht | case pos.intro.intro
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s✝ t✝ : Finset E
x✝ : E
s : Finset E
ih : ∀ t ⊂ s, (convexHull 𝕜) ↑t ⊆ ⋃ t_1, ⋃ (_ : t_1 ⊆ t), combiInterior 𝕜 t_1
x : E
hx : x ∈ (convexHull 𝕜) ↑s
t : Finset E
st : t ⊂ s
ht : x ∈ (convexHull 𝕜) ↑t
⊢ x ∈ ⋃ t, ⋃ (_ : t ⊆ s), combiInterior 𝕜 t | case pos.intro.intro
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s✝ t✝ : Finset E
x✝ : E
s : Finset E
x : E
hx : x ∈ (convexHull 𝕜) ↑s
t : Finset E
st : t ⊂ s
ht : x ∈ (convexHull 𝕜) ↑t
ih : x ∈ ⋃ t_1, ⋃ (_ : t_1 ⊆ t), combiInterior 𝕜 t_1
⊢ x ∈ ⋃ t, ⋃ (_ : t ⊆ s), combiInterior 𝕜 t |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | simplex_combiInteriors_cover | [70, 1] | [82, 75] | simp only [exists_prop, Set.mem_iUnion] at ih ⊢ | case pos.intro.intro
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s✝ t✝ : Finset E
x✝ : E
s : Finset E
x : E
hx : x ∈ (convexHull 𝕜) ↑s
t : Finset E
st : t ⊂ s
ht : x ∈ (convexHull 𝕜) ↑t
ih : x ∈ ⋃ t_1, ⋃ (_ : t_1 ⊆ t), combiInterior 𝕜 t_1
⊢ x ∈ ⋃ t, ⋃ (_ : t ⊆ s), combiInterior 𝕜 t | case pos.intro.intro
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s✝ t✝ : Finset E
x✝ : E
s : Finset E
x : E
hx : x ∈ (convexHull 𝕜) ↑s
t : Finset E
st : t ⊂ s
ht : x ∈ (convexHull 𝕜) ↑t
ih : ∃ i ⊆ t, x ∈ combiInterior 𝕜 i
⊢ ∃ i ⊆ s, x ∈ combiInterior 𝕜 i |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | simplex_combiInteriors_cover | [70, 1] | [82, 75] | obtain ⟨Z, Zt, hZ⟩ := ih | case pos.intro.intro
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s✝ t✝ : Finset E
x✝ : E
s : Finset E
x : E
hx : x ∈ (convexHull 𝕜) ↑s
t : Finset E
st : t ⊂ s
ht : x ∈ (convexHull 𝕜) ↑t
ih : ∃ i ⊆ t, x ∈ combiInterior 𝕜 i
⊢ ∃ i ⊆ s, x ∈ combiInterior 𝕜 i | case pos.intro.intro.intro.intro
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s✝ t✝ : Finset E
x✝ : E
s : Finset E
x : E
hx : x ∈ (convexHull 𝕜) ↑s
t : Finset E
st : t ⊂ s
ht : x ∈ (convexHull 𝕜) ↑t
Z : Finset E
Zt : Z ⊆ t
hZ : x ∈ combiInterior 𝕜 Z
⊢ ∃ i ⊆ s, x ∈ combiInterior 𝕜 i |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | simplex_combiInteriors_cover | [70, 1] | [82, 75] | exact ⟨_, Zt.trans st.1, hZ⟩ | case pos.intro.intro.intro.intro
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s✝ t✝ : Finset E
x✝ : E
s : Finset E
x : E
hx : x ∈ (convexHull 𝕜) ↑s
t : Finset E
st : t ⊂ s
ht : x ∈ (convexHull 𝕜) ↑t
Z : Finset E
Zt : Z ⊆ t
hZ : x ∈ combiInterior 𝕜 Z
⊢ ∃ i ⊆ s, x ∈ combiInterior 𝕜 i | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | simplex_combiInteriors_cover | [70, 1] | [82, 75] | exact subset_iUnion₂ s Subset.rfl ⟨hx, h⟩ | case neg
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s✝ t : Finset E
x✝ : E
s : Finset E
ih : ∀ t ⊂ s, (convexHull 𝕜) ↑t ⊆ ⋃ t_1, ⋃ (_ : t_1 ⊆ t), combiInterior 𝕜 t_1
x : E
hx : x ∈ (convexHull 𝕜) ↑s
h : x ∉ combiFrontier 𝕜 s
⊢ x ∈ ⋃ t, ⋃ (_ : t ⊆ s), combiInterior 𝕜 t | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | simplex_combiInteriors_cover | [70, 1] | [82, 75] | exact iUnion₂_subset fun t ht ↦ diff_subset.trans $ convexHull_mono ht | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
s t : Finset E
x : E
⊢ ⋃ t, ⋃ (_ : t ⊆ s), combiInterior 𝕜 t ⊆ (convexHull 𝕜) ↑s | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | combiFrontier_eq | [90, 1] | [135, 14] | ext 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
⊢ combiFrontier 𝕜 s =
{x | ∃ w, ∃ (_ : ∀ y ∈ s, 0 ≤ w y) (_ : ∑ y ∈ s, w y = 1) (_ : ∃ y ∈ s, w y = 0), s.centerMass w id = x} | case h
𝕜 : 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 ∈ combiFrontier 𝕜 s ↔
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 | combiFrontier_eq | [90, 1] | [135, 14] | simp_rw [combiFrontier, Set.mem_iUnion, Set.mem_setOf_eq] | case h
𝕜 : 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 ∈ combiFrontier 𝕜 s ↔
x ∈ {x | ∃ w, ∃ (_ : ∀ y ∈ s, 0 ≤ w y) (_ : ∑ y ∈ s, w y = 1) (_ : ∃ y ∈ s, w y = 0), s.centerMass w id = x} | case h
𝕜 : 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
⊢ (∃ i, ∃ (_ : i ⊂ s), x ∈ (convexHull 𝕜) ↑i) ↔
∃ 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 | combiFrontier_eq | [90, 1] | [135, 14] | constructor | case h
𝕜 : 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
⊢ (∃ i, ∃ (_ : i ⊂ s), x ∈ (convexHull 𝕜) ↑i) ↔
∃ w, ∃ (_ : ∀ y ∈ s, 0 ≤ w y) (_ : ∑ y ∈ s, w y = 1) (_ : ∃ y ∈ s, w y = 0), s.centerMass w id = x | case h.mp
𝕜 : 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
⊢ (∃ i, ∃ (_ : i ⊂ s), x ∈ (convexHull 𝕜) ↑i) →
∃ w, ∃ (_ : ∀ y ∈ s, 0 ≤ w y) (_ : ∑ y ∈ s, w y = 1) (_ : ∃ y ∈ s, w y = 0), s.centerMass w id = x
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 |
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.mp
𝕜 : 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
⊢ (∃ i, ∃ (_ : i ⊂ s), x ∈ (convexHull 𝕜) ↑i) →
∃ w, ∃ (_ : ∀ y ∈ s, 0 ≤ w y) (_ : ∑ y ∈ s, w y = 1) (_ : ∃ y ∈ s, w y = 0), s.centerMass w id = x | case h.mp
𝕜 : 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 ⊂ s,
x ∈ (convexHull 𝕜) ↑x_1 → ∃ 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 | combiFrontier_eq | [90, 1] | [135, 14] | intro t ts hx | case h.mp
𝕜 : 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 ⊂ s,
x ∈ (convexHull 𝕜) ↑x_1 → ∃ w, (∀ y ∈ s, 0 ≤ w y) ∧ ∑ y ∈ s, w y = 1 ∧ (∃ y ∈ s, w y = 0) ∧ s.centerMass w id = x | case h.mp
𝕜 : 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
t : Finset E
ts : t ⊂ s
hx : x ∈ (convexHull 𝕜) ↑t
⊢ ∃ 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 | combiFrontier_eq | [90, 1] | [135, 14] | rw [Finset.convexHull_eq, Set.mem_setOf_eq] at hx | case h.mp
𝕜 : 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
t : Finset E
ts : t ⊂ s
hx : x ∈ (convexHull 𝕜) ↑t
⊢ ∃ w, (∀ y ∈ s, 0 ≤ w y) ∧ ∑ y ∈ s, w y = 1 ∧ (∃ y ∈ s, w y = 0) ∧ s.centerMass w id = x | case h.mp
𝕜 : 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
t : Finset E
ts : t ⊂ s
hx : ∃ w, (∀ y ∈ t, 0 ≤ w y) ∧ ∑ y ∈ t, w y = 1 ∧ t.centerMass w id = 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 | combiFrontier_eq | [90, 1] | [135, 14] | rcases hx with ⟨w, hw₀, hw₁, hx⟩ | case h.mp
𝕜 : 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
t : Finset E
ts : t ⊂ s
hx : ∃ w, (∀ y ∈ t, 0 ≤ w y) ∧ ∑ y ∈ t, w y = 1 ∧ t.centerMass w id = x
⊢ ∃ w, (∀ y ∈ s, 0 ≤ w y) ∧ ∑ y ∈ s, w y = 1 ∧ (∃ y ∈ s, w y = 0) ∧ s.centerMass w id = x | case h.mp.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✝ x : E
t : Finset E
ts : t ⊂ s
w : E → 𝕜
hw₀ : ∀ y ∈ t, 0 ≤ w y
hw₁ : ∑ y ∈ t, w y = 1
hx : t.centerMass w id = 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 | combiFrontier_eq | [90, 1] | [135, 14] | rcases Finset.exists_of_ssubset ts with ⟨y, hys, hyt⟩ | case h.mp.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✝ x : E
t : Finset E
ts : t ⊂ s
w : E → 𝕜
hw₀ : ∀ y ∈ t, 0 ≤ w y
hw₁ : ∑ y ∈ t, w y = 1
hx : t.centerMass w id = x
⊢ ∃ w, (∀ y ∈ s, 0 ≤ w y) ∧ ∑ y ∈ s, w y = 1 ∧ (∃ y ∈ s, w y = 0) ∧ s.centerMass w id = x | case h.mp.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✝ x : E
t : Finset E
ts : t ⊂ s
w : E → 𝕜
hw₀ : ∀ y ∈ t, 0 ≤ w y
hw₁ : ∑ y ∈ t, w y = 1
hx : t.centerMass w id = x
y : E
hys : y ∈ s
hyt : y ∉ t
⊢ ∃ 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 | combiFrontier_eq | [90, 1] | [135, 14] | let w' z := if z ∈ t then w z else 0 | case h.mp.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✝ x : E
t : Finset E
ts : t ⊂ s
w : E → 𝕜
hw₀ : ∀ y ∈ t, 0 ≤ w y
hw₁ : ∑ y ∈ t, w y = 1
hx : t.centerMass w id = x
y : E
hys : y ∈ s
hyt : y ∉ t
⊢ ∃ w, (∀ y ∈ s, 0 ≤ w y) ∧ ∑ y ∈ s, w y = 1 ∧ (∃ y ∈ s, w y = 0) ∧ s.centerMass w id = x | case h.mp.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✝ x : E
t : Finset E
ts : t ⊂ s
w : E → 𝕜
hw₀ : ∀ y ∈ t, 0 ≤ w y
hw₁ : ∑ y ∈ t, w y = 1
hx : t.centerMass w id = x
y : E
hys : y ∈ s
hyt : y ∉ t
w' : E → 𝕜 := fun z => if z ∈ t then w z else 0
⊢ ∃ 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 | combiFrontier_eq | [90, 1] | [135, 14] | have hw'₁ : s.sum w' = 1 := by
rwa [← Finset.sum_subset ts.1, Finset.sum_extend_by_zero]
simp only [ite_eq_right_iff]
tauto | case h.mp.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✝ x : E
t : Finset E
ts : t ⊂ s
w : E → 𝕜
hw₀ : ∀ y ∈ t, 0 ≤ w y
hw₁ : ∑ y ∈ t, w y = 1
hx : t.centerMass w id = x
y : E
hys : y ∈ s
hyt : y ∉ t
w' : E → 𝕜 := fun z => if z ∈ t then w z else 0
⊢ ∃ w, (∀ y ∈ s, 0 ≤ w y) ∧ ∑ y ∈ s, w y = 1 ∧ (∃ y ∈ s, w y = 0) ∧ s.centerMass w id = x | case h.mp.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✝ x : E
t : Finset E
ts : t ⊂ s
w : E → 𝕜
hw₀ : ∀ y ∈ t, 0 ≤ w y
hw₁ : ∑ y ∈ t, w y = 1
hx : t.centerMass w id = x
y : E
hys : y ∈ s
hyt : y ∉ t
w' : E → 𝕜 := fun z => if z ∈ t then w z else 0
hw'₁ : s.sum w' = 1
⊢ ∃ 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 | combiFrontier_eq | [90, 1] | [135, 14] | refine' ⟨w', _, hw'₁, ⟨_, ‹y ∈ s›, _⟩, _⟩ | case h.mp.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✝ x : E
t : Finset E
ts : t ⊂ s
w : E → 𝕜
hw₀ : ∀ y ∈ t, 0 ≤ w y
hw₁ : ∑ y ∈ t, w y = 1
hx : t.centerMass w id = x
y : E
hys : y ∈ s
hyt : y ∉ t
w' : E → 𝕜 := fun z => if z ∈ t then w z else 0
hw'₁ : s.sum w' = 1
⊢ ∃ w, (∀ y ∈ s, 0 ≤ w y) ∧ ∑ y ∈ s, w y = 1 ∧ (∃ y ∈ s, w y = 0) ∧ s.centerMass w id = x | case h.mp.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✝ x : E
t : Finset E
ts : t ⊂ s
w : E → 𝕜
hw₀ : ∀ y ∈ t, 0 ≤ w y
hw₁ : ∑ y ∈ t, w y = 1
hx : t.centerMass w id = x
y : E
hys : y ∈ s
hyt : y ∉ t
w' : E → 𝕜 := fun z => if z ∈ t then w z else 0
hw'₁ : s.sum w' = 1
⊢ ∀ y ∈ s, 0 ≤ w' y
case h.mp.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✝ x : E
t : Finset E
ts : t ⊂ s
w : E → 𝕜
hw₀ : ∀ y ∈ t, 0 ≤ w y
hw₁ : ∑ y ∈ t, w y = 1
hx : t.centerMass w id = x
y : E
hys : y ∈ s
hyt : y ∉ t
w' : E → 𝕜 := fun z => if z ∈ t then w z else 0
hw'₁ : s.sum w' = 1
⊢ w' y = 0
case h.mp.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✝ x : E
t : Finset E
ts : t ⊂ s
w : E → 𝕜
hw₀ : ∀ y ∈ t, 0 ≤ w y
hw₁ : ∑ y ∈ t, w y = 1
hx : t.centerMass w id = x
y : E
hys : y ∈ s
hyt : y ∉ t
w' : E → 𝕜 := fun z => if z ∈ t then w z else 0
hw'₁ : s.sum w' = 1
⊢ s.centerMass w' id = x |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | combiFrontier_eq | [90, 1] | [135, 14] | rw [← Finset.centerMass_subset id ts.1] | case h.mp.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✝ x : E
t : Finset E
ts : t ⊂ s
w : E → 𝕜
hw₀ : ∀ y ∈ t, 0 ≤ w y
hw₁ : ∑ y ∈ t, w y = 1
hx : t.centerMass w id = x
y : E
hys : y ∈ s
hyt : y ∉ t
w' : E → 𝕜 := fun z => if z ∈ t then w z else 0
hw'₁ : s.sum w' = 1
⊢ s.centerMass w' id = x | case h.mp.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✝ x : E
t : Finset E
ts : t ⊂ s
w : E → 𝕜
hw₀ : ∀ y ∈ t, 0 ≤ w y
hw₁ : ∑ y ∈ t, w y = 1
hx : t.centerMass w id = x
y : E
hys : y ∈ s
hyt : y ∉ t
w' : E → 𝕜 := fun z => if z ∈ t then w z else 0
hw'₁ : s.sum w' = 1
⊢ t.centerMass w' id = x
case h.mp.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✝ x : E
t : Finset E
ts : t ⊂ s
w : E → 𝕜
hw₀ : ∀ y ∈ t, 0 ≤ w y
hw₁ : ∑ y ∈ t, w y = 1
hx : t.centerMass w id = x
y : E
hys : y ∈ s
hyt : y ∉ t
w' : E → 𝕜 := fun z => if z ∈ t then w z else 0
hw'₁ : s.sum w' = 1
⊢ ∀ i ∈ s, i ∉ t → w' i = 0 |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | combiFrontier_eq | [90, 1] | [135, 14] | exact fun i _ hi => if_neg hi | case h.mp.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✝ x : E
t : Finset E
ts : t ⊂ s
w : E → 𝕜
hw₀ : ∀ y ∈ t, 0 ≤ w y
hw₁ : ∑ y ∈ t, w y = 1
hx : t.centerMass w id = x
y : E
hys : y ∈ s
hyt : y ∉ t
w' : E → 𝕜 := fun z => if z ∈ t then w z else 0
hw'₁ : s.sum w' = 1
⊢ ∀ i ∈ s, i ∉ t → w' i = 0 | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | combiFrontier_eq | [90, 1] | [135, 14] | rwa [← Finset.sum_subset ts.1, Finset.sum_extend_by_zero] | 𝕜 : 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
t : Finset E
ts : t ⊂ s
w : E → 𝕜
hw₀ : ∀ y ∈ t, 0 ≤ w y
hw₁ : ∑ y ∈ t, w y = 1
hx : t.centerMass w id = x
y : E
hys : y ∈ s
hyt : y ∉ t
w' : E → 𝕜 := fun z => if z ∈ t then w z else 0
⊢ s.sum w' = 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
t : Finset E
ts : t ⊂ s
w : E → 𝕜
hw₀ : ∀ y ∈ t, 0 ≤ w y
hw₁ : ∑ y ∈ t, w y = 1
hx : t.centerMass w id = x
y : E
hys : y ∈ s
hyt : y ∉ t
w' : E → 𝕜 := fun z => if z ∈ t then w z else 0
⊢ ∀ x ∈ s, x ∉ t → (if x ∈ t then w x else 0) = 0 |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | combiFrontier_eq | [90, 1] | [135, 14] | simp only [ite_eq_right_iff] | 𝕜 : 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
t : Finset E
ts : t ⊂ s
w : E → 𝕜
hw₀ : ∀ y ∈ t, 0 ≤ w y
hw₁ : ∑ y ∈ t, w y = 1
hx : t.centerMass w id = x
y : E
hys : y ∈ s
hyt : y ∉ t
w' : E → 𝕜 := fun z => if z ∈ t then w z else 0
⊢ ∀ x ∈ s, x ∉ t → (if x ∈ t then w x else 0) = 0 | 𝕜 : 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
t : Finset E
ts : t ⊂ s
w : E → 𝕜
hw₀ : ∀ y ∈ t, 0 ≤ w y
hw₁ : ∑ y ∈ t, w y = 1
hx : t.centerMass w id = x
y : E
hys : y ∈ s
hyt : y ∉ t
w' : E → 𝕜 := fun z => if z ∈ t then w z else 0
⊢ ∀ x ∈ s, x ∉ t → x ∈ t → w x = 0 |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SimplicialComplex/Simplex.lean | combiFrontier_eq | [90, 1] | [135, 14] | tauto | 𝕜 : 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
t : Finset E
ts : t ⊂ s
w : E → 𝕜
hw₀ : ∀ y ∈ t, 0 ≤ w y
hw₁ : ∑ y ∈ t, w y = 1
hx : t.centerMass w id = x
y : E
hys : y ∈ s
hyt : y ∉ t
w' : E → 𝕜 := fun z => if z ∈ t then w z else 0
⊢ ∀ x ∈ s, x ∉ t → x ∈ t → w x = 0 | no goals |
Subsets and Splits
No community queries yet
The top public SQL queries from the community will appear here once available.