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
two_implies_three
[530, 1]
[591, 69]
wlog acd : sbtw a c d generalizing a c
case intro.mk.mk.intro.intro.intro 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, SimpleTriangle x y z S : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this : S.Nonempty a b c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line a c ≠ {a, c} d : V hd : d ∈ Line a c hd' : sbtw d a c ∨ sbtw a c d ⊢ False
case intro.mk.mk.intro.intro.intro.inr 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, SimpleTriangle x y z S : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this✝ : S.Nonempty a b c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line a c ≠ {a, c} d : V hd : d ∈ Line a c hd' : sbtw d a c ∨ sbtw a c d this : ∀ (a c : V), SimpleTriangle a b c → (∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c') → Line a c ≠ {a, c} → d ∈ Line a c → sbtw d a c ∨ sbtw a c d → sbtw a c d → False acd : ¬sbtw a c d ⊢ 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, SimpleTriangle x y z S : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this : S.Nonempty b d a c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line a c ≠ {a, c} hd : d ∈ Line a c hd' : sbtw d a c ∨ sbtw a c d acd : sbtw a c d ⊢ False
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/SylvesterChvatal.lean
two_implies_three
[530, 1]
[591, 69]
clear hd'
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, SimpleTriangle x y z S : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this : S.Nonempty b d a c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line a c ≠ {a, c} hd : d ∈ Line a c hd' : sbtw d a c ∨ sbtw a c d acd : sbtw a c d ⊢ 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, SimpleTriangle x y z S : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this : S.Nonempty b d a c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line a c ≠ {a, c} hd : d ∈ Line a c acd : sbtw a c d ⊢ False
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/SylvesterChvatal.lean
two_implies_three
[530, 1]
[591, 69]
let S : Set V := setOf (sbtw a 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, SimpleTriangle x y z S : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this : S.Nonempty b d a c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line a c ≠ {a, c} hd : d ∈ Line a c acd : sbtw a c d ⊢ 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, SimpleTriangle x y z S✝ : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this : S✝.Nonempty b d a c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line a c ≠ {a, c} hd : d ∈ Line a c acd : sbtw a c d S : Set V := setOf (sbtw a c) ⊢ False
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/SylvesterChvatal.lean
two_implies_three
[530, 1]
[591, 69]
obtain ⟨d, hd : sbtw _ _ d, hdmin⟩ := S.toFinite.exists_minimal_wrt (dist c) S ⟨d, acd⟩
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, SimpleTriangle x y z S✝ : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this : S✝.Nonempty b d a c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line a c ≠ {a, c} hd : d ∈ Line a c acd : sbtw a c d S : Set V := setOf (sbtw a c) ⊢ False
case intro.intro 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, SimpleTriangle x y z S✝ : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this : S✝.Nonempty b d✝ a c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line a c ≠ {a, c} hd✝ : d✝ ∈ Line a c acd : sbtw a c d✝ S : Set V := setOf (sbtw a c) d : V hd : sbtw a c d hdmin : ∀ a' ∈ S, dist c a' ≤ dist c d → dist c d = dist c a' ⊢ False
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/SylvesterChvatal.lean
two_implies_three
[530, 1]
[591, 69]
have hbd' : b ≠ d := by rintro rfl have := habc.2.2.2.2.2.2 (Line a c) (Line_isLine hd.ne12) simp [right_extend_mem_Line hd] at this
case intro.intro 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, SimpleTriangle x y z S✝ : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this : S✝.Nonempty b d✝ a c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line a c ≠ {a, c} hd✝ : d✝ ∈ Line a c acd : sbtw a c d✝ S : Set V := setOf (sbtw a c) d : V hd : sbtw a c d hdmin : ∀ a' ∈ S, dist c a' ≤ dist c d → dist c d = dist c a' ⊢ False
case intro.intro 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, SimpleTriangle x y z S✝ : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this : S✝.Nonempty b d✝ a c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line a c ≠ {a, c} hd✝ : d✝ ∈ Line a c acd : sbtw a c d✝ S : Set V := setOf (sbtw a c) d : V hd : sbtw a c d hdmin : ∀ a' ∈ S, dist c a' ≤ dist c d → dist c d = dist c a' hbd' : b ≠ d ⊢ False
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/SylvesterChvatal.lean
two_implies_three
[530, 1]
[591, 69]
replace hdmin : ∀ d', sbtw a c d' → dist c d ≤ dist c d' := by intro d' hd' by_contra! hd'' exact hd''.ne' (hdmin d' hd' hd''.le)
case intro.intro 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, SimpleTriangle x y z S✝ : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this : S✝.Nonempty b d✝ a c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line a c ≠ {a, c} hd✝ : d✝ ∈ Line a c acd : sbtw a c d✝ S : Set V := setOf (sbtw a c) d : V hd : sbtw a c d hdmin : ∀ a' ∈ S, dist c a' ≤ dist c d → dist c d = dist c a' hbd' : b ≠ d ⊢ False
case intro.intro 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, SimpleTriangle x y z S✝ : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this : S✝.Nonempty b d✝ a c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line a c ≠ {a, c} hd✝ : d✝ ∈ Line a c acd : sbtw a c d✝ S : Set V := setOf (sbtw a c) d : V hd : sbtw a c d hbd' : b ≠ d hdmin : ∀ (d' : V), sbtw a c d' → dist c d ≤ dist c d' ⊢ False
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/SylvesterChvatal.lean
two_implies_three
[530, 1]
[591, 69]
have hcd : SimpleEdges.Adj c d := by use hd.2.2.1 intro e he have : 0 ≤ dist e d := dist_nonneg have : dist e d = 0 := by linarith [he.dist, this, hdmin e (hd.right_cancel he)] simp only [dist_eq_zero] at this exact he.ne23 this
case intro.intro 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, SimpleTriangle x y z S✝ : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this : S✝.Nonempty b d✝ a c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line a c ≠ {a, c} hd✝ : d✝ ∈ Line a c acd : sbtw a c d✝ S : Set V := setOf (sbtw a c) d : V hd : sbtw a c d hbd' : b ≠ d hdmin : ∀ (d' : V), sbtw a c d' → dist c d ≤ dist c d' ⊢ False
case intro.intro 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, SimpleTriangle x y z S✝ : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this : S✝.Nonempty b d✝ a c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line a c ≠ {a, c} hd✝ : d✝ ∈ Line a c acd : sbtw a c d✝ S : Set V := setOf (sbtw a c) d : V hd : sbtw a c d hbd' : b ≠ d hdmin : ∀ (d' : V), sbtw a c d' → dist c d ≤ dist c d' hcd : SimpleEdges.Adj c d ⊢ False
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/SylvesterChvatal.lean
two_implies_three
[530, 1]
[591, 69]
have hbd := eqn_7 habc hmin hd hcd
case intro.intro 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, SimpleTriangle x y z S✝ : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this : S✝.Nonempty b d✝ a c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line a c ≠ {a, c} hd✝ : d✝ ∈ Line a c acd : sbtw a c d✝ S : Set V := setOf (sbtw a c) d : V hd : sbtw a c d hbd' : b ≠ d hdmin : ∀ (d' : V), sbtw a c d' → dist c d ≤ dist c d' hcd : SimpleEdges.Adj c d ⊢ False
case intro.intro 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, SimpleTriangle x y z S✝ : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this : S✝.Nonempty b d✝ a c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line a c ≠ {a, c} hd✝ : d✝ ∈ Line a c acd : sbtw a c d✝ S : Set V := setOf (sbtw a c) d : V hd : sbtw a c d hbd' : b ≠ d hdmin : ∀ (d' : V), sbtw a c d' → dist c d ≤ dist c d' hcd : SimpleEdges.Adj c d hbd : ¬SimpleEdges.Adj b d ⊢ False
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/SylvesterChvatal.lean
two_implies_three
[530, 1]
[591, 69]
let S : Set (List V) := setOf (List.Special a b d)
case intro.intro 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, SimpleTriangle x y z S✝ : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this : S✝.Nonempty b d✝ a c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line a c ≠ {a, c} hd✝ : d✝ ∈ Line a c acd : sbtw a c d✝ S : Set V := setOf (sbtw a c) d : V hd : sbtw a c d hbd' : b ≠ d hdmin : ∀ (d' : V), sbtw a c d' → dist c d ≤ dist c d' hcd : SimpleEdges.Adj c d hbd : ¬SimpleEdges.Adj b d ⊢ False
case intro.intro 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, SimpleTriangle x y z S✝¹ : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this : S✝¹.Nonempty b d✝ a c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line a c ≠ {a, c} hd✝ : d✝ ∈ Line a c acd : sbtw a c d✝ S✝ : Set V := setOf (sbtw a c) d : V hd : sbtw a c d hbd' : b ≠ d hdmin : ∀ (d' : V), sbtw a c d' → dist c d ≤ dist c d' hcd : SimpleEdges.Adj c d hbd : ¬SimpleEdges.Adj b d S : Set (List V) := setOf (List.Special a b d) ⊢ False
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/SylvesterChvatal.lean
two_implies_three
[530, 1]
[591, 69]
have : S.Finite := by have ⟨n, hn⟩ := uniformly_bounded_of_chain_ne_of_pathLength_le V [a, b, d].pathLength exact (List.finite_length_le _ _).subset fun l hl => hn l hl.chain_ne hl.pathLength_le
case intro.intro 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, SimpleTriangle x y z S✝¹ : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this : S✝¹.Nonempty b d✝ a c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line a c ≠ {a, c} hd✝ : d✝ ∈ Line a c acd : sbtw a c d✝ S✝ : Set V := setOf (sbtw a c) d : V hd : sbtw a c d hbd' : b ≠ d hdmin : ∀ (d' : V), sbtw a c d' → dist c d ≤ dist c d' hcd : SimpleEdges.Adj c d hbd : ¬SimpleEdges.Adj b d S : Set (List V) := setOf (List.Special a b d) ⊢ False
case intro.intro 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, SimpleTriangle x y z S✝¹ : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this✝ : S✝¹.Nonempty b d✝ a c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line a c ≠ {a, c} hd✝ : d✝ ∈ Line a c acd : sbtw a c d✝ S✝ : Set V := setOf (sbtw a c) d : V hd : sbtw a c d hbd' : b ≠ d hdmin : ∀ (d' : V), sbtw a c d' → dist c d ≤ dist c d' hcd : SimpleEdges.Adj c d hbd : ¬SimpleEdges.Adj b d S : Set (List V) := setOf (List.Special a b d) this : S.Finite ⊢ False
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/SylvesterChvatal.lean
two_implies_three
[530, 1]
[591, 69]
have ⟨P, (hP : P.Special a b d), hPmin⟩ := this.exists_minimal_wrt List.pathLength S ⟨[a, b, d], abd_special habc hd hbd' hbd⟩
case intro.intro 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, SimpleTriangle x y z S✝¹ : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this✝ : S✝¹.Nonempty b d✝ a c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line a c ≠ {a, c} hd✝ : d✝ ∈ Line a c acd : sbtw a c d✝ S✝ : Set V := setOf (sbtw a c) d : V hd : sbtw a c d hbd' : b ≠ d hdmin : ∀ (d' : V), sbtw a c d' → dist c d ≤ dist c d' hcd : SimpleEdges.Adj c d hbd : ¬SimpleEdges.Adj b d S : Set (List V) := setOf (List.Special a b d) this : S.Finite ⊢ False
case intro.intro 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, SimpleTriangle x y z S✝¹ : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this✝ : S✝¹.Nonempty b d✝ a c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line a c ≠ {a, c} hd✝ : d✝ ∈ Line a c acd : sbtw a c d✝ S✝ : Set V := setOf (sbtw a c) d : V hd : sbtw a c d hbd' : b ≠ d hdmin : ∀ (d' : V), sbtw a c d' → dist c d ≤ dist c d' hcd : SimpleEdges.Adj c d hbd : ¬SimpleEdges.Adj b d S : Set (List V) := setOf (List.Special a b d) this : S.Finite P : List V hP : List.Special a b d P hPmin : ∀ a' ∈ S, a'.pathLength ≤ P.pathLength → P.pathLength = a'.pathLength ⊢ False
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/SylvesterChvatal.lean
two_implies_three
[530, 1]
[591, 69]
replace hPmin : ∀ P' : List V, P'.Special a b d → P.pathLength ≤ P'.pathLength := by intro P' hP' by_contra! h exact h.ne' (hPmin P' hP' h.le)
case intro.intro 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, SimpleTriangle x y z S✝¹ : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this✝ : S✝¹.Nonempty b d✝ a c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line a c ≠ {a, c} hd✝ : d✝ ∈ Line a c acd : sbtw a c d✝ S✝ : Set V := setOf (sbtw a c) d : V hd : sbtw a c d hbd' : b ≠ d hdmin : ∀ (d' : V), sbtw a c d' → dist c d ≤ dist c d' hcd : SimpleEdges.Adj c d hbd : ¬SimpleEdges.Adj b d S : Set (List V) := setOf (List.Special a b d) this : S.Finite P : List V hP : List.Special a b d P hPmin : ∀ a' ∈ S, a'.pathLength ≤ P.pathLength → P.pathLength = a'.pathLength ⊢ False
case intro.intro 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, SimpleTriangle x y z S✝¹ : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this✝ : S✝¹.Nonempty b d✝ a c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line a c ≠ {a, c} hd✝ : d✝ ∈ Line a c acd : sbtw a c d✝ S✝ : Set V := setOf (sbtw a c) d : V hd : sbtw a c d hbd' : b ≠ d hdmin : ∀ (d' : V), sbtw a c d' → dist c d ≤ dist c d' hcd : SimpleEdges.Adj c d hbd : ¬SimpleEdges.Adj b d S : Set (List V) := setOf (List.Special a b d) this : S.Finite P : List V hP : List.Special a b d P hPmin : ∀ (P' : List V), List.Special a b d P' → P.pathLength ≤ P'.pathLength ⊢ False
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/SylvesterChvatal.lean
two_implies_three
[530, 1]
[591, 69]
intro a' b' c' h
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, SimpleTriangle x y z S : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this : S.Nonempty a b c : V habc : SimpleTriangle a b c hmin : ∀ a' ∈ S, ((match a' with | (x, y, z) => Delta x y z) ≤ match (a, b, c) with | (x, y, z) => Delta x y z) → (match (a, b, c) with | (x, y, z) => Delta x y z) = match a' with | (x, y, z) => Delta x y z ⊢ ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' 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, SimpleTriangle x y z S : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this : S.Nonempty a b c : V habc : SimpleTriangle a b c hmin : ∀ a' ∈ S, ((match a' with | (x, y, z) => Delta x y z) ≤ match (a, b, c) with | (x, y, z) => Delta x y z) → (match (a, b, c) with | (x, y, z) => Delta x y z) = match a' with | (x, y, z) => Delta x y z a' b' c' : V h : SimpleTriangle a' b' c' ⊢ Delta a b c ≤ Delta a' b' c'
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/SylvesterChvatal.lean
two_implies_three
[530, 1]
[591, 69]
by_contra! h'
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, SimpleTriangle x y z S : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this : S.Nonempty a b c : V habc : SimpleTriangle a b c hmin : ∀ a' ∈ S, ((match a' with | (x, y, z) => Delta x y z) ≤ match (a, b, c) with | (x, y, z) => Delta x y z) → (match (a, b, c) with | (x, y, z) => Delta x y z) = match a' with | (x, y, z) => Delta x y z a' b' c' : V h : SimpleTriangle a' b' c' ⊢ Delta a b c ≤ Delta a' 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, SimpleTriangle x y z S : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this : S.Nonempty a b c : V habc : SimpleTriangle a b c hmin : ∀ a' ∈ S, ((match a' with | (x, y, z) => Delta x y z) ≤ match (a, b, c) with | (x, y, z) => Delta x y z) → (match (a, b, c) with | (x, y, z) => Delta x y z) = match a' with | (x, y, z) => Delta x y z a' b' c' : V h : SimpleTriangle a' b' c' h' : Delta a' b' c' < Delta a b c ⊢ False
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/SylvesterChvatal.lean
two_implies_three
[530, 1]
[591, 69]
exact h'.ne' (hmin (a', b', c') h h'.le)
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, SimpleTriangle x y z S : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this : S.Nonempty a b c : V habc : SimpleTriangle a b c hmin : ∀ a' ∈ S, ((match a' with | (x, y, z) => Delta x y z) ≤ match (a, b, c) with | (x, y, z) => Delta x y z) → (match (a, b, c) with | (x, y, z) => Delta x y z) = match a' with | (x, y, z) => Delta x y z a' b' c' : V h : SimpleTriangle a' b' c' h' : Delta a' b' c' < Delta a b c ⊢ False
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/SylvesterChvatal.lean
two_implies_three
[530, 1]
[591, 69]
rw [Line_comm] at hd h3
case intro.mk.mk.intro.intro.intro.inr 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, SimpleTriangle x y z S : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this✝ : S.Nonempty a b c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line a c ≠ {a, c} d : V hd : d ∈ Line a c hd' : sbtw d a c ∨ sbtw a c d this : ∀ (a c : V), SimpleTriangle a b c → (∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c') → Line a c ≠ {a, c} → d ∈ Line a c → sbtw d a c ∨ sbtw a c d → sbtw a c d → False acd : ¬sbtw a c d ⊢ False
case intro.mk.mk.intro.intro.intro.inr 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, SimpleTriangle x y z S : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this✝ : S.Nonempty a b c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line c a ≠ {a, c} d : V hd : d ∈ Line c a hd' : sbtw d a c ∨ sbtw a c d this : ∀ (a c : V), SimpleTriangle a b c → (∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c') → Line a c ≠ {a, c} → d ∈ Line a c → sbtw d a c ∨ sbtw a c d → sbtw a c d → False acd : ¬sbtw a c d ⊢ False
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/SylvesterChvatal.lean
two_implies_three
[530, 1]
[591, 69]
rw [Set.pair_comm] at h3
case intro.mk.mk.intro.intro.intro.inr 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, SimpleTriangle x y z S : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this✝ : S.Nonempty a b c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line c a ≠ {a, c} d : V hd : d ∈ Line c a hd' : sbtw d a c ∨ sbtw a c d this : ∀ (a c : V), SimpleTriangle a b c → (∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c') → Line a c ≠ {a, c} → d ∈ Line a c → sbtw d a c ∨ sbtw a c d → sbtw a c d → False acd : ¬sbtw a c d ⊢ False
case intro.mk.mk.intro.intro.intro.inr 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, SimpleTriangle x y z S : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this✝ : S.Nonempty a b c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line c a ≠ {c, a} d : V hd : d ∈ Line c a hd' : sbtw d a c ∨ sbtw a c d this : ∀ (a c : V), SimpleTriangle a b c → (∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c') → Line a c ≠ {a, c} → d ∈ Line a c → sbtw d a c ∨ sbtw a c d → sbtw a c d → False acd : ¬sbtw a c d ⊢ False
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/SylvesterChvatal.lean
two_implies_three
[530, 1]
[591, 69]
have h' := hd'.resolve_right acd
case intro.mk.mk.intro.intro.intro.inr 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, SimpleTriangle x y z S : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this✝ : S.Nonempty a b c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line c a ≠ {c, a} d : V hd : d ∈ Line c a hd' : sbtw d a c ∨ sbtw a c d this : ∀ (a c : V), SimpleTriangle a b c → (∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c') → Line a c ≠ {a, c} → d ∈ Line a c → sbtw d a c ∨ sbtw a c d → sbtw a c d → False acd : ¬sbtw a c d ⊢ False
case intro.mk.mk.intro.intro.intro.inr 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, SimpleTriangle x y z S : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this✝ : S.Nonempty a b c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line c a ≠ {c, a} d : V hd : d ∈ Line c a hd' : sbtw d a c ∨ sbtw a c d this : ∀ (a c : V), SimpleTriangle a b c → (∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c') → Line a c ≠ {a, c} → d ∈ Line a c → sbtw d a c ∨ sbtw a c d → sbtw a c d → False acd : ¬sbtw a c d h' : sbtw d a c ⊢ False
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/SylvesterChvatal.lean
two_implies_three
[530, 1]
[591, 69]
refine this c a habc.swap ?_ h3 hd (Or.inr h'.symm) h'.symm
case intro.mk.mk.intro.intro.intro.inr 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, SimpleTriangle x y z S : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this✝ : S.Nonempty a b c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line c a ≠ {c, a} d : V hd : d ∈ Line c a hd' : sbtw d a c ∨ sbtw a c d this : ∀ (a c : V), SimpleTriangle a b c → (∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c') → Line a c ≠ {a, c} → d ∈ Line a c → sbtw d a c ∨ sbtw a c d → sbtw a c d → False acd : ¬sbtw a c d h' : sbtw d a c ⊢ False
case intro.mk.mk.intro.intro.intro.inr 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, SimpleTriangle x y z S : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this✝ : S.Nonempty a b c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line c a ≠ {c, a} d : V hd : d ∈ Line c a hd' : sbtw d a c ∨ sbtw a c d this : ∀ (a c : V), SimpleTriangle a b c → (∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c') → Line a c ≠ {a, c} → d ∈ Line a c → sbtw d a c ∨ sbtw a c d → sbtw a c d → False acd : ¬sbtw a c d h' : sbtw d a c ⊢ ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta c b a ≤ Delta a' b' c'
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/SylvesterChvatal.lean
two_implies_three
[530, 1]
[591, 69]
intro a' b' c' h'
case intro.mk.mk.intro.intro.intro.inr 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, SimpleTriangle x y z S : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this✝ : S.Nonempty a b c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line c a ≠ {c, a} d : V hd : d ∈ Line c a hd' : sbtw d a c ∨ sbtw a c d this : ∀ (a c : V), SimpleTriangle a b c → (∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c') → Line a c ≠ {a, c} → d ∈ Line a c → sbtw d a c ∨ sbtw a c d → sbtw a c d → False acd : ¬sbtw a c d h' : sbtw d a c ⊢ ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta c b a ≤ Delta a' b' c'
case intro.mk.mk.intro.intro.intro.inr 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, SimpleTriangle x y z S : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this✝ : S.Nonempty a b c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line c a ≠ {c, a} d : V hd : d ∈ Line c a hd' : sbtw d a c ∨ sbtw a c d this : ∀ (a c : V), SimpleTriangle a b c → (∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c') → Line a c ≠ {a, c} → d ∈ Line a c → sbtw d a c ∨ sbtw a c d → sbtw a c d → False acd : ¬sbtw a c d h'✝ : sbtw d a c a' b' c' : V h' : SimpleTriangle a' b' c' ⊢ Delta c b a ≤ Delta a' b' c'
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/SylvesterChvatal.lean
two_implies_three
[530, 1]
[591, 69]
rw [Delta_comm]
case intro.mk.mk.intro.intro.intro.inr 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, SimpleTriangle x y z S : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this✝ : S.Nonempty a b c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line c a ≠ {c, a} d : V hd : d ∈ Line c a hd' : sbtw d a c ∨ sbtw a c d this : ∀ (a c : V), SimpleTriangle a b c → (∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c') → Line a c ≠ {a, c} → d ∈ Line a c → sbtw d a c ∨ sbtw a c d → sbtw a c d → False acd : ¬sbtw a c d h'✝ : sbtw d a c a' b' c' : V h' : SimpleTriangle a' b' c' ⊢ Delta c b a ≤ Delta a' b' c'
case intro.mk.mk.intro.intro.intro.inr 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, SimpleTriangle x y z S : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this✝ : S.Nonempty a b c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line c a ≠ {c, a} d : V hd : d ∈ Line c a hd' : sbtw d a c ∨ sbtw a c d this : ∀ (a c : V), SimpleTriangle a b c → (∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c') → Line a c ≠ {a, c} → d ∈ Line a c → sbtw d a c ∨ sbtw a c d → sbtw a c d → False acd : ¬sbtw a c d h'✝ : sbtw d a c a' b' c' : V h' : SimpleTriangle a' b' c' ⊢ Delta a b c ≤ Delta a' b' c'
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/SylvesterChvatal.lean
two_implies_three
[530, 1]
[591, 69]
exact hmin _ _ _ h'
case intro.mk.mk.intro.intro.intro.inr 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, SimpleTriangle x y z S : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this✝ : S.Nonempty a b c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line c a ≠ {c, a} d : V hd : d ∈ Line c a hd' : sbtw d a c ∨ sbtw a c d this : ∀ (a c : V), SimpleTriangle a b c → (∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c') → Line a c ≠ {a, c} → d ∈ Line a c → sbtw d a c ∨ sbtw a c d → sbtw a c d → False acd : ¬sbtw a c d h'✝ : sbtw d a c a' b' c' : V h' : SimpleTriangle a' b' c' ⊢ Delta a b c ≤ Delta a' b' c'
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/SylvesterChvatal.lean
two_implies_three
[530, 1]
[591, 69]
rintro rfl
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, SimpleTriangle x y z S✝ : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this : S✝.Nonempty b d✝ a c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line a c ≠ {a, c} hd✝ : d✝ ∈ Line a c acd : sbtw a c d✝ S : Set V := setOf (sbtw a c) d : V hd : sbtw a c d hdmin : ∀ a' ∈ S, dist c a' ≤ dist c d → dist c d = dist c a' ⊢ b ≠ d
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, SimpleTriangle x y z S✝ : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this : S✝.Nonempty b d a c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line a c ≠ {a, c} hd✝ : d ∈ Line a c acd : sbtw a c d S : Set V := setOf (sbtw a c) hd : sbtw a c b hdmin : ∀ a' ∈ S, dist c a' ≤ dist c b → dist c b = dist c a' ⊢ False
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/SylvesterChvatal.lean
two_implies_three
[530, 1]
[591, 69]
have := habc.2.2.2.2.2.2 (Line a c) (Line_isLine hd.ne12)
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, SimpleTriangle x y z S✝ : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this : S✝.Nonempty b d a c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line a c ≠ {a, c} hd✝ : d ∈ Line a c acd : sbtw a c d S : Set V := setOf (sbtw a c) hd : sbtw a c b hdmin : ∀ a' ∈ S, dist c a' ≤ dist c b → dist c b = dist c a' ⊢ 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, SimpleTriangle x y z S✝ : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this✝ : S✝.Nonempty b d a c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line a c ≠ {a, c} hd✝ : d ∈ Line a c acd : sbtw a c d S : Set V := setOf (sbtw a c) hd : sbtw a c b hdmin : ∀ a' ∈ S, dist c a' ≤ dist c b → dist c b = dist c a' this : ¬{a, b, c} ⊆ Line a c ⊢ False
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/SylvesterChvatal.lean
two_implies_three
[530, 1]
[591, 69]
simp [right_extend_mem_Line hd] at this
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, SimpleTriangle x y z S✝ : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this✝ : S✝.Nonempty b d a c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line a c ≠ {a, c} hd✝ : d ∈ Line a c acd : sbtw a c d S : Set V := setOf (sbtw a c) hd : sbtw a c b hdmin : ∀ a' ∈ S, dist c a' ≤ dist c b → dist c b = dist c a' this : ¬{a, b, c} ⊆ Line a c ⊢ False
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/SylvesterChvatal.lean
two_implies_three
[530, 1]
[591, 69]
intro d' hd'
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, SimpleTriangle x y z S✝ : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this : S✝.Nonempty b d✝ a c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line a c ≠ {a, c} hd✝ : d✝ ∈ Line a c acd : sbtw a c d✝ S : Set V := setOf (sbtw a c) d : V hd : sbtw a c d hdmin : ∀ a' ∈ S, dist c a' ≤ dist c d → dist c d = dist c a' hbd' : b ≠ d ⊢ ∀ (d' : V), sbtw a c d' → dist c d ≤ dist c d'
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, SimpleTriangle x y z S✝ : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this : S✝.Nonempty b d✝ a c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line a c ≠ {a, c} hd✝ : d✝ ∈ Line a c acd : sbtw a c d✝ S : Set V := setOf (sbtw a c) d : V hd : sbtw a c d hdmin : ∀ a' ∈ S, dist c a' ≤ dist c d → dist c d = dist c a' hbd' : b ≠ d d' : V hd' : sbtw a c d' ⊢ dist c d ≤ dist c d'
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/SylvesterChvatal.lean
two_implies_three
[530, 1]
[591, 69]
by_contra! hd''
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, SimpleTriangle x y z S✝ : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this : S✝.Nonempty b d✝ a c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line a c ≠ {a, c} hd✝ : d✝ ∈ Line a c acd : sbtw a c d✝ S : Set V := setOf (sbtw a c) d : V hd : sbtw a c d hdmin : ∀ a' ∈ S, dist c a' ≤ dist c d → dist c d = dist c a' hbd' : b ≠ d d' : V hd' : sbtw a c d' ⊢ dist c d ≤ dist c d'
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, SimpleTriangle x y z S✝ : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this : S✝.Nonempty b d✝ a c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line a c ≠ {a, c} hd✝ : d✝ ∈ Line a c acd : sbtw a c d✝ S : Set V := setOf (sbtw a c) d : V hd : sbtw a c d hdmin : ∀ a' ∈ S, dist c a' ≤ dist c d → dist c d = dist c a' hbd' : b ≠ d d' : V hd' : sbtw a c d' hd'' : dist c d' < dist c d ⊢ False
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/SylvesterChvatal.lean
two_implies_three
[530, 1]
[591, 69]
exact hd''.ne' (hdmin d' hd' hd''.le)
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, SimpleTriangle x y z S✝ : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this : S✝.Nonempty b d✝ a c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line a c ≠ {a, c} hd✝ : d✝ ∈ Line a c acd : sbtw a c d✝ S : Set V := setOf (sbtw a c) d : V hd : sbtw a c d hdmin : ∀ a' ∈ S, dist c a' ≤ dist c d → dist c d = dist c a' hbd' : b ≠ d d' : V hd' : sbtw a c d' hd'' : dist c d' < dist c d ⊢ False
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/SylvesterChvatal.lean
two_implies_three
[530, 1]
[591, 69]
use hd.2.2.1
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, SimpleTriangle x y z S✝ : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this : S✝.Nonempty b d✝ a c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line a c ≠ {a, c} hd✝ : d✝ ∈ Line a c acd : sbtw a c d✝ S : Set V := setOf (sbtw a c) d : V hd : sbtw a c d hbd' : b ≠ d hdmin : ∀ (d' : V), sbtw a c d' → dist c d ≤ dist c d' ⊢ SimpleEdges.Adj c d
case right 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, SimpleTriangle x y z S✝ : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this : S✝.Nonempty b d✝ a c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line a c ≠ {a, c} hd✝ : d✝ ∈ Line a c acd : sbtw a c d✝ S : Set V := setOf (sbtw a c) d : V hd : sbtw a c d hbd' : b ≠ d hdmin : ∀ (d' : V), sbtw a c d' → dist c d ≤ dist c d' ⊢ ∀ (x : V), ¬sbtw c x d
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/SylvesterChvatal.lean
two_implies_three
[530, 1]
[591, 69]
intro e he
case right 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, SimpleTriangle x y z S✝ : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this : S✝.Nonempty b d✝ a c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line a c ≠ {a, c} hd✝ : d✝ ∈ Line a c acd : sbtw a c d✝ S : Set V := setOf (sbtw a c) d : V hd : sbtw a c d hbd' : b ≠ d hdmin : ∀ (d' : V), sbtw a c d' → dist c d ≤ dist c d' ⊢ ∀ (x : V), ¬sbtw c x d
case right 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, SimpleTriangle x y z S✝ : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this : S✝.Nonempty b d✝ a c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line a c ≠ {a, c} hd✝ : d✝ ∈ Line a c acd : sbtw a c d✝ S : Set V := setOf (sbtw a c) d : V hd : sbtw a c d hbd' : b ≠ d hdmin : ∀ (d' : V), sbtw a c d' → dist c d ≤ dist c d' e : V he : sbtw c e d ⊢ False
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/SylvesterChvatal.lean
two_implies_three
[530, 1]
[591, 69]
have : 0 ≤ dist e d := dist_nonneg
case right 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, SimpleTriangle x y z S✝ : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this : S✝.Nonempty b d✝ a c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line a c ≠ {a, c} hd✝ : d✝ ∈ Line a c acd : sbtw a c d✝ S : Set V := setOf (sbtw a c) d : V hd : sbtw a c d hbd' : b ≠ d hdmin : ∀ (d' : V), sbtw a c d' → dist c d ≤ dist c d' e : V he : sbtw c e d ⊢ False
case right 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, SimpleTriangle x y z S✝ : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this✝ : S✝.Nonempty b d✝ a c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line a c ≠ {a, c} hd✝ : d✝ ∈ Line a c acd : sbtw a c d✝ S : Set V := setOf (sbtw a c) d : V hd : sbtw a c d hbd' : b ≠ d hdmin : ∀ (d' : V), sbtw a c d' → dist c d ≤ dist c d' e : V he : sbtw c e d this : 0 ≤ dist e d ⊢ False
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/SylvesterChvatal.lean
two_implies_three
[530, 1]
[591, 69]
have : dist e d = 0 := by linarith [he.dist, this, hdmin e (hd.right_cancel he)]
case right 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, SimpleTriangle x y z S✝ : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this✝ : S✝.Nonempty b d✝ a c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line a c ≠ {a, c} hd✝ : d✝ ∈ Line a c acd : sbtw a c d✝ S : Set V := setOf (sbtw a c) d : V hd : sbtw a c d hbd' : b ≠ d hdmin : ∀ (d' : V), sbtw a c d' → dist c d ≤ dist c d' e : V he : sbtw c e d this : 0 ≤ dist e d ⊢ False
case right 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, SimpleTriangle x y z S✝ : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this✝¹ : S✝.Nonempty b d✝ a c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line a c ≠ {a, c} hd✝ : d✝ ∈ Line a c acd : sbtw a c d✝ S : Set V := setOf (sbtw a c) d : V hd : sbtw a c d hbd' : b ≠ d hdmin : ∀ (d' : V), sbtw a c d' → dist c d ≤ dist c d' e : V he : sbtw c e d this✝ : 0 ≤ dist e d this : dist e d = 0 ⊢ False
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/SylvesterChvatal.lean
two_implies_three
[530, 1]
[591, 69]
simp only [dist_eq_zero] at this
case right 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, SimpleTriangle x y z S✝ : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this✝¹ : S✝.Nonempty b d✝ a c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line a c ≠ {a, c} hd✝ : d✝ ∈ Line a c acd : sbtw a c d✝ S : Set V := setOf (sbtw a c) d : V hd : sbtw a c d hbd' : b ≠ d hdmin : ∀ (d' : V), sbtw a c d' → dist c d ≤ dist c d' e : V he : sbtw c e d this✝ : 0 ≤ dist e d this : dist e d = 0 ⊢ False
case right 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, SimpleTriangle x y z S✝ : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this✝¹ : S✝.Nonempty b d✝ a c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line a c ≠ {a, c} hd✝ : d✝ ∈ Line a c acd : sbtw a c d✝ S : Set V := setOf (sbtw a c) d : V hd : sbtw a c d hbd' : b ≠ d hdmin : ∀ (d' : V), sbtw a c d' → dist c d ≤ dist c d' e : V he : sbtw c e d this✝ : 0 ≤ dist e d this : e = d ⊢ False
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/SylvesterChvatal.lean
two_implies_three
[530, 1]
[591, 69]
exact he.ne23 this
case right 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, SimpleTriangle x y z S✝ : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this✝¹ : S✝.Nonempty b d✝ a c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line a c ≠ {a, c} hd✝ : d✝ ∈ Line a c acd : sbtw a c d✝ S : Set V := setOf (sbtw a c) d : V hd : sbtw a c d hbd' : b ≠ d hdmin : ∀ (d' : V), sbtw a c d' → dist c d ≤ dist c d' e : V he : sbtw c e d this✝ : 0 ≤ dist e d this : e = d ⊢ False
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/SylvesterChvatal.lean
two_implies_three
[530, 1]
[591, 69]
linarith [he.dist, this, hdmin e (hd.right_cancel he)]
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, SimpleTriangle x y z S✝ : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this✝ : S✝.Nonempty b d✝ a c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line a c ≠ {a, c} hd✝ : d✝ ∈ Line a c acd : sbtw a c d✝ S : Set V := setOf (sbtw a c) d : V hd : sbtw a c d hbd' : b ≠ d hdmin : ∀ (d' : V), sbtw a c d' → dist c d ≤ dist c d' e : V he : sbtw c e d this : 0 ≤ dist e d ⊢ dist e d = 0
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/SylvesterChvatal.lean
two_implies_three
[530, 1]
[591, 69]
have ⟨n, hn⟩ := uniformly_bounded_of_chain_ne_of_pathLength_le V [a, b, d].pathLength
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, SimpleTriangle x y z S✝¹ : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this : S✝¹.Nonempty b d✝ a c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line a c ≠ {a, c} hd✝ : d✝ ∈ Line a c acd : sbtw a c d✝ S✝ : Set V := setOf (sbtw a c) d : V hd : sbtw a c d hbd' : b ≠ d hdmin : ∀ (d' : V), sbtw a c d' → dist c d ≤ dist c d' hcd : SimpleEdges.Adj c d hbd : ¬SimpleEdges.Adj b d S : Set (List V) := setOf (List.Special a b d) ⊢ S.Finite
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, SimpleTriangle x y z S✝¹ : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this : S✝¹.Nonempty b d✝ a c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line a c ≠ {a, c} hd✝ : d✝ ∈ Line a c acd : sbtw a c d✝ S✝ : Set V := setOf (sbtw a c) d : V hd : sbtw a c d hbd' : b ≠ d hdmin : ∀ (d' : V), sbtw a c d' → dist c d ≤ dist c d' hcd : SimpleEdges.Adj c d hbd : ¬SimpleEdges.Adj b d S : Set (List V) := setOf (List.Special a b d) n : ℕ hn : ∀ (l : List V), List.Chain' (fun x x_1 => x ≠ x_1) l → l.pathLength ≤ [a, b, d].pathLength → l.length ≤ n ⊢ S.Finite
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/SylvesterChvatal.lean
two_implies_three
[530, 1]
[591, 69]
exact (List.finite_length_le _ _).subset fun l hl => hn l hl.chain_ne hl.pathLength_le
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, SimpleTriangle x y z S✝¹ : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this : S✝¹.Nonempty b d✝ a c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line a c ≠ {a, c} hd✝ : d✝ ∈ Line a c acd : sbtw a c d✝ S✝ : Set V := setOf (sbtw a c) d : V hd : sbtw a c d hbd' : b ≠ d hdmin : ∀ (d' : V), sbtw a c d' → dist c d ≤ dist c d' hcd : SimpleEdges.Adj c d hbd : ¬SimpleEdges.Adj b d S : Set (List V) := setOf (List.Special a b d) n : ℕ hn : ∀ (l : List V), List.Chain' (fun x x_1 => x ≠ x_1) l → l.pathLength ≤ [a, b, d].pathLength → l.length ≤ n ⊢ S.Finite
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/SylvesterChvatal.lean
two_implies_three
[530, 1]
[591, 69]
intro P' hP'
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, SimpleTriangle x y z S✝¹ : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this✝ : S✝¹.Nonempty b d✝ a c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line a c ≠ {a, c} hd✝ : d✝ ∈ Line a c acd : sbtw a c d✝ S✝ : Set V := setOf (sbtw a c) d : V hd : sbtw a c d hbd' : b ≠ d hdmin : ∀ (d' : V), sbtw a c d' → dist c d ≤ dist c d' hcd : SimpleEdges.Adj c d hbd : ¬SimpleEdges.Adj b d S : Set (List V) := setOf (List.Special a b d) this : S.Finite P : List V hP : List.Special a b d P hPmin : ∀ a' ∈ S, a'.pathLength ≤ P.pathLength → P.pathLength = a'.pathLength ⊢ ∀ (P' : List V), List.Special a b d P' → P.pathLength ≤ P'.pathLength
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, SimpleTriangle x y z S✝¹ : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this✝ : S✝¹.Nonempty b d✝ a c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line a c ≠ {a, c} hd✝ : d✝ ∈ Line a c acd : sbtw a c d✝ S✝ : Set V := setOf (sbtw a c) d : V hd : sbtw a c d hbd' : b ≠ d hdmin : ∀ (d' : V), sbtw a c d' → dist c d ≤ dist c d' hcd : SimpleEdges.Adj c d hbd : ¬SimpleEdges.Adj b d S : Set (List V) := setOf (List.Special a b d) this : S.Finite P : List V hP : List.Special a b d P hPmin : ∀ a' ∈ S, a'.pathLength ≤ P.pathLength → P.pathLength = a'.pathLength P' : List V hP' : List.Special a b d P' ⊢ P.pathLength ≤ P'.pathLength
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/SylvesterChvatal.lean
two_implies_three
[530, 1]
[591, 69]
by_contra! h
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, SimpleTriangle x y z S✝¹ : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this✝ : S✝¹.Nonempty b d✝ a c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line a c ≠ {a, c} hd✝ : d✝ ∈ Line a c acd : sbtw a c d✝ S✝ : Set V := setOf (sbtw a c) d : V hd : sbtw a c d hbd' : b ≠ d hdmin : ∀ (d' : V), sbtw a c d' → dist c d ≤ dist c d' hcd : SimpleEdges.Adj c d hbd : ¬SimpleEdges.Adj b d S : Set (List V) := setOf (List.Special a b d) this : S.Finite P : List V hP : List.Special a b d P hPmin : ∀ a' ∈ S, a'.pathLength ≤ P.pathLength → P.pathLength = a'.pathLength P' : List V hP' : List.Special a b d P' ⊢ P.pathLength ≤ P'.pathLength
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, SimpleTriangle x y z S✝¹ : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this✝ : S✝¹.Nonempty b d✝ a c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line a c ≠ {a, c} hd✝ : d✝ ∈ Line a c acd : sbtw a c d✝ S✝ : Set V := setOf (sbtw a c) d : V hd : sbtw a c d hbd' : b ≠ d hdmin : ∀ (d' : V), sbtw a c d' → dist c d ≤ dist c d' hcd : SimpleEdges.Adj c d hbd : ¬SimpleEdges.Adj b d S : Set (List V) := setOf (List.Special a b d) this : S.Finite P : List V hP : List.Special a b d P hPmin : ∀ a' ∈ S, a'.pathLength ≤ P.pathLength → P.pathLength = a'.pathLength P' : List V hP' : List.Special a b d P' h : P'.pathLength < P.pathLength ⊢ False
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/SylvesterChvatal.lean
two_implies_three
[530, 1]
[591, 69]
exact h.ne' (hPmin P' hP' h.le)
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, SimpleTriangle x y z S✝¹ : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this✝ : S✝¹.Nonempty b d✝ a c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line a c ≠ {a, c} hd✝ : d✝ ∈ Line a c acd : sbtw a c d✝ S✝ : Set V := setOf (sbtw a c) d : V hd : sbtw a c d hbd' : b ≠ d hdmin : ∀ (d' : V), sbtw a c d' → dist c d ≤ dist c d' hcd : SimpleEdges.Adj c d hbd : ¬SimpleEdges.Adj b d S : Set (List V) := setOf (List.Special a b d) this : S.Finite P : List V hP : List.Special a b d P hPmin : ∀ a' ∈ S, a'.pathLength ≤ P.pathLength → P.pathLength = a'.pathLength P' : List V hP' : List.Special a b d P' h : P'.pathLength < P.pathLength ⊢ False
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/SylvesterChvatal.lean
two_implies_three
[530, 1]
[591, 69]
simp only [List.Special] at hP
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, SimpleTriangle x y z S✝¹ : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this✝ : S✝¹.Nonempty b d✝ a c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line a c ≠ {a, c} hd✝ : d✝ ∈ Line a c acd : sbtw a c d✝ S✝ : Set V := setOf (sbtw a c) d : V hd : sbtw a c d hbd' : b ≠ d hdmin : ∀ (d' : V), sbtw a c d' → dist c d ≤ dist c d' hcd : SimpleEdges.Adj c d hbd : ¬SimpleEdges.Adj b d S : Set (List V) := setOf (List.Special a b d) this : S.Finite P : List V a₁ a₂ a₃ : V l : List V hP : List.Special a b d (a₁ :: a₂ :: a₃ :: l) hPmin : ∀ (P' : List V), List.Special a b d P' → (a₁ :: a₂ :: a₃ :: l).pathLength ≤ P'.pathLength ⊢ 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, SimpleTriangle x y z S✝¹ : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this✝ : S✝¹.Nonempty b d✝ a c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line a c ≠ {a, c} hd✝ : d✝ ∈ Line a c acd : sbtw a c d✝ S✝ : Set V := setOf (sbtw a c) d : V hd : sbtw a c d hbd' : b ≠ d hdmin : ∀ (d' : V), sbtw a c d' → dist c d ≤ dist c d' hcd : SimpleEdges.Adj c d hbd : ¬SimpleEdges.Adj b d S : Set (List V) := setOf (List.Special a b d) this : S.Finite P : List V a₁ a₂ a₃ : V l : List V hP : a₁ = a ∧ NotCollinear a₁ a₂ a₃ ∧ (¬SimpleEdges.Adj a₁ a₂ ∨ ¬SimpleEdges.Adj a₂ a₃) ∧ (a₁ :: a₂ :: a₃ :: l).getLast ⋯ = d ∧ List.Chain' (fun x x_1 => x ≠ x_1) (a₁ :: a₂ :: a₃ :: l) ∧ (a₁ :: a₂ :: a₃ :: l).pathLength ≤ [a, b, d].pathLength hPmin : ∀ (P' : List V), List.Special a b d P' → (a₁ :: a₂ :: a₃ :: l).pathLength ≤ P'.pathLength ⊢ False
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/SylvesterChvatal.lean
two_implies_three
[530, 1]
[591, 69]
rcases hP with ⟨ha₁, hα, hβ, hPd, hPc, _⟩
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, SimpleTriangle x y z S✝¹ : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this✝ : S✝¹.Nonempty b d✝ a c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line a c ≠ {a, c} hd✝ : d✝ ∈ Line a c acd : sbtw a c d✝ S✝ : Set V := setOf (sbtw a c) d : V hd : sbtw a c d hbd' : b ≠ d hdmin : ∀ (d' : V), sbtw a c d' → dist c d ≤ dist c d' hcd : SimpleEdges.Adj c d hbd : ¬SimpleEdges.Adj b d S : Set (List V) := setOf (List.Special a b d) this : S.Finite P : List V a₁ a₂ a₃ : V l : List V hP : a₁ = a ∧ NotCollinear a₁ a₂ a₃ ∧ (¬SimpleEdges.Adj a₁ a₂ ∨ ¬SimpleEdges.Adj a₂ a₃) ∧ (a₁ :: a₂ :: a₃ :: l).getLast ⋯ = d ∧ List.Chain' (fun x x_1 => x ≠ x_1) (a₁ :: a₂ :: a₃ :: l) ∧ (a₁ :: a₂ :: a₃ :: l).pathLength ≤ [a, b, d].pathLength hPmin : ∀ (P' : List V), List.Special a b d P' → (a₁ :: a₂ :: a₃ :: l).pathLength ≤ P'.pathLength ⊢ False
case intro.intro.intro.intro.intro 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, SimpleTriangle x y z S✝¹ : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this✝ : S✝¹.Nonempty b d✝ a c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line a c ≠ {a, c} hd✝ : d✝ ∈ Line a c acd : sbtw a c d✝ S✝ : Set V := setOf (sbtw a c) d : V hd : sbtw a c d hbd' : b ≠ d hdmin : ∀ (d' : V), sbtw a c d' → dist c d ≤ dist c d' hcd : SimpleEdges.Adj c d hbd : ¬SimpleEdges.Adj b d S : Set (List V) := setOf (List.Special a b d) this : S.Finite P : List V a₁ a₂ a₃ : V l : List V 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₃ hβ : ¬SimpleEdges.Adj a₁ a₂ ∨ ¬SimpleEdges.Adj a₂ a₃ hPd : (a₁ :: a₂ :: a₃ :: l).getLast ⋯ = d hPc : List.Chain' (fun x x_1 => x ≠ x_1) (a₁ :: a₂ :: a₃ :: l) right✝ : (a₁ :: a₂ :: a₃ :: l).pathLength ≤ [a, b, d].pathLength ⊢ False
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/SylvesterChvatal.lean
two_implies_three
[530, 1]
[591, 69]
have : (¬ SimpleEdges.Adj a₁ a₂ ∧ ¬ SimpleEdges.Adj a₂ a₃) ∨ (SimpleEdges.Adj a₁ a₂ ∧ ¬ SimpleEdges.Adj a₂ a₃) ∨ (¬ SimpleEdges.Adj a₁ a₂ ∧ SimpleEdges.Adj a₂ a₃) := by tauto
case intro.intro.intro.intro.intro 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, SimpleTriangle x y z S✝¹ : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this✝ : S✝¹.Nonempty b d✝ a c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line a c ≠ {a, c} hd✝ : d✝ ∈ Line a c acd : sbtw a c d✝ S✝ : Set V := setOf (sbtw a c) d : V hd : sbtw a c d hbd' : b ≠ d hdmin : ∀ (d' : V), sbtw a c d' → dist c d ≤ dist c d' hcd : SimpleEdges.Adj c d hbd : ¬SimpleEdges.Adj b d S : Set (List V) := setOf (List.Special a b d) this : S.Finite P : List V a₁ a₂ a₃ : V l : List V 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₃ hβ : ¬SimpleEdges.Adj a₁ a₂ ∨ ¬SimpleEdges.Adj a₂ a₃ hPd : (a₁ :: a₂ :: a₃ :: l).getLast ⋯ = d hPc : List.Chain' (fun x x_1 => x ≠ x_1) (a₁ :: a₂ :: a₃ :: l) right✝ : (a₁ :: a₂ :: a₃ :: l).pathLength ≤ [a, b, d].pathLength ⊢ False
case intro.intro.intro.intro.intro 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, SimpleTriangle x y z S✝¹ : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this✝¹ : S✝¹.Nonempty b d✝ a c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line a c ≠ {a, c} hd✝ : d✝ ∈ Line a c acd : sbtw a c d✝ S✝ : Set V := setOf (sbtw a c) d : V hd : sbtw a c d hbd' : b ≠ d hdmin : ∀ (d' : V), sbtw a c d' → dist c d ≤ dist c d' hcd : SimpleEdges.Adj c d hbd : ¬SimpleEdges.Adj b d S : Set (List V) := setOf (List.Special a b d) this✝ : S.Finite P : List V a₁ a₂ a₃ : V l : List V 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₃ hβ : ¬SimpleEdges.Adj a₁ a₂ ∨ ¬SimpleEdges.Adj a₂ a₃ hPd : (a₁ :: a₂ :: a₃ :: l).getLast ⋯ = d hPc : List.Chain' (fun x x_1 => x ≠ x_1) (a₁ :: a₂ :: a₃ :: l) right✝ : (a₁ :: a₂ :: a₃ :: l).pathLength ≤ [a, b, d].pathLength this : ¬SimpleEdges.Adj a₁ a₂ ∧ ¬SimpleEdges.Adj a₂ a₃ ∨ SimpleEdges.Adj a₁ a₂ ∧ ¬SimpleEdges.Adj a₂ a₃ ∨ ¬SimpleEdges.Adj a₁ a₂ ∧ SimpleEdges.Adj a₂ a₃ ⊢ False
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/SylvesterChvatal.lean
two_implies_three
[530, 1]
[591, 69]
rcases this with (⟨c₁1, c₁2⟩ | ⟨c₂1, c₂2⟩ | ⟨c₃1, c₃2⟩)
case intro.intro.intro.intro.intro 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, SimpleTriangle x y z S✝¹ : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this✝¹ : S✝¹.Nonempty b d✝ a c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line a c ≠ {a, c} hd✝ : d✝ ∈ Line a c acd : sbtw a c d✝ S✝ : Set V := setOf (sbtw a c) d : V hd : sbtw a c d hbd' : b ≠ d hdmin : ∀ (d' : V), sbtw a c d' → dist c d ≤ dist c d' hcd : SimpleEdges.Adj c d hbd : ¬SimpleEdges.Adj b d S : Set (List V) := setOf (List.Special a b d) this✝ : S.Finite P : List V a₁ a₂ a₃ : V l : List V 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₃ hβ : ¬SimpleEdges.Adj a₁ a₂ ∨ ¬SimpleEdges.Adj a₂ a₃ hPd : (a₁ :: a₂ :: a₃ :: l).getLast ⋯ = d hPc : List.Chain' (fun x x_1 => x ≠ x_1) (a₁ :: a₂ :: a₃ :: l) right✝ : (a₁ :: a₂ :: a₃ :: l).pathLength ≤ [a, b, d].pathLength this : ¬SimpleEdges.Adj a₁ a₂ ∧ ¬SimpleEdges.Adj a₂ a₃ ∨ SimpleEdges.Adj a₁ a₂ ∧ ¬SimpleEdges.Adj a₂ a₃ ∨ ¬SimpleEdges.Adj a₁ a₂ ∧ SimpleEdges.Adj a₂ a₃ ⊢ False
case intro.intro.intro.intro.intro.inl.intro 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, SimpleTriangle x y z S✝¹ : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this✝ : S✝¹.Nonempty b d✝ a c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line a c ≠ {a, c} hd✝ : d✝ ∈ Line a c acd : sbtw a c d✝ S✝ : Set V := setOf (sbtw a c) d : V hd : sbtw a c d hbd' : b ≠ d hdmin : ∀ (d' : V), sbtw a c d' → dist c d ≤ dist c d' hcd : SimpleEdges.Adj c d hbd : ¬SimpleEdges.Adj b d S : Set (List V) := setOf (List.Special a b d) this : S.Finite P : List V a₁ a₂ a₃ : V l : List V 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₃ hβ : ¬SimpleEdges.Adj a₁ a₂ ∨ ¬SimpleEdges.Adj a₂ a₃ hPd : (a₁ :: a₂ :: a₃ :: l).getLast ⋯ = d hPc : List.Chain' (fun x x_1 => x ≠ x_1) (a₁ :: a₂ :: a₃ :: l) right✝ : (a₁ :: a₂ :: a₃ :: l).pathLength ≤ [a, b, d].pathLength c₁1 : ¬SimpleEdges.Adj a₁ a₂ c₁2 : ¬SimpleEdges.Adj a₂ a₃ ⊢ False case intro.intro.intro.intro.intro.inr.inl.intro 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, SimpleTriangle x y z S✝¹ : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this✝ : S✝¹.Nonempty b d✝ a c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line a c ≠ {a, c} hd✝ : d✝ ∈ Line a c acd : sbtw a c d✝ S✝ : Set V := setOf (sbtw a c) d : V hd : sbtw a c d hbd' : b ≠ d hdmin : ∀ (d' : V), sbtw a c d' → dist c d ≤ dist c d' hcd : SimpleEdges.Adj c d hbd : ¬SimpleEdges.Adj b d S : Set (List V) := setOf (List.Special a b d) this : S.Finite P : List V a₁ a₂ a₃ : V l : List V 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₃ hβ : ¬SimpleEdges.Adj a₁ a₂ ∨ ¬SimpleEdges.Adj a₂ a₃ hPd : (a₁ :: a₂ :: a₃ :: l).getLast ⋯ = d hPc : List.Chain' (fun x x_1 => x ≠ x_1) (a₁ :: a₂ :: a₃ :: l) right✝ : (a₁ :: a₂ :: a₃ :: l).pathLength ≤ [a, b, d].pathLength c₂1 : SimpleEdges.Adj a₁ a₂ c₂2 : ¬SimpleEdges.Adj a₂ a₃ ⊢ False case intro.intro.intro.intro.intro.inr.inr.intro 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, SimpleTriangle x y z S✝¹ : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this✝ : S✝¹.Nonempty b d✝ a c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line a c ≠ {a, c} hd✝ : d✝ ∈ Line a c acd : sbtw a c d✝ S✝ : Set V := setOf (sbtw a c) d : V hd : sbtw a c d hbd' : b ≠ d hdmin : ∀ (d' : V), sbtw a c d' → dist c d ≤ dist c d' hcd : SimpleEdges.Adj c d hbd : ¬SimpleEdges.Adj b d S : Set (List V) := setOf (List.Special a b d) this : S.Finite P : List V a₁ a₂ a₃ : V l : List V 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₃ hβ : ¬SimpleEdges.Adj a₁ a₂ ∨ ¬SimpleEdges.Adj a₂ a₃ hPd : (a₁ :: a₂ :: a₃ :: l).getLast ⋯ = d hPc : List.Chain' (fun x x_1 => x ≠ x_1) (a₁ :: a₂ :: a₃ :: l) right✝ : (a₁ :: a₂ :: a₃ :: l).pathLength ≤ [a, b, d].pathLength c₃1 : ¬SimpleEdges.Adj a₁ a₂ c₃2 : SimpleEdges.Adj a₂ a₃ ⊢ False
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/SylvesterChvatal.lean
two_implies_three
[530, 1]
[591, 69]
tauto
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, SimpleTriangle x y z S✝¹ : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this✝ : S✝¹.Nonempty b d✝ a c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line a c ≠ {a, c} hd✝ : d✝ ∈ Line a c acd : sbtw a c d✝ S✝ : Set V := setOf (sbtw a c) d : V hd : sbtw a c d hbd' : b ≠ d hdmin : ∀ (d' : V), sbtw a c d' → dist c d ≤ dist c d' hcd : SimpleEdges.Adj c d hbd : ¬SimpleEdges.Adj b d S : Set (List V) := setOf (List.Special a b d) this : S.Finite P : List V a₁ a₂ a₃ : V l : List V 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₃ hβ : ¬SimpleEdges.Adj a₁ a₂ ∨ ¬SimpleEdges.Adj a₂ a₃ hPd : (a₁ :: a₂ :: a₃ :: l).getLast ⋯ = d hPc : List.Chain' (fun x x_1 => x ≠ x_1) (a₁ :: a₂ :: a₃ :: l) right✝ : (a₁ :: a₂ :: a₃ :: l).pathLength ≤ [a, b, d].pathLength ⊢ ¬SimpleEdges.Adj a₁ a₂ ∧ ¬SimpleEdges.Adj a₂ a₃ ∨ SimpleEdges.Adj a₁ a₂ ∧ ¬SimpleEdges.Adj a₂ a₃ ∨ ¬SimpleEdges.Adj a₁ a₂ ∧ SimpleEdges.Adj a₂ a₃
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/SylvesterChvatal.lean
two_implies_three
[530, 1]
[591, 69]
exact case1 habc hmin hd hbd' hbd hPmin ha₁ hα hPd hPc c₁1 c₁2
case intro.intro.intro.intro.intro.inl.intro 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, SimpleTriangle x y z S✝¹ : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this✝ : S✝¹.Nonempty b d✝ a c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line a c ≠ {a, c} hd✝ : d✝ ∈ Line a c acd : sbtw a c d✝ S✝ : Set V := setOf (sbtw a c) d : V hd : sbtw a c d hbd' : b ≠ d hdmin : ∀ (d' : V), sbtw a c d' → dist c d ≤ dist c d' hcd : SimpleEdges.Adj c d hbd : ¬SimpleEdges.Adj b d S : Set (List V) := setOf (List.Special a b d) this : S.Finite P : List V a₁ a₂ a₃ : V l : List V 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₃ hβ : ¬SimpleEdges.Adj a₁ a₂ ∨ ¬SimpleEdges.Adj a₂ a₃ hPd : (a₁ :: a₂ :: a₃ :: l).getLast ⋯ = d hPc : List.Chain' (fun x x_1 => x ≠ x_1) (a₁ :: a₂ :: a₃ :: l) right✝ : (a₁ :: a₂ :: a₃ :: l).pathLength ≤ [a, b, d].pathLength c₁1 : ¬SimpleEdges.Adj a₁ a₂ c₁2 : ¬SimpleEdges.Adj a₂ a₃ ⊢ False
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/SylvesterChvatal.lean
two_implies_three
[530, 1]
[591, 69]
exact case2 habc hmin hd hbd' hbd hPmin ha₁ hα hPd hPc c₂1 c₂2
case intro.intro.intro.intro.intro.inr.inl.intro 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, SimpleTriangle x y z S✝¹ : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this✝ : S✝¹.Nonempty b d✝ a c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line a c ≠ {a, c} hd✝ : d✝ ∈ Line a c acd : sbtw a c d✝ S✝ : Set V := setOf (sbtw a c) d : V hd : sbtw a c d hbd' : b ≠ d hdmin : ∀ (d' : V), sbtw a c d' → dist c d ≤ dist c d' hcd : SimpleEdges.Adj c d hbd : ¬SimpleEdges.Adj b d S : Set (List V) := setOf (List.Special a b d) this : S.Finite P : List V a₁ a₂ a₃ : V l : List V 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₃ hβ : ¬SimpleEdges.Adj a₁ a₂ ∨ ¬SimpleEdges.Adj a₂ a₃ hPd : (a₁ :: a₂ :: a₃ :: l).getLast ⋯ = d hPc : List.Chain' (fun x x_1 => x ≠ x_1) (a₁ :: a₂ :: a₃ :: l) right✝ : (a₁ :: a₂ :: a₃ :: l).pathLength ≤ [a, b, d].pathLength c₂1 : SimpleEdges.Adj a₁ a₂ c₂2 : ¬SimpleEdges.Adj a₂ a₃ ⊢ False
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/SylvesterChvatal.lean
two_implies_three
[530, 1]
[591, 69]
exact case3 habc hmin hd hbd' hbd hPmin ha₁ hα hPd hPc c₃1 c₃2
case intro.intro.intro.intro.intro.inr.inr.intro 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, SimpleTriangle x y z S✝¹ : Set (V × V × V) := {(x, y, z) | SimpleTriangle x y z} this✝ : S✝¹.Nonempty b d✝ a c : V habc : SimpleTriangle a b c hmin : ∀ (a' b' c' : V), SimpleTriangle a' b' c' → Delta a b c ≤ Delta a' b' c' h3 : Line a c ≠ {a, c} hd✝ : d✝ ∈ Line a c acd : sbtw a c d✝ S✝ : Set V := setOf (sbtw a c) d : V hd : sbtw a c d hbd' : b ≠ d hdmin : ∀ (d' : V), sbtw a c d' → dist c d ≤ dist c d' hcd : SimpleEdges.Adj c d hbd : ¬SimpleEdges.Adj b d S : Set (List V) := setOf (List.Special a b d) this : S.Finite P : List V a₁ a₂ a₃ : V l : List V 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₃ hβ : ¬SimpleEdges.Adj a₁ a₂ ∨ ¬SimpleEdges.Adj a₂ a₃ hPd : (a₁ :: a₂ :: a₃ :: l).getLast ⋯ = d hPc : List.Chain' (fun x x_1 => x ≠ x_1) (a₁ :: a₂ :: a₃ :: l) right✝ : (a₁ :: a₂ :: a₃ :: l).pathLength ≤ [a, b, d].pathLength c₃1 : ¬SimpleEdges.Adj a₁ a₂ c₃2 : SimpleEdges.Adj a₂ a₃ ⊢ False
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/SylvesterChvatal.lean
sylvester_chvatal
[593, 1]
[601, 29]
by_cases h : ∀ x y z : V, ¬ NotCollinear x y z
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✝¹ : Nontrivial V inst✝ : Finite V ⊢ ∃ a b, a ≠ b ∧ (Line a b = {a, b} ∨ Line a b = Set.univ)
case pos 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✝¹ : Nontrivial V inst✝ : Finite V h : ∀ (x y z : V), ¬NotCollinear x y z ⊢ ∃ a b, a ≠ b ∧ (Line a b = {a, b} ∨ Line a b = Set.univ) case neg 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✝¹ : Nontrivial V inst✝ : Finite V h : ¬∀ (x y z : V), ¬NotCollinear x y z ⊢ ∃ a b, a ≠ b ∧ (Line a b = {a, b} ∨ Line a b = Set.univ)
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/SylvesterChvatal.lean
sylvester_chvatal
[593, 1]
[601, 29]
push_neg at h
case neg 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✝¹ : Nontrivial V inst✝ : Finite V h : ¬∀ (x y z : V), ¬NotCollinear x y z ⊢ ∃ a b, a ≠ b ∧ (Line a b = {a, b} ∨ Line a b = Set.univ)
case neg 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✝¹ : Nontrivial V inst✝ : Finite V h : ∃ x y z, NotCollinear x y z ⊢ ∃ a b, a ≠ b ∧ (Line a b = {a, b} ∨ Line a b = Set.univ)
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/SylvesterChvatal.lean
sylvester_chvatal
[593, 1]
[601, 29]
replace h := one_implies_two h
case neg 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✝¹ : Nontrivial V inst✝ : Finite V h : ∃ x y z, NotCollinear x y z ⊢ ∃ a b, a ≠ b ∧ (Line a b = {a, b} ∨ Line a b = Set.univ)
case neg 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✝¹ : Nontrivial V inst✝ : Finite V h : ∃ x y z, SimpleTriangle x y z ⊢ ∃ a b, a ≠ b ∧ (Line a b = {a, b} ∨ Line a b = Set.univ)
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/SylvesterChvatal.lean
sylvester_chvatal
[593, 1]
[601, 29]
obtain ⟨a, b, h, hl⟩ := two_implies_three h
case neg 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✝¹ : Nontrivial V inst✝ : Finite V h : ∃ x y z, SimpleTriangle x y z ⊢ ∃ a b, a ≠ b ∧ (Line a b = {a, b} ∨ Line a b = Set.univ)
case neg.intro.intro.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✝¹ : Nontrivial V inst✝ : Finite V h✝ : ∃ x y z, SimpleTriangle x y z a b : V h : a ≠ b hl : Line a b = {a, b} ⊢ ∃ a b, a ≠ b ∧ (Line a b = {a, b} ∨ Line a b = Set.univ)
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/SylvesterChvatal.lean
sylvester_chvatal
[593, 1]
[601, 29]
exact ⟨a, b, h, Or.inl hl⟩
case neg.intro.intro.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✝¹ : Nontrivial V inst✝ : Finite V h✝ : ∃ x y z, SimpleTriangle x y z a b : V h : a ≠ b hl : Line a b = {a, b} ⊢ ∃ a b, a ≠ b ∧ (Line a b = {a, b} ∨ Line a b = Set.univ)
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/SylvesterChvatal.lean
sylvester_chvatal
[593, 1]
[601, 29]
obtain ⟨L, hL, a, b, hab, rfl⟩ := thm_two' h
case pos 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✝¹ : Nontrivial V inst✝ : Finite V h : ∀ (x y z : V), ¬NotCollinear x y z ⊢ ∃ a b, a ≠ b ∧ (Line a b = {a, b} ∨ Line a b = Set.univ)
case pos.intro.intro.intro.intro.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✝¹ : Nontrivial V inst✝ : Finite V h : ∀ (x y z : V), ¬NotCollinear x y z a b : V hab : a ≠ b hL : Line a b = Set.univ ⊢ ∃ a b, a ≠ b ∧ (Line a b = {a, b} ∨ Line a b = Set.univ)
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/SylvesterChvatal.lean
sylvester_chvatal
[593, 1]
[601, 29]
exact ⟨a, b, hab, Or.inr hL⟩
case pos.intro.intro.intro.intro.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✝¹ : Nontrivial V inst✝ : Finite V h : ∀ (x y z : V), ¬NotCollinear x y z a b : V hab : a ≠ b hL : Line a b = Set.univ ⊢ ∃ a b, a ≠ b ∧ (Line a b = {a, b} ∨ Line a b = Set.univ)
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/ErdosRenyi/Basic.lean
ErdosRenyi.meas
[51, 1]
[54, 35]
simpa using hG.meas H.edgeFinset
α : Type u_1 Ω : Type u_2 inst✝⁵ : MeasurableSpace Ω G : Ω → SimpleGraph α H : SimpleGraph α inst✝⁴ : (ω : Ω) → DecidableRel (G ω).Adj p : ℝ≥0 μ : Measure Ω inst✝³ : IsProbabilityMeasure μ hG : ErdosRenyi G p μ inst✝² : Fintype α inst✝¹ : DecidableEq α inst✝ : DecidableRel H.Adj ⊢ μ {ω | G ω = H} = ↑p ^ H.edgeFinset.card * (1 - ↑p) ^ (Fintype.card (Sym2 α) - H.edgeFinset.card)
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/MinkowskiCaratheodory.lean
convexHull_extremePoints
[20, 1]
[23, 53]
sorry
E : Type u_1 inst✝² : NormedAddCommGroup E inst✝¹ : NormedSpace ℝ E inst✝ : FiniteDimensional ℝ E x : E s B : Set E hscomp : IsCompact s hsconv : Convex ℝ s ⊢ (convexHull ℝ) (extremePoints ℝ s) = s
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/MinkowskiCaratheodory.lean
closed_convexHull_extremePoints_of_compact_of_convex
[32, 1]
[35, 96]
rw [closure_convexHull_extremePoints hscomp hsconv, convexHull_extremePoints hscomp hsconv]
E : Type u_1 inst✝² : NormedAddCommGroup E inst✝¹ : NormedSpace ℝ E inst✝ : FiniteDimensional ℝ E x : E s B : Set E hscomp : IsCompact s hsconv : Convex ℝ s ⊢ closure ((convexHull ℝ) (extremePoints ℝ s)) = (convexHull ℝ) (extremePoints ℝ s)
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/ConvexContinuous.lean
Real.closedBall_eq_segment
[26, 1]
[27, 96]
rw [closedBall_eq_Icc, segment_eq_Icc ((sub_le_self _ hε).trans $ le_add_of_nonneg_right hε)]
ε r : ℝ hε : 0 ≤ ε ⊢ closedBall r ε = segment ℝ (r - ε) (r + ε)
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/ConvexContinuous.lean
IsOpen.exists_mem_intrinsicInterior_convexHull_finset
[52, 1]
[68, 8]
classical lift x to affineSpan ℝ s using subset_affineSpan _ _ hx set x : affineSpan ℝ s := x with hx clear_value x subst hx obtain ⟨ε, hε, hεx⟩ := (Metric.nhds_basis_closedBall.1 _).1 (isOpen_iff_mem_nhds.1 hs _ hx) set f : Finset (Fin $ finrank ℝ $ vectorSpan ℝ s) → vectorSpan ℝ s := fun u ↦ (ε / ∑ i, ‖finBasis ℝ (vectorSpan ℝ s) i‖) • ∑ i, if i ∈ u then finBasis ℝ (vectorSpan ℝ s) i else -finBasis ℝ (vectorSpan ℝ s) i with hf sorry
E : Type u_1 inst✝² : NormedAddCommGroup E inst✝¹ : NormedSpace ℝ E inst✝ : FiniteDimensional ℝ E s : Set E x : E hs : IsOpen (Subtype.val ⁻¹' s) hx : x ∈ s ⊢ ∃ t, x ∈ intrinsicInterior ℝ ((convexHull ℝ) ↑t) ∧ (convexHull ℝ) ↑t ⊆ s
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/ConvexContinuous.lean
IsOpen.exists_mem_intrinsicInterior_convexHull_finset
[52, 1]
[68, 8]
lift x to affineSpan ℝ s using subset_affineSpan _ _ hx
E : Type u_1 inst✝² : NormedAddCommGroup E inst✝¹ : NormedSpace ℝ E inst✝ : FiniteDimensional ℝ E s : Set E x : E hs : IsOpen (Subtype.val ⁻¹' s) hx : x ∈ s ⊢ ∃ t, x ∈ intrinsicInterior ℝ ((convexHull ℝ) ↑t) ∧ (convexHull ℝ) ↑t ⊆ s
case intro E : Type u_1 inst✝² : NormedAddCommGroup E inst✝¹ : NormedSpace ℝ E inst✝ : FiniteDimensional ℝ E s : Set E hs : IsOpen (Subtype.val ⁻¹' s) x : ↥(affineSpan ℝ s) hx : ↑x ∈ s ⊢ ∃ t, ↑x ∈ intrinsicInterior ℝ ((convexHull ℝ) ↑t) ∧ (convexHull ℝ) ↑t ⊆ s
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/ConvexContinuous.lean
IsOpen.exists_mem_intrinsicInterior_convexHull_finset
[52, 1]
[68, 8]
set x : affineSpan ℝ s := x with hx
case intro E : Type u_1 inst✝² : NormedAddCommGroup E inst✝¹ : NormedSpace ℝ E inst✝ : FiniteDimensional ℝ E s : Set E hs : IsOpen (Subtype.val ⁻¹' s) x : ↥(affineSpan ℝ s) hx : ↑x ∈ s ⊢ ∃ t, ↑x ∈ intrinsicInterior ℝ ((convexHull ℝ) ↑t) ∧ (convexHull ℝ) ↑t ⊆ s
case intro E : Type u_1 inst✝² : NormedAddCommGroup E inst✝¹ : NormedSpace ℝ E inst✝ : FiniteDimensional ℝ E s : Set E hs : IsOpen (Subtype.val ⁻¹' s) x✝ : ↥(affineSpan ℝ s) x : ↥(affineSpan ℝ s) := x✝ hx✝ : ↑x ∈ s hx : x = x✝ ⊢ ∃ t, ↑x ∈ intrinsicInterior ℝ ((convexHull ℝ) ↑t) ∧ (convexHull ℝ) ↑t ⊆ s
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/ConvexContinuous.lean
IsOpen.exists_mem_intrinsicInterior_convexHull_finset
[52, 1]
[68, 8]
clear_value x
case intro E : Type u_1 inst✝² : NormedAddCommGroup E inst✝¹ : NormedSpace ℝ E inst✝ : FiniteDimensional ℝ E s : Set E hs : IsOpen (Subtype.val ⁻¹' s) x✝ : ↥(affineSpan ℝ s) x : ↥(affineSpan ℝ s) := x✝ hx✝ : ↑x ∈ s hx : x = x✝ ⊢ ∃ t, ↑x ∈ intrinsicInterior ℝ ((convexHull ℝ) ↑t) ∧ (convexHull ℝ) ↑t ⊆ s
case intro E : Type u_1 inst✝² : NormedAddCommGroup E inst✝¹ : NormedSpace ℝ E inst✝ : FiniteDimensional ℝ E s : Set E hs : IsOpen (Subtype.val ⁻¹' s) x✝ x : ↥(affineSpan ℝ s) hx✝ : ↑x ∈ s hx : x = x✝ ⊢ ∃ t, ↑x ∈ intrinsicInterior ℝ ((convexHull ℝ) ↑t) ∧ (convexHull ℝ) ↑t ⊆ s
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/ConvexContinuous.lean
IsOpen.exists_mem_intrinsicInterior_convexHull_finset
[52, 1]
[68, 8]
subst hx
case intro E : Type u_1 inst✝² : NormedAddCommGroup E inst✝¹ : NormedSpace ℝ E inst✝ : FiniteDimensional ℝ E s : Set E hs : IsOpen (Subtype.val ⁻¹' s) x✝ x : ↥(affineSpan ℝ s) hx✝ : ↑x ∈ s hx : x = x✝ ⊢ ∃ t, ↑x ∈ intrinsicInterior ℝ ((convexHull ℝ) ↑t) ∧ (convexHull ℝ) ↑t ⊆ s
case intro E : Type u_1 inst✝² : NormedAddCommGroup E inst✝¹ : NormedSpace ℝ E inst✝ : FiniteDimensional ℝ E s : Set E hs : IsOpen (Subtype.val ⁻¹' s) x : ↥(affineSpan ℝ s) hx : ↑x ∈ s ⊢ ∃ t, ↑x ∈ intrinsicInterior ℝ ((convexHull ℝ) ↑t) ∧ (convexHull ℝ) ↑t ⊆ s
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/ConvexContinuous.lean
IsOpen.exists_mem_intrinsicInterior_convexHull_finset
[52, 1]
[68, 8]
obtain ⟨ε, hε, hεx⟩ := (Metric.nhds_basis_closedBall.1 _).1 (isOpen_iff_mem_nhds.1 hs _ hx)
case intro E : Type u_1 inst✝² : NormedAddCommGroup E inst✝¹ : NormedSpace ℝ E inst✝ : FiniteDimensional ℝ E s : Set E hs : IsOpen (Subtype.val ⁻¹' s) x : ↥(affineSpan ℝ s) hx : ↑x ∈ s ⊢ ∃ t, ↑x ∈ intrinsicInterior ℝ ((convexHull ℝ) ↑t) ∧ (convexHull ℝ) ↑t ⊆ s
case intro.intro.intro E : Type u_1 inst✝² : NormedAddCommGroup E inst✝¹ : NormedSpace ℝ E inst✝ : FiniteDimensional ℝ E s : Set E hs : IsOpen (Subtype.val ⁻¹' s) x : ↥(affineSpan ℝ s) hx : ↑x ∈ s ε : ℝ hε : 0 < ε hεx : closedBall x ε ⊆ Subtype.val ⁻¹' s ⊢ ∃ t, ↑x ∈ intrinsicInterior ℝ ((convexHull ℝ) ↑t) ∧ (convexHull ℝ) ↑t ⊆ s
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/ConvexContinuous.lean
IsOpen.exists_mem_intrinsicInterior_convexHull_finset
[52, 1]
[68, 8]
set f : Finset (Fin $ finrank ℝ $ vectorSpan ℝ s) → vectorSpan ℝ s := fun u ↦ (ε / ∑ i, ‖finBasis ℝ (vectorSpan ℝ s) i‖) • ∑ i, if i ∈ u then finBasis ℝ (vectorSpan ℝ s) i else -finBasis ℝ (vectorSpan ℝ s) i with hf
case intro.intro.intro E : Type u_1 inst✝² : NormedAddCommGroup E inst✝¹ : NormedSpace ℝ E inst✝ : FiniteDimensional ℝ E s : Set E hs : IsOpen (Subtype.val ⁻¹' s) x : ↥(affineSpan ℝ s) hx : ↑x ∈ s ε : ℝ hε : 0 < ε hεx : closedBall x ε ⊆ Subtype.val ⁻¹' s ⊢ ∃ t, ↑x ∈ intrinsicInterior ℝ ((convexHull ℝ) ↑t) ∧ (convexHull ℝ) ↑t ⊆ s
case intro.intro.intro E : Type u_1 inst✝² : NormedAddCommGroup E inst✝¹ : NormedSpace ℝ E inst✝ : FiniteDimensional ℝ E s : Set E hs : IsOpen (Subtype.val ⁻¹' s) x : ↥(affineSpan ℝ s) hx : ↑x ∈ s ε : ℝ hε : 0 < ε hεx : closedBall x ε ⊆ Subtype.val ⁻¹' s f : Finset (Fin (finrank ℝ ↥(vectorSpan ℝ s))) → ↥(vectorSpan ℝ s) := fun u => (ε / ∑ i : Fin (finrank ℝ ↥(vectorSpan ℝ s)), ‖(finBasis ℝ ↥(vectorSpan ℝ s)) i‖) • ∑ i : Fin (finrank ℝ ↥(vectorSpan ℝ s)), if i ∈ u then (finBasis ℝ ↥(vectorSpan ℝ s)) i else -(finBasis ℝ ↥(vectorSpan ℝ s)) i hf : f = fun u => (ε / ∑ i : Fin (finrank ℝ ↥(vectorSpan ℝ s)), ‖(finBasis ℝ ↥(vectorSpan ℝ s)) i‖) • ∑ i : Fin (finrank ℝ ↥(vectorSpan ℝ s)), if i ∈ u then (finBasis ℝ ↥(vectorSpan ℝ s)) i else -(finBasis ℝ ↥(vectorSpan ℝ s)) i ⊢ ∃ t, ↑x ∈ intrinsicInterior ℝ ((convexHull ℝ) ↑t) ∧ (convexHull ℝ) ↑t ⊆ s
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/ConvexContinuous.lean
IsOpen.exists_mem_intrinsicInterior_convexHull_finset
[52, 1]
[68, 8]
sorry
case intro.intro.intro E : Type u_1 inst✝² : NormedAddCommGroup E inst✝¹ : NormedSpace ℝ E inst✝ : FiniteDimensional ℝ E s : Set E hs : IsOpen (Subtype.val ⁻¹' s) x : ↥(affineSpan ℝ s) hx : ↑x ∈ s ε : ℝ hε : 0 < ε hεx : closedBall x ε ⊆ Subtype.val ⁻¹' s f : Finset (Fin (finrank ℝ ↥(vectorSpan ℝ s))) → ↥(vectorSpan ℝ s) := fun u => (ε / ∑ i : Fin (finrank ℝ ↥(vectorSpan ℝ s)), ‖(finBasis ℝ ↥(vectorSpan ℝ s)) i‖) • ∑ i : Fin (finrank ℝ ↥(vectorSpan ℝ s)), if i ∈ u then (finBasis ℝ ↥(vectorSpan ℝ s)) i else -(finBasis ℝ ↥(vectorSpan ℝ s)) i hf : f = fun u => (ε / ∑ i : Fin (finrank ℝ ↥(vectorSpan ℝ s)), ‖(finBasis ℝ ↥(vectorSpan ℝ s)) i‖) • ∑ i : Fin (finrank ℝ ↥(vectorSpan ℝ s)), if i ∈ u then (finBasis ℝ ↥(vectorSpan ℝ s)) i else -(finBasis ℝ ↥(vectorSpan ℝ s)) i ⊢ ∃ t, ↑x ∈ intrinsicInterior ℝ ((convexHull ℝ) ↑t) ∧ (convexHull ℝ) ↑t ⊆ s
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/ConvexContinuous.lean
ConvexOn.continuousOn
[104, 1]
[115, 8]
classical sorry
E : Type u_1 inst✝² : NormedAddCommGroup E inst✝¹ : NormedSpace ℝ E inst✝ : FiniteDimensional ℝ E s : Set E f : E → ℝ hf : ConvexOn ℝ s f ⊢ ContinuousOn f (intrinsicInterior ℝ s)
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/ConvexContinuous.lean
ConvexOn.continuousOn
[104, 1]
[115, 8]
sorry
E : Type u_1 inst✝² : NormedAddCommGroup E inst✝¹ : NormedSpace ℝ E inst✝ : FiniteDimensional ℝ E s : Set E f : E → ℝ hf : ConvexOn ℝ s f ⊢ ContinuousOn f (intrinsicInterior ℝ s)
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Mathlib/RingTheory/Int/Basic.lean
Nat.prime_composite_induction
[5, 1]
[12, 69]
refine induction_on_primes zero one ?_ _
P : ℕ → Prop zero : P 0 one : P 1 prime : ∀ (p : ℕ), p.Prime → P p composite : ∀ (a : ℕ), 2 ≤ a → P a → ∀ (b : ℕ), 2 ≤ b → P b → P (a * b) n : ℕ ⊢ P n
P : ℕ → Prop zero : P 0 one : P 1 prime : ∀ (p : ℕ), p.Prime → P p composite : ∀ (a : ℕ), 2 ≤ a → P a → ∀ (b : ℕ), 2 ≤ b → P b → P (a * b) n : ℕ ⊢ ∀ (p a : ℕ), p.Prime → P a → P (p * a)
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Mathlib/RingTheory/Int/Basic.lean
Nat.prime_composite_induction
[5, 1]
[12, 69]
rintro p (_ | _ | a) hp ha
P : ℕ → Prop zero : P 0 one : P 1 prime : ∀ (p : ℕ), p.Prime → P p composite : ∀ (a : ℕ), 2 ≤ a → P a → ∀ (b : ℕ), 2 ≤ b → P b → P (a * b) n : ℕ ⊢ ∀ (p a : ℕ), p.Prime → P a → P (p * a)
case zero P : ℕ → Prop zero : P 0 one : P 1 prime : ∀ (p : ℕ), p.Prime → P p composite : ∀ (a : ℕ), 2 ≤ a → P a → ∀ (b : ℕ), 2 ≤ b → P b → P (a * b) n p : ℕ hp : p.Prime ha : P 0 ⊢ P (p * 0) case succ.zero P : ℕ → Prop zero : P 0 one : P 1 prime : ∀ (p : ℕ), p.Prime → P p composite : ∀ (a : ℕ), 2 ≤ a → P a → ∀ (b : ℕ), 2 ≤ b → P b → P (a * b) n p : ℕ hp : p.Prime ha : P (0 + 1) ⊢ P (p * (0 + 1)) case succ.succ P : ℕ → Prop zero : P 0 one : P 1 prime : ∀ (p : ℕ), p.Prime → P p composite : ∀ (a : ℕ), 2 ≤ a → P a → ∀ (b : ℕ), 2 ≤ b → P b → P (a * b) n p a : ℕ hp : p.Prime ha : P (a + 1 + 1) ⊢ P (p * (a + 1 + 1))
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Mathlib/RingTheory/Int/Basic.lean
Nat.prime_composite_induction
[5, 1]
[12, 69]
simpa
case zero P : ℕ → Prop zero : P 0 one : P 1 prime : ∀ (p : ℕ), p.Prime → P p composite : ∀ (a : ℕ), 2 ≤ a → P a → ∀ (b : ℕ), 2 ≤ b → P b → P (a * b) n p : ℕ hp : p.Prime ha : P 0 ⊢ P (p * 0)
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Mathlib/RingTheory/Int/Basic.lean
Nat.prime_composite_induction
[5, 1]
[12, 69]
simpa using prime _ hp
case succ.zero P : ℕ → Prop zero : P 0 one : P 1 prime : ∀ (p : ℕ), p.Prime → P p composite : ∀ (a : ℕ), 2 ≤ a → P a → ∀ (b : ℕ), 2 ≤ b → P b → P (a * b) n p : ℕ hp : p.Prime ha : P (0 + 1) ⊢ P (p * (0 + 1))
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Mathlib/RingTheory/Int/Basic.lean
Nat.prime_composite_induction
[5, 1]
[12, 69]
exact composite _ hp.two_le (prime _ hp) _ a.one_lt_succ_succ ha
case succ.succ P : ℕ → Prop zero : P 0 one : P 1 prime : ∀ (p : ℕ), p.Prime → P p composite : ∀ (a : ℕ), 2 ≤ a → P a → ∀ (b : ℕ), 2 ≤ b → P b → P (a * b) n p a : ℕ hp : p.Prime ha : P (a + 1 + 1) ⊢ P (p * (a + 1 + 1))
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Incidence.lean
IncidenceAlgebra.ext
[97, 1]
[102, 66]
refine' DFunLike.coe_injective' (funext₂ fun a b ↦ _)
𝕄 : Type u_1 F : Type u_2 𝕜 : Type u_3 𝕝 : Type u_4 𝕞 : Type u_5 α : Type u_6 β : Type u_7 inst✝¹ : Zero 𝕜 inst✝ : LE α a b : α f g : IncidenceAlgebra 𝕜 α h : ∀ (a b : α), a ≤ b → f a b = g a b ⊢ f = g
𝕄 : Type u_1 F : Type u_2 𝕜 : Type u_3 𝕝 : Type u_4 𝕞 : Type u_5 α : Type u_6 β : Type u_7 inst✝¹ : Zero 𝕜 inst✝ : LE α a✝ b✝ : α f g : IncidenceAlgebra 𝕜 α h : ∀ (a b : α), a ≤ b → f a b = g a b a b : α ⊢ f a b = g a b
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Incidence.lean
IncidenceAlgebra.ext
[97, 1]
[102, 66]
by_cases hab : a ≤ b
𝕄 : Type u_1 F : Type u_2 𝕜 : Type u_3 𝕝 : Type u_4 𝕞 : Type u_5 α : Type u_6 β : Type u_7 inst✝¹ : Zero 𝕜 inst✝ : LE α a✝ b✝ : α f g : IncidenceAlgebra 𝕜 α h : ∀ (a b : α), a ≤ b → f a b = g a b a b : α ⊢ f a b = g a b
case pos 𝕄 : Type u_1 F : Type u_2 𝕜 : Type u_3 𝕝 : Type u_4 𝕞 : Type u_5 α : Type u_6 β : Type u_7 inst✝¹ : Zero 𝕜 inst✝ : LE α a✝ b✝ : α f g : IncidenceAlgebra 𝕜 α h : ∀ (a b : α), a ≤ b → f a b = g a b a b : α hab : a ≤ b ⊢ f a b = g a b case neg 𝕄 : Type u_1 F : Type u_2 𝕜 : Type u_3 𝕝 : Type u_4 𝕞 : Type u_5 α : Type u_6 β : Type u_7 inst✝¹ : Zero 𝕜 inst✝ : LE α a✝ b✝ : α f g : IncidenceAlgebra 𝕜 α h : ∀ (a b : α), a ≤ b → f a b = g a b a b : α hab : ¬a ≤ b ⊢ f a b = g a b
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Incidence.lean
IncidenceAlgebra.ext
[97, 1]
[102, 66]
exact h _ _ hab
case pos 𝕄 : Type u_1 F : Type u_2 𝕜 : Type u_3 𝕝 : Type u_4 𝕞 : Type u_5 α : Type u_6 β : Type u_7 inst✝¹ : Zero 𝕜 inst✝ : LE α a✝ b✝ : α f g : IncidenceAlgebra 𝕜 α h : ∀ (a b : α), a ≤ b → f a b = g a b a b : α hab : a ≤ b ⊢ f a b = g a b
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Incidence.lean
IncidenceAlgebra.ext
[97, 1]
[102, 66]
rw [apply_eq_zero_of_not_le hab, apply_eq_zero_of_not_le hab]
case neg 𝕄 : Type u_1 F : Type u_2 𝕜 : Type u_3 𝕝 : Type u_4 𝕞 : Type u_5 α : Type u_6 β : Type u_7 inst✝¹ : Zero 𝕜 inst✝ : LE α a✝ b✝ : α f g : IncidenceAlgebra 𝕜 α h : ∀ (a b : α), a ≤ b → f a b = g a b a b : α hab : ¬a ≤ b ⊢ f a b = g a b
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Incidence.lean
IncidenceAlgebra.zeta_mul_zeta
[345, 1]
[350, 49]
rw [mul_apply, card_eq_sum_ones, Nat.cast_sum, Nat.cast_one]
𝕄 : Type u_1 F : Type u_2 𝕜 : Type u_3 𝕝 : Type u_4 𝕞 : Type u_5 α : Type u_6 β : Type u_7 inst✝³ : Semiring 𝕜 inst✝² : Preorder α inst✝¹ : LocallyFiniteOrder α inst✝ : DecidableRel fun x x_1 => x ≤ x_1 a b : α ⊢ (zeta 𝕜 * zeta 𝕜) a b = ↑(Icc a b).card
𝕄 : Type u_1 F : Type u_2 𝕜 : Type u_3 𝕝 : Type u_4 𝕞 : Type u_5 α : Type u_6 β : Type u_7 inst✝³ : Semiring 𝕜 inst✝² : Preorder α inst✝¹ : LocallyFiniteOrder α inst✝ : DecidableRel fun x x_1 => x ≤ x_1 a b : α ⊢ ∑ x ∈ Icc a b, (zeta 𝕜) a x * (zeta 𝕜) x b = ∑ x ∈ Icc a b, 1
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Incidence.lean
IncidenceAlgebra.zeta_mul_zeta
[345, 1]
[350, 49]
refine' sum_congr rfl fun x hx ↦ _
𝕄 : Type u_1 F : Type u_2 𝕜 : Type u_3 𝕝 : Type u_4 𝕞 : Type u_5 α : Type u_6 β : Type u_7 inst✝³ : Semiring 𝕜 inst✝² : Preorder α inst✝¹ : LocallyFiniteOrder α inst✝ : DecidableRel fun x x_1 => x ≤ x_1 a b : α ⊢ ∑ x ∈ Icc a b, (zeta 𝕜) a x * (zeta 𝕜) x b = ∑ x ∈ Icc a b, 1
𝕄 : Type u_1 F : Type u_2 𝕜 : Type u_3 𝕝 : Type u_4 𝕞 : Type u_5 α : Type u_6 β : Type u_7 inst✝³ : Semiring 𝕜 inst✝² : Preorder α inst✝¹ : LocallyFiniteOrder α inst✝ : DecidableRel fun x x_1 => x ≤ x_1 a b x : α hx : x ∈ Icc a b ⊢ (zeta 𝕜) a x * (zeta 𝕜) x b = 1
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Incidence.lean
IncidenceAlgebra.zeta_mul_zeta
[345, 1]
[350, 49]
rw [mem_Icc] at hx
𝕄 : Type u_1 F : Type u_2 𝕜 : Type u_3 𝕝 : Type u_4 𝕞 : Type u_5 α : Type u_6 β : Type u_7 inst✝³ : Semiring 𝕜 inst✝² : Preorder α inst✝¹ : LocallyFiniteOrder α inst✝ : DecidableRel fun x x_1 => x ≤ x_1 a b x : α hx : x ∈ Icc a b ⊢ (zeta 𝕜) a x * (zeta 𝕜) x b = 1
𝕄 : Type u_1 F : Type u_2 𝕜 : Type u_3 𝕝 : Type u_4 𝕞 : Type u_5 α : Type u_6 β : Type u_7 inst✝³ : Semiring 𝕜 inst✝² : Preorder α inst✝¹ : LocallyFiniteOrder α inst✝ : DecidableRel fun x x_1 => x ≤ x_1 a b x : α hx : a ≤ x ∧ x ≤ b ⊢ (zeta 𝕜) a x * (zeta 𝕜) x b = 1
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Incidence.lean
IncidenceAlgebra.zeta_mul_zeta
[345, 1]
[350, 49]
rw [zeta_of_le hx.1, zeta_of_le hx.2, one_mul]
𝕄 : Type u_1 F : Type u_2 𝕜 : Type u_3 𝕝 : Type u_4 𝕞 : Type u_5 α : Type u_6 β : Type u_7 inst✝³ : Semiring 𝕜 inst✝² : Preorder α inst✝¹ : LocallyFiniteOrder α inst✝ : DecidableRel fun x x_1 => x ≤ x_1 a b x : α hx : a ≤ x ∧ x ≤ b ⊢ (zeta 𝕜) a x * (zeta 𝕜) x b = 1
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Incidence.lean
IncidenceAlgebra.zeta_mul_kappa
[352, 1]
[357, 49]
rw [mul_apply, card_eq_sum_ones, Nat.cast_sum, Nat.cast_one]
𝕄 : Type u_1 F : Type u_2 𝕜 : Type u_3 𝕝 : Type u_4 𝕞 : Type u_5 α : Type u_6 β : Type u_7 inst✝³ : Semiring 𝕜 inst✝² : Preorder α inst✝¹ : LocallyFiniteOrder α inst✝ : DecidableRel fun x x_1 => x ≤ x_1 a b : α ⊢ (zeta 𝕜 * zeta 𝕜) a b = ↑(Icc a b).card
𝕄 : Type u_1 F : Type u_2 𝕜 : Type u_3 𝕝 : Type u_4 𝕞 : Type u_5 α : Type u_6 β : Type u_7 inst✝³ : Semiring 𝕜 inst✝² : Preorder α inst✝¹ : LocallyFiniteOrder α inst✝ : DecidableRel fun x x_1 => x ≤ x_1 a b : α ⊢ ∑ x ∈ Icc a b, (zeta 𝕜) a x * (zeta 𝕜) x b = ∑ x ∈ Icc a b, 1
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Incidence.lean
IncidenceAlgebra.zeta_mul_kappa
[352, 1]
[357, 49]
refine' sum_congr rfl fun x hx ↦ _
𝕄 : Type u_1 F : Type u_2 𝕜 : Type u_3 𝕝 : Type u_4 𝕞 : Type u_5 α : Type u_6 β : Type u_7 inst✝³ : Semiring 𝕜 inst✝² : Preorder α inst✝¹ : LocallyFiniteOrder α inst✝ : DecidableRel fun x x_1 => x ≤ x_1 a b : α ⊢ ∑ x ∈ Icc a b, (zeta 𝕜) a x * (zeta 𝕜) x b = ∑ x ∈ Icc a b, 1
𝕄 : Type u_1 F : Type u_2 𝕜 : Type u_3 𝕝 : Type u_4 𝕞 : Type u_5 α : Type u_6 β : Type u_7 inst✝³ : Semiring 𝕜 inst✝² : Preorder α inst✝¹ : LocallyFiniteOrder α inst✝ : DecidableRel fun x x_1 => x ≤ x_1 a b x : α hx : x ∈ Icc a b ⊢ (zeta 𝕜) a x * (zeta 𝕜) x b = 1
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Incidence.lean
IncidenceAlgebra.zeta_mul_kappa
[352, 1]
[357, 49]
rw [mem_Icc] at hx
𝕄 : Type u_1 F : Type u_2 𝕜 : Type u_3 𝕝 : Type u_4 𝕞 : Type u_5 α : Type u_6 β : Type u_7 inst✝³ : Semiring 𝕜 inst✝² : Preorder α inst✝¹ : LocallyFiniteOrder α inst✝ : DecidableRel fun x x_1 => x ≤ x_1 a b x : α hx : x ∈ Icc a b ⊢ (zeta 𝕜) a x * (zeta 𝕜) x b = 1
𝕄 : Type u_1 F : Type u_2 𝕜 : Type u_3 𝕝 : Type u_4 𝕞 : Type u_5 α : Type u_6 β : Type u_7 inst✝³ : Semiring 𝕜 inst✝² : Preorder α inst✝¹ : LocallyFiniteOrder α inst✝ : DecidableRel fun x x_1 => x ≤ x_1 a b x : α hx : a ≤ x ∧ x ≤ b ⊢ (zeta 𝕜) a x * (zeta 𝕜) x b = 1
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Incidence.lean
IncidenceAlgebra.zeta_mul_kappa
[352, 1]
[357, 49]
rw [zeta_of_le hx.1, zeta_of_le hx.2, one_mul]
𝕄 : Type u_1 F : Type u_2 𝕜 : Type u_3 𝕝 : Type u_4 𝕞 : Type u_5 α : Type u_6 β : Type u_7 inst✝³ : Semiring 𝕜 inst✝² : Preorder α inst✝¹ : LocallyFiniteOrder α inst✝ : DecidableRel fun x x_1 => x ≤ x_1 a b x : α hx : a ≤ x ∧ x ≤ b ⊢ (zeta 𝕜) a x * (zeta 𝕜) x b = 1
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Incidence.lean
IncidenceAlgebra.muAux_apply
[375, 1]
[377, 13]
rw [muAux]
𝕄 : Type u_1 F : Type u_2 𝕜 : Type u_3 𝕝 : Type u_4 𝕞 : Type u_5 α : Type u_6 β : Type u_7 inst✝⁴ : AddCommGroup 𝕜 inst✝³ : One 𝕜 inst✝² : Preorder α inst✝¹ : LocallyFiniteOrder α inst✝ : DecidableEq α a b : α ⊢ muAux 𝕜 a b = if a = b then 1 else -∑ x ∈ (Ico a b).attach, muAux 𝕜 a ↑x
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Incidence.lean
IncidenceAlgebra.mu_apply
[392, 1]
[393, 43]
rw [mu, coe_mk, muAux_apply, sum_attach]
𝕄 : Type u_1 F : Type u_2 𝕜 : Type u_3 𝕝 : Type u_4 𝕞 : Type u_5 α : Type u_6 β : Type u_7 inst✝⁴ : AddCommGroup 𝕜 inst✝³ : One 𝕜 inst✝² : Preorder α inst✝¹ : LocallyFiniteOrder α inst✝ : DecidableEq α a b : α ⊢ (mu 𝕜) a b = if a = b then 1 else -∑ x ∈ Ico a b, (mu 𝕜) a x
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Incidence.lean
IncidenceAlgebra.mu_apply_of_eq
[395, 1]
[395, 88]
rw [mu_apply, if_pos h]
𝕄 : Type u_1 F : Type u_2 𝕜 : Type u_3 𝕝 : Type u_4 𝕞 : Type u_5 α : Type u_6 β : Type u_7 inst✝⁴ : AddCommGroup 𝕜 inst✝³ : One 𝕜 inst✝² : Preorder α inst✝¹ : LocallyFiniteOrder α inst✝ : DecidableEq α a b : α h : a = b ⊢ (mu 𝕜) a b = 1
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Incidence.lean
IncidenceAlgebra.mu_apply_of_ne
[399, 1]
[400, 26]
rw [mu_apply, if_neg h]
𝕄 : Type u_1 F : Type u_2 𝕜 : Type u_3 𝕝 : Type u_4 𝕞 : Type u_5 α : Type u_6 β : Type u_7 inst✝⁴ : AddCommGroup 𝕜 inst✝³ : One 𝕜 inst✝² : Preorder α inst✝¹ : LocallyFiniteOrder α inst✝ : DecidableEq α a b : α h : a ≠ b ⊢ (mu 𝕜) a b = -∑ x ∈ Ico a b, (mu 𝕜) a x
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Incidence.lean
IncidenceAlgebra.mu_spec_of_ne_right
[408, 1]
[419, 50]
have : mu 𝕜 a b = _ := mu_apply_of_ne h
𝕄 : Type u_1 F : Type u_2 𝕜 : Type u_3 𝕝 : Type u_4 𝕞 : Type u_5 α : Type u_6 β : Type u_7 inst✝⁴ : AddCommGroup 𝕜 inst✝³ : One 𝕜 inst✝² : PartialOrder α inst✝¹ : LocallyFiniteOrder α inst✝ : DecidableEq α a b : α h : a ≠ b ⊢ ∑ x ∈ Icc a b, (mu 𝕜) a x = 0
𝕄 : Type u_1 F : Type u_2 𝕜 : Type u_3 𝕝 : Type u_4 𝕞 : Type u_5 α : Type u_6 β : Type u_7 inst✝⁴ : AddCommGroup 𝕜 inst✝³ : One 𝕜 inst✝² : PartialOrder α inst✝¹ : LocallyFiniteOrder α inst✝ : DecidableEq α a b : α h : a ≠ b this : (mu 𝕜) a b = -∑ x ∈ Ico a b, (mu 𝕜) a x ⊢ ∑ x ∈ Icc a b, (mu 𝕜) a x = 0
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Incidence.lean
IncidenceAlgebra.mu_spec_of_ne_right
[408, 1]
[419, 50]
by_cases hab : a ≤ b
𝕄 : Type u_1 F : Type u_2 𝕜 : Type u_3 𝕝 : Type u_4 𝕞 : Type u_5 α : Type u_6 β : Type u_7 inst✝⁴ : AddCommGroup 𝕜 inst✝³ : One 𝕜 inst✝² : PartialOrder α inst✝¹ : LocallyFiniteOrder α inst✝ : DecidableEq α a b : α h : a ≠ b this : (mu 𝕜) a b = -∑ x ∈ Ico a b, (mu 𝕜) a x ⊢ ∑ x ∈ Icc a b, (mu 𝕜) a x = 0
case pos 𝕄 : Type u_1 F : Type u_2 𝕜 : Type u_3 𝕝 : Type u_4 𝕞 : Type u_5 α : Type u_6 β : Type u_7 inst✝⁴ : AddCommGroup 𝕜 inst✝³ : One 𝕜 inst✝² : PartialOrder α inst✝¹ : LocallyFiniteOrder α inst✝ : DecidableEq α a b : α h : a ≠ b this : (mu 𝕜) a b = -∑ x ∈ Ico a b, (mu 𝕜) a x hab : a ≤ b ⊢ ∑ x ∈ Icc a b, (mu 𝕜) a x = 0 case neg 𝕄 : Type u_1 F : Type u_2 𝕜 : Type u_3 𝕝 : Type u_4 𝕞 : Type u_5 α : Type u_6 β : Type u_7 inst✝⁴ : AddCommGroup 𝕜 inst✝³ : One 𝕜 inst✝² : PartialOrder α inst✝¹ : LocallyFiniteOrder α inst✝ : DecidableEq α a b : α h : a ≠ b this : (mu 𝕜) a b = -∑ x ∈ Ico a b, (mu 𝕜) a x hab : ¬a ≤ b ⊢ ∑ x ∈ Icc a b, (mu 𝕜) a x = 0
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Incidence.lean
IncidenceAlgebra.mu_spec_of_ne_right
[408, 1]
[419, 50]
rw [Icc_eq_cons_Ico hab]
case pos 𝕄 : Type u_1 F : Type u_2 𝕜 : Type u_3 𝕝 : Type u_4 𝕞 : Type u_5 α : Type u_6 β : Type u_7 inst✝⁴ : AddCommGroup 𝕜 inst✝³ : One 𝕜 inst✝² : PartialOrder α inst✝¹ : LocallyFiniteOrder α inst✝ : DecidableEq α a b : α h : a ≠ b this : (mu 𝕜) a b = -∑ x ∈ Ico a b, (mu 𝕜) a x hab : a ≤ b ⊢ ∑ x ∈ Icc a b, (mu 𝕜) a x = 0
case pos 𝕄 : Type u_1 F : Type u_2 𝕜 : Type u_3 𝕝 : Type u_4 𝕞 : Type u_5 α : Type u_6 β : Type u_7 inst✝⁴ : AddCommGroup 𝕜 inst✝³ : One 𝕜 inst✝² : PartialOrder α inst✝¹ : LocallyFiniteOrder α inst✝ : DecidableEq α a b : α h : a ≠ b this : (mu 𝕜) a b = -∑ x ∈ Ico a b, (mu 𝕜) a x hab : a ≤ b ⊢ ∑ x ∈ cons b (Ico a b) ⋯, (mu 𝕜) a x = 0
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Incidence.lean
IncidenceAlgebra.mu_spec_of_ne_right
[408, 1]
[419, 50]
simp [this, neg_add_self]
case pos 𝕄 : Type u_1 F : Type u_2 𝕜 : Type u_3 𝕝 : Type u_4 𝕞 : Type u_5 α : Type u_6 β : Type u_7 inst✝⁴ : AddCommGroup 𝕜 inst✝³ : One 𝕜 inst✝² : PartialOrder α inst✝¹ : LocallyFiniteOrder α inst✝ : DecidableEq α a b : α h : a ≠ b this : (mu 𝕜) a b = -∑ x ∈ Ico a b, (mu 𝕜) a x hab : a ≤ b ⊢ ∑ x ∈ cons b (Ico a b) ⋯, (mu 𝕜) a x = 0
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Incidence.lean
IncidenceAlgebra.mu_spec_of_ne_right
[408, 1]
[419, 50]
have : ∀ x ∈ Icc a b, ¬a ≤ x := by intro x hx hn apply hab rw [mem_Icc] at hx exact le_trans hn hx.2
case neg 𝕄 : Type u_1 F : Type u_2 𝕜 : Type u_3 𝕝 : Type u_4 𝕞 : Type u_5 α : Type u_6 β : Type u_7 inst✝⁴ : AddCommGroup 𝕜 inst✝³ : One 𝕜 inst✝² : PartialOrder α inst✝¹ : LocallyFiniteOrder α inst✝ : DecidableEq α a b : α h : a ≠ b this : (mu 𝕜) a b = -∑ x ∈ Ico a b, (mu 𝕜) a x hab : ¬a ≤ b ⊢ ∑ x ∈ Icc a b, (mu 𝕜) a x = 0
case neg 𝕄 : Type u_1 F : Type u_2 𝕜 : Type u_3 𝕝 : Type u_4 𝕞 : Type u_5 α : Type u_6 β : Type u_7 inst✝⁴ : AddCommGroup 𝕜 inst✝³ : One 𝕜 inst✝² : PartialOrder α inst✝¹ : LocallyFiniteOrder α inst✝ : DecidableEq α a b : α h : a ≠ b this✝ : (mu 𝕜) a b = -∑ x ∈ Ico a b, (mu 𝕜) a x hab : ¬a ≤ b this : ∀ x ∈ Icc a b, ¬a ≤ x ⊢ ∑ x ∈ Icc a b, (mu 𝕜) a x = 0
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Incidence.lean
IncidenceAlgebra.mu_spec_of_ne_right
[408, 1]
[419, 50]
convert sum_const_zero
case neg 𝕄 : Type u_1 F : Type u_2 𝕜 : Type u_3 𝕝 : Type u_4 𝕞 : Type u_5 α : Type u_6 β : Type u_7 inst✝⁴ : AddCommGroup 𝕜 inst✝³ : One 𝕜 inst✝² : PartialOrder α inst✝¹ : LocallyFiniteOrder α inst✝ : DecidableEq α a b : α h : a ≠ b this✝ : (mu 𝕜) a b = -∑ x ∈ Ico a b, (mu 𝕜) a x hab : ¬a ≤ b this : ∀ x ∈ Icc a b, ¬a ≤ x ⊢ ∑ x ∈ Icc a b, (mu 𝕜) a x = 0
case h.e'_2.a 𝕄 : Type u_1 F : Type u_2 𝕜 : Type u_3 𝕝 : Type u_4 𝕞 : Type u_5 α : Type u_6 β : Type u_7 inst✝⁴ : AddCommGroup 𝕜 inst✝³ : One 𝕜 inst✝² : PartialOrder α inst✝¹ : LocallyFiniteOrder α inst✝ : DecidableEq α a b : α h : a ≠ b this✝ : (mu 𝕜) a b = -∑ x ∈ Ico a b, (mu 𝕜) a x hab : ¬a ≤ b this : ∀ x ∈ Icc a b, ¬a ≤ x x✝ : α a✝ : x✝ ∈ Icc a b ⊢ (mu 𝕜) a x✝ = 0
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Incidence.lean
IncidenceAlgebra.mu_spec_of_ne_right
[408, 1]
[419, 50]
simp [apply_eq_zero_of_not_le (this ‹_› ‹_›)]
case h.e'_2.a 𝕄 : Type u_1 F : Type u_2 𝕜 : Type u_3 𝕝 : Type u_4 𝕞 : Type u_5 α : Type u_6 β : Type u_7 inst✝⁴ : AddCommGroup 𝕜 inst✝³ : One 𝕜 inst✝² : PartialOrder α inst✝¹ : LocallyFiniteOrder α inst✝ : DecidableEq α a b : α h : a ≠ b this✝ : (mu 𝕜) a b = -∑ x ∈ Ico a b, (mu 𝕜) a x hab : ¬a ≤ b this : ∀ x ∈ Icc a b, ¬a ≤ x x✝ : α a✝ : x✝ ∈ Icc a b ⊢ (mu 𝕜) a x✝ = 0
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Incidence.lean
IncidenceAlgebra.mu_spec_of_ne_right
[408, 1]
[419, 50]
intro x hx hn
𝕄 : Type u_1 F : Type u_2 𝕜 : Type u_3 𝕝 : Type u_4 𝕞 : Type u_5 α : Type u_6 β : Type u_7 inst✝⁴ : AddCommGroup 𝕜 inst✝³ : One 𝕜 inst✝² : PartialOrder α inst✝¹ : LocallyFiniteOrder α inst✝ : DecidableEq α a b : α h : a ≠ b this : (mu 𝕜) a b = -∑ x ∈ Ico a b, (mu 𝕜) a x hab : ¬a ≤ b ⊢ ∀ x ∈ Icc a b, ¬a ≤ x
𝕄 : Type u_1 F : Type u_2 𝕜 : Type u_3 𝕝 : Type u_4 𝕞 : Type u_5 α : Type u_6 β : Type u_7 inst✝⁴ : AddCommGroup 𝕜 inst✝³ : One 𝕜 inst✝² : PartialOrder α inst✝¹ : LocallyFiniteOrder α inst✝ : DecidableEq α a b : α h : a ≠ b this : (mu 𝕜) a b = -∑ x ∈ Ico a b, (mu 𝕜) a x hab : ¬a ≤ b x : α hx : x ∈ Icc a b hn : a ≤ x ⊢ False
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Incidence.lean
IncidenceAlgebra.mu_spec_of_ne_right
[408, 1]
[419, 50]
apply hab
𝕄 : Type u_1 F : Type u_2 𝕜 : Type u_3 𝕝 : Type u_4 𝕞 : Type u_5 α : Type u_6 β : Type u_7 inst✝⁴ : AddCommGroup 𝕜 inst✝³ : One 𝕜 inst✝² : PartialOrder α inst✝¹ : LocallyFiniteOrder α inst✝ : DecidableEq α a b : α h : a ≠ b this : (mu 𝕜) a b = -∑ x ∈ Ico a b, (mu 𝕜) a x hab : ¬a ≤ b x : α hx : x ∈ Icc a b hn : a ≤ x ⊢ False
𝕄 : Type u_1 F : Type u_2 𝕜 : Type u_3 𝕝 : Type u_4 𝕞 : Type u_5 α : Type u_6 β : Type u_7 inst✝⁴ : AddCommGroup 𝕜 inst✝³ : One 𝕜 inst✝² : PartialOrder α inst✝¹ : LocallyFiniteOrder α inst✝ : DecidableEq α a b : α h : a ≠ b this : (mu 𝕜) a b = -∑ x ∈ Ico a b, (mu 𝕜) a x hab : ¬a ≤ b x : α hx : x ∈ Icc a b hn : a ≤ x ⊢ a ≤ b
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Incidence.lean
IncidenceAlgebra.mu_spec_of_ne_right
[408, 1]
[419, 50]
rw [mem_Icc] at hx
𝕄 : Type u_1 F : Type u_2 𝕜 : Type u_3 𝕝 : Type u_4 𝕞 : Type u_5 α : Type u_6 β : Type u_7 inst✝⁴ : AddCommGroup 𝕜 inst✝³ : One 𝕜 inst✝² : PartialOrder α inst✝¹ : LocallyFiniteOrder α inst✝ : DecidableEq α a b : α h : a ≠ b this : (mu 𝕜) a b = -∑ x ∈ Ico a b, (mu 𝕜) a x hab : ¬a ≤ b x : α hx : x ∈ Icc a b hn : a ≤ x ⊢ a ≤ b
𝕄 : Type u_1 F : Type u_2 𝕜 : Type u_3 𝕝 : Type u_4 𝕞 : Type u_5 α : Type u_6 β : Type u_7 inst✝⁴ : AddCommGroup 𝕜 inst✝³ : One 𝕜 inst✝² : PartialOrder α inst✝¹ : LocallyFiniteOrder α inst✝ : DecidableEq α a b : α h : a ≠ b this : (mu 𝕜) a b = -∑ x ∈ Ico a b, (mu 𝕜) a x hab : ¬a ≤ b x : α hx : a ≤ x ∧ x ≤ b hn : a ≤ x ⊢ a ≤ b