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/SylvesterChvatal.lean | one_implies_two | [153, 1] | [194, 30] | ring | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z : V
h✝ : ∃ x y z, NotCollinear x y z
S : Set (V × V × V) := {(a, b, c) | NotCollinear a b c}
this✝ : S.Nonempty
f : V × V × V → ℝ :=
fun x =>
match x with
| (a, b, c) => dist a b + dist b c + dist c a
a b c : V
h₁ : NotCollinear a b c
h₂ : ∀ (a' b' c' : V), NotCollinear a' b' c' → dist a b + dist b c + dist c a ≤ dist a' b' + dist b' c' + dist c' a'
cont : ∀ (x y z : V), SimpleEdges.Adj x y → SimpleEdges.Adj y z → SimpleEdges.Adj z x → ¬NotCollinear x y z
this :
∀ (a b c : V),
NotCollinear a b c →
(∀ (a' b' c' : V),
NotCollinear a' b' c' → dist a b + dist b c + dist c a ≤ dist a' b' + dist b' c' + dist c' a') →
¬SimpleEdges.Adj a b → False
hab : SimpleEdges.Adj a b
x✝² x✝¹ x✝ : V
h : NotCollinear x✝² x✝¹ x✝
⊢ dist c a + dist a b + dist b c = dist a b + dist b c + dist c a | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | one_implies_two | [153, 1] | [194, 30] | simp [left_mem_Line, right_mem_Line, hc] | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z : V
h : ∃ x y z, NotCollinear x y z
S : Set (V × V × V) := {(a, b, c) | NotCollinear a b c}
this : S.Nonempty
f : V × V × V → ℝ :=
fun x =>
match x with
| (a, b, c) => dist a b + dist b c + dist c a
cont : ∀ (x y z : V), SimpleEdges.Adj x y → SimpleEdges.Adj y z → SimpleEdges.Adj z x → ¬NotCollinear x y z
a b c : V
h₁ : NotCollinear a b c
h₂ : ∀ (a' b' c' : V), NotCollinear a' b' c' → dist a b + dist b c + dist c a ≤ dist a' b' + dist b' c' + dist c' a'
d : V
adb : sbtw a d b
hc : c ∈ Line a b
⊢ {a, b, c} ⊆ Line a b | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | one_implies_two | [153, 1] | [194, 30] | by_contra! | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z : V
h : ∃ x y z, NotCollinear x y z
S : Set (V × V × V) := {(a, b, c) | NotCollinear a b c}
this : S.Nonempty
f : V × V × V → ℝ :=
fun x =>
match x with
| (a, b, c) => dist a b + dist b c + dist c a
cont : ∀ (x y z : V), SimpleEdges.Adj x y → SimpleEdges.Adj y z → SimpleEdges.Adj z x → ¬NotCollinear x y z
a b c : V
h₁ : NotCollinear a b c
h₂ : ∀ (a' b' c' : V), NotCollinear a' b' c' → dist a b + dist b c + dist c a ≤ dist a' b' + dist b' c' + dist c' a'
d : V
adb : sbtw a d b
habc : c ∉ Line a b
hdab : d ∈ Line a b
hcd : c ≠ d
⊢ dist d c < dist d b + dist b c | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z : V
h : ∃ x y z, NotCollinear x y z
S : Set (V × V × V) := {(a, b, c) | NotCollinear a b c}
this✝ : S.Nonempty
f : V × V × V → ℝ :=
fun x =>
match x with
| (a, b, c) => dist a b + dist b c + dist c a
cont : ∀ (x y z : V), SimpleEdges.Adj x y → SimpleEdges.Adj y z → SimpleEdges.Adj z x → ¬NotCollinear x y z
a b c : V
h₁ : NotCollinear a b c
h₂ : ∀ (a' b' c' : V), NotCollinear a' b' c' → dist a b + dist b c + dist c a ≤ dist a' b' + dist b' c' + dist c' a'
d : V
adb : sbtw a d b
habc : c ∉ Line a b
hdab : d ∈ Line a b
hcd : c ≠ d
this : dist d b + dist b c ≤ dist d c
⊢ False |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | one_implies_two | [153, 1] | [194, 30] | refine habc (generateLine_close_right hdab right_mem_Line ?_) | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z : V
h : ∃ x y z, NotCollinear x y z
S : Set (V × V × V) := {(a, b, c) | NotCollinear a b c}
this✝ : S.Nonempty
f : V × V × V → ℝ :=
fun x =>
match x with
| (a, b, c) => dist a b + dist b c + dist c a
cont : ∀ (x y z : V), SimpleEdges.Adj x y → SimpleEdges.Adj y z → SimpleEdges.Adj z x → ¬NotCollinear x y z
a b c : V
h₁ : NotCollinear a b c
h₂ : ∀ (a' b' c' : V), NotCollinear a' b' c' → dist a b + dist b c + dist c a ≤ dist a' b' + dist b' c' + dist c' a'
d : V
adb : sbtw a d b
habc : c ∉ Line a b
hdab : d ∈ Line a b
hcd : c ≠ d
this : dist d b + dist b c ≤ dist d c
⊢ False | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z : V
h : ∃ x y z, NotCollinear x y z
S : Set (V × V × V) := {(a, b, c) | NotCollinear a b c}
this✝ : S.Nonempty
f : V × V × V → ℝ :=
fun x =>
match x with
| (a, b, c) => dist a b + dist b c + dist c a
cont : ∀ (x y z : V), SimpleEdges.Adj x y → SimpleEdges.Adj y z → SimpleEdges.Adj z x → ¬NotCollinear x y z
a b c : V
h₁ : NotCollinear a b c
h₂ : ∀ (a' b' c' : V), NotCollinear a' b' c' → dist a b + dist b c + dist c a ≤ dist a' b' + dist b' c' + dist c' a'
d : V
adb : sbtw a d b
habc : c ∉ Line a b
hdab : d ∈ Line a b
hcd : c ≠ d
this : dist d b + dist b c ≤ dist d c
⊢ sbtw d b c |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | one_implies_two | [153, 1] | [194, 30] | exact ⟨adb.ne23, hcd.symm, h₁.2.2.1, this.antisymm (dist_triangle _ _ _)⟩ | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z : V
h : ∃ x y z, NotCollinear x y z
S : Set (V × V × V) := {(a, b, c) | NotCollinear a b c}
this✝ : S.Nonempty
f : V × V × V → ℝ :=
fun x =>
match x with
| (a, b, c) => dist a b + dist b c + dist c a
cont : ∀ (x y z : V), SimpleEdges.Adj x y → SimpleEdges.Adj y z → SimpleEdges.Adj z x → ¬NotCollinear x y z
a b c : V
h₁ : NotCollinear a b c
h₂ : ∀ (a' b' c' : V), NotCollinear a' b' c' → dist a b + dist b c + dist c a ≤ dist a' b' + dist b' c' + dist c' a'
d : V
adb : sbtw a d b
habc : c ∉ Line a b
hdab : d ∈ Line a b
hcd : c ≠ d
this : dist d b + dist b c ≤ dist d c
⊢ sbtw d b c | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | one_implies_two | [153, 1] | [194, 30] | linarith only [this, adb.2.2.2] | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z : V
h : ∃ x y z, NotCollinear x y z
S : Set (V × V × V) := {(a, b, c) | NotCollinear a b c}
this✝ : S.Nonempty
f : V × V × V → ℝ :=
fun x =>
match x with
| (a, b, c) => dist a b + dist b c + dist c a
cont : ∀ (x y z : V), SimpleEdges.Adj x y → SimpleEdges.Adj y z → SimpleEdges.Adj z x → ¬NotCollinear x y z
a b c : V
h₁ : NotCollinear a b c
h₂ : ∀ (a' b' c' : V), NotCollinear a' b' c' → dist a b + dist b c + dist c a ≤ dist a' b' + dist b' c' + dist c' a'
d : V
adb : sbtw a d b
habc : c ∉ Line a b
hdab : d ∈ Line a b
hcd : c ≠ d
this : dist d c < dist d b + dist b c
⊢ dist a d + dist d c + dist c a < dist a b + dist b c + dist c a | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | Delta_comm | [198, 1] | [199, 41] | simp only [Delta, add_comm, dist_comm] | V : Type u_1
inst✝² : MetricSpace V
u✝ v✝ w✝ : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z u v w : V
⊢ Delta u v w = Delta w v u | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | Delta_pos_of | [201, 1] | [205, 90] | rw [Delta] | V : Type u_1
inst✝² : MetricSpace V
u✝ v✝ w✝ : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z u v w : V
h : NotCollinear u v w
⊢ 0 < Delta u v w | V : Type u_1
inst✝² : MetricSpace V
u✝ v✝ w✝ : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z u v w : V
h : NotCollinear u v w
⊢ 0 < dist u v + dist v w - dist u w |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | Delta_pos_of | [201, 1] | [205, 90] | by_contra! | V : Type u_1
inst✝² : MetricSpace V
u✝ v✝ w✝ : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z u v w : V
h : NotCollinear u v w
⊢ 0 < dist u v + dist v w - dist u w | V : Type u_1
inst✝² : MetricSpace V
u✝ v✝ w✝ : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z u v w : V
h : NotCollinear u v w
this : dist u v + dist v w - dist u w ≤ 0
⊢ False |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | Delta_pos_of | [201, 1] | [205, 90] | have : sbtw u v w := sbtw_mk h.1 h.2.2.1 (by linarith only [this]) | V : Type u_1
inst✝² : MetricSpace V
u✝ v✝ w✝ : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z u v w : V
h : NotCollinear u v w
this : dist u v + dist v w - dist u w ≤ 0
⊢ False | V : Type u_1
inst✝² : MetricSpace V
u✝ v✝ w✝ : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z u v w : V
h : NotCollinear u v w
this✝ : dist u v + dist v w - dist u w ≤ 0
this : sbtw u v w
⊢ False |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | Delta_pos_of | [201, 1] | [205, 90] | exact h.2.2.2 (Line u v) (Line_isLine this.ne12) (by simp [right_extend_mem_Line this]) | V : Type u_1
inst✝² : MetricSpace V
u✝ v✝ w✝ : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z u v w : V
h : NotCollinear u v w
this✝ : dist u v + dist v w - dist u w ≤ 0
this : sbtw u v w
⊢ False | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | Delta_pos_of | [201, 1] | [205, 90] | linarith only [this] | V : Type u_1
inst✝² : MetricSpace V
u✝ v✝ w✝ : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z u v w : V
h : NotCollinear u v w
this : dist u v + dist v w - dist u w ≤ 0
⊢ dist u v + dist v w ≤ dist u w | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | Delta_pos_of | [201, 1] | [205, 90] | simp [right_extend_mem_Line this] | V : Type u_1
inst✝² : MetricSpace V
u✝ v✝ w✝ : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z u v w : V
h : NotCollinear u v w
this✝ : dist u v + dist v w - dist u w ≤ 0
this : sbtw u v w
⊢ {u, v, w} ⊆ Line u v | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | exists_third | [207, 1] | [224, 15] | by_contra! h' | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b : V
hab : a ≠ b
h : Line a b ≠ {a, b}
⊢ ∃ c ∈ Line a b, sbtw c a b ∨ sbtw a c b ∨ sbtw a b c | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b : V
hab : a ≠ b
h : Line a b ≠ {a, b}
h' : ∀ c ∈ Line a b, ¬sbtw c a b ∧ ¬sbtw a c b ∧ ¬sbtw a b c
⊢ False |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | exists_third | [207, 1] | [224, 15] | exact h this | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b : V
hab : a ≠ b
h : Line a b ≠ {a, b}
h' : ∀ c ∈ Line a b, ¬sbtw c a b ∧ ¬sbtw a c b ∧ ¬sbtw a b c
this : Line a b = {a, b}
⊢ False | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | exists_third | [207, 1] | [224, 15] | refine (subset_generateLine _).antisymm' ?_ | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b : V
hab : a ≠ b
h : Line a b ≠ {a, b}
h' : ∀ c ∈ Line a b, ¬sbtw c a b ∧ ¬sbtw a c b ∧ ¬sbtw a b c
⊢ Line a b = {a, b} | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b : V
hab : a ≠ b
h : Line a b ≠ {a, b}
h' : ∀ c ∈ Line a b, ¬sbtw c a b ∧ ¬sbtw a c b ∧ ¬sbtw a b c
⊢ GenerateLine {a, b} ⊆ {a, b} |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | exists_third | [207, 1] | [224, 15] | change Line a b ⊆ {a, b} | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b : V
hab : a ≠ b
h : Line a b ≠ {a, b}
h' : ∀ c ∈ Line a b, ¬sbtw c a b ∧ ¬sbtw a c b ∧ ¬sbtw a b c
⊢ GenerateLine {a, b} ⊆ {a, b} | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b : V
hab : a ≠ b
h : Line a b ≠ {a, b}
h' : ∀ c ∈ Line a b, ¬sbtw c a b ∧ ¬sbtw a c b ∧ ¬sbtw a b c
⊢ Line a b ⊆ {a, b} |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | exists_third | [207, 1] | [224, 15] | refine generateLine_minimal le_rfl ?_ ?_ | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b : V
hab : a ≠ b
h : Line a b ≠ {a, b}
h' : ∀ c ∈ Line a b, ¬sbtw c a b ∧ ¬sbtw a c b ∧ ¬sbtw a b c
⊢ Line a b ⊆ {a, b} | case refine_1
V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b : V
hab : a ≠ b
h : Line a b ≠ {a, b}
h' : ∀ c ∈ Line a b, ¬sbtw c a b ∧ ¬sbtw a c b ∧ ¬sbtw a b c
⊢ ∀ {x y z : V}, x ∈ {a, b} → y ∈ {a, b} → sbtw x y z → z ∈ {a, b}
case refine_2
V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b : V
hab : a ≠ b
h : Line a b ≠ {a, b}
h' : ∀ c ∈ Line a b, ¬sbtw c a b ∧ ¬sbtw a c b ∧ ¬sbtw a b c
⊢ ∀ {x y z : V}, x ∈ {a, b} → y ∈ {a, b} → sbtw x z y → z ∈ {a, b} |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | exists_third | [207, 1] | [224, 15] | rintro x y z (rfl | rfl) (rfl | rfl) h | case refine_1
V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b : V
hab : a ≠ b
h : Line a b ≠ {a, b}
h' : ∀ c ∈ Line a b, ¬sbtw c a b ∧ ¬sbtw a c b ∧ ¬sbtw a b c
⊢ ∀ {x y z : V}, x ∈ {a, b} → y ∈ {a, b} → sbtw x y z → z ∈ {a, b} | case refine_1.inl.inl
V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y✝ z✝ b y z : V
hab : y ≠ b
h✝ : Line y b ≠ {y, b}
h' : ∀ c ∈ Line y b, ¬sbtw c y b ∧ ¬sbtw y c b ∧ ¬sbtw y b c
h : sbtw y y z
⊢ z ∈ {y, b}
case refine_1.inl.inr
V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x✝ y✝ z✝ x y z : V
hab : x ≠ y
h✝ : Line x y ≠ {x, y}
h' : ∀ c ∈ Line x y, ¬sbtw c x y ∧ ¬sbtw x c y ∧ ¬sbtw x y c
h : sbtw x y z
⊢ z ∈ {x, y}
case refine_1.inr.inl
V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x✝ y✝ z✝ x y z : V
hab : y ≠ x
h✝ : Line y x ≠ {y, x}
h' : ∀ c ∈ Line y x, ¬sbtw c y x ∧ ¬sbtw y c x ∧ ¬sbtw y x c
h : sbtw x y z
⊢ z ∈ {y, x}
case refine_1.inr.inr
V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y✝ z✝ a y z : V
hab : a ≠ y
h✝ : Line a y ≠ {a, y}
h' : ∀ c ∈ Line a y, ¬sbtw c a y ∧ ¬sbtw a c y ∧ ¬sbtw a y c
h : sbtw y y z
⊢ z ∈ {a, y} |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | exists_third | [207, 1] | [224, 15] | exact (h.ne12 rfl).elim | case refine_1.inl.inl
V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y✝ z✝ b y z : V
hab : y ≠ b
h✝ : Line y b ≠ {y, b}
h' : ∀ c ∈ Line y b, ¬sbtw c y b ∧ ¬sbtw y c b ∧ ¬sbtw y b c
h : sbtw y y z
⊢ z ∈ {y, b} | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | exists_third | [207, 1] | [224, 15] | exact ((h' z (right_extend_mem_Line h)).2.2 h).elim | case refine_1.inl.inr
V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x✝ y✝ z✝ x y z : V
hab : x ≠ y
h✝ : Line x y ≠ {x, y}
h' : ∀ c ∈ Line x y, ¬sbtw c x y ∧ ¬sbtw x c y ∧ ¬sbtw x y c
h : sbtw x y z
⊢ z ∈ {x, y} | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | exists_third | [207, 1] | [224, 15] | exact ((h' z (left_extend_mem_Line h.symm)).1 h.symm).elim | case refine_1.inr.inl
V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x✝ y✝ z✝ x y z : V
hab : y ≠ x
h✝ : Line y x ≠ {y, x}
h' : ∀ c ∈ Line y x, ¬sbtw c y x ∧ ¬sbtw y c x ∧ ¬sbtw y x c
h : sbtw x y z
⊢ z ∈ {y, x} | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | exists_third | [207, 1] | [224, 15] | exact (h.ne12 rfl).elim | case refine_1.inr.inr
V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y✝ z✝ a y z : V
hab : a ≠ y
h✝ : Line a y ≠ {a, y}
h' : ∀ c ∈ Line a y, ¬sbtw c a y ∧ ¬sbtw a c y ∧ ¬sbtw a y c
h : sbtw y y z
⊢ z ∈ {a, y} | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | exists_third | [207, 1] | [224, 15] | rintro x y z (rfl | rfl) (rfl | rfl) h | case refine_2
V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b : V
hab : a ≠ b
h : Line a b ≠ {a, b}
h' : ∀ c ∈ Line a b, ¬sbtw c a b ∧ ¬sbtw a c b ∧ ¬sbtw a b c
⊢ ∀ {x y z : V}, x ∈ {a, b} → y ∈ {a, b} → sbtw x z y → z ∈ {a, b} | case refine_2.inl.inl
V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y✝ z✝ b y z : V
hab : y ≠ b
h✝ : Line y b ≠ {y, b}
h' : ∀ c ∈ Line y b, ¬sbtw c y b ∧ ¬sbtw y c b ∧ ¬sbtw y b c
h : sbtw y z y
⊢ z ∈ {y, b}
case refine_2.inl.inr
V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x✝ y✝ z✝ x y z : V
hab : x ≠ y
h✝ : Line x y ≠ {x, y}
h' : ∀ c ∈ Line x y, ¬sbtw c x y ∧ ¬sbtw x c y ∧ ¬sbtw x y c
h : sbtw x z y
⊢ z ∈ {x, y}
case refine_2.inr.inl
V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x✝ y✝ z✝ x y z : V
hab : y ≠ x
h✝ : Line y x ≠ {y, x}
h' : ∀ c ∈ Line y x, ¬sbtw c y x ∧ ¬sbtw y c x ∧ ¬sbtw y x c
h : sbtw x z y
⊢ z ∈ {y, x}
case refine_2.inr.inr
V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y✝ z✝ a y z : V
hab : a ≠ y
h✝ : Line a y ≠ {a, y}
h' : ∀ c ∈ Line a y, ¬sbtw c a y ∧ ¬sbtw a c y ∧ ¬sbtw a y c
h : sbtw y z y
⊢ z ∈ {a, y} |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | exists_third | [207, 1] | [224, 15] | exact (h.ne13 rfl).elim | case refine_2.inl.inl
V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y✝ z✝ b y z : V
hab : y ≠ b
h✝ : Line y b ≠ {y, b}
h' : ∀ c ∈ Line y b, ¬sbtw c y b ∧ ¬sbtw y c b ∧ ¬sbtw y b c
h : sbtw y z y
⊢ z ∈ {y, b} | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | exists_third | [207, 1] | [224, 15] | exact ((h' z (middle_extend_mem_Line h)).2.1 h).elim | case refine_2.inl.inr
V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x✝ y✝ z✝ x y z : V
hab : x ≠ y
h✝ : Line x y ≠ {x, y}
h' : ∀ c ∈ Line x y, ¬sbtw c x y ∧ ¬sbtw x c y ∧ ¬sbtw x y c
h : sbtw x z y
⊢ z ∈ {x, y} | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | exists_third | [207, 1] | [224, 15] | exact ((h' z (middle_extend_mem_Line h.symm)).2.1 h.symm).elim | case refine_2.inr.inl
V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x✝ y✝ z✝ x y z : V
hab : y ≠ x
h✝ : Line y x ≠ {y, x}
h' : ∀ c ∈ Line y x, ¬sbtw c y x ∧ ¬sbtw y c x ∧ ¬sbtw y x c
h : sbtw x z y
⊢ z ∈ {y, x} | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | exists_third | [207, 1] | [224, 15] | exact (h.ne13 rfl).elim | case refine_2.inr.inr
V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y✝ z✝ a y z : V
hab : a ≠ y
h✝ : Line a y ≠ {a, y}
h' : ∀ c ∈ Line a y, ¬sbtw c a y ∧ ¬sbtw a c y ∧ ¬sbtw a y c
h : sbtw y z y
⊢ z ∈ {a, y} | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | eqn_7 | [226, 1] | [243, 44] | intro h | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b c d : V
habc : SimpleTriangle a b c
habc_min : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c'
hacd : sbtw a c d
hcd : SimpleEdges.Adj c d
⊢ ¬SimpleEdges.Adj b d | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b c d : V
habc : SimpleTriangle a b c
habc_min : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c'
hacd : sbtw a c d
hcd : SimpleEdges.Adj c d
h : SimpleEdges.Adj b d
⊢ False |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | eqn_7 | [226, 1] | [243, 44] | have hbcd : NotCollinear b c d := by
refine ⟨habc.2.1.ne, h.ne, hcd.ne, fun l hl h ↦ ?_⟩
simp only [Set.mem_singleton_iff, Set.mem_insert_iff, Set.subset_def, forall_eq_or_imp,
forall_eq] at h
refine habc.2.2.2.2.2.2 l hl (by simp [*, hl.close_left h.2.1 h.2.2 hacd]) | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b c d : V
habc : SimpleTriangle a b c
habc_min : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c'
hacd : sbtw a c d
hcd : SimpleEdges.Adj c d
h : SimpleEdges.Adj b d
⊢ False | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b c d : V
habc : SimpleTriangle a b c
habc_min : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c'
hacd : sbtw a c d
hcd : SimpleEdges.Adj c d
h : SimpleEdges.Adj b d
hbcd : NotCollinear b c d
⊢ False |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | eqn_7 | [226, 1] | [243, 44] | replace hbcd : SimpleTriangle b c d := ⟨habc.2.1, hcd, h.symm, hbcd⟩ | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b c d : V
habc : SimpleTriangle a b c
habc_min : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c'
hacd : sbtw a c d
hcd : SimpleEdges.Adj c d
h : SimpleEdges.Adj b d
hbcd : NotCollinear b c d
⊢ False | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b c d : V
habc : SimpleTriangle a b c
habc_min : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c'
hacd : sbtw a c d
hcd : SimpleEdges.Adj c d
h : SimpleEdges.Adj b d
hbcd : SimpleTriangle b c d
⊢ False |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | eqn_7 | [226, 1] | [243, 44] | have habd : sbtw a b d := by
refine sbtw_mk habc.1.ne h.ne ?_
have := habc_min _ _ _ hbcd
rw [Delta, Delta] at this
linarith [hacd.dist] | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b c d : V
habc : SimpleTriangle a b c
habc_min : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c'
hacd : sbtw a c d
hcd : SimpleEdges.Adj c d
h : SimpleEdges.Adj b d
hbcd : SimpleTriangle b c d
⊢ False | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b c d : V
habc : SimpleTriangle a b c
habc_min : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c'
hacd : sbtw a c d
hcd : SimpleEdges.Adj c d
h : SimpleEdges.Adj b d
hbcd : SimpleTriangle b c d
habd : sbtw a b d
⊢ False |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | eqn_7 | [226, 1] | [243, 44] | refine habc.2.2.2.2.2.2 (Line a d) (Line_isLine habd.ne13) ?_ | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b c d : V
habc : SimpleTriangle a b c
habc_min : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c'
hacd : sbtw a c d
hcd : SimpleEdges.Adj c d
h : SimpleEdges.Adj b d
hbcd : SimpleTriangle b c d
habd : sbtw a b d
⊢ False | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b c d : V
habc : SimpleTriangle a b c
habc_min : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c'
hacd : sbtw a c d
hcd : SimpleEdges.Adj c d
h : SimpleEdges.Adj b d
hbcd : SimpleTriangle b c d
habd : sbtw a b d
⊢ {a, b, c} ⊆ Line a d |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | eqn_7 | [226, 1] | [243, 44] | simp [middle_extend_mem_Line, hacd, habd] | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b c d : V
habc : SimpleTriangle a b c
habc_min : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c'
hacd : sbtw a c d
hcd : SimpleEdges.Adj c d
h : SimpleEdges.Adj b d
hbcd : SimpleTriangle b c d
habd : sbtw a b d
⊢ {a, b, c} ⊆ Line a d | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | eqn_7 | [226, 1] | [243, 44] | refine ⟨habc.2.1.ne, h.ne, hcd.ne, fun l hl h ↦ ?_⟩ | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b c d : V
habc : SimpleTriangle a b c
habc_min : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c'
hacd : sbtw a c d
hcd : SimpleEdges.Adj c d
h : SimpleEdges.Adj b d
⊢ NotCollinear b c d | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b c d : V
habc : SimpleTriangle a b c
habc_min : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c'
hacd : sbtw a c d
hcd : SimpleEdges.Adj c d
h✝ : SimpleEdges.Adj b d
l : Set V
hl : l.IsLine
h : {b, c, d} ⊆ l
⊢ False |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | eqn_7 | [226, 1] | [243, 44] | simp only [Set.mem_singleton_iff, Set.mem_insert_iff, Set.subset_def, forall_eq_or_imp,
forall_eq] at h | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b c d : V
habc : SimpleTriangle a b c
habc_min : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c'
hacd : sbtw a c d
hcd : SimpleEdges.Adj c d
h✝ : SimpleEdges.Adj b d
l : Set V
hl : l.IsLine
h : {b, c, d} ⊆ l
⊢ False | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b c d : V
habc : SimpleTriangle a b c
habc_min : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c'
hacd : sbtw a c d
hcd : SimpleEdges.Adj c d
h✝ : SimpleEdges.Adj b d
l : Set V
hl : l.IsLine
h : b ∈ l ∧ c ∈ l ∧ d ∈ l
⊢ False |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | eqn_7 | [226, 1] | [243, 44] | refine habc.2.2.2.2.2.2 l hl (by simp [*, hl.close_left h.2.1 h.2.2 hacd]) | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b c d : V
habc : SimpleTriangle a b c
habc_min : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c'
hacd : sbtw a c d
hcd : SimpleEdges.Adj c d
h✝ : SimpleEdges.Adj b d
l : Set V
hl : l.IsLine
h : b ∈ l ∧ c ∈ l ∧ d ∈ l
⊢ False | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | eqn_7 | [226, 1] | [243, 44] | simp [*, hl.close_left h.2.1 h.2.2 hacd] | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b c d : V
habc : SimpleTriangle a b c
habc_min : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c'
hacd : sbtw a c d
hcd : SimpleEdges.Adj c d
h✝ : SimpleEdges.Adj b d
l : Set V
hl : l.IsLine
h : b ∈ l ∧ c ∈ l ∧ d ∈ l
⊢ {a, b, c} ⊆ l | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | eqn_7 | [226, 1] | [243, 44] | refine sbtw_mk habc.1.ne h.ne ?_ | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b c d : V
habc : SimpleTriangle a b c
habc_min : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c'
hacd : sbtw a c d
hcd : SimpleEdges.Adj c d
h : SimpleEdges.Adj b d
hbcd : SimpleTriangle b c d
⊢ sbtw a b d | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b c d : V
habc : SimpleTriangle a b c
habc_min : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c'
hacd : sbtw a c d
hcd : SimpleEdges.Adj c d
h : SimpleEdges.Adj b d
hbcd : SimpleTriangle b c d
⊢ dist a b + dist b d ≤ dist a d |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | eqn_7 | [226, 1] | [243, 44] | have := habc_min _ _ _ hbcd | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b c d : V
habc : SimpleTriangle a b c
habc_min : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c'
hacd : sbtw a c d
hcd : SimpleEdges.Adj c d
h : SimpleEdges.Adj b d
hbcd : SimpleTriangle b c d
⊢ dist a b + dist b d ≤ dist a d | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b c d : V
habc : SimpleTriangle a b c
habc_min : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c'
hacd : sbtw a c d
hcd : SimpleEdges.Adj c d
h : SimpleEdges.Adj b d
hbcd : SimpleTriangle b c d
this : Delta a b c ≤ Delta b c d
⊢ dist a b + dist b d ≤ dist a d |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | eqn_7 | [226, 1] | [243, 44] | rw [Delta, Delta] at this | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b c d : V
habc : SimpleTriangle a b c
habc_min : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c'
hacd : sbtw a c d
hcd : SimpleEdges.Adj c d
h : SimpleEdges.Adj b d
hbcd : SimpleTriangle b c d
this : Delta a b c ≤ Delta b c d
⊢ dist a b + dist b d ≤ dist a d | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b c d : V
habc : SimpleTriangle a b c
habc_min : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c'
hacd : sbtw a c d
hcd : SimpleEdges.Adj c d
h : SimpleEdges.Adj b d
hbcd : SimpleTriangle b c d
this : dist a b + dist b c - dist a c ≤ dist b c + dist c d - dist b d
⊢ dist a b + dist b d ≤ dist a d |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | eqn_7 | [226, 1] | [243, 44] | linarith [hacd.dist] | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b c d : V
habc : SimpleTriangle a b c
habc_min : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c'
hacd : sbtw a c d
hcd : SimpleEdges.Adj c d
h : SimpleEdges.Adj b d
hbcd : SimpleTriangle b c d
this : dist a b + dist b c - dist a c ≤ dist b c + dist c d - dist b d
⊢ dist a b + dist b d ≤ dist a d | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | eqn_8 | [245, 1] | [253, 42] | by_contra! | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b c d : V
habc : SimpleTriangle a b c
hacd : sbtw a c d
⊢ dist a b + dist b d < dist a d + Delta a b c | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b c d : V
habc : SimpleTriangle a b c
hacd : sbtw a c d
this : dist a d + Delta a b c ≤ dist a b + dist b d
⊢ False |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | eqn_8 | [245, 1] | [253, 42] | have hbcd : sbtw b c d := by
refine sbtw_mk habc.2.1.ne hacd.ne23 ?_
rw [Delta] at this
linarith [hacd.dist] | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b c d : V
habc : SimpleTriangle a b c
hacd : sbtw a c d
this : dist a d + Delta a b c ≤ dist a b + dist b d
⊢ False | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b c d : V
habc : SimpleTriangle a b c
hacd : sbtw a c d
this : dist a d + Delta a b c ≤ dist a b + dist b d
hbcd : sbtw b c d
⊢ False |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | eqn_8 | [245, 1] | [253, 42] | refine habc.2.2.2.2.2.2 (Line c d) (Line_isLine hbcd.ne23) ?_ | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b c d : V
habc : SimpleTriangle a b c
hacd : sbtw a c d
this : dist a d + Delta a b c ≤ dist a b + dist b d
hbcd : sbtw b c d
⊢ False | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b c d : V
habc : SimpleTriangle a b c
hacd : sbtw a c d
this : dist a d + Delta a b c ≤ dist a b + dist b d
hbcd : sbtw b c d
⊢ {a, b, c} ⊆ Line c d |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | eqn_8 | [245, 1] | [253, 42] | simp [left_extend_mem_Line, hacd, hbcd] | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b c d : V
habc : SimpleTriangle a b c
hacd : sbtw a c d
this : dist a d + Delta a b c ≤ dist a b + dist b d
hbcd : sbtw b c d
⊢ {a, b, c} ⊆ Line c d | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | eqn_8 | [245, 1] | [253, 42] | refine sbtw_mk habc.2.1.ne hacd.ne23 ?_ | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b c d : V
habc : SimpleTriangle a b c
hacd : sbtw a c d
this : dist a d + Delta a b c ≤ dist a b + dist b d
⊢ sbtw b c d | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b c d : V
habc : SimpleTriangle a b c
hacd : sbtw a c d
this : dist a d + Delta a b c ≤ dist a b + dist b d
⊢ dist b c + dist c d ≤ dist b d |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | eqn_8 | [245, 1] | [253, 42] | rw [Delta] at this | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b c d : V
habc : SimpleTriangle a b c
hacd : sbtw a c d
this : dist a d + Delta a b c ≤ dist a b + dist b d
⊢ dist b c + dist c d ≤ dist b d | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b c d : V
habc : SimpleTriangle a b c
hacd : sbtw a c d
this : dist a d + (dist a b + dist b c - dist a c) ≤ dist a b + dist b d
⊢ dist b c + dist c d ≤ dist b d |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | eqn_8 | [245, 1] | [253, 42] | linarith [hacd.dist] | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b c d : V
habc : SimpleTriangle a b c
hacd : sbtw a c d
this : dist a d + (dist a b + dist b c - dist a c) ≤ dist a b + dist b d
⊢ dist b c + dist c d ≤ dist b d | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | List.pathLength_nonneg | [259, 1] | [261, 72] | simp [pathLength] | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z head✝ : V
⊢ 0 ≤ [head✝].pathLength | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | exists_min_dist | [297, 1] | [305, 100] | cases subsingleton_or_nontrivial V | V✝ : Type u_1
inst✝⁴ : MetricSpace V✝
u v w : V✝
inst✝³ : Finite V✝
inst✝² : Nontrivial V✝
x y z : V✝
V : Type u_2
inst✝¹ : MetricSpace V
inst✝ : Finite V
⊢ ∃ r, 0 < r ∧ ∀ (x y : V), x ≠ y → r ≤ dist x y | case inl
V✝ : Type u_1
inst✝⁴ : MetricSpace V✝
u v w : V✝
inst✝³ : Finite V✝
inst✝² : Nontrivial V✝
x y z : V✝
V : Type u_2
inst✝¹ : MetricSpace V
inst✝ : Finite V
h✝ : Subsingleton V
⊢ ∃ r, 0 < r ∧ ∀ (x y : V), x ≠ y → r ≤ dist x y
case inr
V✝ : Type u_1
inst✝⁴ : MetricSpace V✝
u v w : V✝
inst✝³ : Finite V✝
inst✝² : Nontrivial V✝
x y z : V✝
V : Type u_2
inst✝¹ : MetricSpace V
inst✝ : Finite V
h✝ : Nontrivial V
⊢ ∃ r, 0 < r ∧ ∀ (x y : V), x ≠ y → r ≤ dist x y |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | exists_min_dist | [297, 1] | [305, 100] | let S : Set (V × V) := (Set.diagonal V)ᶜ | case inr
V✝ : Type u_1
inst✝⁴ : MetricSpace V✝
u v w : V✝
inst✝³ : Finite V✝
inst✝² : Nontrivial V✝
x y z : V✝
V : Type u_2
inst✝¹ : MetricSpace V
inst✝ : Finite V
h✝ : Nontrivial V
⊢ ∃ r, 0 < r ∧ ∀ (x y : V), x ≠ y → r ≤ dist x y | case inr
V✝ : Type u_1
inst✝⁴ : MetricSpace V✝
u v w : V✝
inst✝³ : Finite V✝
inst✝² : Nontrivial V✝
x y z : V✝
V : Type u_2
inst✝¹ : MetricSpace V
inst✝ : Finite V
h✝ : Nontrivial V
S : Set (V × V) := (Set.diagonal V)ᶜ
⊢ ∃ r, 0 < r ∧ ∀ (x y : V), x ≠ y → r ≤ dist x y |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | exists_min_dist | [297, 1] | [305, 100] | have : S.Nonempty := have ⟨x, y, hxy⟩ := exists_pair_ne V; ⟨(x, y), by simp [S, hxy]⟩ | case inr
V✝ : Type u_1
inst✝⁴ : MetricSpace V✝
u v w : V✝
inst✝³ : Finite V✝
inst✝² : Nontrivial V✝
x y z : V✝
V : Type u_2
inst✝¹ : MetricSpace V
inst✝ : Finite V
h✝ : Nontrivial V
S : Set (V × V) := (Set.diagonal V)ᶜ
⊢ ∃ r, 0 < r ∧ ∀ (x y : V), x ≠ y → r ≤ dist x y | case inr
V✝ : Type u_1
inst✝⁴ : MetricSpace V✝
u v w : V✝
inst✝³ : Finite V✝
inst✝² : Nontrivial V✝
x y z : V✝
V : Type u_2
inst✝¹ : MetricSpace V
inst✝ : Finite V
h✝ : Nontrivial V
S : Set (V × V) := (Set.diagonal V)ᶜ
this : S.Nonempty
⊢ ∃ r, 0 < r ∧ ∀ (x y : V), x ≠ y → r ≤ dist x y |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | exists_min_dist | [297, 1] | [305, 100] | obtain ⟨⟨x, y⟩, (hxy : x ≠ y), h⟩ := S.toFinite.exists_minimal_wrt (Function.uncurry dist) _ this | case inr
V✝ : Type u_1
inst✝⁴ : MetricSpace V✝
u v w : V✝
inst✝³ : Finite V✝
inst✝² : Nontrivial V✝
x y z : V✝
V : Type u_2
inst✝¹ : MetricSpace V
inst✝ : Finite V
h✝ : Nontrivial V
S : Set (V × V) := (Set.diagonal V)ᶜ
this : S.Nonempty
⊢ ∃ r, 0 < r ∧ ∀ (x y : V), x ≠ y → r ≤ dist x y | case inr.intro.mk.intro
V✝ : Type u_1
inst✝⁴ : MetricSpace V✝
u v w : V✝
inst✝³ : Finite V✝
inst✝² : Nontrivial V✝
x✝ y✝ z : V✝
V : Type u_2
inst✝¹ : MetricSpace V
inst✝ : Finite V
h✝ : Nontrivial V
S : Set (V × V) := (Set.diagonal V)ᶜ
this : S.Nonempty
x y : V
hxy : x ≠ y
h :
∀ a' ∈ S,
Function.uncurry dist a' ≤ Function.uncurry dist (x, y) → Function.uncurry dist (x, y) = Function.uncurry dist a'
⊢ ∃ r, 0 < r ∧ ∀ (x y : V), x ≠ y → r ≤ dist x y |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | exists_min_dist | [297, 1] | [305, 100] | simp only [Set.mem_compl_iff, Set.mem_diagonal_iff, Function.uncurry_apply_pair, Prod.forall] at h | case inr.intro.mk.intro
V✝ : Type u_1
inst✝⁴ : MetricSpace V✝
u v w : V✝
inst✝³ : Finite V✝
inst✝² : Nontrivial V✝
x✝ y✝ z : V✝
V : Type u_2
inst✝¹ : MetricSpace V
inst✝ : Finite V
h✝ : Nontrivial V
S : Set (V × V) := (Set.diagonal V)ᶜ
this : S.Nonempty
x y : V
hxy : x ≠ y
h :
∀ a' ∈ S,
Function.uncurry dist a' ≤ Function.uncurry dist (x, y) → Function.uncurry dist (x, y) = Function.uncurry dist a'
⊢ ∃ r, 0 < r ∧ ∀ (x y : V), x ≠ y → r ≤ dist x y | case inr.intro.mk.intro
V✝ : Type u_1
inst✝⁴ : MetricSpace V✝
u v w : V✝
inst✝³ : Finite V✝
inst✝² : Nontrivial V✝
x✝ y✝ z : V✝
V : Type u_2
inst✝¹ : MetricSpace V
inst✝ : Finite V
h✝ : Nontrivial V
S : Set (V × V) := (Set.diagonal V)ᶜ
this : S.Nonempty
x y : V
hxy : x ≠ y
h : ∀ (a b : V), (a, b) ∈ S → dist a b ≤ dist x y → dist x y = dist a b
⊢ ∃ r, 0 < r ∧ ∀ (x y : V), x ≠ y → r ≤ dist x y |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | exists_min_dist | [297, 1] | [305, 100] | exact ⟨dist x y, by simp [hxy], fun a b hab => le_of_not_lt (fun h' => h'.ne' (h _ _ hab h'.le))⟩ | case inr.intro.mk.intro
V✝ : Type u_1
inst✝⁴ : MetricSpace V✝
u v w : V✝
inst✝³ : Finite V✝
inst✝² : Nontrivial V✝
x✝ y✝ z : V✝
V : Type u_2
inst✝¹ : MetricSpace V
inst✝ : Finite V
h✝ : Nontrivial V
S : Set (V × V) := (Set.diagonal V)ᶜ
this : S.Nonempty
x y : V
hxy : x ≠ y
h : ∀ (a b : V), (a, b) ∈ S → dist a b ≤ dist x y → dist x y = dist a b
⊢ ∃ r, 0 < r ∧ ∀ (x y : V), x ≠ y → r ≤ dist x y | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | exists_min_dist | [297, 1] | [305, 100] | exact ⟨1, zero_lt_one, fun x y ↦ by simp [Subsingleton.elim x y]⟩ | case inl
V✝ : Type u_1
inst✝⁴ : MetricSpace V✝
u v w : V✝
inst✝³ : Finite V✝
inst✝² : Nontrivial V✝
x y z : V✝
V : Type u_2
inst✝¹ : MetricSpace V
inst✝ : Finite V
h✝ : Subsingleton V
⊢ ∃ r, 0 < r ∧ ∀ (x y : V), x ≠ y → r ≤ dist x y | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | exists_min_dist | [297, 1] | [305, 100] | simp [Subsingleton.elim x y] | V✝ : Type u_1
inst✝⁴ : MetricSpace V✝
u v w : V✝
inst✝³ : Finite V✝
inst✝² : Nontrivial V✝
x✝ y✝ z : V✝
V : Type u_2
inst✝¹ : MetricSpace V
inst✝ : Finite V
h✝ : Subsingleton V
x y : V
⊢ x ≠ y → 1 ≤ dist x y | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | exists_min_dist | [297, 1] | [305, 100] | simp [S, hxy] | V✝ : Type u_1
inst✝⁴ : MetricSpace V✝
u v w : V✝
inst✝³ : Finite V✝
inst✝² : Nontrivial V✝
x✝ y✝ z : V✝
V : Type u_2
inst✝¹ : MetricSpace V
inst✝ : Finite V
h✝ : Nontrivial V
S : Set (V × V) := (Set.diagonal V)ᶜ
x y : V
hxy : x ≠ y
⊢ (x, y) ∈ S | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | exists_min_dist | [297, 1] | [305, 100] | simp [hxy] | V✝ : Type u_1
inst✝⁴ : MetricSpace V✝
u v w : V✝
inst✝³ : Finite V✝
inst✝² : Nontrivial V✝
x✝ y✝ z : V✝
V : Type u_2
inst✝¹ : MetricSpace V
inst✝ : Finite V
h✝ : Nontrivial V
S : Set (V × V) := (Set.diagonal V)ᶜ
this : S.Nonempty
x y : V
hxy : x ≠ y
h : ∀ (a b : V), (a, b) ∈ S → dist a b ≤ dist x y → dist x y = dist a b
⊢ 0 < dist x y | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | length_mul_le_pathLength_add | [307, 1] | [316, 77] | simp [List.pathLength, hr] | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z : V
r : ℝ
hr : 0 ≤ r
h : ∀ (x y : V), x ≠ y → r ≤ dist x y
x✝ : List.Chain' (fun x x_1 => x ≠ x_1) []
⊢ ↑[].length * r ≤ [].pathLength + r | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | length_mul_le_pathLength_add | [307, 1] | [316, 77] | simp [List.pathLength] | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z : V
r : ℝ
hr : 0 ≤ r
h : ∀ (x y : V), x ≠ y → r ≤ dist x y
head✝ : V
x✝ : List.Chain' (fun x x_1 => x ≠ x_1) [head✝]
⊢ ↑[head✝].length * r ≤ [head✝].pathLength + r | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | length_mul_le_pathLength_add | [307, 1] | [316, 77] | simp only [List.chain'_cons] at h' | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x✝ y✝ z : V
r : ℝ
hr : 0 ≤ r
h : ∀ (x y : V), x ≠ y → r ≤ dist x y
x y : V
xs : List V
h' : List.Chain' (fun x x_1 => x ≠ x_1) (x :: y :: xs)
⊢ ↑(x :: y :: xs).length * r ≤ (x :: y :: xs).pathLength + r | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x✝ y✝ z : V
r : ℝ
hr : 0 ≤ r
h : ∀ (x y : V), x ≠ y → r ≤ dist x y
x y : V
xs : List V
h' : x ≠ y ∧ List.Chain' (fun x x_1 => x ≠ x_1) (y :: xs)
⊢ ↑(x :: y :: xs).length * r ≤ (x :: y :: xs).pathLength + r |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | length_mul_le_pathLength_add | [307, 1] | [316, 77] | rw [List.pathLength, List.length, Nat.cast_add_one, add_one_mul (α := ℝ), add_assoc,
add_comm] | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x✝ y✝ z : V
r : ℝ
hr : 0 ≤ r
h : ∀ (x y : V), x ≠ y → r ≤ dist x y
x y : V
xs : List V
h' : x ≠ y ∧ List.Chain' (fun x x_1 => x ≠ x_1) (y :: xs)
⊢ ↑(x :: y :: xs).length * r ≤ (x :: y :: xs).pathLength + r | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x✝ y✝ z : V
r : ℝ
hr : 0 ≤ r
h : ∀ (x y : V), x ≠ y → r ≤ dist x y
x y : V
xs : List V
h' : x ≠ y ∧ List.Chain' (fun x x_1 => x ≠ x_1) (y :: xs)
⊢ r + ↑(y :: xs).length * r ≤ dist x y + ((y :: xs).pathLength + r) |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | length_mul_le_pathLength_add | [307, 1] | [316, 77] | exact add_le_add (h _ _ h'.1) (length_mul_le_pathLength_add hr h h'.2) | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x✝ y✝ z : V
r : ℝ
hr : 0 ≤ r
h : ∀ (x y : V), x ≠ y → r ≤ dist x y
x y : V
xs : List V
h' : x ≠ y ∧ List.Chain' (fun x x_1 => x ≠ x_1) (y :: xs)
⊢ r + ↑(y :: xs).length * r ≤ dist x y + ((y :: xs).pathLength + r) | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | uniformly_bounded_of_chain_ne_of_pathLength_le | [318, 1] | [328, 15] | have ⟨r, hr, hr'⟩ := exists_min_dist V | V✝ : Type u_1
inst✝⁴ : MetricSpace V✝
u v w : V✝
inst✝³ : Finite V✝
inst✝² : Nontrivial V✝
x y z : V✝
V : Type u_2
inst✝¹ : MetricSpace V
inst✝ : Finite V
R : ℝ
⊢ ∃ n, ∀ (l : List V), List.Chain' (fun x x_1 => x ≠ x_1) l → l.pathLength ≤ R → l.length ≤ n | V✝ : Type u_1
inst✝⁴ : MetricSpace V✝
u v w : V✝
inst✝³ : Finite V✝
inst✝² : Nontrivial V✝
x y z : V✝
V : Type u_2
inst✝¹ : MetricSpace V
inst✝ : Finite V
R r : ℝ
hr : 0 < r
hr' : ∀ (x y : V), x ≠ y → r ≤ dist x y
⊢ ∃ n, ∀ (l : List V), List.Chain' (fun x x_1 => x ≠ x_1) l → l.pathLength ≤ R → l.length ≤ n |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | uniformly_bounded_of_chain_ne_of_pathLength_le | [318, 1] | [328, 15] | refine ⟨⌊R / r + 1⌋₊, ?_⟩ | V✝ : Type u_1
inst✝⁴ : MetricSpace V✝
u v w : V✝
inst✝³ : Finite V✝
inst✝² : Nontrivial V✝
x y z : V✝
V : Type u_2
inst✝¹ : MetricSpace V
inst✝ : Finite V
R r : ℝ
hr : 0 < r
hr' : ∀ (x y : V), x ≠ y → r ≤ dist x y
⊢ ∃ n, ∀ (l : List V), List.Chain' (fun x x_1 => x ≠ x_1) l → l.pathLength ≤ R → l.length ≤ n | V✝ : Type u_1
inst✝⁴ : MetricSpace V✝
u v w : V✝
inst✝³ : Finite V✝
inst✝² : Nontrivial V✝
x y z : V✝
V : Type u_2
inst✝¹ : MetricSpace V
inst✝ : Finite V
R r : ℝ
hr : 0 < r
hr' : ∀ (x y : V), x ≠ y → r ≤ dist x y
⊢ ∀ (l : List V), List.Chain' (fun x x_1 => x ≠ x_1) l → l.pathLength ≤ R → l.length ≤ ⌊R / r + 1⌋₊ |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | uniformly_bounded_of_chain_ne_of_pathLength_le | [318, 1] | [328, 15] | intro l hl hl' | V✝ : Type u_1
inst✝⁴ : MetricSpace V✝
u v w : V✝
inst✝³ : Finite V✝
inst✝² : Nontrivial V✝
x y z : V✝
V : Type u_2
inst✝¹ : MetricSpace V
inst✝ : Finite V
R r : ℝ
hr : 0 < r
hr' : ∀ (x y : V), x ≠ y → r ≤ dist x y
⊢ ∀ (l : List V), List.Chain' (fun x x_1 => x ≠ x_1) l → l.pathLength ≤ R → l.length ≤ ⌊R / r + 1⌋₊ | V✝ : Type u_1
inst✝⁴ : MetricSpace V✝
u v w : V✝
inst✝³ : Finite V✝
inst✝² : Nontrivial V✝
x y z : V✝
V : Type u_2
inst✝¹ : MetricSpace V
inst✝ : Finite V
R r : ℝ
hr : 0 < r
hr' : ∀ (x y : V), x ≠ y → r ≤ dist x y
l : List V
hl : List.Chain' (fun x x_1 => x ≠ x_1) l
hl' : l.pathLength ≤ R
⊢ l.length ≤ ⌊R / r + 1⌋₊ |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | uniformly_bounded_of_chain_ne_of_pathLength_le | [318, 1] | [328, 15] | have hR : 0 ≤ R := l.pathLength_nonneg.trans hl' | V✝ : Type u_1
inst✝⁴ : MetricSpace V✝
u v w : V✝
inst✝³ : Finite V✝
inst✝² : Nontrivial V✝
x y z : V✝
V : Type u_2
inst✝¹ : MetricSpace V
inst✝ : Finite V
R r : ℝ
hr : 0 < r
hr' : ∀ (x y : V), x ≠ y → r ≤ dist x y
l : List V
hl : List.Chain' (fun x x_1 => x ≠ x_1) l
hl' : l.pathLength ≤ R
⊢ l.length ≤ ⌊R / r + 1⌋₊ | V✝ : Type u_1
inst✝⁴ : MetricSpace V✝
u v w : V✝
inst✝³ : Finite V✝
inst✝² : Nontrivial V✝
x y z : V✝
V : Type u_2
inst✝¹ : MetricSpace V
inst✝ : Finite V
R r : ℝ
hr : 0 < r
hr' : ∀ (x y : V), x ≠ y → r ≤ dist x y
l : List V
hl : List.Chain' (fun x x_1 => x ≠ x_1) l
hl' : l.pathLength ≤ R
hR : 0 ≤ R
⊢ l.length ≤ ⌊R / r + 1⌋₊ |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | uniformly_bounded_of_chain_ne_of_pathLength_le | [318, 1] | [328, 15] | have := length_mul_le_pathLength_add hr.le hr' hl | V✝ : Type u_1
inst✝⁴ : MetricSpace V✝
u v w : V✝
inst✝³ : Finite V✝
inst✝² : Nontrivial V✝
x y z : V✝
V : Type u_2
inst✝¹ : MetricSpace V
inst✝ : Finite V
R r : ℝ
hr : 0 < r
hr' : ∀ (x y : V), x ≠ y → r ≤ dist x y
l : List V
hl : List.Chain' (fun x x_1 => x ≠ x_1) l
hl' : l.pathLength ≤ R
hR : 0 ≤ R
⊢ l.length ≤ ⌊R / r + 1⌋₊ | V✝ : Type u_1
inst✝⁴ : MetricSpace V✝
u v w : V✝
inst✝³ : Finite V✝
inst✝² : Nontrivial V✝
x y z : V✝
V : Type u_2
inst✝¹ : MetricSpace V
inst✝ : Finite V
R r : ℝ
hr : 0 < r
hr' : ∀ (x y : V), x ≠ y → r ≤ dist x y
l : List V
hl : List.Chain' (fun x x_1 => x ≠ x_1) l
hl' : l.pathLength ≤ R
hR : 0 ≤ R
this : ↑l.length * r ≤ l.pathLength + r
⊢ l.length ≤ ⌊R / r + 1⌋₊ |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | uniformly_bounded_of_chain_ne_of_pathLength_le | [318, 1] | [328, 15] | rw [Nat.le_floor_iff, div_add_one hr.ne', le_div_iff hr] | V✝ : Type u_1
inst✝⁴ : MetricSpace V✝
u v w : V✝
inst✝³ : Finite V✝
inst✝² : Nontrivial V✝
x y z : V✝
V : Type u_2
inst✝¹ : MetricSpace V
inst✝ : Finite V
R r : ℝ
hr : 0 < r
hr' : ∀ (x y : V), x ≠ y → r ≤ dist x y
l : List V
hl : List.Chain' (fun x x_1 => x ≠ x_1) l
hl' : l.pathLength ≤ R
hR : 0 ≤ R
this : ↑l.length * r ≤ l.pathLength + r
⊢ l.length ≤ ⌊R / r + 1⌋₊ | V✝ : Type u_1
inst✝⁴ : MetricSpace V✝
u v w : V✝
inst✝³ : Finite V✝
inst✝² : Nontrivial V✝
x y z : V✝
V : Type u_2
inst✝¹ : MetricSpace V
inst✝ : Finite V
R r : ℝ
hr : 0 < r
hr' : ∀ (x y : V), x ≠ y → r ≤ dist x y
l : List V
hl : List.Chain' (fun x x_1 => x ≠ x_1) l
hl' : l.pathLength ≤ R
hR : 0 ≤ R
this : ↑l.length * r ≤ l.pathLength + r
⊢ ↑l.length * r ≤ R + r
V✝ : Type u_1
inst✝⁴ : MetricSpace V✝
u v w : V✝
inst✝³ : Finite V✝
inst✝² : Nontrivial V✝
x y z : V✝
V : Type u_2
inst✝¹ : MetricSpace V
inst✝ : Finite V
R r : ℝ
hr : 0 < r
hr' : ∀ (x y : V), x ≠ y → r ≤ dist x y
l : List V
hl : List.Chain' (fun x x_1 => x ≠ x_1) l
hl' : l.pathLength ≤ R
hR : 0 ≤ R
this : ↑l.length * r ≤ l.pathLength + r
⊢ 0 ≤ R / r + 1 |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | uniformly_bounded_of_chain_ne_of_pathLength_le | [318, 1] | [328, 15] | linarith | V✝ : Type u_1
inst✝⁴ : MetricSpace V✝
u v w : V✝
inst✝³ : Finite V✝
inst✝² : Nontrivial V✝
x y z : V✝
V : Type u_2
inst✝¹ : MetricSpace V
inst✝ : Finite V
R r : ℝ
hr : 0 < r
hr' : ∀ (x y : V), x ≠ y → r ≤ dist x y
l : List V
hl : List.Chain' (fun x x_1 => x ≠ x_1) l
hl' : l.pathLength ≤ R
hR : 0 ≤ R
this : ↑l.length * r ≤ l.pathLength + r
⊢ ↑l.length * r ≤ R + r | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | uniformly_bounded_of_chain_ne_of_pathLength_le | [318, 1] | [328, 15] | positivity | V✝ : Type u_1
inst✝⁴ : MetricSpace V✝
u v w : V✝
inst✝³ : Finite V✝
inst✝² : Nontrivial V✝
x y z : V✝
V : Type u_2
inst✝¹ : MetricSpace V
inst✝ : Finite V
R r : ℝ
hr : 0 < r
hr' : ∀ (x y : V), x ≠ y → r ≤ dist x y
l : List V
hl : List.Chain' (fun x x_1 => x ≠ x_1) l
hl' : l.pathLength ≤ R
hR : 0 ≤ R
this : ↑l.length * r ≤ l.pathLength + r
⊢ 0 ≤ R / r + 1 | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | abd_special | [330, 1] | [339, 80] | simp only [List.Special, ne_eq, List.getLast_cons, List.getLast_singleton', and_true, hbd,
or_true, true_and, List.nodup_cons, List.nodup_nil, List.not_mem_nil, List.mem_cons,
List.mem_singleton, or_false, hbd', hacd.ne13, notCollinear_iff, habc.1.ne, Set.subset_def,
Set.mem_singleton_iff, Set.mem_insert_iff, forall_eq_or_imp, forall_eq, le_refl,
List.chain'_cons, List.chain'_singleton, not_false_eq_true] | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b c d : V
habc : SimpleTriangle a b c
hacd : sbtw a c d
hbd' : b ≠ d
hbd : ¬SimpleEdges.Adj b d
⊢ List.Special a b d [a, b, d] | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b c d : V
habc : SimpleTriangle a b c
hacd : sbtw a c d
hbd' : b ≠ d
hbd : ¬SimpleEdges.Adj b d
⊢ ∀ (l : Set V), l.IsLine → ¬(a ∈ l ∧ b ∈ l ∧ d ∈ l) |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | abd_special | [330, 1] | [339, 80] | intro l hl hl' | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b c d : V
habc : SimpleTriangle a b c
hacd : sbtw a c d
hbd' : b ≠ d
hbd : ¬SimpleEdges.Adj b d
⊢ ∀ (l : Set V), l.IsLine → ¬(a ∈ l ∧ b ∈ l ∧ d ∈ l) | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b c d : V
habc : SimpleTriangle a b c
hacd : sbtw a c d
hbd' : b ≠ d
hbd : ¬SimpleEdges.Adj b d
l : Set V
hl : l.IsLine
hl' : a ∈ l ∧ b ∈ l ∧ d ∈ l
⊢ False |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | abd_special | [330, 1] | [339, 80] | exact habc.2.2.2.2.2.2 l hl $ by simp [*, hl.close_middle hl'.1 hl'.2.2 hacd] | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b c d : V
habc : SimpleTriangle a b c
hacd : sbtw a c d
hbd' : b ≠ d
hbd : ¬SimpleEdges.Adj b d
l : Set V
hl : l.IsLine
hl' : a ∈ l ∧ b ∈ l ∧ d ∈ l
⊢ False | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | abd_special | [330, 1] | [339, 80] | simp [*, hl.close_middle hl'.1 hl'.2.2 hacd] | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b c d : V
habc : SimpleTriangle a b c
hacd : sbtw a c d
hbd' : b ≠ d
hbd : ¬SimpleEdges.Adj b d
l : Set V
hl : l.IsLine
hl' : a ∈ l ∧ b ∈ l ∧ d ∈ l
⊢ {a, b, c} ⊆ l | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | eqn_9 | [341, 1] | [347, 24] | refine (hP' [a, b, d] (abd_special habc hacd hbd' hbd)).trans_lt ?_ | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b c d : V
P : List V
habc : SimpleTriangle a b c
hacd : sbtw a c d
hbd' : b ≠ d
hbd : ¬SimpleEdges.Adj b d
hP' : ∀ (P' : List V), List.Special a b d P' → P.pathLength ≤ P'.pathLength
⊢ P.pathLength < dist a d + Delta a b c | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b c d : V
P : List V
habc : SimpleTriangle a b c
hacd : sbtw a c d
hbd' : b ≠ d
hbd : ¬SimpleEdges.Adj b d
hP' : ∀ (P' : List V), List.Special a b d P' → P.pathLength ≤ P'.pathLength
⊢ [a, b, d].pathLength < dist a d + Delta a b c |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | eqn_9 | [341, 1] | [347, 24] | rw [List.pathLength, List.pathLength, List.pathLength, add_zero] | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b c d : V
P : List V
habc : SimpleTriangle a b c
hacd : sbtw a c d
hbd' : b ≠ d
hbd : ¬SimpleEdges.Adj b d
hP' : ∀ (P' : List V), List.Special a b d P' → P.pathLength ≤ P'.pathLength
⊢ [a, b, d].pathLength < dist a d + Delta a b c | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b c d : V
P : List V
habc : SimpleTriangle a b c
hacd : sbtw a c d
hbd' : b ≠ d
hbd : ¬SimpleEdges.Adj b d
hP' : ∀ (P' : List V), List.Special a b d P' → P.pathLength ≤ P'.pathLength
⊢ dist a b + dist b d < dist a d + Delta a b c |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | eqn_9 | [341, 1] | [347, 24] | exact eqn_8 habc hacd | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b c d : V
P : List V
habc : SimpleTriangle a b c
hacd : sbtw a c d
hbd' : b ≠ d
hbd : ¬SimpleEdges.Adj b d
hP' : ∀ (P' : List V), List.Special a b d P' → P.pathLength ≤ P'.pathLength
⊢ dist a b + dist b d < dist a d + Delta a b c | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | exists_simple_split_right | [349, 1] | [361, 22] | simp only [SimpleEdges_adj, hab, not_false_eq_true, true_and, ne_eq, not_forall, not_not] at hab' | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b : V
hab : a ≠ b
hab' : ¬SimpleEdges.Adj a b
⊢ ∃ c, sbtw a c b ∧ SimpleEdges.Adj c b | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b : V
hab : a ≠ b
hab' : ∃ x, sbtw a x b
⊢ ∃ c, sbtw a c b ∧ SimpleEdges.Adj c b |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | exists_simple_split_right | [349, 1] | [361, 22] | obtain ⟨c', hc'⟩ := hab' | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b : V
hab : a ≠ b
hab' : ∃ x, sbtw a x b
⊢ ∃ c, sbtw a c b ∧ SimpleEdges.Adj c b | case intro
V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b : V
hab : a ≠ b
c' : V
hc' : sbtw a c' b
⊢ ∃ c, sbtw a c b ∧ SimpleEdges.Adj c b |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | exists_simple_split_right | [349, 1] | [361, 22] | obtain ⟨c, hc : sbtw _ c _, hcmin⟩ := S.toFinite.exists_minimal_wrt (dist b) _ ⟨c', hc'⟩ | case intro
V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b : V
hab : a ≠ b
c' : V
hc' : sbtw a c' b
S : Set V := {x | sbtw a x b}
⊢ ∃ c, sbtw a c b ∧ SimpleEdges.Adj c b | case intro.intro.intro
V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b : V
hab : a ≠ b
c' : V
hc' : sbtw a c' b
S : Set V := {x | sbtw a x b}
c : V
hc : sbtw a c b
hcmin : ∀ a' ∈ S, dist b a' ≤ dist b c → dist b c = dist b a'
⊢ ∃ c, sbtw a c b ∧ SimpleEdges.Adj c b |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | exists_simple_split_right | [349, 1] | [361, 22] | refine ⟨c, hc, hc.ne23, fun c' hc' => ?_⟩ | case intro.intro.intro
V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b : V
hab : a ≠ b
c' : V
hc' : sbtw a c' b
S : Set V := {x | sbtw a x b}
c : V
hc : sbtw a c b
hcmin : ∀ a' ∈ S, dist b a' ≤ dist b c → dist b c = dist b a'
⊢ ∃ c, sbtw a c b ∧ SimpleEdges.Adj c b | case intro.intro.intro
V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b : V
hab : a ≠ b
c'✝ : V
hc'✝ : sbtw a c'✝ b
S : Set V := {x | sbtw a x b}
c : V
hc : sbtw a c b
hcmin : ∀ a' ∈ S, dist b a' ≤ dist b c → dist b c = dist b a'
c' : V
hc' : sbtw c c' b
⊢ False |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | exists_simple_split_right | [349, 1] | [361, 22] | have : dist b c ≤ dist b c' :=
le_of_not_lt fun h => h.ne' <| hcmin _ (hc.trans_right' hc') h.le | case intro.intro.intro
V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b : V
hab : a ≠ b
c'✝ : V
hc'✝ : sbtw a c'✝ b
S : Set V := {x | sbtw a x b}
c : V
hc : sbtw a c b
hcmin : ∀ a' ∈ S, dist b a' ≤ dist b c → dist b c = dist b a'
c' : V
hc' : sbtw c c' b
⊢ False | case intro.intro.intro
V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b : V
hab : a ≠ b
c'✝ : V
hc'✝ : sbtw a c'✝ b
S : Set V := {x | sbtw a x b}
c : V
hc : sbtw a c b
hcmin : ∀ a' ∈ S, dist b a' ≤ dist b c → dist b c = dist b a'
c' : V
hc' : sbtw c c' b
this : dist b c ≤ dist b c'
⊢ False |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | exists_simple_split_right | [349, 1] | [361, 22] | rw [dist_comm b, dist_comm b] at this | case intro.intro.intro
V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b : V
hab : a ≠ b
c'✝ : V
hc'✝ : sbtw a c'✝ b
S : Set V := {x | sbtw a x b}
c : V
hc : sbtw a c b
hcmin : ∀ a' ∈ S, dist b a' ≤ dist b c → dist b c = dist b a'
c' : V
hc' : sbtw c c' b
this : dist b c ≤ dist b c'
⊢ False | case intro.intro.intro
V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b : V
hab : a ≠ b
c'✝ : V
hc'✝ : sbtw a c'✝ b
S : Set V := {x | sbtw a x b}
c : V
hc : sbtw a c b
hcmin : ∀ a' ∈ S, dist b a' ≤ dist b c → dist b c = dist b a'
c' : V
hc' : sbtw c c' b
this : dist c b ≤ dist c' b
⊢ False |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | exists_simple_split_right | [349, 1] | [361, 22] | have : dist c c' ≤ 0 := by linarith [hc'.dist] | case intro.intro.intro
V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b : V
hab : a ≠ b
c'✝ : V
hc'✝ : sbtw a c'✝ b
S : Set V := {x | sbtw a x b}
c : V
hc : sbtw a c b
hcmin : ∀ a' ∈ S, dist b a' ≤ dist b c → dist b c = dist b a'
c' : V
hc' : sbtw c c' b
this : dist c b ≤ dist c' b
⊢ False | case intro.intro.intro
V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b : V
hab : a ≠ b
c'✝ : V
hc'✝ : sbtw a c'✝ b
S : Set V := {x | sbtw a x b}
c : V
hc : sbtw a c b
hcmin : ∀ a' ∈ S, dist b a' ≤ dist b c → dist b c = dist b a'
c' : V
hc' : sbtw c c' b
this✝ : dist c b ≤ dist c' b
this : dist c c' ≤ 0
⊢ False |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | exists_simple_split_right | [349, 1] | [361, 22] | simp only [dist_le_zero] at this | case intro.intro.intro
V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b : V
hab : a ≠ b
c'✝ : V
hc'✝ : sbtw a c'✝ b
S : Set V := {x | sbtw a x b}
c : V
hc : sbtw a c b
hcmin : ∀ a' ∈ S, dist b a' ≤ dist b c → dist b c = dist b a'
c' : V
hc' : sbtw c c' b
this✝ : dist c b ≤ dist c' b
this : dist c c' ≤ 0
⊢ False | case intro.intro.intro
V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b : V
hab : a ≠ b
c'✝ : V
hc'✝ : sbtw a c'✝ b
S : Set V := {x | sbtw a x b}
c : V
hc : sbtw a c b
hcmin : ∀ a' ∈ S, dist b a' ≤ dist b c → dist b c = dist b a'
c' : V
hc' : sbtw c c' b
this✝ : dist c b ≤ dist c' b
this : c = c'
⊢ False |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | exists_simple_split_right | [349, 1] | [361, 22] | exact hc'.ne12 this | case intro.intro.intro
V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b : V
hab : a ≠ b
c'✝ : V
hc'✝ : sbtw a c'✝ b
S : Set V := {x | sbtw a x b}
c : V
hc : sbtw a c b
hcmin : ∀ a' ∈ S, dist b a' ≤ dist b c → dist b c = dist b a'
c' : V
hc' : sbtw c c' b
this✝ : dist c b ≤ dist c' b
this : c = c'
⊢ False | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | exists_simple_split_right | [349, 1] | [361, 22] | linarith [hc'.dist] | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b : V
hab : a ≠ b
c'✝ : V
hc'✝ : sbtw a c'✝ b
S : Set V := {x | sbtw a x b}
c : V
hc : sbtw a c b
hcmin : ∀ a' ∈ S, dist b a' ≤ dist b c → dist b c = dist b a'
c' : V
hc' : sbtw c c' b
this : dist c b ≤ dist c' b
⊢ dist c c' ≤ 0 | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | case1 | [367, 1] | [423, 59] | simp | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b c d a₁ a₂ a₃ : V
l : List V
habc : SimpleTriangle a b c
habc_min : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c'
hacd : sbtw a c d
hbd' : b ≠ d
hbd : ¬SimpleEdges.Adj b d
hPmin : ∀ (P' : List V), List.Special a b d P' → (a₁ :: a₂ :: a₃ :: l).pathLength ≤ P'.pathLength
ha₁ : a₁ = a
hα : NotCollinear a₁ a₂ a₃
⊢ a₁ :: a₂ :: a₃ :: l ≠ [] | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | case1 | [367, 1] | [423, 59] | have ⟨b₁₂, hb₁₂, hba⟩ := exists_simple_split_right hα.1 c₁1 | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b c d a₁ a₂ a₃ : V
l : List V
habc : SimpleTriangle a b c
habc_min : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c'
hacd : sbtw a c d
hbd' : b ≠ d
hbd : ¬SimpleEdges.Adj b d
hPmin : ∀ (P' : List V), List.Special a b d P' → (a₁ :: a₂ :: a₃ :: l).pathLength ≤ P'.pathLength
ha₁ : a₁ = a
hα : NotCollinear a₁ a₂ a₃
hPd : (a₁ :: a₂ :: a₃ :: l).getLast ⋯ = d
hPc : List.Chain' (fun x x_1 => x ≠ x_1) (a₁ :: a₂ :: a₃ :: l)
c₁1 : ¬SimpleEdges.Adj a₁ a₂
c₁2 : ¬SimpleEdges.Adj a₂ a₃
⊢ False | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b c d a₁ a₂ a₃ : V
l : List V
habc : SimpleTriangle a b c
habc_min : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c'
hacd : sbtw a c d
hbd' : b ≠ d
hbd : ¬SimpleEdges.Adj b d
hPmin : ∀ (P' : List V), List.Special a b d P' → (a₁ :: a₂ :: a₃ :: l).pathLength ≤ P'.pathLength
ha₁ : a₁ = a
hα : NotCollinear a₁ a₂ a₃
hPd : (a₁ :: a₂ :: a₃ :: l).getLast ⋯ = d
hPc : List.Chain' (fun x x_1 => x ≠ x_1) (a₁ :: a₂ :: a₃ :: l)
c₁1 : ¬SimpleEdges.Adj a₁ a₂
c₁2 : ¬SimpleEdges.Adj a₂ a₃
b₁₂ : V
hb₁₂ : sbtw a₁ b₁₂ a₂
hba : SimpleEdges.Adj b₁₂ a₂
⊢ False |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | case1 | [367, 1] | [423, 59] | have ⟨b₂₃, hb₂₃, hab⟩ := exists_simple_split_left hα.2.2.1 c₁2 | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b c d a₁ a₂ a₃ : V
l : List V
habc : SimpleTriangle a b c
habc_min : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c'
hacd : sbtw a c d
hbd' : b ≠ d
hbd : ¬SimpleEdges.Adj b d
hPmin : ∀ (P' : List V), List.Special a b d P' → (a₁ :: a₂ :: a₃ :: l).pathLength ≤ P'.pathLength
ha₁ : a₁ = a
hα : NotCollinear a₁ a₂ a₃
hPd : (a₁ :: a₂ :: a₃ :: l).getLast ⋯ = d
hPc : List.Chain' (fun x x_1 => x ≠ x_1) (a₁ :: a₂ :: a₃ :: l)
c₁1 : ¬SimpleEdges.Adj a₁ a₂
c₁2 : ¬SimpleEdges.Adj a₂ a₃
b₁₂ : V
hb₁₂ : sbtw a₁ b₁₂ a₂
hba : SimpleEdges.Adj b₁₂ a₂
⊢ False | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b c d a₁ a₂ a₃ : V
l : List V
habc : SimpleTriangle a b c
habc_min : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c'
hacd : sbtw a c d
hbd' : b ≠ d
hbd : ¬SimpleEdges.Adj b d
hPmin : ∀ (P' : List V), List.Special a b d P' → (a₁ :: a₂ :: a₃ :: l).pathLength ≤ P'.pathLength
ha₁ : a₁ = a
hα : NotCollinear a₁ a₂ a₃
hPd : (a₁ :: a₂ :: a₃ :: l).getLast ⋯ = d
hPc : List.Chain' (fun x x_1 => x ≠ x_1) (a₁ :: a₂ :: a₃ :: l)
c₁1 : ¬SimpleEdges.Adj a₁ a₂
c₁2 : ¬SimpleEdges.Adj a₂ a₃
b₁₂ : V
hb₁₂ : sbtw a₁ b₁₂ a₂
hba : SimpleEdges.Adj b₁₂ a₂
b₂₃ : V
hb₂₃ : sbtw a₂ b₂₃ a₃
hab : SimpleEdges.Adj a₂ b₂₃
⊢ False |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | case1 | [367, 1] | [423, 59] | have hb : NotCollinear b₁₂ a₂ b₂₃ := by
refine NotCollinear.mk fun l hl hl' ↦ ?_
simp only [Set.mem_singleton_iff, Set.mem_insert_iff, Set.subset_def, forall_eq_or_imp,
forall_eq] at hl'
have : a₁ ∈ l := hl.close_left hl'.1 hl'.2.1 hb₁₂
have : a₃ ∈ l := hl.close_right hl'.2.1 hl'.2.2 hb₂₃
exact hα.2.2.2 l hl (by simp [*, -ha₁]) | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b c d a₁ a₂ a₃ : V
l : List V
habc : SimpleTriangle a b c
habc_min : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c'
hacd : sbtw a c d
hbd' : b ≠ d
hbd : ¬SimpleEdges.Adj b d
hPmin : ∀ (P' : List V), List.Special a b d P' → (a₁ :: a₂ :: a₃ :: l).pathLength ≤ P'.pathLength
ha₁ : a₁ = a
hα : NotCollinear a₁ a₂ a₃
hPd : (a₁ :: a₂ :: a₃ :: l).getLast ⋯ = d
hPc : List.Chain' (fun x x_1 => x ≠ x_1) (a₁ :: a₂ :: a₃ :: l)
c₁1 : ¬SimpleEdges.Adj a₁ a₂
c₁2 : ¬SimpleEdges.Adj a₂ a₃
b₁₂ : V
hb₁₂ : sbtw a₁ b₁₂ a₂
hba : SimpleEdges.Adj b₁₂ a₂
b₂₃ : V
hb₂₃ : sbtw a₂ b₂₃ a₃
hab : SimpleEdges.Adj a₂ b₂₃
⊢ False | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b c d a₁ a₂ a₃ : V
l : List V
habc : SimpleTriangle a b c
habc_min : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c'
hacd : sbtw a c d
hbd' : b ≠ d
hbd : ¬SimpleEdges.Adj b d
hPmin : ∀ (P' : List V), List.Special a b d P' → (a₁ :: a₂ :: a₃ :: l).pathLength ≤ P'.pathLength
ha₁ : a₁ = a
hα : NotCollinear a₁ a₂ a₃
hPd : (a₁ :: a₂ :: a₃ :: l).getLast ⋯ = d
hPc : List.Chain' (fun x x_1 => x ≠ x_1) (a₁ :: a₂ :: a₃ :: l)
c₁1 : ¬SimpleEdges.Adj a₁ a₂
c₁2 : ¬SimpleEdges.Adj a₂ a₃
b₁₂ : V
hb₁₂ : sbtw a₁ b₁₂ a₂
hba : SimpleEdges.Adj b₁₂ a₂
b₂₃ : V
hb₂₃ : sbtw a₂ b₂₃ a₃
hab : SimpleEdges.Adj a₂ b₂₃
hb : NotCollinear b₁₂ a₂ b₂₃
⊢ False |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | case1 | [367, 1] | [423, 59] | refine NotCollinear.mk fun l hl hl' ↦ ?_ | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b c d a₁ a₂ a₃ : V
l : List V
habc : SimpleTriangle a b c
habc_min : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c'
hacd : sbtw a c d
hbd' : b ≠ d
hbd : ¬SimpleEdges.Adj b d
hPmin : ∀ (P' : List V), List.Special a b d P' → (a₁ :: a₂ :: a₃ :: l).pathLength ≤ P'.pathLength
ha₁ : a₁ = a
hα : NotCollinear a₁ a₂ a₃
hPd : (a₁ :: a₂ :: a₃ :: l).getLast ⋯ = d
hPc : List.Chain' (fun x x_1 => x ≠ x_1) (a₁ :: a₂ :: a₃ :: l)
c₁1 : ¬SimpleEdges.Adj a₁ a₂
c₁2 : ¬SimpleEdges.Adj a₂ a₃
b₁₂ : V
hb₁₂ : sbtw a₁ b₁₂ a₂
hba : SimpleEdges.Adj b₁₂ a₂
b₂₃ : V
hb₂₃ : sbtw a₂ b₂₃ a₃
hab : SimpleEdges.Adj a₂ b₂₃
⊢ NotCollinear b₁₂ a₂ b₂₃ | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b c d a₁ a₂ a₃ : V
l✝ : List V
habc : SimpleTriangle a b c
habc_min : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c'
hacd : sbtw a c d
hbd' : b ≠ d
hbd : ¬SimpleEdges.Adj b d
hPmin : ∀ (P' : List V), List.Special a b d P' → (a₁ :: a₂ :: a₃ :: l✝).pathLength ≤ P'.pathLength
ha₁ : a₁ = a
hα : NotCollinear a₁ a₂ a₃
hPd : (a₁ :: a₂ :: a₃ :: l✝).getLast ⋯ = d
hPc : List.Chain' (fun x x_1 => x ≠ x_1) (a₁ :: a₂ :: a₃ :: l✝)
c₁1 : ¬SimpleEdges.Adj a₁ a₂
c₁2 : ¬SimpleEdges.Adj a₂ a₃
b₁₂ : V
hb₁₂ : sbtw a₁ b₁₂ a₂
hba : SimpleEdges.Adj b₁₂ a₂
b₂₃ : V
hb₂₃ : sbtw a₂ b₂₃ a₃
hab : SimpleEdges.Adj a₂ b₂₃
l : Set V
hl : l.IsLine
hl' : {b₁₂, a₂, b₂₃} ⊆ l
⊢ False |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | case1 | [367, 1] | [423, 59] | simp only [Set.mem_singleton_iff, Set.mem_insert_iff, Set.subset_def, forall_eq_or_imp,
forall_eq] at hl' | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b c d a₁ a₂ a₃ : V
l✝ : List V
habc : SimpleTriangle a b c
habc_min : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c'
hacd : sbtw a c d
hbd' : b ≠ d
hbd : ¬SimpleEdges.Adj b d
hPmin : ∀ (P' : List V), List.Special a b d P' → (a₁ :: a₂ :: a₃ :: l✝).pathLength ≤ P'.pathLength
ha₁ : a₁ = a
hα : NotCollinear a₁ a₂ a₃
hPd : (a₁ :: a₂ :: a₃ :: l✝).getLast ⋯ = d
hPc : List.Chain' (fun x x_1 => x ≠ x_1) (a₁ :: a₂ :: a₃ :: l✝)
c₁1 : ¬SimpleEdges.Adj a₁ a₂
c₁2 : ¬SimpleEdges.Adj a₂ a₃
b₁₂ : V
hb₁₂ : sbtw a₁ b₁₂ a₂
hba : SimpleEdges.Adj b₁₂ a₂
b₂₃ : V
hb₂₃ : sbtw a₂ b₂₃ a₃
hab : SimpleEdges.Adj a₂ b₂₃
l : Set V
hl : l.IsLine
hl' : {b₁₂, a₂, b₂₃} ⊆ l
⊢ False | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b c d a₁ a₂ a₃ : V
l✝ : List V
habc : SimpleTriangle a b c
habc_min : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c'
hacd : sbtw a c d
hbd' : b ≠ d
hbd : ¬SimpleEdges.Adj b d
hPmin : ∀ (P' : List V), List.Special a b d P' → (a₁ :: a₂ :: a₃ :: l✝).pathLength ≤ P'.pathLength
ha₁ : a₁ = a
hα : NotCollinear a₁ a₂ a₃
hPd : (a₁ :: a₂ :: a₃ :: l✝).getLast ⋯ = d
hPc : List.Chain' (fun x x_1 => x ≠ x_1) (a₁ :: a₂ :: a₃ :: l✝)
c₁1 : ¬SimpleEdges.Adj a₁ a₂
c₁2 : ¬SimpleEdges.Adj a₂ a₃
b₁₂ : V
hb₁₂ : sbtw a₁ b₁₂ a₂
hba : SimpleEdges.Adj b₁₂ a₂
b₂₃ : V
hb₂₃ : sbtw a₂ b₂₃ a₃
hab : SimpleEdges.Adj a₂ b₂₃
l : Set V
hl : l.IsLine
hl' : b₁₂ ∈ l ∧ a₂ ∈ l ∧ b₂₃ ∈ l
⊢ False |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | case1 | [367, 1] | [423, 59] | have : a₁ ∈ l := hl.close_left hl'.1 hl'.2.1 hb₁₂ | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b c d a₁ a₂ a₃ : V
l✝ : List V
habc : SimpleTriangle a b c
habc_min : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c'
hacd : sbtw a c d
hbd' : b ≠ d
hbd : ¬SimpleEdges.Adj b d
hPmin : ∀ (P' : List V), List.Special a b d P' → (a₁ :: a₂ :: a₃ :: l✝).pathLength ≤ P'.pathLength
ha₁ : a₁ = a
hα : NotCollinear a₁ a₂ a₃
hPd : (a₁ :: a₂ :: a₃ :: l✝).getLast ⋯ = d
hPc : List.Chain' (fun x x_1 => x ≠ x_1) (a₁ :: a₂ :: a₃ :: l✝)
c₁1 : ¬SimpleEdges.Adj a₁ a₂
c₁2 : ¬SimpleEdges.Adj a₂ a₃
b₁₂ : V
hb₁₂ : sbtw a₁ b₁₂ a₂
hba : SimpleEdges.Adj b₁₂ a₂
b₂₃ : V
hb₂₃ : sbtw a₂ b₂₃ a₃
hab : SimpleEdges.Adj a₂ b₂₃
l : Set V
hl : l.IsLine
hl' : b₁₂ ∈ l ∧ a₂ ∈ l ∧ b₂₃ ∈ l
⊢ False | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b c d a₁ a₂ a₃ : V
l✝ : List V
habc : SimpleTriangle a b c
habc_min : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c'
hacd : sbtw a c d
hbd' : b ≠ d
hbd : ¬SimpleEdges.Adj b d
hPmin : ∀ (P' : List V), List.Special a b d P' → (a₁ :: a₂ :: a₃ :: l✝).pathLength ≤ P'.pathLength
ha₁ : a₁ = a
hα : NotCollinear a₁ a₂ a₃
hPd : (a₁ :: a₂ :: a₃ :: l✝).getLast ⋯ = d
hPc : List.Chain' (fun x x_1 => x ≠ x_1) (a₁ :: a₂ :: a₃ :: l✝)
c₁1 : ¬SimpleEdges.Adj a₁ a₂
c₁2 : ¬SimpleEdges.Adj a₂ a₃
b₁₂ : V
hb₁₂ : sbtw a₁ b₁₂ a₂
hba : SimpleEdges.Adj b₁₂ a₂
b₂₃ : V
hb₂₃ : sbtw a₂ b₂₃ a₃
hab : SimpleEdges.Adj a₂ b₂₃
l : Set V
hl : l.IsLine
hl' : b₁₂ ∈ l ∧ a₂ ∈ l ∧ b₂₃ ∈ l
this : a₁ ∈ l
⊢ False |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | case1 | [367, 1] | [423, 59] | have : a₃ ∈ l := hl.close_right hl'.2.1 hl'.2.2 hb₂₃ | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b c d a₁ a₂ a₃ : V
l✝ : List V
habc : SimpleTriangle a b c
habc_min : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c'
hacd : sbtw a c d
hbd' : b ≠ d
hbd : ¬SimpleEdges.Adj b d
hPmin : ∀ (P' : List V), List.Special a b d P' → (a₁ :: a₂ :: a₃ :: l✝).pathLength ≤ P'.pathLength
ha₁ : a₁ = a
hα : NotCollinear a₁ a₂ a₃
hPd : (a₁ :: a₂ :: a₃ :: l✝).getLast ⋯ = d
hPc : List.Chain' (fun x x_1 => x ≠ x_1) (a₁ :: a₂ :: a₃ :: l✝)
c₁1 : ¬SimpleEdges.Adj a₁ a₂
c₁2 : ¬SimpleEdges.Adj a₂ a₃
b₁₂ : V
hb₁₂ : sbtw a₁ b₁₂ a₂
hba : SimpleEdges.Adj b₁₂ a₂
b₂₃ : V
hb₂₃ : sbtw a₂ b₂₃ a₃
hab : SimpleEdges.Adj a₂ b₂₃
l : Set V
hl : l.IsLine
hl' : b₁₂ ∈ l ∧ a₂ ∈ l ∧ b₂₃ ∈ l
this : a₁ ∈ l
⊢ False | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b c d a₁ a₂ a₃ : V
l✝ : List V
habc : SimpleTriangle a b c
habc_min : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c'
hacd : sbtw a c d
hbd' : b ≠ d
hbd : ¬SimpleEdges.Adj b d
hPmin : ∀ (P' : List V), List.Special a b d P' → (a₁ :: a₂ :: a₃ :: l✝).pathLength ≤ P'.pathLength
ha₁ : a₁ = a
hα : NotCollinear a₁ a₂ a₃
hPd : (a₁ :: a₂ :: a₃ :: l✝).getLast ⋯ = d
hPc : List.Chain' (fun x x_1 => x ≠ x_1) (a₁ :: a₂ :: a₃ :: l✝)
c₁1 : ¬SimpleEdges.Adj a₁ a₂
c₁2 : ¬SimpleEdges.Adj a₂ a₃
b₁₂ : V
hb₁₂ : sbtw a₁ b₁₂ a₂
hba : SimpleEdges.Adj b₁₂ a₂
b₂₃ : V
hb₂₃ : sbtw a₂ b₂₃ a₃
hab : SimpleEdges.Adj a₂ b₂₃
l : Set V
hl : l.IsLine
hl' : b₁₂ ∈ l ∧ a₂ ∈ l ∧ b₂₃ ∈ l
this✝ : a₁ ∈ l
this : a₃ ∈ l
⊢ False |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | case1 | [367, 1] | [423, 59] | exact hα.2.2.2 l hl (by simp [*, -ha₁]) | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b c d a₁ a₂ a₃ : V
l✝ : List V
habc : SimpleTriangle a b c
habc_min : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c'
hacd : sbtw a c d
hbd' : b ≠ d
hbd : ¬SimpleEdges.Adj b d
hPmin : ∀ (P' : List V), List.Special a b d P' → (a₁ :: a₂ :: a₃ :: l✝).pathLength ≤ P'.pathLength
ha₁ : a₁ = a
hα : NotCollinear a₁ a₂ a₃
hPd : (a₁ :: a₂ :: a₃ :: l✝).getLast ⋯ = d
hPc : List.Chain' (fun x x_1 => x ≠ x_1) (a₁ :: a₂ :: a₃ :: l✝)
c₁1 : ¬SimpleEdges.Adj a₁ a₂
c₁2 : ¬SimpleEdges.Adj a₂ a₃
b₁₂ : V
hb₁₂ : sbtw a₁ b₁₂ a₂
hba : SimpleEdges.Adj b₁₂ a₂
b₂₃ : V
hb₂₃ : sbtw a₂ b₂₃ a₃
hab : SimpleEdges.Adj a₂ b₂₃
l : Set V
hl : l.IsLine
hl' : b₁₂ ∈ l ∧ a₂ ∈ l ∧ b₂₃ ∈ l
this✝ : a₁ ∈ l
this : a₃ ∈ l
⊢ False | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | case1 | [367, 1] | [423, 59] | simp [*, -ha₁] | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b c d a₁ a₂ a₃ : V
l✝ : List V
habc : SimpleTriangle a b c
habc_min : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c'
hacd : sbtw a c d
hbd' : b ≠ d
hbd : ¬SimpleEdges.Adj b d
hPmin : ∀ (P' : List V), List.Special a b d P' → (a₁ :: a₂ :: a₃ :: l✝).pathLength ≤ P'.pathLength
ha₁ : a₁ = a
hα : NotCollinear a₁ a₂ a₃
hPd : (a₁ :: a₂ :: a₃ :: l✝).getLast ⋯ = d
hPc : List.Chain' (fun x x_1 => x ≠ x_1) (a₁ :: a₂ :: a₃ :: l✝)
c₁1 : ¬SimpleEdges.Adj a₁ a₂
c₁2 : ¬SimpleEdges.Adj a₂ a₃
b₁₂ : V
hb₁₂ : sbtw a₁ b₁₂ a₂
hba : SimpleEdges.Adj b₁₂ a₂
b₂₃ : V
hb₂₃ : sbtw a₂ b₂₃ a₃
hab : SimpleEdges.Adj a₂ b₂₃
l : Set V
hl : l.IsLine
hl' : b₁₂ ∈ l ∧ a₂ ∈ l ∧ b₂₃ ∈ l
this✝ : a₁ ∈ l
this : a₃ ∈ l
⊢ {a₁, a₂, a₃} ⊆ l | no goals |
Subsets and Splits
No community queries yet
The top public SQL queries from the community will appear here once available.