url
stringclasses 147
values | commit
stringclasses 147
values | file_path
stringlengths 7
101
| full_name
stringlengths 1
94
| start
stringlengths 6
10
| end
stringlengths 6
11
| tactic
stringlengths 1
11.2k
| state_before
stringlengths 3
2.09M
| state_after
stringlengths 6
2.09M
|
---|---|---|---|---|---|---|---|---|
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Analysis/Convex/SimplicialComplex/Basic.lean | Geometry.SimplicialComplex.facets_singleton | [64, 1] | [66, 74] | rw [Set.eq_singleton_iff_unique_mem] at hK ⊢ | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x y : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
hK : K.faces = {s}
⊢ K.facets = {s} | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x y : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
hK : s ∈ K.faces ∧ ∀ x ∈ K.faces, x = s
⊢ s ∈ K.facets ∧ ∀ x ∈ K.facets, x = s |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Analysis/Convex/SimplicialComplex/Basic.lean | Geometry.SimplicialComplex.facets_singleton | [64, 1] | [66, 74] | exact ⟨⟨hK.1, fun t ht _ => (hK.2 _ ht).symm⟩, fun t ht => hK.2 _ ht.1⟩ | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x y : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
hK : s ∈ K.faces ∧ ∀ x ∈ K.faces, x = s
⊢ s ∈ K.facets ∧ ∀ x ∈ K.facets, x = s | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Analysis/Convex/SimplicialComplex/Basic.lean | Geometry.SimplicialComplex.mem_of_mem_convexHull | [86, 1] | [91, 38] | have h := K.inter_subset_convexHull hx hs ⟨by simp, hxs⟩ | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x y : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
hx : x ∈ K.vertices
hs : s ∈ K
hxs : x ∈ (convexHull 𝕜) ↑s
⊢ x ∈ s | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x y : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
hx : x ∈ K.vertices
hs : s ∈ K
hxs : x ∈ (convexHull 𝕜) ↑s
h : x ∈ (convexHull 𝕜) (↑{x} ∩ ↑s)
⊢ x ∈ s |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Analysis/Convex/SimplicialComplex/Basic.lean | Geometry.SimplicialComplex.mem_of_mem_convexHull | [86, 1] | [91, 38] | by_contra H | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x y : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
hx : x ∈ K.vertices
hs : s ∈ K
hxs : x ∈ (convexHull 𝕜) ↑s
h : x ∈ (convexHull 𝕜) (↑{x} ∩ ↑s)
⊢ x ∈ s | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x y : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
hx : x ∈ K.vertices
hs : s ∈ K
hxs : x ∈ (convexHull 𝕜) ↑s
h : x ∈ (convexHull 𝕜) (↑{x} ∩ ↑s)
H : ¬x ∈ s
⊢ False |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Analysis/Convex/SimplicialComplex/Basic.lean | Geometry.SimplicialComplex.mem_of_mem_convexHull | [86, 1] | [91, 38] | rwa [← coe_inter, inter_comm, disjoint_iff_inter_eq_empty.1 (disjoint_singleton_right.2 H),
coe_empty, convexHull_empty] at h | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x y : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
hx : x ∈ K.vertices
hs : s ∈ K
hxs : x ∈ (convexHull 𝕜) ↑s
h : x ∈ (convexHull 𝕜) (↑{x} ∩ ↑s)
H : ¬x ∈ s
⊢ False | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Analysis/Convex/SimplicialComplex/Basic.lean | Geometry.SimplicialComplex.mem_of_mem_convexHull | [86, 1] | [91, 38] | simp | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : OrderedRing 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
K K₁ K₂ : SimplicialComplex 𝕜 E
x y : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
hx : x ∈ K.vertices
hs : s ∈ K
hxs : x ∈ (convexHull 𝕜) ↑s
⊢ x ∈ (convexHull 𝕜) ↑{x} | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Analysis/Convex/SimplicialComplex/Basic.lean | Geometry.SimplicialComplex.mem_ofSimplex | [145, 1] | [149, 18] | refine' ⟨_, fun h => ⟨h.1, s, rfl, h.2⟩⟩ | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
K : SimplicialComplex 𝕜 E
x y : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
hs : AffineIndependent 𝕜 Subtype.val
⊢ t ∈ ofSimplex hs ↔ t.Nonempty ∧ t ⊆ s | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
K : SimplicialComplex 𝕜 E
x y : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
hs : AffineIndependent 𝕜 Subtype.val
⊢ t ∈ ofSimplex hs → t.Nonempty ∧ t ⊆ s |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Analysis/Convex/SimplicialComplex/Basic.lean | Geometry.SimplicialComplex.mem_ofSimplex | [145, 1] | [149, 18] | rintro ⟨ht, u, rfl : u = s, hts⟩ | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
K : SimplicialComplex 𝕜 E
x y : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
hs : AffineIndependent 𝕜 Subtype.val
⊢ t ∈ ofSimplex hs → t.Nonempty ∧ t ⊆ s | case intro.intro.intro
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
K : SimplicialComplex 𝕜 E
x y : E
t : Finset E
A : Set (Finset E)
m n : ℕ
ht : t.Nonempty
u : Finset E
hts : t ⊆ u
hs : AffineIndependent 𝕜 Subtype.val
⊢ t.Nonempty ∧ t ⊆ u |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Analysis/Convex/SimplicialComplex/Basic.lean | Geometry.SimplicialComplex.mem_ofSimplex | [145, 1] | [149, 18] | exact ⟨ht, hts⟩ | case intro.intro.intro
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝² : LinearOrderedField 𝕜
inst✝¹ : AddCommGroup E
inst✝ : Module 𝕜 E
K : SimplicialComplex 𝕜 E
x y : E
t : Finset E
A : Set (Finset E)
m n : ℕ
ht : t.Nonempty
u : Finset E
hts : t ⊆ u
hs : AffineIndependent 𝕜 Subtype.val
⊢ t.Nonempty ∧ t ⊆ u | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Analysis/Convex/SimplicialComplex/Basic.lean | Geometry.SimplicialComplex.face_dimension_le_space_dimension | [152, 1] | [154, 100] | simpa using (K.indep hs).card_le_finrank_succ.trans (add_le_add_right (Submodule.finrank_le _) _) | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : LinearOrderedField 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K : SimplicialComplex 𝕜 E
x y : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : FiniteDimensional 𝕜 E
hs : s ∈ K
⊢ s.card ≤ FiniteDimensional.finrank 𝕜 E + 1 | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Analysis/Convex/SimplicialComplex/Basic.lean | Geometry.SimplicialComplex.subfacet | [156, 1] | [165, 36] | have := id hs | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : LinearOrderedField 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K : SimplicialComplex 𝕜 E
x y : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : FiniteDimensional 𝕜 E
hs : s ∈ K
⊢ ∃ t ∈ K.facets, s ⊆ t | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : LinearOrderedField 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K : SimplicialComplex 𝕜 E
x y : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : FiniteDimensional 𝕜 E
hs this : s ∈ K
⊢ ∃ t ∈ K.facets, s ⊆ t |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Analysis/Convex/SimplicialComplex/Basic.lean | Geometry.SimplicialComplex.subfacet | [156, 1] | [165, 36] | revert this | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : LinearOrderedField 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K : SimplicialComplex 𝕜 E
x y : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : FiniteDimensional 𝕜 E
hs this : s ∈ K
⊢ ∃ t ∈ K.facets, s ⊆ t | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : LinearOrderedField 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K : SimplicialComplex 𝕜 E
x y : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : FiniteDimensional 𝕜 E
hs : s ∈ K
⊢ s ∈ K → ∃ t ∈ K.facets, s ⊆ t |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Analysis/Convex/SimplicialComplex/Basic.lean | Geometry.SimplicialComplex.subfacet | [156, 1] | [165, 36] | refine strongDownwardInductionOn s ?_ (face_dimension_le_space_dimension hs) | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : LinearOrderedField 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K : SimplicialComplex 𝕜 E
x y : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : FiniteDimensional 𝕜 E
hs : s ∈ K
⊢ s ∈ K → ∃ t ∈ K.facets, s ⊆ t | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : LinearOrderedField 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K : SimplicialComplex 𝕜 E
x y : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : FiniteDimensional 𝕜 E
hs : s ∈ K
⊢ ∀ (t₁ : Finset E),
(∀ {t₂ : Finset E}, t₂.card ≤ FiniteDimensional.finrank 𝕜 E + 1 → t₁ ⊂ t₂ → t₂ ∈ K → ∃ t ∈ K.facets, t₂ ⊆ t) →
t₁.card ≤ FiniteDimensional.finrank 𝕜 E + 1 → t₁ ∈ K → ∃ t ∈ K.facets, t₁ ⊆ t |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Analysis/Convex/SimplicialComplex/Basic.lean | Geometry.SimplicialComplex.subfacet | [156, 1] | [165, 36] | rintro t h - ht | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : LinearOrderedField 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K : SimplicialComplex 𝕜 E
x y : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : FiniteDimensional 𝕜 E
hs : s ∈ K
⊢ ∀ (t₁ : Finset E),
(∀ {t₂ : Finset E}, t₂.card ≤ FiniteDimensional.finrank 𝕜 E + 1 → t₁ ⊂ t₂ → t₂ ∈ K → ∃ t ∈ K.facets, t₂ ⊆ t) →
t₁.card ≤ FiniteDimensional.finrank 𝕜 E + 1 → t₁ ∈ K → ∃ t ∈ K.facets, t₁ ⊆ t | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : LinearOrderedField 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K : SimplicialComplex 𝕜 E
x y : E
s t✝ : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : FiniteDimensional 𝕜 E
hs : s ∈ K
t : Finset E
h : ∀ {t₂ : Finset E}, t₂.card ≤ FiniteDimensional.finrank 𝕜 E + 1 → t ⊂ t₂ → t₂ ∈ K → ∃ t ∈ K.facets, t₂ ⊆ t
ht : t ∈ K
⊢ ∃ t_1 ∈ K.facets, t ⊆ t_1 |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Analysis/Convex/SimplicialComplex/Basic.lean | Geometry.SimplicialComplex.subfacet | [156, 1] | [165, 36] | by_cases htfacet : t ∈ K.facets | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : LinearOrderedField 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K : SimplicialComplex 𝕜 E
x y : E
s t✝ : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : FiniteDimensional 𝕜 E
hs : s ∈ K
t : Finset E
h : ∀ {t₂ : Finset E}, t₂.card ≤ FiniteDimensional.finrank 𝕜 E + 1 → t ⊂ t₂ → t₂ ∈ K → ∃ t ∈ K.facets, t₂ ⊆ t
ht : t ∈ K
⊢ ∃ t_1 ∈ K.facets, t ⊆ t_1 | case pos
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : LinearOrderedField 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K : SimplicialComplex 𝕜 E
x y : E
s t✝ : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : FiniteDimensional 𝕜 E
hs : s ∈ K
t : Finset E
h : ∀ {t₂ : Finset E}, t₂.card ≤ FiniteDimensional.finrank 𝕜 E + 1 → t ⊂ t₂ → t₂ ∈ K → ∃ t ∈ K.facets, t₂ ⊆ t
ht : t ∈ K
htfacet : t ∈ K.facets
⊢ ∃ t_1 ∈ K.facets, t ⊆ t_1
case neg
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : LinearOrderedField 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K : SimplicialComplex 𝕜 E
x y : E
s t✝ : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : FiniteDimensional 𝕜 E
hs : s ∈ K
t : Finset E
h : ∀ {t₂ : Finset E}, t₂.card ≤ FiniteDimensional.finrank 𝕜 E + 1 → t ⊂ t₂ → t₂ ∈ K → ∃ t ∈ K.facets, t₂ ⊆ t
ht : t ∈ K
htfacet : t ∉ K.facets
⊢ ∃ t_1 ∈ K.facets, t ⊆ t_1 |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Analysis/Convex/SimplicialComplex/Basic.lean | Geometry.SimplicialComplex.subfacet | [156, 1] | [165, 36] | obtain ⟨u, hu, htu⟩ := (not_facet_iff_subface ht).mp htfacet | case neg
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : LinearOrderedField 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K : SimplicialComplex 𝕜 E
x y : E
s t✝ : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : FiniteDimensional 𝕜 E
hs : s ∈ K
t : Finset E
h : ∀ {t₂ : Finset E}, t₂.card ≤ FiniteDimensional.finrank 𝕜 E + 1 → t ⊂ t₂ → t₂ ∈ K → ∃ t ∈ K.facets, t₂ ⊆ t
ht : t ∈ K
htfacet : t ∉ K.facets
⊢ ∃ t_1 ∈ K.facets, t ⊆ t_1 | case neg.intro.intro
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : LinearOrderedField 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K : SimplicialComplex 𝕜 E
x y : E
s t✝ : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : FiniteDimensional 𝕜 E
hs : s ∈ K
t : Finset E
h : ∀ {t₂ : Finset E}, t₂.card ≤ FiniteDimensional.finrank 𝕜 E + 1 → t ⊂ t₂ → t₂ ∈ K → ∃ t ∈ K.facets, t₂ ⊆ t
ht : t ∈ K
htfacet : t ∉ K.facets
u : Finset E
hu : u ∈ K.faces
htu : t ⊂ u
⊢ ∃ t_1 ∈ K.facets, t ⊆ t_1 |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Analysis/Convex/SimplicialComplex/Basic.lean | Geometry.SimplicialComplex.subfacet | [156, 1] | [165, 36] | obtain ⟨v, hv⟩ := h (face_dimension_le_space_dimension hu) htu hu | case neg.intro.intro
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : LinearOrderedField 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K : SimplicialComplex 𝕜 E
x y : E
s t✝ : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : FiniteDimensional 𝕜 E
hs : s ∈ K
t : Finset E
h : ∀ {t₂ : Finset E}, t₂.card ≤ FiniteDimensional.finrank 𝕜 E + 1 → t ⊂ t₂ → t₂ ∈ K → ∃ t ∈ K.facets, t₂ ⊆ t
ht : t ∈ K
htfacet : t ∉ K.facets
u : Finset E
hu : u ∈ K.faces
htu : t ⊂ u
⊢ ∃ t_1 ∈ K.facets, t ⊆ t_1 | case neg.intro.intro.intro
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : LinearOrderedField 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K : SimplicialComplex 𝕜 E
x y : E
s t✝ : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : FiniteDimensional 𝕜 E
hs : s ∈ K
t : Finset E
h : ∀ {t₂ : Finset E}, t₂.card ≤ FiniteDimensional.finrank 𝕜 E + 1 → t ⊂ t₂ → t₂ ∈ K → ∃ t ∈ K.facets, t₂ ⊆ t
ht : t ∈ K
htfacet : t ∉ K.facets
u : Finset E
hu : u ∈ K.faces
htu : t ⊂ u
v : Finset E
hv : v ∈ K.facets ∧ u ⊆ v
⊢ ∃ t_1 ∈ K.facets, t ⊆ t_1 |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Analysis/Convex/SimplicialComplex/Basic.lean | Geometry.SimplicialComplex.subfacet | [156, 1] | [165, 36] | exact ⟨v, hv.1, htu.1.trans hv.2⟩ | case neg.intro.intro.intro
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : LinearOrderedField 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K : SimplicialComplex 𝕜 E
x y : E
s t✝ : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : FiniteDimensional 𝕜 E
hs : s ∈ K
t : Finset E
h : ∀ {t₂ : Finset E}, t₂.card ≤ FiniteDimensional.finrank 𝕜 E + 1 → t ⊂ t₂ → t₂ ∈ K → ∃ t ∈ K.facets, t₂ ⊆ t
ht : t ∈ K
htfacet : t ∉ K.facets
u : Finset E
hu : u ∈ K.faces
htu : t ⊂ u
v : Finset E
hv : v ∈ K.facets ∧ u ⊆ v
⊢ ∃ t_1 ∈ K.facets, t ⊆ t_1 | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Analysis/Convex/SimplicialComplex/Basic.lean | Geometry.SimplicialComplex.subfacet | [156, 1] | [165, 36] | exact ⟨t, htfacet, Subset.rfl⟩ | case pos
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : LinearOrderedField 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K : SimplicialComplex 𝕜 E
x y : E
s t✝ : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : FiniteDimensional 𝕜 E
hs : s ∈ K
t : Finset E
h : ∀ {t₂ : Finset E}, t₂.card ≤ FiniteDimensional.finrank 𝕜 E + 1 → t ⊂ t₂ → t₂ ∈ K → ∃ t ∈ K.facets, t₂ ⊆ t
ht : t ∈ K
htfacet : t ∈ K.facets
⊢ ∃ t_1 ∈ K.facets, t ⊆ t_1 | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Analysis/Convex/SimplicialComplex/Basic.lean | Geometry.SimplicialComplex.facets_eq_empty_iff | [167, 1] | [174, 21] | refine' ⟨fun h => _, _⟩ | 𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : LinearOrderedField 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K : SimplicialComplex 𝕜 E
x y : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : FiniteDimensional 𝕜 E
⊢ K.facets = ∅ ↔ K = ⊥ | case refine'_1
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : LinearOrderedField 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K : SimplicialComplex 𝕜 E
x y : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : FiniteDimensional 𝕜 E
h : K.facets = ∅
⊢ K = ⊥
case refine'_2
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : LinearOrderedField 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K : SimplicialComplex 𝕜 E
x y : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : FiniteDimensional 𝕜 E
⊢ K = ⊥ → K.facets = ∅ |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Analysis/Convex/SimplicialComplex/Basic.lean | Geometry.SimplicialComplex.facets_eq_empty_iff | [167, 1] | [174, 21] | ext s | case refine'_1
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : LinearOrderedField 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K : SimplicialComplex 𝕜 E
x y : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : FiniteDimensional 𝕜 E
h : K.facets = ∅
⊢ K = ⊥ | case refine'_1.faces.h
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : LinearOrderedField 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K : SimplicialComplex 𝕜 E
x y : E
s✝ t : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : FiniteDimensional 𝕜 E
h : K.facets = ∅
s : Finset E
⊢ s ∈ K.faces ↔ s ∈ ⊥.faces |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Analysis/Convex/SimplicialComplex/Basic.lean | Geometry.SimplicialComplex.facets_eq_empty_iff | [167, 1] | [174, 21] | refine' iff_of_false (fun hs => _) (Set.not_mem_empty _) | case refine'_1.faces.h
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : LinearOrderedField 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K : SimplicialComplex 𝕜 E
x y : E
s✝ t : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : FiniteDimensional 𝕜 E
h : K.facets = ∅
s : Finset E
⊢ s ∈ K.faces ↔ s ∈ ⊥.faces | case refine'_1.faces.h
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : LinearOrderedField 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K : SimplicialComplex 𝕜 E
x y : E
s✝ t : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : FiniteDimensional 𝕜 E
h : K.facets = ∅
s : Finset E
hs : s ∈ K.faces
⊢ False |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Analysis/Convex/SimplicialComplex/Basic.lean | Geometry.SimplicialComplex.facets_eq_empty_iff | [167, 1] | [174, 21] | obtain ⟨t, ht, -⟩ := subfacet hs | case refine'_1.faces.h
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : LinearOrderedField 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K : SimplicialComplex 𝕜 E
x y : E
s✝ t : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : FiniteDimensional 𝕜 E
h : K.facets = ∅
s : Finset E
hs : s ∈ K.faces
⊢ False | case refine'_1.faces.h.intro.intro
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : LinearOrderedField 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K : SimplicialComplex 𝕜 E
x y : E
s✝ t✝ : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : FiniteDimensional 𝕜 E
h : K.facets = ∅
s : Finset E
hs : s ∈ K.faces
t : Finset E
ht : t ∈ K.facets
⊢ False |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Analysis/Convex/SimplicialComplex/Basic.lean | Geometry.SimplicialComplex.facets_eq_empty_iff | [167, 1] | [174, 21] | exact h.subset ht | case refine'_1.faces.h.intro.intro
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : LinearOrderedField 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K : SimplicialComplex 𝕜 E
x y : E
s✝ t✝ : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : FiniteDimensional 𝕜 E
h : K.facets = ∅
s : Finset E
hs : s ∈ K.faces
t : Finset E
ht : t ∈ K.facets
⊢ False | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Analysis/Convex/SimplicialComplex/Basic.lean | Geometry.SimplicialComplex.facets_eq_empty_iff | [167, 1] | [174, 21] | rintro rfl | case refine'_2
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : LinearOrderedField 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
K : SimplicialComplex 𝕜 E
x y : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : FiniteDimensional 𝕜 E
⊢ K = ⊥ → K.facets = ∅ | case refine'_2
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : LinearOrderedField 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
x y : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : FiniteDimensional 𝕜 E
⊢ ⊥.facets = ∅ |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Analysis/Convex/SimplicialComplex/Basic.lean | Geometry.SimplicialComplex.facets_eq_empty_iff | [167, 1] | [174, 21] | exact facets_bot | case refine'_2
𝕜 : Type u_1
E : Type u_2
ι : Type u_3
inst✝³ : LinearOrderedField 𝕜
inst✝² : AddCommGroup E
inst✝¹ : Module 𝕜 E
x y : E
s t : Finset E
A : Set (Finset E)
m n : ℕ
inst✝ : FiniteDimensional 𝕜 E
⊢ ⊥.facets = ∅ | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Combinatorics/Colex.lean | Finset.Colex.cons_le_cons | [11, 1] | [16, 27] | obtain rfl | hab := eq_or_ne a b | α : Type u_1
β : Type u_2
inst✝¹ : PartialOrder α
inst✝ : PartialOrder β
f : α → β
𝒜 𝒜₁ 𝒜₂ : Finset (Finset α)
s t u : Finset α
a b : α
ha : a ∉ s
hb : b ∉ s
⊢ { ofColex := cons a s ha } ≤ { ofColex := cons b s hb } ↔ a ≤ b | case inl
α : Type u_1
β : Type u_2
inst✝¹ : PartialOrder α
inst✝ : PartialOrder β
f : α → β
𝒜 𝒜₁ 𝒜₂ : Finset (Finset α)
s t u : Finset α
a : α
ha hb : a ∉ s
⊢ { ofColex := cons a s ha } ≤ { ofColex := cons a s hb } ↔ a ≤ a
case inr
α : Type u_1
β : Type u_2
inst✝¹ : PartialOrder α
inst✝ : PartialOrder β
f : α → β
𝒜 𝒜₁ 𝒜₂ : Finset (Finset α)
s t u : Finset α
a b : α
ha : a ∉ s
hb : b ∉ s
hab : a ≠ b
⊢ { ofColex := cons a s ha } ≤ { ofColex := cons b s hb } ↔ a ≤ b |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Combinatorics/Colex.lean | Finset.Colex.cons_le_cons | [11, 1] | [16, 27] | classical
rw [← toColex_sdiff_le_toColex_sdiff', cons_sdiff_cons hab, cons_sdiff_cons hab.symm,
singleton_le_singleton] | case inr
α : Type u_1
β : Type u_2
inst✝¹ : PartialOrder α
inst✝ : PartialOrder β
f : α → β
𝒜 𝒜₁ 𝒜₂ : Finset (Finset α)
s t u : Finset α
a b : α
ha : a ∉ s
hb : b ∉ s
hab : a ≠ b
⊢ { ofColex := cons a s ha } ≤ { ofColex := cons b s hb } ↔ a ≤ b | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Combinatorics/Colex.lean | Finset.Colex.cons_le_cons | [11, 1] | [16, 27] | simp | case inl
α : Type u_1
β : Type u_2
inst✝¹ : PartialOrder α
inst✝ : PartialOrder β
f : α → β
𝒜 𝒜₁ 𝒜₂ : Finset (Finset α)
s t u : Finset α
a : α
ha hb : a ∉ s
⊢ { ofColex := cons a s ha } ≤ { ofColex := cons a s hb } ↔ a ≤ a | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Combinatorics/Colex.lean | Finset.Colex.cons_le_cons | [11, 1] | [16, 27] | rw [← toColex_sdiff_le_toColex_sdiff', cons_sdiff_cons hab, cons_sdiff_cons hab.symm,
singleton_le_singleton] | case inr
α : Type u_1
β : Type u_2
inst✝¹ : PartialOrder α
inst✝ : PartialOrder β
f : α → β
𝒜 𝒜₁ 𝒜₂ : Finset (Finset α)
s t u : Finset α
a b : α
ha : a ∉ s
hb : b ∉ s
hab : a ≠ b
⊢ { ofColex := cons a s ha } ≤ { ofColex := cons b s hb } ↔ a ≤ b | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Combinatorics/Colex.lean | Finset.Colex.insert_le_insert | [23, 1] | [25, 70] | rw [← cons_eq_insert _ _ ha, ← cons_eq_insert _ _ hb, cons_le_cons] | α : Type u_1
β : Type u_2
inst✝² : PartialOrder α
inst✝¹ : PartialOrder β
f : α → β
𝒜 𝒜₁ 𝒜₂ : Finset (Finset α)
s t u : Finset α
a b : α
inst✝ : DecidableEq α
ha : a ∉ s
hb : b ∉ s
⊢ { ofColex := insert a s } ≤ { ofColex := insert b s } ↔ a ≤ b | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Combinatorics/Colex.lean | Finset.Colex.insert_lt_insert | [27, 1] | [29, 70] | rw [← cons_eq_insert _ _ ha, ← cons_eq_insert _ _ hb, cons_lt_cons] | α : Type u_1
β : Type u_2
inst✝² : PartialOrder α
inst✝¹ : PartialOrder β
f : α → β
𝒜 𝒜₁ 𝒜₂ : Finset (Finset α)
s t u : Finset α
a b : α
inst✝ : DecidableEq α
ha : a ∉ s
hb : b ∉ s
⊢ { ofColex := insert a s } < { ofColex := insert b s } ↔ a < b | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Combinatorics/Colex.lean | Finset.Colex.erase_le_erase | [31, 1] | [37, 27] | obtain rfl | hab := eq_or_ne a b | α : Type u_1
β : Type u_2
inst✝² : PartialOrder α
inst✝¹ : PartialOrder β
f : α → β
𝒜 𝒜₁ 𝒜₂ : Finset (Finset α)
s t u : Finset α
a b : α
inst✝ : DecidableEq α
ha : a ∈ s
hb : b ∈ s
⊢ { ofColex := s.erase a } ≤ { ofColex := s.erase b } ↔ b ≤ a | case inl
α : Type u_1
β : Type u_2
inst✝² : PartialOrder α
inst✝¹ : PartialOrder β
f : α → β
𝒜 𝒜₁ 𝒜₂ : Finset (Finset α)
s t u : Finset α
a : α
inst✝ : DecidableEq α
ha hb : a ∈ s
⊢ { ofColex := s.erase a } ≤ { ofColex := s.erase a } ↔ a ≤ a
case inr
α : Type u_1
β : Type u_2
inst✝² : PartialOrder α
inst✝¹ : PartialOrder β
f : α → β
𝒜 𝒜₁ 𝒜₂ : Finset (Finset α)
s t u : Finset α
a b : α
inst✝ : DecidableEq α
ha : a ∈ s
hb : b ∈ s
hab : a ≠ b
⊢ { ofColex := s.erase a } ≤ { ofColex := s.erase b } ↔ b ≤ a |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Combinatorics/Colex.lean | Finset.Colex.erase_le_erase | [31, 1] | [37, 27] | classical
rw [← toColex_sdiff_le_toColex_sdiff', erase_sdiff_erase hab hb, erase_sdiff_erase hab.symm ha,
singleton_le_singleton] | case inr
α : Type u_1
β : Type u_2
inst✝² : PartialOrder α
inst✝¹ : PartialOrder β
f : α → β
𝒜 𝒜₁ 𝒜₂ : Finset (Finset α)
s t u : Finset α
a b : α
inst✝ : DecidableEq α
ha : a ∈ s
hb : b ∈ s
hab : a ≠ b
⊢ { ofColex := s.erase a } ≤ { ofColex := s.erase b } ↔ b ≤ a | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Combinatorics/Colex.lean | Finset.Colex.erase_le_erase | [31, 1] | [37, 27] | simp | case inl
α : Type u_1
β : Type u_2
inst✝² : PartialOrder α
inst✝¹ : PartialOrder β
f : α → β
𝒜 𝒜₁ 𝒜₂ : Finset (Finset α)
s t u : Finset α
a : α
inst✝ : DecidableEq α
ha hb : a ∈ s
⊢ { ofColex := s.erase a } ≤ { ofColex := s.erase a } ↔ a ≤ a | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Combinatorics/Colex.lean | Finset.Colex.erase_le_erase | [31, 1] | [37, 27] | rw [← toColex_sdiff_le_toColex_sdiff', erase_sdiff_erase hab hb, erase_sdiff_erase hab.symm ha,
singleton_le_singleton] | case inr
α : Type u_1
β : Type u_2
inst✝² : PartialOrder α
inst✝¹ : PartialOrder β
f : α → β
𝒜 𝒜₁ 𝒜₂ : Finset (Finset α)
s t u : Finset α
a b : α
inst✝ : DecidableEq α
ha : a ∈ s
hb : b ∈ s
hab : a ≠ b
⊢ { ofColex := s.erase a } ≤ { ofColex := s.erase b } ↔ b ≤ a | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Combinatorics/Colex.lean | Finset.Colex.lt_iff_exists_forall_lt_mem_iff_mem | [55, 1] | [71, 73] | simp only [lt_iff_exists_forall_lt] | α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a : α
⊢ { ofColex := s } < { ofColex := t } ↔ ∃ w ∈ t, w ∉ s ∧ ∀ ⦃a : α⦄, w < a → (a ∈ s ↔ a ∈ t) | α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a : α
⊢ (∃ a ∈ t, a ∉ s ∧ ∀ b ∈ s, b ∉ t → b < a) ↔ ∃ w ∈ t, w ∉ s ∧ ∀ ⦃a : α⦄, w < a → (a ∈ s ↔ a ∈ t) |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Combinatorics/Colex.lean | Finset.Colex.lt_iff_exists_forall_lt_mem_iff_mem | [55, 1] | [71, 73] | refine ⟨fun h ↦ ?_, ?_⟩ | α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a : α
⊢ (∃ a ∈ t, a ∉ s ∧ ∀ b ∈ s, b ∉ t → b < a) ↔ ∃ w ∈ t, w ∉ s ∧ ∀ ⦃a : α⦄, w < a → (a ∈ s ↔ a ∈ t) | case refine_1
α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a : α
h : ∃ a ∈ t, a ∉ s ∧ ∀ b ∈ s, b ∉ t → b < a
⊢ ∃ w ∈ t, w ∉ s ∧ ∀ ⦃a : α⦄, w < a → (a ∈ s ↔ a ∈ t)
case refine_2
α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a : α
⊢ (∃ w ∈ t, w ∉ s ∧ ∀ ⦃a : α⦄, w < a → (a ∈ s ↔ a ∈ t)) → ∃ a ∈ t, a ∉ s ∧ ∀ b ∈ s, b ∉ t → b < a |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Combinatorics/Colex.lean | Finset.Colex.lt_iff_exists_forall_lt_mem_iff_mem | [55, 1] | [71, 73] | let u := (t \ s).filter fun w ↦ ∀ a ∈ s, a ∉ t → a < w | case refine_1
α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a : α
h : ∃ a ∈ t, a ∉ s ∧ ∀ b ∈ s, b ∉ t → b < a
⊢ ∃ w ∈ t, w ∉ s ∧ ∀ ⦃a : α⦄, w < a → (a ∈ s ↔ a ∈ t) | case refine_1
α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a : α
h : ∃ a ∈ t, a ∉ s ∧ ∀ b ∈ s, b ∉ t → b < a
u : Finset α := filter (fun w => ∀ a ∈ s, a ∉ t → a < w) (t \ s)
⊢ ∃ w ∈ t, w ∉ s ∧ ∀ ⦃a : α⦄, w < a → (a ∈ s ↔ a ∈ t) |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Combinatorics/Colex.lean | Finset.Colex.lt_iff_exists_forall_lt_mem_iff_mem | [55, 1] | [71, 73] | have mem_u {w : α} : w ∈ u ↔ w ∈ t ∧ w ∉ s ∧ ∀ a ∈ s, a ∉ t → a < w := by simp [u, and_assoc] | case refine_1
α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a : α
h : ∃ a ∈ t, a ∉ s ∧ ∀ b ∈ s, b ∉ t → b < a
u : Finset α := filter (fun w => ∀ a ∈ s, a ∉ t → a < w) (t \ s)
⊢ ∃ w ∈ t, w ∉ s ∧ ∀ ⦃a : α⦄, w < a → (a ∈ s ↔ a ∈ t) | case refine_1
α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a : α
h : ∃ a ∈ t, a ∉ s ∧ ∀ b ∈ s, b ∉ t → b < a
u : Finset α := filter (fun w => ∀ a ∈ s, a ∉ t → a < w) (t \ s)
mem_u : ∀ {w : α}, w ∈ u ↔ w ∈ t ∧ w ∉ s ∧ ∀ a ∈ s, a ∉ t → a < w
⊢ ∃ w ∈ t, w ∉ s ∧ ∀ ⦃a : α⦄, w < a → (a ∈ s ↔ a ∈ t) |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Combinatorics/Colex.lean | Finset.Colex.lt_iff_exists_forall_lt_mem_iff_mem | [55, 1] | [71, 73] | have hu : u.Nonempty := h.imp fun _ ↦ mem_u.2 | case refine_1
α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a : α
h : ∃ a ∈ t, a ∉ s ∧ ∀ b ∈ s, b ∉ t → b < a
u : Finset α := filter (fun w => ∀ a ∈ s, a ∉ t → a < w) (t \ s)
mem_u : ∀ {w : α}, w ∈ u ↔ w ∈ t ∧ w ∉ s ∧ ∀ a ∈ s, a ∉ t → a < w
⊢ ∃ w ∈ t, w ∉ s ∧ ∀ ⦃a : α⦄, w < a → (a ∈ s ↔ a ∈ t) | case refine_1
α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a : α
h : ∃ a ∈ t, a ∉ s ∧ ∀ b ∈ s, b ∉ t → b < a
u : Finset α := filter (fun w => ∀ a ∈ s, a ∉ t → a < w) (t \ s)
mem_u : ∀ {w : α}, w ∈ u ↔ w ∈ t ∧ w ∉ s ∧ ∀ a ∈ s, a ∉ t → a < w
hu : u.Nonempty
⊢ ∃ w ∈ t, w ∉ s ∧ ∀ ⦃a : α⦄, w < a → (a ∈ s ↔ a ∈ t) |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Combinatorics/Colex.lean | Finset.Colex.lt_iff_exists_forall_lt_mem_iff_mem | [55, 1] | [71, 73] | let m := max' _ hu | case refine_1
α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a : α
h : ∃ a ∈ t, a ∉ s ∧ ∀ b ∈ s, b ∉ t → b < a
u : Finset α := filter (fun w => ∀ a ∈ s, a ∉ t → a < w) (t \ s)
mem_u : ∀ {w : α}, w ∈ u ↔ w ∈ t ∧ w ∉ s ∧ ∀ a ∈ s, a ∉ t → a < w
hu : u.Nonempty
⊢ ∃ w ∈ t, w ∉ s ∧ ∀ ⦃a : α⦄, w < a → (a ∈ s ↔ a ∈ t) | case refine_1
α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a : α
h : ∃ a ∈ t, a ∉ s ∧ ∀ b ∈ s, b ∉ t → b < a
u : Finset α := filter (fun w => ∀ a ∈ s, a ∉ t → a < w) (t \ s)
mem_u : ∀ {w : α}, w ∈ u ↔ w ∈ t ∧ w ∉ s ∧ ∀ a ∈ s, a ∉ t → a < w
hu : u.Nonempty
m : α := u.max' hu
⊢ ∃ w ∈ t, w ∉ s ∧ ∀ ⦃a : α⦄, w < a → (a ∈ s ↔ a ∈ t) |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Combinatorics/Colex.lean | Finset.Colex.lt_iff_exists_forall_lt_mem_iff_mem | [55, 1] | [71, 73] | have ⟨hmt, hms, hm⟩ : m ∈ t ∧ m ∉ s ∧ ∀ a ∈ s, a ∉ t → a < m := mem_u.1 $ max'_mem _ _ | case refine_1
α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a : α
h : ∃ a ∈ t, a ∉ s ∧ ∀ b ∈ s, b ∉ t → b < a
u : Finset α := filter (fun w => ∀ a ∈ s, a ∉ t → a < w) (t \ s)
mem_u : ∀ {w : α}, w ∈ u ↔ w ∈ t ∧ w ∉ s ∧ ∀ a ∈ s, a ∉ t → a < w
hu : u.Nonempty
m : α := u.max' hu
⊢ ∃ w ∈ t, w ∉ s ∧ ∀ ⦃a : α⦄, w < a → (a ∈ s ↔ a ∈ t) | case refine_1
α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a : α
h : ∃ a ∈ t, a ∉ s ∧ ∀ b ∈ s, b ∉ t → b < a
u : Finset α := filter (fun w => ∀ a ∈ s, a ∉ t → a < w) (t \ s)
mem_u : ∀ {w : α}, w ∈ u ↔ w ∈ t ∧ w ∉ s ∧ ∀ a ∈ s, a ∉ t → a < w
hu : u.Nonempty
m : α := u.max' hu
hmt : m ∈ t
hms : m ∉ s
hm : ∀ a ∈ s, a ∉ t → a < m
⊢ ∃ w ∈ t, w ∉ s ∧ ∀ ⦃a : α⦄, w < a → (a ∈ s ↔ a ∈ t) |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Combinatorics/Colex.lean | Finset.Colex.lt_iff_exists_forall_lt_mem_iff_mem | [55, 1] | [71, 73] | refine ⟨m, hmt, hms, fun a hma ↦ ⟨fun has ↦ not_imp_comm.1 (hm _ has) hma.asymm, fun hat ↦ ?_⟩⟩ | case refine_1
α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a : α
h : ∃ a ∈ t, a ∉ s ∧ ∀ b ∈ s, b ∉ t → b < a
u : Finset α := filter (fun w => ∀ a ∈ s, a ∉ t → a < w) (t \ s)
mem_u : ∀ {w : α}, w ∈ u ↔ w ∈ t ∧ w ∉ s ∧ ∀ a ∈ s, a ∉ t → a < w
hu : u.Nonempty
m : α := u.max' hu
hmt : m ∈ t
hms : m ∉ s
hm : ∀ a ∈ s, a ∉ t → a < m
⊢ ∃ w ∈ t, w ∉ s ∧ ∀ ⦃a : α⦄, w < a → (a ∈ s ↔ a ∈ t) | case refine_1
α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a✝ : α
h : ∃ a ∈ t, a ∉ s ∧ ∀ b ∈ s, b ∉ t → b < a
u : Finset α := filter (fun w => ∀ a ∈ s, a ∉ t → a < w) (t \ s)
mem_u : ∀ {w : α}, w ∈ u ↔ w ∈ t ∧ w ∉ s ∧ ∀ a ∈ s, a ∉ t → a < w
hu : u.Nonempty
m : α := u.max' hu
hmt : m ∈ t
hms : m ∉ s
hm : ∀ a ∈ s, a ∉ t → a < m
a : α
hma : m < a
hat : a ∈ t
⊢ a ∈ s |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Combinatorics/Colex.lean | Finset.Colex.lt_iff_exists_forall_lt_mem_iff_mem | [55, 1] | [71, 73] | by_contra has | case refine_1
α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a✝ : α
h : ∃ a ∈ t, a ∉ s ∧ ∀ b ∈ s, b ∉ t → b < a
u : Finset α := filter (fun w => ∀ a ∈ s, a ∉ t → a < w) (t \ s)
mem_u : ∀ {w : α}, w ∈ u ↔ w ∈ t ∧ w ∉ s ∧ ∀ a ∈ s, a ∉ t → a < w
hu : u.Nonempty
m : α := u.max' hu
hmt : m ∈ t
hms : m ∉ s
hm : ∀ a ∈ s, a ∉ t → a < m
a : α
hma : m < a
hat : a ∈ t
⊢ a ∈ s | case refine_1
α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a✝ : α
h : ∃ a ∈ t, a ∉ s ∧ ∀ b ∈ s, b ∉ t → b < a
u : Finset α := filter (fun w => ∀ a ∈ s, a ∉ t → a < w) (t \ s)
mem_u : ∀ {w : α}, w ∈ u ↔ w ∈ t ∧ w ∉ s ∧ ∀ a ∈ s, a ∉ t → a < w
hu : u.Nonempty
m : α := u.max' hu
hmt : m ∈ t
hms : m ∉ s
hm : ∀ a ∈ s, a ∉ t → a < m
a : α
hma : m < a
hat : a ∈ t
has : a ∉ s
⊢ False |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Combinatorics/Colex.lean | Finset.Colex.lt_iff_exists_forall_lt_mem_iff_mem | [55, 1] | [71, 73] | have hau : a ∈ u := mem_u.2 ⟨hat, has, fun b hbs hbt ↦ (hm _ hbs hbt).trans hma⟩ | case refine_1
α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a✝ : α
h : ∃ a ∈ t, a ∉ s ∧ ∀ b ∈ s, b ∉ t → b < a
u : Finset α := filter (fun w => ∀ a ∈ s, a ∉ t → a < w) (t \ s)
mem_u : ∀ {w : α}, w ∈ u ↔ w ∈ t ∧ w ∉ s ∧ ∀ a ∈ s, a ∉ t → a < w
hu : u.Nonempty
m : α := u.max' hu
hmt : m ∈ t
hms : m ∉ s
hm : ∀ a ∈ s, a ∉ t → a < m
a : α
hma : m < a
hat : a ∈ t
has : a ∉ s
⊢ False | case refine_1
α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a✝ : α
h : ∃ a ∈ t, a ∉ s ∧ ∀ b ∈ s, b ∉ t → b < a
u : Finset α := filter (fun w => ∀ a ∈ s, a ∉ t → a < w) (t \ s)
mem_u : ∀ {w : α}, w ∈ u ↔ w ∈ t ∧ w ∉ s ∧ ∀ a ∈ s, a ∉ t → a < w
hu : u.Nonempty
m : α := u.max' hu
hmt : m ∈ t
hms : m ∉ s
hm : ∀ a ∈ s, a ∉ t → a < m
a : α
hma : m < a
hat : a ∈ t
has : a ∉ s
hau : a ∈ u
⊢ False |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Combinatorics/Colex.lean | Finset.Colex.lt_iff_exists_forall_lt_mem_iff_mem | [55, 1] | [71, 73] | exact hma.not_le $ le_max' _ _ hau | case refine_1
α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a✝ : α
h : ∃ a ∈ t, a ∉ s ∧ ∀ b ∈ s, b ∉ t → b < a
u : Finset α := filter (fun w => ∀ a ∈ s, a ∉ t → a < w) (t \ s)
mem_u : ∀ {w : α}, w ∈ u ↔ w ∈ t ∧ w ∉ s ∧ ∀ a ∈ s, a ∉ t → a < w
hu : u.Nonempty
m : α := u.max' hu
hmt : m ∈ t
hms : m ∉ s
hm : ∀ a ∈ s, a ∉ t → a < m
a : α
hma : m < a
hat : a ∈ t
has : a ∉ s
hau : a ∈ u
⊢ False | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Combinatorics/Colex.lean | Finset.Colex.lt_iff_exists_forall_lt_mem_iff_mem | [55, 1] | [71, 73] | simp [u, and_assoc] | α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a : α
h : ∃ a ∈ t, a ∉ s ∧ ∀ b ∈ s, b ∉ t → b < a
u : Finset α := filter (fun w => ∀ a ∈ s, a ∉ t → a < w) (t \ s)
w : α
⊢ w ∈ u ↔ w ∈ t ∧ w ∉ s ∧ ∀ a ∈ s, a ∉ t → a < w | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Combinatorics/Colex.lean | Finset.Colex.lt_iff_exists_forall_lt_mem_iff_mem | [55, 1] | [71, 73] | rintro ⟨w, hwt, hws, hw⟩ | case refine_2
α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a : α
⊢ (∃ w ∈ t, w ∉ s ∧ ∀ ⦃a : α⦄, w < a → (a ∈ s ↔ a ∈ t)) → ∃ a ∈ t, a ∉ s ∧ ∀ b ∈ s, b ∉ t → b < a | case refine_2.intro.intro.intro
α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a w : α
hwt : w ∈ t
hws : w ∉ s
hw : ∀ ⦃a : α⦄, w < a → (a ∈ s ↔ a ∈ t)
⊢ ∃ a ∈ t, a ∉ s ∧ ∀ b ∈ s, b ∉ t → b < a |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Combinatorics/Colex.lean | Finset.Colex.lt_iff_exists_forall_lt_mem_iff_mem | [55, 1] | [71, 73] | refine ⟨w, hwt, hws, fun a has hat ↦ ?_⟩ | case refine_2.intro.intro.intro
α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a w : α
hwt : w ∈ t
hws : w ∉ s
hw : ∀ ⦃a : α⦄, w < a → (a ∈ s ↔ a ∈ t)
⊢ ∃ a ∈ t, a ∉ s ∧ ∀ b ∈ s, b ∉ t → b < a | case refine_2.intro.intro.intro
α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a✝ w : α
hwt : w ∈ t
hws : w ∉ s
hw : ∀ ⦃a : α⦄, w < a → (a ∈ s ↔ a ∈ t)
a : α
has : a ∈ s
hat : a ∉ t
⊢ a < w |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Combinatorics/Colex.lean | Finset.Colex.lt_iff_exists_forall_lt_mem_iff_mem | [55, 1] | [71, 73] | by_contra! hwa | case refine_2.intro.intro.intro
α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a✝ w : α
hwt : w ∈ t
hws : w ∉ s
hw : ∀ ⦃a : α⦄, w < a → (a ∈ s ↔ a ∈ t)
a : α
has : a ∈ s
hat : a ∉ t
⊢ a < w | case refine_2.intro.intro.intro
α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a✝ w : α
hwt : w ∈ t
hws : w ∉ s
hw : ∀ ⦃a : α⦄, w < a → (a ∈ s ↔ a ∈ t)
a : α
has : a ∈ s
hat : a ∉ t
hwa : w ≤ a
⊢ False |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Combinatorics/Colex.lean | Finset.Colex.lt_iff_exists_forall_lt_mem_iff_mem | [55, 1] | [71, 73] | exact hat $ (hw $ hwa.lt_of_ne $ ne_of_mem_of_not_mem hwt hat).1 has | case refine_2.intro.intro.intro
α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a✝ w : α
hwt : w ∈ t
hws : w ∉ s
hw : ∀ ⦃a : α⦄, w < a → (a ∈ s ↔ a ∈ t)
a : α
has : a ∈ s
hat : a ∉ t
hwa : w ≤ a
⊢ False | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Combinatorics/Colex.lean | Finset.Colex.erase_le_erase_min' | [73, 1] | [115, 94] | generalize_proofs ht | α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a : α
hst : { ofColex := s } ≤ { ofColex := t }
hcard : s.card ≤ t.card
ha : a ∈ s
⊢ { ofColex := s.erase a } ≤ { ofColex := t.erase (t.min' ⋯) } | α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a : α
hst : { ofColex := s } ≤ { ofColex := t }
hcard : s.card ≤ t.card
ha : a ∈ s
ht : t.Nonempty
⊢ { ofColex := s.erase a } ≤ { ofColex := t.erase (t.min' ht) } |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Combinatorics/Colex.lean | Finset.Colex.erase_le_erase_min' | [73, 1] | [115, 94] | set m := min' t ht | α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a : α
hst : { ofColex := s } ≤ { ofColex := t }
hcard : s.card ≤ t.card
ha : a ∈ s
ht : t.Nonempty
⊢ { ofColex := s.erase a } ≤ { ofColex := t.erase (t.min' ht) } | α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a : α
hst : { ofColex := s } ≤ { ofColex := t }
hcard : s.card ≤ t.card
ha : a ∈ s
ht : t.Nonempty
m : α := t.min' ht
⊢ { ofColex := s.erase a } ≤ { ofColex := t.erase m } |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Combinatorics/Colex.lean | Finset.Colex.erase_le_erase_min' | [73, 1] | [115, 94] | obtain rfl | h' := eq_or_ne s t | α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a : α
hst : { ofColex := s } ≤ { ofColex := t }
hcard : s.card ≤ t.card
ha : a ∈ s
ht : t.Nonempty
m : α := t.min' ht
⊢ { ofColex := s.erase a } ≤ { ofColex := t.erase m } | case inl
α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s : Finset α
a : α
ha : a ∈ s
hst : { ofColex := s } ≤ { ofColex := s }
hcard : s.card ≤ s.card
ht : s.Nonempty
m : α := s.min' ht
⊢ { ofColex := s.erase a } ≤ { ofColex := s.erase m }
case inr
α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a : α
hst : { ofColex := s } ≤ { ofColex := t }
hcard : s.card ≤ t.card
ha : a ∈ s
ht : t.Nonempty
m : α := t.min' ht
h' : s ≠ t
⊢ { ofColex := s.erase a } ≤ { ofColex := t.erase m } |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Combinatorics/Colex.lean | Finset.Colex.erase_le_erase_min' | [73, 1] | [115, 94] | replace hst := hst.lt_of_ne $ toColex_inj.not.2 h' | case inr
α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a : α
hst : { ofColex := s } ≤ { ofColex := t }
hcard : s.card ≤ t.card
ha : a ∈ s
ht : t.Nonempty
m : α := t.min' ht
h' : s ≠ t
⊢ { ofColex := s.erase a } ≤ { ofColex := t.erase m } | case inr
α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a : α
hcard : s.card ≤ t.card
ha : a ∈ s
ht : t.Nonempty
m : α := t.min' ht
h' : s ≠ t
hst : { ofColex := s } < { ofColex := t }
⊢ { ofColex := s.erase a } ≤ { ofColex := t.erase m } |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Combinatorics/Colex.lean | Finset.Colex.erase_le_erase_min' | [73, 1] | [115, 94] | simp only [lt_iff_exists_forall_lt_mem_iff_mem] at hst | case inr
α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a : α
hcard : s.card ≤ t.card
ha : a ∈ s
ht : t.Nonempty
m : α := t.min' ht
h' : s ≠ t
hst : { ofColex := s } < { ofColex := t }
⊢ { ofColex := s.erase a } ≤ { ofColex := t.erase m } | case inr
α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a : α
hcard : s.card ≤ t.card
ha : a ∈ s
ht : t.Nonempty
m : α := t.min' ht
h' : s ≠ t
hst : ∃ w ∈ t, w ∉ s ∧ ∀ ⦃a : α⦄, w < a → (a ∈ s ↔ a ∈ t)
⊢ { ofColex := s.erase a } ≤ { ofColex := t.erase m } |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Combinatorics/Colex.lean | Finset.Colex.erase_le_erase_min' | [73, 1] | [115, 94] | obtain ⟨w, hwt, hws, hw⟩ := hst | case inr
α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a : α
hcard : s.card ≤ t.card
ha : a ∈ s
ht : t.Nonempty
m : α := t.min' ht
h' : s ≠ t
hst : ∃ w ∈ t, w ∉ s ∧ ∀ ⦃a : α⦄, w < a → (a ∈ s ↔ a ∈ t)
⊢ { ofColex := s.erase a } ≤ { ofColex := t.erase m } | case inr.intro.intro.intro
α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a : α
hcard : s.card ≤ t.card
ha : a ∈ s
ht : t.Nonempty
m : α := t.min' ht
h' : s ≠ t
w : α
hwt : w ∈ t
hws : w ∉ s
hw : ∀ ⦃a : α⦄, w < a → (a ∈ s ↔ a ∈ t)
⊢ { ofColex := s.erase a } ≤ { ofColex := t.erase m } |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Combinatorics/Colex.lean | Finset.Colex.erase_le_erase_min' | [73, 1] | [115, 94] | obtain hwa | haw := (ne_of_mem_of_not_mem ha hws).symm.lt_or_lt | case inr.intro.intro.intro
α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a : α
hcard : s.card ≤ t.card
ha : a ∈ s
ht : t.Nonempty
m : α := t.min' ht
h' : s ≠ t
w : α
hwt : w ∈ t
hws : w ∉ s
hw : ∀ ⦃a : α⦄, w < a → (a ∈ s ↔ a ∈ t)
⊢ { ofColex := s.erase a } ≤ { ofColex := t.erase m } | case inr.intro.intro.intro.inl
α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a : α
hcard : s.card ≤ t.card
ha : a ∈ s
ht : t.Nonempty
m : α := t.min' ht
h' : s ≠ t
w : α
hwt : w ∈ t
hws : w ∉ s
hw : ∀ ⦃a : α⦄, w < a → (a ∈ s ↔ a ∈ t)
hwa : w < a
⊢ { ofColex := s.erase a } ≤ { ofColex := t.erase m }
case inr.intro.intro.intro.inr
α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a : α
hcard : s.card ≤ t.card
ha : a ∈ s
ht : t.Nonempty
m : α := t.min' ht
h' : s ≠ t
w : α
hwt : w ∈ t
hws : w ∉ s
hw : ∀ ⦃a : α⦄, w < a → (a ∈ s ↔ a ∈ t)
haw : a < w
⊢ { ofColex := s.erase a } ≤ { ofColex := t.erase m } |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Combinatorics/Colex.lean | Finset.Colex.erase_le_erase_min' | [73, 1] | [115, 94] | obtain rfl | hmw : m = w ∨ m < w := (min'_le _ _ hwt).eq_or_lt | case inr.intro.intro.intro.inr
α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a : α
hcard : s.card ≤ t.card
ha : a ∈ s
ht : t.Nonempty
m : α := t.min' ht
h' : s ≠ t
w : α
hwt : w ∈ t
hws : w ∉ s
hw : ∀ ⦃a : α⦄, w < a → (a ∈ s ↔ a ∈ t)
haw : a < w
⊢ { ofColex := s.erase a } ≤ { ofColex := t.erase m } | case inr.intro.intro.intro.inr.inl
α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a : α
hcard : s.card ≤ t.card
ha : a ∈ s
ht : t.Nonempty
m : α := t.min' ht
h' : s ≠ t
hwt : m ∈ t
hws : m ∉ s
hw : ∀ ⦃a : α⦄, m < a → (a ∈ s ↔ a ∈ t)
haw : a < m
⊢ { ofColex := s.erase a } ≤ { ofColex := t.erase m }
case inr.intro.intro.intro.inr.inr
α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a : α
hcard : s.card ≤ t.card
ha : a ∈ s
ht : t.Nonempty
m : α := t.min' ht
h' : s ≠ t
w : α
hwt : w ∈ t
hws : w ∉ s
hw : ∀ ⦃a : α⦄, w < a → (a ∈ s ↔ a ∈ t)
haw : a < w
hmw : m < w
⊢ { ofColex := s.erase a } ≤ { ofColex := t.erase m } |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Combinatorics/Colex.lean | Finset.Colex.erase_le_erase_min' | [73, 1] | [115, 94] | exact (erase_le_erase ha $ min'_mem _ _).2 $ min'_le _ _ $ ha | case inl
α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s : Finset α
a : α
ha : a ∈ s
hst : { ofColex := s } ≤ { ofColex := s }
hcard : s.card ≤ s.card
ht : s.Nonempty
m : α := s.min' ht
⊢ { ofColex := s.erase a } ≤ { ofColex := s.erase m } | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Combinatorics/Colex.lean | Finset.Colex.erase_le_erase_min' | [73, 1] | [115, 94] | have hma : m < a := (min'_le _ _ hwt).trans_lt hwa | case inr.intro.intro.intro.inl
α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a : α
hcard : s.card ≤ t.card
ha : a ∈ s
ht : t.Nonempty
m : α := t.min' ht
h' : s ≠ t
w : α
hwt : w ∈ t
hws : w ∉ s
hw : ∀ ⦃a : α⦄, w < a → (a ∈ s ↔ a ∈ t)
hwa : w < a
⊢ { ofColex := s.erase a } ≤ { ofColex := t.erase m } | case inr.intro.intro.intro.inl
α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a : α
hcard : s.card ≤ t.card
ha : a ∈ s
ht : t.Nonempty
m : α := t.min' ht
h' : s ≠ t
w : α
hwt : w ∈ t
hws : w ∉ s
hw : ∀ ⦃a : α⦄, w < a → (a ∈ s ↔ a ∈ t)
hwa : w < a
hma : m < a
⊢ { ofColex := s.erase a } ≤ { ofColex := t.erase m } |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Combinatorics/Colex.lean | Finset.Colex.erase_le_erase_min' | [73, 1] | [115, 94] | refine (lt_iff_exists_forall_lt.2 ⟨a, mem_erase.2 ⟨hma.ne', (hw hwa).1 ha⟩,
not_mem_erase _ _, fun b hbs hbt ↦ ?_⟩).le | case inr.intro.intro.intro.inl
α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a : α
hcard : s.card ≤ t.card
ha : a ∈ s
ht : t.Nonempty
m : α := t.min' ht
h' : s ≠ t
w : α
hwt : w ∈ t
hws : w ∉ s
hw : ∀ ⦃a : α⦄, w < a → (a ∈ s ↔ a ∈ t)
hwa : w < a
hma : m < a
⊢ { ofColex := s.erase a } ≤ { ofColex := t.erase m } | case inr.intro.intro.intro.inl
α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a : α
hcard : s.card ≤ t.card
ha : a ∈ s
ht : t.Nonempty
m : α := t.min' ht
h' : s ≠ t
w : α
hwt : w ∈ t
hws : w ∉ s
hw : ∀ ⦃a : α⦄, w < a → (a ∈ s ↔ a ∈ t)
hwa : w < a
hma : m < a
b : α
hbs : b ∈ { ofColex := { val := s.val.erase a, nodup := ⋯ } }.ofColex
hbt : b ∉ { ofColex := { val := t.val.erase m, nodup := ⋯ } }.ofColex
⊢ b < a |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Combinatorics/Colex.lean | Finset.Colex.erase_le_erase_min' | [73, 1] | [115, 94] | change b ∉ t.erase m at hbt | case inr.intro.intro.intro.inl
α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a : α
hcard : s.card ≤ t.card
ha : a ∈ s
ht : t.Nonempty
m : α := t.min' ht
h' : s ≠ t
w : α
hwt : w ∈ t
hws : w ∉ s
hw : ∀ ⦃a : α⦄, w < a → (a ∈ s ↔ a ∈ t)
hwa : w < a
hma : m < a
b : α
hbs : b ∈ { ofColex := { val := s.val.erase a, nodup := ⋯ } }.ofColex
hbt : b ∉ { ofColex := { val := t.val.erase m, nodup := ⋯ } }.ofColex
⊢ b < a | case inr.intro.intro.intro.inl
α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a : α
hcard : s.card ≤ t.card
ha : a ∈ s
ht : t.Nonempty
m : α := t.min' ht
h' : s ≠ t
w : α
hwt : w ∈ t
hws : w ∉ s
hw : ∀ ⦃a : α⦄, w < a → (a ∈ s ↔ a ∈ t)
hwa : w < a
hma : m < a
b : α
hbs : b ∈ { ofColex := { val := s.val.erase a, nodup := ⋯ } }.ofColex
hbt : b ∉ t.erase m
⊢ b < a |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Combinatorics/Colex.lean | Finset.Colex.erase_le_erase_min' | [73, 1] | [115, 94] | rw [mem_erase, not_and_or, not_ne_iff] at hbt | case inr.intro.intro.intro.inl
α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a : α
hcard : s.card ≤ t.card
ha : a ∈ s
ht : t.Nonempty
m : α := t.min' ht
h' : s ≠ t
w : α
hwt : w ∈ t
hws : w ∉ s
hw : ∀ ⦃a : α⦄, w < a → (a ∈ s ↔ a ∈ t)
hwa : w < a
hma : m < a
b : α
hbs : b ∈ { ofColex := { val := s.val.erase a, nodup := ⋯ } }.ofColex
hbt : b ∉ t.erase m
⊢ b < a | case inr.intro.intro.intro.inl
α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a : α
hcard : s.card ≤ t.card
ha : a ∈ s
ht : t.Nonempty
m : α := t.min' ht
h' : s ≠ t
w : α
hwt : w ∈ t
hws : w ∉ s
hw : ∀ ⦃a : α⦄, w < a → (a ∈ s ↔ a ∈ t)
hwa : w < a
hma : m < a
b : α
hbs : b ∈ { ofColex := { val := s.val.erase a, nodup := ⋯ } }.ofColex
hbt : b = m ∨ b ∉ t
⊢ b < a |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Combinatorics/Colex.lean | Finset.Colex.erase_le_erase_min' | [73, 1] | [115, 94] | obtain rfl | hbt := hbt | case inr.intro.intro.intro.inl
α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a : α
hcard : s.card ≤ t.card
ha : a ∈ s
ht : t.Nonempty
m : α := t.min' ht
h' : s ≠ t
w : α
hwt : w ∈ t
hws : w ∉ s
hw : ∀ ⦃a : α⦄, w < a → (a ∈ s ↔ a ∈ t)
hwa : w < a
hma : m < a
b : α
hbs : b ∈ { ofColex := { val := s.val.erase a, nodup := ⋯ } }.ofColex
hbt : b = m ∨ b ∉ t
⊢ b < a | case inr.intro.intro.intro.inl.inl
α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a : α
hcard : s.card ≤ t.card
ha : a ∈ s
ht : t.Nonempty
m : α := t.min' ht
h' : s ≠ t
w : α
hwt : w ∈ t
hws : w ∉ s
hw : ∀ ⦃a : α⦄, w < a → (a ∈ s ↔ a ∈ t)
hwa : w < a
hma : m < a
hbs : m ∈ { ofColex := { val := s.val.erase a, nodup := ⋯ } }.ofColex
⊢ m < a
case inr.intro.intro.intro.inl.inr
α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a : α
hcard : s.card ≤ t.card
ha : a ∈ s
ht : t.Nonempty
m : α := t.min' ht
h' : s ≠ t
w : α
hwt : w ∈ t
hws : w ∉ s
hw : ∀ ⦃a : α⦄, w < a → (a ∈ s ↔ a ∈ t)
hwa : w < a
hma : m < a
b : α
hbs : b ∈ { ofColex := { val := s.val.erase a, nodup := ⋯ } }.ofColex
hbt : b ∉ t
⊢ b < a |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Combinatorics/Colex.lean | Finset.Colex.erase_le_erase_min' | [73, 1] | [115, 94] | assumption | case inr.intro.intro.intro.inl.inl
α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a : α
hcard : s.card ≤ t.card
ha : a ∈ s
ht : t.Nonempty
m : α := t.min' ht
h' : s ≠ t
w : α
hwt : w ∈ t
hws : w ∉ s
hw : ∀ ⦃a : α⦄, w < a → (a ∈ s ↔ a ∈ t)
hwa : w < a
hma : m < a
hbs : m ∈ { ofColex := { val := s.val.erase a, nodup := ⋯ } }.ofColex
⊢ m < a | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Combinatorics/Colex.lean | Finset.Colex.erase_le_erase_min' | [73, 1] | [115, 94] | by_contra! hab | case inr.intro.intro.intro.inl.inr
α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a : α
hcard : s.card ≤ t.card
ha : a ∈ s
ht : t.Nonempty
m : α := t.min' ht
h' : s ≠ t
w : α
hwt : w ∈ t
hws : w ∉ s
hw : ∀ ⦃a : α⦄, w < a → (a ∈ s ↔ a ∈ t)
hwa : w < a
hma : m < a
b : α
hbs : b ∈ { ofColex := { val := s.val.erase a, nodup := ⋯ } }.ofColex
hbt : b ∉ t
⊢ b < a | case inr.intro.intro.intro.inl.inr
α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a : α
hcard : s.card ≤ t.card
ha : a ∈ s
ht : t.Nonempty
m : α := t.min' ht
h' : s ≠ t
w : α
hwt : w ∈ t
hws : w ∉ s
hw : ∀ ⦃a : α⦄, w < a → (a ∈ s ↔ a ∈ t)
hwa : w < a
hma : m < a
b : α
hbs : b ∈ { ofColex := { val := s.val.erase a, nodup := ⋯ } }.ofColex
hbt : b ∉ t
hab : a ≤ b
⊢ False |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Combinatorics/Colex.lean | Finset.Colex.erase_le_erase_min' | [73, 1] | [115, 94] | exact hbt $ (hw $ hwa.trans_le hab).1 $ mem_of_mem_erase hbs | case inr.intro.intro.intro.inl.inr
α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a : α
hcard : s.card ≤ t.card
ha : a ∈ s
ht : t.Nonempty
m : α := t.min' ht
h' : s ≠ t
w : α
hwt : w ∈ t
hws : w ∉ s
hw : ∀ ⦃a : α⦄, w < a → (a ∈ s ↔ a ∈ t)
hwa : w < a
hma : m < a
b : α
hbs : b ∈ { ofColex := { val := s.val.erase a, nodup := ⋯ } }.ofColex
hbt : b ∉ t
hab : a ≤ b
⊢ False | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Combinatorics/Colex.lean | Finset.Colex.erase_le_erase_min' | [73, 1] | [115, 94] | have : erase t m ⊆ erase s a := by
rintro b hb
rw [mem_erase] at hb ⊢
exact ⟨(haw.trans_le $ min'_le _ _ hb.2).ne', (hw $ hb.1.lt_of_le' $ min'_le _ _ hb.2).2 hb.2⟩ | case inr.intro.intro.intro.inr.inl
α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a : α
hcard : s.card ≤ t.card
ha : a ∈ s
ht : t.Nonempty
m : α := t.min' ht
h' : s ≠ t
hwt : m ∈ t
hws : m ∉ s
hw : ∀ ⦃a : α⦄, m < a → (a ∈ s ↔ a ∈ t)
haw : a < m
⊢ { ofColex := s.erase a } ≤ { ofColex := t.erase m } | case inr.intro.intro.intro.inr.inl
α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a : α
hcard : s.card ≤ t.card
ha : a ∈ s
ht : t.Nonempty
m : α := t.min' ht
h' : s ≠ t
hwt : m ∈ t
hws : m ∉ s
hw : ∀ ⦃a : α⦄, m < a → (a ∈ s ↔ a ∈ t)
haw : a < m
this : t.erase m ⊆ s.erase a
⊢ { ofColex := s.erase a } ≤ { ofColex := t.erase m } |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Combinatorics/Colex.lean | Finset.Colex.erase_le_erase_min' | [73, 1] | [115, 94] | rw [eq_of_subset_of_card_le this] | case inr.intro.intro.intro.inr.inl
α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a : α
hcard : s.card ≤ t.card
ha : a ∈ s
ht : t.Nonempty
m : α := t.min' ht
h' : s ≠ t
hwt : m ∈ t
hws : m ∉ s
hw : ∀ ⦃a : α⦄, m < a → (a ∈ s ↔ a ∈ t)
haw : a < m
this : t.erase m ⊆ s.erase a
⊢ { ofColex := s.erase a } ≤ { ofColex := t.erase m } | case inr.intro.intro.intro.inr.inl
α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a : α
hcard : s.card ≤ t.card
ha : a ∈ s
ht : t.Nonempty
m : α := t.min' ht
h' : s ≠ t
hwt : m ∈ t
hws : m ∉ s
hw : ∀ ⦃a : α⦄, m < a → (a ∈ s ↔ a ∈ t)
haw : a < m
this : t.erase m ⊆ s.erase a
⊢ (s.erase a).card ≤ (t.erase m).card |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Combinatorics/Colex.lean | Finset.Colex.erase_le_erase_min' | [73, 1] | [115, 94] | rw [card_erase_of_mem ha, card_erase_of_mem (min'_mem _ _)] | case inr.intro.intro.intro.inr.inl
α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a : α
hcard : s.card ≤ t.card
ha : a ∈ s
ht : t.Nonempty
m : α := t.min' ht
h' : s ≠ t
hwt : m ∈ t
hws : m ∉ s
hw : ∀ ⦃a : α⦄, m < a → (a ∈ s ↔ a ∈ t)
haw : a < m
this : t.erase m ⊆ s.erase a
⊢ (s.erase a).card ≤ (t.erase m).card | case inr.intro.intro.intro.inr.inl
α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a : α
hcard : s.card ≤ t.card
ha : a ∈ s
ht : t.Nonempty
m : α := t.min' ht
h' : s ≠ t
hwt : m ∈ t
hws : m ∉ s
hw : ∀ ⦃a : α⦄, m < a → (a ∈ s ↔ a ∈ t)
haw : a < m
this : t.erase m ⊆ s.erase a
⊢ s.card - 1 ≤ t.card - 1 |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Combinatorics/Colex.lean | Finset.Colex.erase_le_erase_min' | [73, 1] | [115, 94] | exact tsub_le_tsub_right hcard _ | case inr.intro.intro.intro.inr.inl
α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a : α
hcard : s.card ≤ t.card
ha : a ∈ s
ht : t.Nonempty
m : α := t.min' ht
h' : s ≠ t
hwt : m ∈ t
hws : m ∉ s
hw : ∀ ⦃a : α⦄, m < a → (a ∈ s ↔ a ∈ t)
haw : a < m
this : t.erase m ⊆ s.erase a
⊢ s.card - 1 ≤ t.card - 1 | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Combinatorics/Colex.lean | Finset.Colex.erase_le_erase_min' | [73, 1] | [115, 94] | rintro b hb | α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a : α
hcard : s.card ≤ t.card
ha : a ∈ s
ht : t.Nonempty
m : α := t.min' ht
h' : s ≠ t
hwt : m ∈ t
hws : m ∉ s
hw : ∀ ⦃a : α⦄, m < a → (a ∈ s ↔ a ∈ t)
haw : a < m
⊢ t.erase m ⊆ s.erase a | α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a : α
hcard : s.card ≤ t.card
ha : a ∈ s
ht : t.Nonempty
m : α := t.min' ht
h' : s ≠ t
hwt : m ∈ t
hws : m ∉ s
hw : ∀ ⦃a : α⦄, m < a → (a ∈ s ↔ a ∈ t)
haw : a < m
b : α
hb : b ∈ t.erase m
⊢ b ∈ s.erase a |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Combinatorics/Colex.lean | Finset.Colex.erase_le_erase_min' | [73, 1] | [115, 94] | rw [mem_erase] at hb ⊢ | α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a : α
hcard : s.card ≤ t.card
ha : a ∈ s
ht : t.Nonempty
m : α := t.min' ht
h' : s ≠ t
hwt : m ∈ t
hws : m ∉ s
hw : ∀ ⦃a : α⦄, m < a → (a ∈ s ↔ a ∈ t)
haw : a < m
b : α
hb : b ∈ t.erase m
⊢ b ∈ s.erase a | α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a : α
hcard : s.card ≤ t.card
ha : a ∈ s
ht : t.Nonempty
m : α := t.min' ht
h' : s ≠ t
hwt : m ∈ t
hws : m ∉ s
hw : ∀ ⦃a : α⦄, m < a → (a ∈ s ↔ a ∈ t)
haw : a < m
b : α
hb : b ≠ m ∧ b ∈ t
⊢ b ≠ a ∧ b ∈ s |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Combinatorics/Colex.lean | Finset.Colex.erase_le_erase_min' | [73, 1] | [115, 94] | exact ⟨(haw.trans_le $ min'_le _ _ hb.2).ne', (hw $ hb.1.lt_of_le' $ min'_le _ _ hb.2).2 hb.2⟩ | α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a : α
hcard : s.card ≤ t.card
ha : a ∈ s
ht : t.Nonempty
m : α := t.min' ht
h' : s ≠ t
hwt : m ∈ t
hws : m ∉ s
hw : ∀ ⦃a : α⦄, m < a → (a ∈ s ↔ a ∈ t)
haw : a < m
b : α
hb : b ≠ m ∧ b ∈ t
⊢ b ≠ a ∧ b ∈ s | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Combinatorics/Colex.lean | Finset.Colex.erase_le_erase_min' | [73, 1] | [115, 94] | refine (lt_iff_exists_forall_lt.2 ⟨w, mem_erase.2 ⟨hmw.ne', hwt⟩, mt mem_of_mem_erase hws,
fun b hbs hbt ↦ ?_⟩).le | case inr.intro.intro.intro.inr.inr
α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a : α
hcard : s.card ≤ t.card
ha : a ∈ s
ht : t.Nonempty
m : α := t.min' ht
h' : s ≠ t
w : α
hwt : w ∈ t
hws : w ∉ s
hw : ∀ ⦃a : α⦄, w < a → (a ∈ s ↔ a ∈ t)
haw : a < w
hmw : m < w
⊢ { ofColex := s.erase a } ≤ { ofColex := t.erase m } | case inr.intro.intro.intro.inr.inr
α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a : α
hcard : s.card ≤ t.card
ha : a ∈ s
ht : t.Nonempty
m : α := t.min' ht
h' : s ≠ t
w : α
hwt : w ∈ t
hws : w ∉ s
hw : ∀ ⦃a : α⦄, w < a → (a ∈ s ↔ a ∈ t)
haw : a < w
hmw : m < w
b : α
hbs : b ∈ { ofColex := { val := s.val.erase a, nodup := ⋯ } }.ofColex
hbt : b ∉ { ofColex := { val := t.val.erase m, nodup := ⋯ } }.ofColex
⊢ b < w |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Combinatorics/Colex.lean | Finset.Colex.erase_le_erase_min' | [73, 1] | [115, 94] | change b ∉ t.erase m at hbt | case inr.intro.intro.intro.inr.inr
α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a : α
hcard : s.card ≤ t.card
ha : a ∈ s
ht : t.Nonempty
m : α := t.min' ht
h' : s ≠ t
w : α
hwt : w ∈ t
hws : w ∉ s
hw : ∀ ⦃a : α⦄, w < a → (a ∈ s ↔ a ∈ t)
haw : a < w
hmw : m < w
b : α
hbs : b ∈ { ofColex := { val := s.val.erase a, nodup := ⋯ } }.ofColex
hbt : b ∉ { ofColex := { val := t.val.erase m, nodup := ⋯ } }.ofColex
⊢ b < w | case inr.intro.intro.intro.inr.inr
α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a : α
hcard : s.card ≤ t.card
ha : a ∈ s
ht : t.Nonempty
m : α := t.min' ht
h' : s ≠ t
w : α
hwt : w ∈ t
hws : w ∉ s
hw : ∀ ⦃a : α⦄, w < a → (a ∈ s ↔ a ∈ t)
haw : a < w
hmw : m < w
b : α
hbs : b ∈ { ofColex := { val := s.val.erase a, nodup := ⋯ } }.ofColex
hbt : b ∉ t.erase m
⊢ b < w |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Combinatorics/Colex.lean | Finset.Colex.erase_le_erase_min' | [73, 1] | [115, 94] | rw [mem_erase, not_and_or, not_ne_iff] at hbt | case inr.intro.intro.intro.inr.inr
α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a : α
hcard : s.card ≤ t.card
ha : a ∈ s
ht : t.Nonempty
m : α := t.min' ht
h' : s ≠ t
w : α
hwt : w ∈ t
hws : w ∉ s
hw : ∀ ⦃a : α⦄, w < a → (a ∈ s ↔ a ∈ t)
haw : a < w
hmw : m < w
b : α
hbs : b ∈ { ofColex := { val := s.val.erase a, nodup := ⋯ } }.ofColex
hbt : b ∉ t.erase m
⊢ b < w | case inr.intro.intro.intro.inr.inr
α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a : α
hcard : s.card ≤ t.card
ha : a ∈ s
ht : t.Nonempty
m : α := t.min' ht
h' : s ≠ t
w : α
hwt : w ∈ t
hws : w ∉ s
hw : ∀ ⦃a : α⦄, w < a → (a ∈ s ↔ a ∈ t)
haw : a < w
hmw : m < w
b : α
hbs : b ∈ { ofColex := { val := s.val.erase a, nodup := ⋯ } }.ofColex
hbt : b = m ∨ b ∉ t
⊢ b < w |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Combinatorics/Colex.lean | Finset.Colex.erase_le_erase_min' | [73, 1] | [115, 94] | obtain rfl | hbt := hbt | case inr.intro.intro.intro.inr.inr
α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a : α
hcard : s.card ≤ t.card
ha : a ∈ s
ht : t.Nonempty
m : α := t.min' ht
h' : s ≠ t
w : α
hwt : w ∈ t
hws : w ∉ s
hw : ∀ ⦃a : α⦄, w < a → (a ∈ s ↔ a ∈ t)
haw : a < w
hmw : m < w
b : α
hbs : b ∈ { ofColex := { val := s.val.erase a, nodup := ⋯ } }.ofColex
hbt : b = m ∨ b ∉ t
⊢ b < w | case inr.intro.intro.intro.inr.inr.inl
α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a : α
hcard : s.card ≤ t.card
ha : a ∈ s
ht : t.Nonempty
m : α := t.min' ht
h' : s ≠ t
w : α
hwt : w ∈ t
hws : w ∉ s
hw : ∀ ⦃a : α⦄, w < a → (a ∈ s ↔ a ∈ t)
haw : a < w
hmw : m < w
hbs : m ∈ { ofColex := { val := s.val.erase a, nodup := ⋯ } }.ofColex
⊢ m < w
case inr.intro.intro.intro.inr.inr.inr
α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a : α
hcard : s.card ≤ t.card
ha : a ∈ s
ht : t.Nonempty
m : α := t.min' ht
h' : s ≠ t
w : α
hwt : w ∈ t
hws : w ∉ s
hw : ∀ ⦃a : α⦄, w < a → (a ∈ s ↔ a ∈ t)
haw : a < w
hmw : m < w
b : α
hbs : b ∈ { ofColex := { val := s.val.erase a, nodup := ⋯ } }.ofColex
hbt : b ∉ t
⊢ b < w |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Combinatorics/Colex.lean | Finset.Colex.erase_le_erase_min' | [73, 1] | [115, 94] | assumption | case inr.intro.intro.intro.inr.inr.inl
α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a : α
hcard : s.card ≤ t.card
ha : a ∈ s
ht : t.Nonempty
m : α := t.min' ht
h' : s ≠ t
w : α
hwt : w ∈ t
hws : w ∉ s
hw : ∀ ⦃a : α⦄, w < a → (a ∈ s ↔ a ∈ t)
haw : a < w
hmw : m < w
hbs : m ∈ { ofColex := { val := s.val.erase a, nodup := ⋯ } }.ofColex
⊢ m < w | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Combinatorics/Colex.lean | Finset.Colex.erase_le_erase_min' | [73, 1] | [115, 94] | by_contra! hwb | case inr.intro.intro.intro.inr.inr.inr
α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a : α
hcard : s.card ≤ t.card
ha : a ∈ s
ht : t.Nonempty
m : α := t.min' ht
h' : s ≠ t
w : α
hwt : w ∈ t
hws : w ∉ s
hw : ∀ ⦃a : α⦄, w < a → (a ∈ s ↔ a ∈ t)
haw : a < w
hmw : m < w
b : α
hbs : b ∈ { ofColex := { val := s.val.erase a, nodup := ⋯ } }.ofColex
hbt : b ∉ t
⊢ b < w | case inr.intro.intro.intro.inr.inr.inr
α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a : α
hcard : s.card ≤ t.card
ha : a ∈ s
ht : t.Nonempty
m : α := t.min' ht
h' : s ≠ t
w : α
hwt : w ∈ t
hws : w ∉ s
hw : ∀ ⦃a : α⦄, w < a → (a ∈ s ↔ a ∈ t)
haw : a < w
hmw : m < w
b : α
hbs : b ∈ { ofColex := { val := s.val.erase a, nodup := ⋯ } }.ofColex
hbt : b ∉ t
hwb : w ≤ b
⊢ False |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/Mathlib/Combinatorics/Colex.lean | Finset.Colex.erase_le_erase_min' | [73, 1] | [115, 94] | exact hbt $ (hw $ hwb.lt_of_ne $ ne_of_mem_of_not_mem hwt hbt).1 $ mem_of_mem_erase hbs | case inr.intro.intro.intro.inr.inr.inr
α : Type u_1
β : Type u_2
inst✝ : LinearOrder α
s t : Finset α
a : α
hcard : s.card ≤ t.card
ha : a ∈ s
ht : t.Nonempty
m : α := t.min' ht
h' : s ≠ t
w : α
hwt : w ∈ t
hws : w ∉ s
hw : ∀ ⦃a : α⦄, w < a → (a ∈ s ↔ a ∈ t)
haw : a < w
hmw : m < w
b : α
hbs : b ∈ { ofColex := { val := s.val.erase a, nodup := ⋯ } }.ofColex
hbt : b ∉ t
hwb : w ≤ b
⊢ False | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | generateLine_minimal | [36, 1] | [44, 61] | intro x hx | V : Type u_1
inst✝ : MetricSpace V
u v w : V
S L : Set V
hL₀ : S ⊆ L
out_closed : ∀ {x y z : V}, x ∈ L → y ∈ L → sbtw x y z → z ∈ L
in_closed : ∀ {x y z : V}, x ∈ L → y ∈ L → sbtw x z y → z ∈ L
⊢ GenerateLine S ⊆ L | V : Type u_1
inst✝ : MetricSpace V
u v w : V
S L : Set V
hL₀ : S ⊆ L
out_closed : ∀ {x y z : V}, x ∈ L → y ∈ L → sbtw x y z → z ∈ L
in_closed : ∀ {x y z : V}, x ∈ L → y ∈ L → sbtw x z y → z ∈ L
x : V
hx : x ∈ GenerateLine S
⊢ x ∈ L |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | generateLine_minimal | [36, 1] | [44, 61] | induction hx with
| basic h => exact hL₀ h
| extend_out u v w _ _ hw hu hv => exact out_closed hu hv hw
| extend_in u v w _ _ hw hu hv => exact in_closed hu hv hw | V : Type u_1
inst✝ : MetricSpace V
u v w : V
S L : Set V
hL₀ : S ⊆ L
out_closed : ∀ {x y z : V}, x ∈ L → y ∈ L → sbtw x y z → z ∈ L
in_closed : ∀ {x y z : V}, x ∈ L → y ∈ L → sbtw x z y → z ∈ L
x : V
hx : x ∈ GenerateLine S
⊢ x ∈ L | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | generateLine_minimal | [36, 1] | [44, 61] | exact hL₀ h | case basic
V : Type u_1
inst✝ : MetricSpace V
u v w : V
S L : Set V
hL₀ : S ⊆ L
out_closed : ∀ {x y z : V}, x ∈ L → y ∈ L → sbtw x y z → z ∈ L
in_closed : ∀ {x y z : V}, x ∈ L → y ∈ L → sbtw x z y → z ∈ L
x x✝ : V
h : x✝ ∈ S
⊢ x✝ ∈ L | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | generateLine_minimal | [36, 1] | [44, 61] | exact out_closed hu hv hw | case extend_out
V : Type u_1
inst✝ : MetricSpace V
u✝ v✝ w✝ : V
S L : Set V
hL₀ : S ⊆ L
out_closed : ∀ {x y z : V}, x ∈ L → y ∈ L → sbtw x y z → z ∈ L
in_closed : ∀ {x y z : V}, x ∈ L → y ∈ L → sbtw x z y → z ∈ L
x u v w : V
a✝¹ : GenerateLine S u
a✝ : GenerateLine S v
hw : sbtw u v w
hu : u ∈ L
hv : v ∈ L
⊢ w ∈ L | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | generateLine_minimal | [36, 1] | [44, 61] | exact in_closed hu hv hw | case extend_in
V : Type u_1
inst✝ : MetricSpace V
u✝ v✝ w✝ : V
S L : Set V
hL₀ : S ⊆ L
out_closed : ∀ {x y z : V}, x ∈ L → y ∈ L → sbtw x y z → z ∈ L
in_closed : ∀ {x y z : V}, x ∈ L → y ∈ L → sbtw x z y → z ∈ L
x u v w : V
a✝¹ : GenerateLine S u
a✝ : GenerateLine S v
hw : sbtw u w v
hu : u ∈ L
hv : v ∈ L
⊢ w ∈ L | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | left_mem_Line | [48, 1] | [48, 88] | simp | V : Type u_1
inst✝ : MetricSpace V
u v w a b : V
⊢ a ∈ {a, b} | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | right_mem_Line | [49, 1] | [49, 89] | simp | V : Type u_1
inst✝ : MetricSpace V
u v w a b : V
⊢ b ∈ {a, b} | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | Line_comm | [57, 1] | [57, 75] | rw [Line, Line, Set.pair_comm] | V : Type u_1
inst✝ : MetricSpace V
u v w : V
⊢ Line u v = Line v u | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | Set.IsLine.close_right | [63, 1] | [66, 42] | obtain ⟨x, y, _, rfl⟩ := hL | V : Type u_1
inst✝ : MetricSpace V
u v w : V
L : Set V
hL : L.IsLine
a b c : V
ha : a ∈ L
hb : b ∈ L
hc : sbtw a b c
⊢ c ∈ L | case intro.intro.intro
V : Type u_1
inst✝ : MetricSpace V
u v w a b c : V
hc : sbtw a b c
x y : V
left✝ : x ≠ y
ha : a ∈ Line x y
hb : b ∈ Line x y
⊢ c ∈ Line x y |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | Set.IsLine.close_right | [63, 1] | [66, 42] | exact generateLine_close_right ha hb hc | case intro.intro.intro
V : Type u_1
inst✝ : MetricSpace V
u v w a b c : V
hc : sbtw a b c
x y : V
left✝ : x ≠ y
ha : a ∈ Line x y
hb : b ∈ Line x y
⊢ c ∈ Line x y | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | Set.IsLine.close_left | [68, 1] | [71, 41] | obtain ⟨x, y, _, rfl⟩ := hL | V : Type u_1
inst✝ : MetricSpace V
u v w : V
L : Set V
hL : L.IsLine
a b c : V
ha : a ∈ L
hb : b ∈ L
hc : sbtw c a b
⊢ c ∈ L | case intro.intro.intro
V : Type u_1
inst✝ : MetricSpace V
u v w a b c : V
hc : sbtw c a b
x y : V
left✝ : x ≠ y
ha : a ∈ Line x y
hb : b ∈ Line x y
⊢ c ∈ Line x y |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | Set.IsLine.close_left | [68, 1] | [71, 41] | exact generateLine_close_left ha hb hc | case intro.intro.intro
V : Type u_1
inst✝ : MetricSpace V
u v w a b c : V
hc : sbtw c a b
x y : V
left✝ : x ≠ y
ha : a ∈ Line x y
hb : b ∈ Line x y
⊢ c ∈ Line x y | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | Set.IsLine.close_middle | [73, 1] | [76, 43] | obtain ⟨x, y, _, rfl⟩ := hL | V : Type u_1
inst✝ : MetricSpace V
u v w : V
L : Set V
hL : L.IsLine
a b c : V
ha : a ∈ L
hb : b ∈ L
hc : sbtw a c b
⊢ c ∈ L | case intro.intro.intro
V : Type u_1
inst✝ : MetricSpace V
u v w a b c : V
hc : sbtw a c b
x y : V
left✝ : x ≠ y
ha : a ∈ Line x y
hb : b ∈ Line x y
⊢ c ∈ Line x y |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | Set.IsLine.close_middle | [73, 1] | [76, 43] | exact generateLine_close_middle ha hb hc | case intro.intro.intro
V : Type u_1
inst✝ : MetricSpace V
u v w a b c : V
hc : sbtw a c b
x y : V
left✝ : x ≠ y
ha : a ∈ Line x y
hb : b ∈ Line x y
⊢ c ∈ Line x y | no goals |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | exists_isLine | [86, 1] | [90, 48] | rcases ne_or_eq a b with h | rfl | V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b : V
⊢ ∃ L, L.IsLine ∧ {a, b} ⊆ L | case inl
V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b : V
h : a ≠ b
⊢ ∃ L, L.IsLine ∧ {a, b} ⊆ L
case inr
V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a : V
⊢ ∃ L, L.IsLine ∧ {a, a} ⊆ L |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | exists_isLine | [86, 1] | [90, 48] | have ⟨b, h⟩ := exists_ne a | case inr
V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a : V
⊢ ∃ L, L.IsLine ∧ {a, a} ⊆ L | case inr
V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b : V
h : b ≠ a
⊢ ∃ L, L.IsLine ∧ {a, a} ⊆ L |
https://github.com/YaelDillies/LeanCamCombi.git | 034199694e3b91536d03bc4a8b0cdbd659cdf50f | LeanCamCombi/SylvesterChvatal.lean | exists_isLine | [86, 1] | [90, 48] | exact ⟨Line a b, Line_isLine h.symm, by simp⟩ | case inr
V : Type u_1
inst✝² : MetricSpace V
u v w : V
inst✝¹ : Finite V
inst✝ : Nontrivial V
x y z a b : V
h : b ≠ a
⊢ ∃ L, L.IsLine ∧ {a, a} ⊆ L | no goals |
Subsets and Splits
No community queries yet
The top public SQL queries from the community will appear here once available.