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/Independence.lean
AffineIndependent.convexIndependent
[11, 1]
[15, 8]
sorry
𝕜 : Type u_1 E : Type u_2 ι : Type u_3 inst✝² : OrderedRing 𝕜 inst✝¹ : AddCommGroup E inst✝ : Module 𝕜 E p : ι → E hp : AffineIndependent 𝕜 p s : Set ι x : ι hx : p x ∈ (convexHull 𝕜) (p '' s) x✝ : x ∉ s ⊢ False
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Mathlib/Data/Finset/PosDiffs.lean
Finset.mem_posDiffs
[55, 1]
[56, 98]
simp_rw [posDiffs, mem_image, mem_filter, mem_product, Prod.exists, and_assoc, exists_and_left]
α : Type u_1 inst✝² : GeneralizedBooleanAlgebra α inst✝¹ : DecidableRel fun x x_1 => x ≤ x_1 inst✝ : DecidableEq α s t : Finset α a : α ⊢ a ∈ s \₊ t ↔ ∃ b ∈ s, ∃ c ∈ t, c ≤ b ∧ b \ c = a
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Mathlib/Data/Finset/PosDiffs.lean
Finset.posDiffs_empty
[58, 1]
[58, 79]
simp [posDiffs]
α : Type u_1 inst✝² : GeneralizedBooleanAlgebra α inst✝¹ : DecidableRel fun x x_1 => x ≤ x_1 inst✝ : DecidableEq α s✝ t : Finset α a : α s : Finset α ⊢ s \₊ ∅ = ∅
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Mathlib/Data/Finset/PosDiffs.lean
Finset.empty_posDiffs
[59, 1]
[59, 79]
simp [posDiffs]
α : Type u_1 inst✝² : GeneralizedBooleanAlgebra α inst✝¹ : DecidableRel fun x x_1 => x ≤ x_1 inst✝ : DecidableEq α s✝ t : Finset α a : α s : Finset α ⊢ ∅ \₊ s = ∅
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Mathlib/Data/Finset/PosDiffs.lean
Finset.posDiffs_subset_diffs
[61, 1]
[63, 57]
simp only [subset_iff, mem_posDiffs, mem_diffs]
α : Type u_1 inst✝² : GeneralizedBooleanAlgebra α inst✝¹ : DecidableRel fun x x_1 => x ≤ x_1 inst✝ : DecidableEq α s t : Finset α a : α ⊢ s \₊ t ⊆ s \\ t
α : Type u_1 inst✝² : GeneralizedBooleanAlgebra α inst✝¹ : DecidableRel fun x x_1 => x ≤ x_1 inst✝ : DecidableEq α s t : Finset α a : α ⊢ ∀ ⦃x : α⦄, (∃ b ∈ s, ∃ c ∈ t, c ≤ b ∧ b \ c = x) → ∃ a ∈ s, ∃ b ∈ t, a \ b = x
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Mathlib/Data/Finset/PosDiffs.lean
Finset.posDiffs_subset_diffs
[61, 1]
[63, 57]
exact fun a ⟨b, hb, c, hc, _, ha⟩ ↦ ⟨b, hb, c, hc, ha⟩
α : Type u_1 inst✝² : GeneralizedBooleanAlgebra α inst✝¹ : DecidableRel fun x x_1 => x ≤ x_1 inst✝ : DecidableEq α s t : Finset α a : α ⊢ ∀ ⦃x : α⦄, (∃ b ∈ s, ∃ c ∈ t, c ≤ b ∧ b \ c = x) → ∃ a ∈ s, ∃ b ∈ t, a \ b = x
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Mathlib/Data/Finset/PosDiffs.lean
Finset.card_posDiffs_self_le
[73, 1]
[81, 10]
revert h𝒜
α : Type u_1 inst✝ : DecidableEq α 𝒜 ℬ : Finset (Finset α) h𝒜 : (↑𝒜).OrdConnected ⊢ (𝒜 \₊ 𝒜).card ≤ 𝒜.card
α : Type u_1 inst✝ : DecidableEq α 𝒜 ℬ : Finset (Finset α) ⊢ (↑𝒜).OrdConnected → (𝒜 \₊ 𝒜).card ≤ 𝒜.card
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Mathlib/Data/Finset/PosDiffs.lean
Finset.card_posDiffs_self_le
[73, 1]
[81, 10]
refine' Finset.memberFamily_induction_on 𝒜 _ _ _
α : Type u_1 inst✝ : DecidableEq α 𝒜 ℬ : Finset (Finset α) ⊢ (↑𝒜).OrdConnected → (𝒜 \₊ 𝒜).card ≤ 𝒜.card
case refine'_1 α : Type u_1 inst✝ : DecidableEq α 𝒜 ℬ : Finset (Finset α) ⊢ (↑∅).OrdConnected → (∅ \₊ ∅).card ≤ ∅.card case refine'_2 α : Type u_1 inst✝ : DecidableEq α 𝒜 ℬ : Finset (Finset α) ⊢ (↑{∅}).OrdConnected → ({∅} \₊ {∅}).card ≤ {∅}.card case refine'_3 α : Type u_1 inst✝ : DecidableEq α 𝒜 ℬ : Finset (Finset α) ⊢ ∀ (a : α) ⦃𝒜 : Finset (Finset α)⦄, ((↑(nonMemberSubfamily a 𝒜)).OrdConnected → (nonMemberSubfamily a 𝒜 \₊ nonMemberSubfamily a 𝒜).card ≤ (nonMemberSubfamily a 𝒜).card) → ((↑(memberSubfamily a 𝒜)).OrdConnected → (memberSubfamily a 𝒜 \₊ memberSubfamily a 𝒜).card ≤ (memberSubfamily a 𝒜).card) → (↑𝒜).OrdConnected → (𝒜 \₊ 𝒜).card ≤ 𝒜.card
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Mathlib/Data/Finset/PosDiffs.lean
Finset.card_posDiffs_self_le
[73, 1]
[81, 10]
simp
case refine'_1 α : Type u_1 inst✝ : DecidableEq α 𝒜 ℬ : Finset (Finset α) ⊢ (↑∅).OrdConnected → (∅ \₊ ∅).card ≤ ∅.card
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Mathlib/Data/Finset/PosDiffs.lean
Finset.card_posDiffs_self_le
[73, 1]
[81, 10]
intro
case refine'_2 α : Type u_1 inst✝ : DecidableEq α 𝒜 ℬ : Finset (Finset α) ⊢ (↑{∅}).OrdConnected → ({∅} \₊ {∅}).card ≤ {∅}.card
case refine'_2 α : Type u_1 inst✝ : DecidableEq α 𝒜 ℬ : Finset (Finset α) h𝒜✝ : (↑{∅}).OrdConnected ⊢ ({∅} \₊ {∅}).card ≤ {∅}.card
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Mathlib/Data/Finset/PosDiffs.lean
Finset.card_posDiffs_self_le
[73, 1]
[81, 10]
rfl
case refine'_2 α : Type u_1 inst✝ : DecidableEq α 𝒜 ℬ : Finset (Finset α) h𝒜✝ : (↑{∅}).OrdConnected ⊢ ({∅} \₊ {∅}).card ≤ {∅}.card
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Mathlib/Data/Finset/PosDiffs.lean
Finset.card_posDiffs_self_le
[73, 1]
[81, 10]
rintro a 𝒜 h𝒜₀ h𝒜₁ h𝒜
case refine'_3 α : Type u_1 inst✝ : DecidableEq α 𝒜 ℬ : Finset (Finset α) ⊢ ∀ (a : α) ⦃𝒜 : Finset (Finset α)⦄, ((↑(nonMemberSubfamily a 𝒜)).OrdConnected → (nonMemberSubfamily a 𝒜 \₊ nonMemberSubfamily a 𝒜).card ≤ (nonMemberSubfamily a 𝒜).card) → ((↑(memberSubfamily a 𝒜)).OrdConnected → (memberSubfamily a 𝒜 \₊ memberSubfamily a 𝒜).card ≤ (memberSubfamily a 𝒜).card) → (↑𝒜).OrdConnected → (𝒜 \₊ 𝒜).card ≤ 𝒜.card
case refine'_3 α : Type u_1 inst✝ : DecidableEq α 𝒜✝ ℬ : Finset (Finset α) a : α 𝒜 : Finset (Finset α) h𝒜₀ : (↑(nonMemberSubfamily a 𝒜)).OrdConnected → (nonMemberSubfamily a 𝒜 \₊ nonMemberSubfamily a 𝒜).card ≤ (nonMemberSubfamily a 𝒜).card h𝒜₁ : (↑(memberSubfamily a 𝒜)).OrdConnected → (memberSubfamily a 𝒜 \₊ memberSubfamily a 𝒜).card ≤ (memberSubfamily a 𝒜).card h𝒜 : (↑𝒜).OrdConnected ⊢ (𝒜 \₊ 𝒜).card ≤ 𝒜.card
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Mathlib/Data/Finset/PosDiffs.lean
Finset.card_posDiffs_self_le
[73, 1]
[81, 10]
sorry
case refine'_3 α : Type u_1 inst✝ : DecidableEq α 𝒜✝ ℬ : Finset (Finset α) a : α 𝒜 : Finset (Finset α) h𝒜₀ : (↑(nonMemberSubfamily a 𝒜)).OrdConnected → (nonMemberSubfamily a 𝒜 \₊ nonMemberSubfamily a 𝒜).card ≤ (nonMemberSubfamily a 𝒜).card h𝒜₁ : (↑(memberSubfamily a 𝒜)).OrdConnected → (memberSubfamily a 𝒜 \₊ memberSubfamily a 𝒜).card ≤ (memberSubfamily a 𝒜).card h𝒜 : (↑𝒜).OrdConnected ⊢ (𝒜 \₊ 𝒜).card ≤ 𝒜.card
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Mathlib/Data/Finset/PosDiffs.lean
Finset.le_card_upper_inter_lower
[83, 1]
[91, 48]
refine' (card_le_card _).trans (card_posDiffs_self_le _)
α : Type u_1 inst✝ : DecidableEq α 𝒜 ℬ : Finset (Finset α) h𝒜 : IsLowerSet ↑𝒜 hℬ : IsUpperSet ↑ℬ ⊢ (𝒜 \₊ ℬ).card ≤ (𝒜 ∩ ℬ).card
case refine'_1 α : Type u_1 inst✝ : DecidableEq α 𝒜 ℬ : Finset (Finset α) h𝒜 : IsLowerSet ↑𝒜 hℬ : IsUpperSet ↑ℬ ⊢ 𝒜 \₊ ℬ ⊆ 𝒜 ∩ ℬ \₊ (𝒜 ∩ ℬ) case refine'_2 α : Type u_1 inst✝ : DecidableEq α 𝒜 ℬ : Finset (Finset α) h𝒜 : IsLowerSet ↑𝒜 hℬ : IsUpperSet ↑ℬ ⊢ (↑(𝒜 ∩ ℬ)).OrdConnected
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Mathlib/Data/Finset/PosDiffs.lean
Finset.le_card_upper_inter_lower
[83, 1]
[91, 48]
simp_rw [subset_iff, mem_posDiffs, mem_inter]
case refine'_1 α : Type u_1 inst✝ : DecidableEq α 𝒜 ℬ : Finset (Finset α) h𝒜 : IsLowerSet ↑𝒜 hℬ : IsUpperSet ↑ℬ ⊢ 𝒜 \₊ ℬ ⊆ 𝒜 ∩ ℬ \₊ (𝒜 ∩ ℬ)
case refine'_1 α : Type u_1 inst✝ : DecidableEq α 𝒜 ℬ : Finset (Finset α) h𝒜 : IsLowerSet ↑𝒜 hℬ : IsUpperSet ↑ℬ ⊢ ∀ ⦃x : Finset α⦄, (∃ b ∈ 𝒜, ∃ c ∈ ℬ, c ≤ b ∧ b \ c = x) → ∃ b, (b ∈ 𝒜 ∧ b ∈ ℬ) ∧ ∃ c, (c ∈ 𝒜 ∧ c ∈ ℬ) ∧ c ≤ b ∧ b \ c = x
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Mathlib/Data/Finset/PosDiffs.lean
Finset.le_card_upper_inter_lower
[83, 1]
[91, 48]
rintro _ ⟨s, hs, t, ht, hts, rfl⟩
case refine'_1 α : Type u_1 inst✝ : DecidableEq α 𝒜 ℬ : Finset (Finset α) h𝒜 : IsLowerSet ↑𝒜 hℬ : IsUpperSet ↑ℬ ⊢ ∀ ⦃x : Finset α⦄, (∃ b ∈ 𝒜, ∃ c ∈ ℬ, c ≤ b ∧ b \ c = x) → ∃ b, (b ∈ 𝒜 ∧ b ∈ ℬ) ∧ ∃ c, (c ∈ 𝒜 ∧ c ∈ ℬ) ∧ c ≤ b ∧ b \ c = x
case refine'_1.intro.intro.intro.intro.intro α : Type u_1 inst✝ : DecidableEq α 𝒜 ℬ : Finset (Finset α) h𝒜 : IsLowerSet ↑𝒜 hℬ : IsUpperSet ↑ℬ s : Finset α hs : s ∈ 𝒜 t : Finset α ht : t ∈ ℬ hts : t ≤ s ⊢ ∃ b, (b ∈ 𝒜 ∧ b ∈ ℬ) ∧ ∃ c, (c ∈ 𝒜 ∧ c ∈ ℬ) ∧ c ≤ b ∧ b \ c = s \ t
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Mathlib/Data/Finset/PosDiffs.lean
Finset.le_card_upper_inter_lower
[83, 1]
[91, 48]
exact ⟨s, ⟨hs, hℬ hts ht⟩, t, ⟨h𝒜 hts hs, ht⟩, hts, rfl⟩
case refine'_1.intro.intro.intro.intro.intro α : Type u_1 inst✝ : DecidableEq α 𝒜 ℬ : Finset (Finset α) h𝒜 : IsLowerSet ↑𝒜 hℬ : IsUpperSet ↑ℬ s : Finset α hs : s ∈ 𝒜 t : Finset α ht : t ∈ ℬ hts : t ≤ s ⊢ ∃ b, (b ∈ 𝒜 ∧ b ∈ ℬ) ∧ ∃ c, (c ∈ 𝒜 ∧ c ∈ ℬ) ∧ c ≤ b ∧ b \ c = s \ t
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Mathlib/Data/Finset/PosDiffs.lean
Finset.le_card_upper_inter_lower
[83, 1]
[91, 48]
rw [coe_inter]
case refine'_2 α : Type u_1 inst✝ : DecidableEq α 𝒜 ℬ : Finset (Finset α) h𝒜 : IsLowerSet ↑𝒜 hℬ : IsUpperSet ↑ℬ ⊢ (↑(𝒜 ∩ ℬ)).OrdConnected
case refine'_2 α : Type u_1 inst✝ : DecidableEq α 𝒜 ℬ : Finset (Finset α) h𝒜 : IsLowerSet ↑𝒜 hℬ : IsUpperSet ↑ℬ ⊢ (↑𝒜 ∩ ↑ℬ).OrdConnected
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Mathlib/Data/Finset/PosDiffs.lean
Finset.le_card_upper_inter_lower
[83, 1]
[91, 48]
exact h𝒜.ordConnected.inter hℬ.ordConnected
case refine'_2 α : Type u_1 inst✝ : DecidableEq α 𝒜 ℬ : Finset (Finset α) h𝒜 : IsLowerSet ↑𝒜 hℬ : IsUpperSet ↑ℬ ⊢ (↑𝒜 ∩ ↑ℬ).OrdConnected
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Mathlib/Data/Finset/PosDiffs.lean
Finset.mem_posSub
[111, 1]
[112, 96]
simp_rw [posSub, mem_image, mem_filter, mem_product, Prod.exists, and_assoc, exists_and_left]
α : Type u_1 inst✝³ : Sub α inst✝² : Preorder α inst✝¹ : DecidableRel fun x x_1 => x ≤ x_1 inst✝ : DecidableEq α s t : Finset α a : α ⊢ a ∈ s -₊ t ↔ ∃ b ∈ s, ∃ c ∈ t, c ≤ b ∧ b - c = a
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Mathlib/Data/Finset/PosDiffs.lean
Finset.posSub_subset_sub
[114, 1]
[115, 79]
rw [mem_posSub, mem_sub]
α : Type u_1 inst✝³ : Sub α inst✝² : Preorder α inst✝¹ : DecidableRel fun x x_1 => x ≤ x_1 inst✝ : DecidableEq α s t : Finset α a x : α ⊢ x ∈ s -₊ t → x ∈ s - t
α : Type u_1 inst✝³ : Sub α inst✝² : Preorder α inst✝¹ : DecidableRel fun x x_1 => x ≤ x_1 inst✝ : DecidableEq α s t : Finset α a x : α ⊢ (∃ b ∈ s, ∃ c ∈ t, c ≤ b ∧ b - c = x) → ∃ b ∈ s, ∃ c ∈ t, b - c = x
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Mathlib/Data/Finset/PosDiffs.lean
Finset.posSub_subset_sub
[114, 1]
[115, 79]
exact fun ⟨b, hb, c, hc, _, h⟩ ↦ ⟨b, hb, c, hc, h⟩
α : Type u_1 inst✝³ : Sub α inst✝² : Preorder α inst✝¹ : DecidableRel fun x x_1 => x ≤ x_1 inst✝ : DecidableEq α s t : Finset α a x : α ⊢ (∃ b ∈ s, ∃ c ∈ t, c ≤ b ∧ b - c = x) → ∃ b ∈ s, ∃ c ∈ t, b - c = x
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Mathlib/Combinatorics/SimpleGraph/Basic.lean
SimpleGraph.deleteEdges_eq_self
[13, 1]
[15, 56]
rw [deleteEdges, sdiff_eq_left, disjoint_fromEdgeSet]
α : Type u_1 β : Type u_2 G H : SimpleGraph α s✝ s : Set (Sym2 α) ⊢ G.deleteEdges s = G ↔ Disjoint G.edgeSet s
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Mathlib/Combinatorics/SimpleGraph/Basic.lean
SimpleGraph.ind_empty
[30, 1]
[30, 74]
ext
α : Type u_1 β : Type u_2 G✝ H : SimpleGraph α s✝ : Set (Sym2 α) s t : Set α a b : α G : SimpleGraph α ⊢ G.ind ∅ = ⊥
case Adj.h.h.a α : Type u_1 β : Type u_2 G✝ H : SimpleGraph α s✝ : Set (Sym2 α) s t : Set α a b : α G : SimpleGraph α x✝¹ x✝ : α ⊢ (G.ind ∅).Adj x✝¹ x✝ ↔ ⊥.Adj x✝¹ x✝
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Mathlib/Combinatorics/SimpleGraph/Basic.lean
SimpleGraph.ind_empty
[30, 1]
[30, 74]
simp
case Adj.h.h.a α : Type u_1 β : Type u_2 G✝ H : SimpleGraph α s✝ : Set (Sym2 α) s t : Set α a b : α G : SimpleGraph α x✝¹ x✝ : α ⊢ (G.ind ∅).Adj x✝¹ x✝ ↔ ⊥.Adj x✝¹ x✝
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Mathlib/Combinatorics/SimpleGraph/Basic.lean
SimpleGraph.ind_univ
[31, 1]
[31, 76]
ext
α : Type u_1 β : Type u_2 G✝ H : SimpleGraph α s✝ : Set (Sym2 α) s t : Set α a b : α G : SimpleGraph α ⊢ G.ind univ = G
case Adj.h.h.a α : Type u_1 β : Type u_2 G✝ H : SimpleGraph α s✝ : Set (Sym2 α) s t : Set α a b : α G : SimpleGraph α x✝¹ x✝ : α ⊢ (G.ind univ).Adj x✝¹ x✝ ↔ G.Adj x✝¹ x✝
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Mathlib/Combinatorics/SimpleGraph/Basic.lean
SimpleGraph.ind_univ
[31, 1]
[31, 76]
simp
case Adj.h.h.a α : Type u_1 β : Type u_2 G✝ H : SimpleGraph α s✝ : Set (Sym2 α) s t : Set α a b : α G : SimpleGraph α x✝¹ x✝ : α ⊢ (G.ind univ).Adj x✝¹ x✝ ↔ G.Adj x✝¹ x✝
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Mathlib/Combinatorics/SimpleGraph/Basic.lean
SimpleGraph.ind_singleton
[33, 1]
[35, 39]
ext
α : Type u_1 β : Type u_2 G✝ H : SimpleGraph α s✝ : Set (Sym2 α) s t : Set α a✝ b : α G : SimpleGraph α a : α ⊢ G.ind {a} = ⊥
case Adj.h.h.a α : Type u_1 β : Type u_2 G✝ H : SimpleGraph α s✝ : Set (Sym2 α) s t : Set α a✝ b : α G : SimpleGraph α a x✝¹ x✝ : α ⊢ (G.ind {a}).Adj x✝¹ x✝ ↔ ⊥.Adj x✝¹ x✝
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Mathlib/Combinatorics/SimpleGraph/Basic.lean
SimpleGraph.ind_singleton
[33, 1]
[35, 39]
simp
case Adj.h.h.a α : Type u_1 β : Type u_2 G✝ H : SimpleGraph α s✝ : Set (Sym2 α) s t : Set α a✝ b : α G : SimpleGraph α a x✝¹ x✝ : α ⊢ (G.ind {a}).Adj x✝¹ x✝ ↔ ⊥.Adj x✝¹ x✝
case Adj.h.h.a α : Type u_1 β : Type u_2 G✝ H : SimpleGraph α s✝ : Set (Sym2 α) s t : Set α a✝ b : α G : SimpleGraph α a x✝¹ x✝ : α ⊢ G.Adj x✝¹ x✝ → x✝¹ = a → ¬x✝ = a
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Mathlib/Combinatorics/SimpleGraph/Basic.lean
SimpleGraph.ind_singleton
[33, 1]
[35, 39]
rintro h rfl
case Adj.h.h.a α : Type u_1 β : Type u_2 G✝ H : SimpleGraph α s✝ : Set (Sym2 α) s t : Set α a✝ b : α G : SimpleGraph α a x✝¹ x✝ : α ⊢ G.Adj x✝¹ x✝ → x✝¹ = a → ¬x✝ = a
case Adj.h.h.a α : Type u_1 β : Type u_2 G✝ H : SimpleGraph α s✝ : Set (Sym2 α) s t : Set α a b : α G : SimpleGraph α x✝¹ x✝ : α h : G.Adj x✝¹ x✝ ⊢ ¬x✝ = x✝¹
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Mathlib/Combinatorics/SimpleGraph/Basic.lean
SimpleGraph.ind_singleton
[33, 1]
[35, 39]
exact h.ne'
case Adj.h.h.a α : Type u_1 β : Type u_2 G✝ H : SimpleGraph α s✝ : Set (Sym2 α) s t : Set α a b : α G : SimpleGraph α x✝¹ x✝ : α h : G.Adj x✝¹ x✝ ⊢ ¬x✝ = x✝¹
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Mathlib/Combinatorics/SimpleGraph/Basic.lean
SimpleGraph.ind_inter
[37, 1]
[39, 19]
ext
α : Type u_1 β : Type u_2 G✝ H : SimpleGraph α s✝¹ : Set (Sym2 α) s✝ t✝ : Set α a b : α G : SimpleGraph α s t : Set α ⊢ G.ind (s ∩ t) = G.ind s ⊓ G.ind t
case Adj.h.h.a α : Type u_1 β : Type u_2 G✝ H : SimpleGraph α s✝¹ : Set (Sym2 α) s✝ t✝ : Set α a b : α G : SimpleGraph α s t : Set α x✝¹ x✝ : α ⊢ (G.ind (s ∩ t)).Adj x✝¹ x✝ ↔ (G.ind s ⊓ G.ind t).Adj x✝¹ x✝
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Mathlib/Combinatorics/SimpleGraph/Basic.lean
SimpleGraph.ind_inter
[37, 1]
[39, 19]
simp
case Adj.h.h.a α : Type u_1 β : Type u_2 G✝ H : SimpleGraph α s✝¹ : Set (Sym2 α) s✝ t✝ : Set α a b : α G : SimpleGraph α s t : Set α x✝¹ x✝ : α ⊢ (G.ind (s ∩ t)).Adj x✝¹ x✝ ↔ (G.ind s ⊓ G.ind t).Adj x✝¹ x✝
case Adj.h.h.a α : Type u_1 β : Type u_2 G✝ H : SimpleGraph α s✝¹ : Set (Sym2 α) s✝ t✝ : Set α a b : α G : SimpleGraph α s t : Set α x✝¹ x✝ : α ⊢ G.Adj x✝¹ x✝ ∧ (x✝¹ ∈ s ∧ x✝¹ ∈ t) ∧ x✝ ∈ s ∧ x✝ ∈ t ↔ (G.Adj x✝¹ x✝ ∧ x✝¹ ∈ s ∧ x✝ ∈ s) ∧ G.Adj x✝¹ x✝ ∧ x✝¹ ∈ t ∧ x✝ ∈ t
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Mathlib/Combinatorics/SimpleGraph/Basic.lean
SimpleGraph.ind_inter
[37, 1]
[39, 19]
tauto
case Adj.h.h.a α : Type u_1 β : Type u_2 G✝ H : SimpleGraph α s✝¹ : Set (Sym2 α) s✝ t✝ : Set α a b : α G : SimpleGraph α s t : Set α x✝¹ x✝ : α ⊢ G.Adj x✝¹ x✝ ∧ (x✝¹ ∈ s ∧ x✝¹ ∈ t) ∧ x✝ ∈ s ∧ x✝ ∈ t ↔ (G.Adj x✝¹ x✝ ∧ x✝¹ ∈ s ∧ x✝ ∈ s) ∧ G.Adj x✝¹ x✝ ∧ x✝¹ ∈ t ∧ x✝ ∈ t
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/Mathlib/Combinatorics/SimpleGraph/Basic.lean
SimpleGraph.disjoint_ind
[41, 1]
[43, 77]
rw [disjoint_iff, ← ind_inter, disjoint_iff_inter_eq_empty.1 h, ind_empty]
α : Type u_1 β : Type u_2 G H : SimpleGraph α s✝ : Set (Sym2 α) s t : Set α a b : α h : Disjoint s t ⊢ Disjoint (G.ind s) (G.ind t)
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/KruskalKatona.lean
Finset.Colex.shadow_initSeg
[83, 1]
[131, 20]
ext t
α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t : Finset α r : ℕ inst✝ : Fintype α hs : s.Nonempty ⊢ ∂ (initSeg s) = initSeg (s.erase (s.min' hs))
case a α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t✝ : Finset α r : ℕ inst✝ : Fintype α hs : s.Nonempty t : Finset α ⊢ t ∈ ∂ (initSeg s) ↔ t ∈ initSeg (s.erase (s.min' hs))
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/KruskalKatona.lean
Finset.Colex.shadow_initSeg
[83, 1]
[131, 20]
simp only [mem_shadow_iff_insert_mem, mem_initSeg, exists_prop]
case a α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t✝ : Finset α r : ℕ inst✝ : Fintype α hs : s.Nonempty t : Finset α ⊢ t ∈ ∂ (initSeg s) ↔ t ∈ initSeg (s.erase (s.min' hs))
case a α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t✝ : Finset α r : ℕ inst✝ : Fintype α hs : s.Nonempty t : Finset α ⊢ (∃ a ∉ t, s.card = (insert a t).card ∧ { ofColex := insert a t } ≤ { ofColex := s }) ↔ (s.erase (s.min' hs)).card = t.card ∧ { ofColex := t } ≤ { ofColex := s.erase (s.min' hs) }
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/KruskalKatona.lean
Finset.Colex.shadow_initSeg
[83, 1]
[131, 20]
constructor
case a α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t✝ : Finset α r : ℕ inst✝ : Fintype α hs : s.Nonempty t : Finset α ⊢ (∃ a ∉ t, s.card = (insert a t).card ∧ { ofColex := insert a t } ≤ { ofColex := s }) ↔ (s.erase (s.min' hs)).card = t.card ∧ { ofColex := t } ≤ { ofColex := s.erase (s.min' hs) }
case a.mp α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t✝ : Finset α r : ℕ inst✝ : Fintype α hs : s.Nonempty t : Finset α ⊢ (∃ a ∉ t, s.card = (insert a t).card ∧ { ofColex := insert a t } ≤ { ofColex := s }) → (s.erase (s.min' hs)).card = t.card ∧ { ofColex := t } ≤ { ofColex := s.erase (s.min' hs) } case a.mpr α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t✝ : Finset α r : ℕ inst✝ : Fintype α hs : s.Nonempty t : Finset α ⊢ (s.erase (s.min' hs)).card = t.card ∧ { ofColex := t } ≤ { ofColex := s.erase (s.min' hs) } → ∃ a ∉ t, s.card = (insert a t).card ∧ { ofColex := insert a t } ≤ { ofColex := s }
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/KruskalKatona.lean
Finset.Colex.shadow_initSeg
[83, 1]
[131, 20]
simp_rw [le_iff_eq_or_lt, lt_iff_exists_forall_lt_mem_iff_mem]
case a.mpr α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t✝ : Finset α r : ℕ inst✝ : Fintype α hs : s.Nonempty t : Finset α ⊢ (s.erase (s.min' hs)).card = t.card ∧ { ofColex := t } ≤ { ofColex := s.erase (s.min' hs) } → ∃ a ∉ t, s.card = (insert a t).card ∧ { ofColex := insert a t } ≤ { ofColex := s }
case a.mpr α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t✝ : Finset α r : ℕ inst✝ : Fintype α hs : s.Nonempty t : Finset α ⊢ (s.erase (s.min' hs)).card = t.card ∧ ({ ofColex := t } = { ofColex := s.erase (s.min' hs) } ∨ ∃ w ∈ s.erase (s.min' hs), w ∉ t ∧ ∀ ⦃a : α⦄, w < a → (a ∈ t ↔ a ∈ s.erase (s.min' hs))) → ∃ a ∉ t, s.card = (insert a t).card ∧ ({ ofColex := insert a t } = { ofColex := s } ∨ ∃ w ∈ s, w ∉ insert a t ∧ ∀ ⦃a_1 : α⦄, w < a_1 → (a_1 ∈ insert a t ↔ a_1 ∈ s))
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/KruskalKatona.lean
Finset.Colex.shadow_initSeg
[83, 1]
[131, 20]
simp only [toColex_inj, ofColex_toColex, ne_eq, and_imp]
case a.mpr α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t✝ : Finset α r : ℕ inst✝ : Fintype α hs : s.Nonempty t : Finset α ⊢ (s.erase (s.min' hs)).card = t.card ∧ ({ ofColex := t } = { ofColex := s.erase (s.min' hs) } ∨ ∃ w ∈ s.erase (s.min' hs), w ∉ t ∧ ∀ ⦃a : α⦄, w < a → (a ∈ t ↔ a ∈ s.erase (s.min' hs))) → ∃ a ∉ t, s.card = (insert a t).card ∧ ({ ofColex := insert a t } = { ofColex := s } ∨ ∃ w ∈ s, w ∉ insert a t ∧ ∀ ⦃a_1 : α⦄, w < a_1 → (a_1 ∈ insert a t ↔ a_1 ∈ s))
case a.mpr α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t✝ : Finset α r : ℕ inst✝ : Fintype α hs : s.Nonempty t : Finset α ⊢ (s.erase (s.min' hs)).card = t.card → (t = s.erase (s.min' hs) ∨ ∃ w ∈ s.erase (s.min' hs), w ∉ t ∧ ∀ ⦃a : α⦄, w < a → (a ∈ t ↔ a ∈ s.erase (s.min' hs))) → ∃ a ∉ t, s.card = (insert a t).card ∧ (insert a t = s ∨ ∃ w ∈ s, w ∉ insert a t ∧ ∀ ⦃a_1 : α⦄, w < a_1 → (a_1 ∈ insert a t ↔ a_1 ∈ s))
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/KruskalKatona.lean
Finset.Colex.shadow_initSeg
[83, 1]
[131, 20]
rintro cards' (rfl | ⟨k, hks, hkt, z⟩)
case a.mpr α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t✝ : Finset α r : ℕ inst✝ : Fintype α hs : s.Nonempty t : Finset α ⊢ (s.erase (s.min' hs)).card = t.card → (t = s.erase (s.min' hs) ∨ ∃ w ∈ s.erase (s.min' hs), w ∉ t ∧ ∀ ⦃a : α⦄, w < a → (a ∈ t ↔ a ∈ s.erase (s.min' hs))) → ∃ a ∉ t, s.card = (insert a t).card ∧ (insert a t = s ∨ ∃ w ∈ s, w ∉ insert a t ∧ ∀ ⦃a_1 : α⦄, w < a_1 → (a_1 ∈ insert a t ↔ a_1 ∈ s))
case a.mpr.inl α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t : Finset α r : ℕ inst✝ : Fintype α hs : s.Nonempty cards' : (s.erase (s.min' hs)).card = (s.erase (s.min' hs)).card ⊢ ∃ a ∉ s.erase (s.min' hs), s.card = (insert a (s.erase (s.min' hs))).card ∧ (insert a (s.erase (s.min' hs)) = s ∨ ∃ w ∈ s, w ∉ insert a (s.erase (s.min' hs)) ∧ ∀ ⦃a_1 : α⦄, w < a_1 → (a_1 ∈ insert a (s.erase (s.min' hs)) ↔ a_1 ∈ s)) case a.mpr.inr.intro.intro.intro α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t✝ : Finset α r : ℕ inst✝ : Fintype α hs : s.Nonempty t : Finset α cards' : (s.erase (s.min' hs)).card = t.card k : α hks : k ∈ s.erase (s.min' hs) hkt : k ∉ t z : ∀ ⦃a : α⦄, k < a → (a ∈ t ↔ a ∈ s.erase (s.min' hs)) ⊢ ∃ a ∉ t, s.card = (insert a t).card ∧ (insert a t = s ∨ ∃ w ∈ s, w ∉ insert a t ∧ ∀ ⦃a_1 : α⦄, w < a_1 → (a_1 ∈ insert a t ↔ a_1 ∈ s))
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/KruskalKatona.lean
Finset.Colex.shadow_initSeg
[83, 1]
[131, 20]
set j := min' tᶜ ⟨k, mem_compl.2 hkt⟩
case a.mpr.inr.intro.intro.intro α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t✝ : Finset α r : ℕ inst✝ : Fintype α hs : s.Nonempty t : Finset α cards' : (s.erase (s.min' hs)).card = t.card k : α hks : k ∈ s.erase (s.min' hs) hkt : k ∉ t z : ∀ ⦃a : α⦄, k < a → (a ∈ t ↔ a ∈ s.erase (s.min' hs)) ⊢ ∃ a ∉ t, s.card = (insert a t).card ∧ (insert a t = s ∨ ∃ w ∈ s, w ∉ insert a t ∧ ∀ ⦃a_1 : α⦄, w < a_1 → (a_1 ∈ insert a t ↔ a_1 ∈ s))
case a.mpr.inr.intro.intro.intro α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t✝ : Finset α r : ℕ inst✝ : Fintype α hs : s.Nonempty t : Finset α cards' : (s.erase (s.min' hs)).card = t.card k : α hks : k ∈ s.erase (s.min' hs) hkt : k ∉ t z : ∀ ⦃a : α⦄, k < a → (a ∈ t ↔ a ∈ s.erase (s.min' hs)) j : α := tᶜ.min' ⋯ ⊢ ∃ a ∉ t, s.card = (insert a t).card ∧ (insert a t = s ∨ ∃ w ∈ s, w ∉ insert a t ∧ ∀ ⦃a_1 : α⦄, w < a_1 → (a_1 ∈ insert a t ↔ a_1 ∈ s))
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/KruskalKatona.lean
Finset.Colex.shadow_initSeg
[83, 1]
[131, 20]
have hjk : j ≤ k := min'_le _ _ (mem_compl.2 ‹k ∉ t›)
case a.mpr.inr.intro.intro.intro α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t✝ : Finset α r : ℕ inst✝ : Fintype α hs : s.Nonempty t : Finset α cards' : (s.erase (s.min' hs)).card = t.card k : α hks : k ∈ s.erase (s.min' hs) hkt : k ∉ t z : ∀ ⦃a : α⦄, k < a → (a ∈ t ↔ a ∈ s.erase (s.min' hs)) j : α := tᶜ.min' ⋯ ⊢ ∃ a ∉ t, s.card = (insert a t).card ∧ (insert a t = s ∨ ∃ w ∈ s, w ∉ insert a t ∧ ∀ ⦃a_1 : α⦄, w < a_1 → (a_1 ∈ insert a t ↔ a_1 ∈ s))
case a.mpr.inr.intro.intro.intro α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t✝ : Finset α r : ℕ inst✝ : Fintype α hs : s.Nonempty t : Finset α cards' : (s.erase (s.min' hs)).card = t.card k : α hks : k ∈ s.erase (s.min' hs) hkt : k ∉ t z : ∀ ⦃a : α⦄, k < a → (a ∈ t ↔ a ∈ s.erase (s.min' hs)) j : α := tᶜ.min' ⋯ hjk : j ≤ k ⊢ ∃ a ∉ t, s.card = (insert a t).card ∧ (insert a t = s ∨ ∃ w ∈ s, w ∉ insert a t ∧ ∀ ⦃a_1 : α⦄, w < a_1 → (a_1 ∈ insert a t ↔ a_1 ∈ s))
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/KruskalKatona.lean
Finset.Colex.shadow_initSeg
[83, 1]
[131, 20]
have : j ∉ t := mem_compl.1 (min'_mem _ _)
case a.mpr.inr.intro.intro.intro α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t✝ : Finset α r : ℕ inst✝ : Fintype α hs : s.Nonempty t : Finset α cards' : (s.erase (s.min' hs)).card = t.card k : α hks : k ∈ s.erase (s.min' hs) hkt : k ∉ t z : ∀ ⦃a : α⦄, k < a → (a ∈ t ↔ a ∈ s.erase (s.min' hs)) j : α := tᶜ.min' ⋯ hjk : j ≤ k ⊢ ∃ a ∉ t, s.card = (insert a t).card ∧ (insert a t = s ∨ ∃ w ∈ s, w ∉ insert a t ∧ ∀ ⦃a_1 : α⦄, w < a_1 → (a_1 ∈ insert a t ↔ a_1 ∈ s))
case a.mpr.inr.intro.intro.intro α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t✝ : Finset α r : ℕ inst✝ : Fintype α hs : s.Nonempty t : Finset α cards' : (s.erase (s.min' hs)).card = t.card k : α hks : k ∈ s.erase (s.min' hs) hkt : k ∉ t z : ∀ ⦃a : α⦄, k < a → (a ∈ t ↔ a ∈ s.erase (s.min' hs)) j : α := tᶜ.min' ⋯ hjk : j ≤ k this : j ∉ t ⊢ ∃ a ∉ t, s.card = (insert a t).card ∧ (insert a t = s ∨ ∃ w ∈ s, w ∉ insert a t ∧ ∀ ⦃a_1 : α⦄, w < a_1 → (a_1 ∈ insert a t ↔ a_1 ∈ s))
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/KruskalKatona.lean
Finset.Colex.shadow_initSeg
[83, 1]
[131, 20]
have hcard : card s = card (insert j t) := by rw [card_insert_of_not_mem ‹j ∉ t›, ← ‹_ = card t›, card_erase_add_one (min'_mem _ _)]
case a.mpr.inr.intro.intro.intro α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t✝ : Finset α r : ℕ inst✝ : Fintype α hs : s.Nonempty t : Finset α cards' : (s.erase (s.min' hs)).card = t.card k : α hks : k ∈ s.erase (s.min' hs) hkt : k ∉ t z : ∀ ⦃a : α⦄, k < a → (a ∈ t ↔ a ∈ s.erase (s.min' hs)) j : α := tᶜ.min' ⋯ hjk : j ≤ k this : j ∉ t ⊢ ∃ a ∉ t, s.card = (insert a t).card ∧ (insert a t = s ∨ ∃ w ∈ s, w ∉ insert a t ∧ ∀ ⦃a_1 : α⦄, w < a_1 → (a_1 ∈ insert a t ↔ a_1 ∈ s))
case a.mpr.inr.intro.intro.intro α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t✝ : Finset α r : ℕ inst✝ : Fintype α hs : s.Nonempty t : Finset α cards' : (s.erase (s.min' hs)).card = t.card k : α hks : k ∈ s.erase (s.min' hs) hkt : k ∉ t z : ∀ ⦃a : α⦄, k < a → (a ∈ t ↔ a ∈ s.erase (s.min' hs)) j : α := tᶜ.min' ⋯ hjk : j ≤ k this : j ∉ t hcard : s.card = (insert j t).card ⊢ ∃ a ∉ t, s.card = (insert a t).card ∧ (insert a t = s ∨ ∃ w ∈ s, w ∉ insert a t ∧ ∀ ⦃a_1 : α⦄, w < a_1 → (a_1 ∈ insert a t ↔ a_1 ∈ s))
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/KruskalKatona.lean
Finset.Colex.shadow_initSeg
[83, 1]
[131, 20]
refine' ⟨j, ‹_›, hcard, _⟩
case a.mpr.inr.intro.intro.intro α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t✝ : Finset α r : ℕ inst✝ : Fintype α hs : s.Nonempty t : Finset α cards' : (s.erase (s.min' hs)).card = t.card k : α hks : k ∈ s.erase (s.min' hs) hkt : k ∉ t z : ∀ ⦃a : α⦄, k < a → (a ∈ t ↔ a ∈ s.erase (s.min' hs)) j : α := tᶜ.min' ⋯ hjk : j ≤ k this : j ∉ t hcard : s.card = (insert j t).card ⊢ ∃ a ∉ t, s.card = (insert a t).card ∧ (insert a t = s ∨ ∃ w ∈ s, w ∉ insert a t ∧ ∀ ⦃a_1 : α⦄, w < a_1 → (a_1 ∈ insert a t ↔ a_1 ∈ s))
case a.mpr.inr.intro.intro.intro α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t✝ : Finset α r : ℕ inst✝ : Fintype α hs : s.Nonempty t : Finset α cards' : (s.erase (s.min' hs)).card = t.card k : α hks : k ∈ s.erase (s.min' hs) hkt : k ∉ t z : ∀ ⦃a : α⦄, k < a → (a ∈ t ↔ a ∈ s.erase (s.min' hs)) j : α := tᶜ.min' ⋯ hjk : j ≤ k this : j ∉ t hcard : s.card = (insert j t).card ⊢ insert j t = s ∨ ∃ w ∈ s, w ∉ insert j t ∧ ∀ ⦃a : α⦄, w < a → (a ∈ insert j t ↔ a ∈ s)
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/KruskalKatona.lean
Finset.Colex.shadow_initSeg
[83, 1]
[131, 20]
obtain hjk | r₁ := hjk.lt_or_eq
case a.mpr.inr.intro.intro.intro α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t✝ : Finset α r : ℕ inst✝ : Fintype α hs : s.Nonempty t : Finset α cards' : (s.erase (s.min' hs)).card = t.card k : α hks : k ∈ s.erase (s.min' hs) hkt : k ∉ t z : ∀ ⦃a : α⦄, k < a → (a ∈ t ↔ a ∈ s.erase (s.min' hs)) j : α := tᶜ.min' ⋯ hjk : j ≤ k this : j ∉ t hcard : s.card = (insert j t).card ⊢ insert j t = s ∨ ∃ w ∈ s, w ∉ insert j t ∧ ∀ ⦃a : α⦄, w < a → (a ∈ insert j t ↔ a ∈ s)
case a.mpr.inr.intro.intro.intro.inl α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t✝ : Finset α r : ℕ inst✝ : Fintype α hs : s.Nonempty t : Finset α cards' : (s.erase (s.min' hs)).card = t.card k : α hks : k ∈ s.erase (s.min' hs) hkt : k ∉ t z : ∀ ⦃a : α⦄, k < a → (a ∈ t ↔ a ∈ s.erase (s.min' hs)) j : α := tᶜ.min' ⋯ hjk✝ : j ≤ k this : j ∉ t hcard : s.card = (insert j t).card hjk : j < k ⊢ insert j t = s ∨ ∃ w ∈ s, w ∉ insert j t ∧ ∀ ⦃a : α⦄, w < a → (a ∈ insert j t ↔ a ∈ s) case a.mpr.inr.intro.intro.intro.inr α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t✝ : Finset α r : ℕ inst✝ : Fintype α hs : s.Nonempty t : Finset α cards' : (s.erase (s.min' hs)).card = t.card k : α hks : k ∈ s.erase (s.min' hs) hkt : k ∉ t z : ∀ ⦃a : α⦄, k < a → (a ∈ t ↔ a ∈ s.erase (s.min' hs)) j : α := tᶜ.min' ⋯ hjk : j ≤ k this : j ∉ t hcard : s.card = (insert j t).card r₁ : j = k ⊢ insert j t = s ∨ ∃ w ∈ s, w ∉ insert j t ∧ ∀ ⦃a : α⦄, w < a → (a ∈ insert j t ↔ a ∈ s)
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/KruskalKatona.lean
Finset.Colex.shadow_initSeg
[83, 1]
[131, 20]
refine' Or.inl (eq_of_subset_of_card_le (fun a ha ↦ _) hcard.ge).symm
case a.mpr.inr.intro.intro.intro.inr α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t✝ : Finset α r : ℕ inst✝ : Fintype α hs : s.Nonempty t : Finset α cards' : (s.erase (s.min' hs)).card = t.card k : α hks : k ∈ s.erase (s.min' hs) hkt : k ∉ t z : ∀ ⦃a : α⦄, k < a → (a ∈ t ↔ a ∈ s.erase (s.min' hs)) j : α := tᶜ.min' ⋯ hjk : j ≤ k this : j ∉ t hcard : s.card = (insert j t).card r₁ : j = k ⊢ insert j t = s ∨ ∃ w ∈ s, w ∉ insert j t ∧ ∀ ⦃a : α⦄, w < a → (a ∈ insert j t ↔ a ∈ s)
case a.mpr.inr.intro.intro.intro.inr α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t✝ : Finset α r : ℕ inst✝ : Fintype α hs : s.Nonempty t : Finset α cards' : (s.erase (s.min' hs)).card = t.card k : α hks : k ∈ s.erase (s.min' hs) hkt : k ∉ t z : ∀ ⦃a : α⦄, k < a → (a ∈ t ↔ a ∈ s.erase (s.min' hs)) j : α := tᶜ.min' ⋯ hjk : j ≤ k this : j ∉ t hcard : s.card = (insert j t).card r₁ : j = k a : α ha : a ∈ s ⊢ a ∈ insert j t
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/KruskalKatona.lean
Finset.Colex.shadow_initSeg
[83, 1]
[131, 20]
rcases lt_trichotomy k a with (lt | rfl | gt)
case a.mpr.inr.intro.intro.intro.inr α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t✝ : Finset α r : ℕ inst✝ : Fintype α hs : s.Nonempty t : Finset α cards' : (s.erase (s.min' hs)).card = t.card k : α hks : k ∈ s.erase (s.min' hs) hkt : k ∉ t z : ∀ ⦃a : α⦄, k < a → (a ∈ t ↔ a ∈ s.erase (s.min' hs)) j : α := tᶜ.min' ⋯ hjk : j ≤ k this : j ∉ t hcard : s.card = (insert j t).card r₁ : j = k a : α ha : a ∈ s ⊢ a ∈ insert j t
case a.mpr.inr.intro.intro.intro.inr.inl α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t✝ : Finset α r : ℕ inst✝ : Fintype α hs : s.Nonempty t : Finset α cards' : (s.erase (s.min' hs)).card = t.card k : α hks : k ∈ s.erase (s.min' hs) hkt : k ∉ t z : ∀ ⦃a : α⦄, k < a → (a ∈ t ↔ a ∈ s.erase (s.min' hs)) j : α := tᶜ.min' ⋯ hjk : j ≤ k this : j ∉ t hcard : s.card = (insert j t).card r₁ : j = k a : α ha : a ∈ s lt : k < a ⊢ a ∈ insert j t case a.mpr.inr.intro.intro.intro.inr.inr.inl α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t✝ : Finset α r : ℕ inst✝ : Fintype α hs : s.Nonempty t : Finset α cards' : (s.erase (s.min' hs)).card = t.card k : α hks : k ∈ s.erase (s.min' hs) hkt : k ∉ t z : ∀ ⦃a : α⦄, k < a → (a ∈ t ↔ a ∈ s.erase (s.min' hs)) j : α := tᶜ.min' ⋯ hjk : j ≤ k this : j ∉ t hcard : s.card = (insert j t).card r₁ : j = k ha : k ∈ s ⊢ k ∈ insert j t case a.mpr.inr.intro.intro.intro.inr.inr.inr α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t✝ : Finset α r : ℕ inst✝ : Fintype α hs : s.Nonempty t : Finset α cards' : (s.erase (s.min' hs)).card = t.card k : α hks : k ∈ s.erase (s.min' hs) hkt : k ∉ t z : ∀ ⦃a : α⦄, k < a → (a ∈ t ↔ a ∈ s.erase (s.min' hs)) j : α := tᶜ.min' ⋯ hjk : j ≤ k this : j ∉ t hcard : s.card = (insert j t).card r₁ : j = k a : α ha : a ∈ s gt : a < k ⊢ a ∈ insert j t
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/KruskalKatona.lean
Finset.Colex.shadow_initSeg
[83, 1]
[131, 20]
rintro ⟨a, ha, hst, hts⟩
case a.mp α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t✝ : Finset α r : ℕ inst✝ : Fintype α hs : s.Nonempty t : Finset α ⊢ (∃ a ∉ t, s.card = (insert a t).card ∧ { ofColex := insert a t } ≤ { ofColex := s }) → (s.erase (s.min' hs)).card = t.card ∧ { ofColex := t } ≤ { ofColex := s.erase (s.min' hs) }
case a.mp.intro.intro.intro α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t✝ : Finset α r : ℕ inst✝ : Fintype α hs : s.Nonempty t : Finset α a : α ha : a ∉ t hst : s.card = (insert a t).card hts : { ofColex := insert a t } ≤ { ofColex := s } ⊢ (s.erase (s.min' hs)).card = t.card ∧ { ofColex := t } ≤ { ofColex := s.erase (s.min' hs) }
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/KruskalKatona.lean
Finset.Colex.shadow_initSeg
[83, 1]
[131, 20]
constructor
case a.mp.intro.intro.intro α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t✝ : Finset α r : ℕ inst✝ : Fintype α hs : s.Nonempty t : Finset α a : α ha : a ∉ t hst : s.card = (insert a t).card hts : { ofColex := insert a t } ≤ { ofColex := s } ⊢ (s.erase (s.min' hs)).card = t.card ∧ { ofColex := t } ≤ { ofColex := s.erase (s.min' hs) }
case a.mp.intro.intro.intro.left α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t✝ : Finset α r : ℕ inst✝ : Fintype α hs : s.Nonempty t : Finset α a : α ha : a ∉ t hst : s.card = (insert a t).card hts : { ofColex := insert a t } ≤ { ofColex := s } ⊢ (s.erase (s.min' hs)).card = t.card case a.mp.intro.intro.intro.right α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t✝ : Finset α r : ℕ inst✝ : Fintype α hs : s.Nonempty t : Finset α a : α ha : a ∉ t hst : s.card = (insert a t).card hts : { ofColex := insert a t } ≤ { ofColex := s } ⊢ { ofColex := t } ≤ { ofColex := s.erase (s.min' hs) }
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/KruskalKatona.lean
Finset.Colex.shadow_initSeg
[83, 1]
[131, 20]
rw [card_erase_of_mem (min'_mem _ _), hst, card_insert_of_not_mem ha, add_tsub_cancel_right]
case a.mp.intro.intro.intro.left α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t✝ : Finset α r : ℕ inst✝ : Fintype α hs : s.Nonempty t : Finset α a : α ha : a ∉ t hst : s.card = (insert a t).card hts : { ofColex := insert a t } ≤ { ofColex := s } ⊢ (s.erase (s.min' hs)).card = t.card
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/KruskalKatona.lean
Finset.Colex.shadow_initSeg
[83, 1]
[131, 20]
simpa [ha] using erase_le_erase_min' hts hst.ge (mem_insert_self _ _)
case a.mp.intro.intro.intro.right α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t✝ : Finset α r : ℕ inst✝ : Fintype α hs : s.Nonempty t : Finset α a : α ha : a ∉ t hst : s.card = (insert a t).card hts : { ofColex := insert a t } ≤ { ofColex := s } ⊢ { ofColex := t } ≤ { ofColex := s.erase (s.min' hs) }
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/KruskalKatona.lean
Finset.Colex.shadow_initSeg
[83, 1]
[131, 20]
refine' ⟨min' s hs, not_mem_erase _ _, _⟩
case a.mpr.inl α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t : Finset α r : ℕ inst✝ : Fintype α hs : s.Nonempty cards' : (s.erase (s.min' hs)).card = (s.erase (s.min' hs)).card ⊢ ∃ a ∉ s.erase (s.min' hs), s.card = (insert a (s.erase (s.min' hs))).card ∧ (insert a (s.erase (s.min' hs)) = s ∨ ∃ w ∈ s, w ∉ insert a (s.erase (s.min' hs)) ∧ ∀ ⦃a_1 : α⦄, w < a_1 → (a_1 ∈ insert a (s.erase (s.min' hs)) ↔ a_1 ∈ s))
case a.mpr.inl α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t : Finset α r : ℕ inst✝ : Fintype α hs : s.Nonempty cards' : (s.erase (s.min' hs)).card = (s.erase (s.min' hs)).card ⊢ s.card = (insert (s.min' hs) (s.erase (s.min' hs))).card ∧ (insert (s.min' hs) (s.erase (s.min' hs)) = s ∨ ∃ w ∈ s, w ∉ insert (s.min' hs) (s.erase (s.min' hs)) ∧ ∀ ⦃a : α⦄, w < a → (a ∈ insert (s.min' hs) (s.erase (s.min' hs)) ↔ a ∈ s))
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/KruskalKatona.lean
Finset.Colex.shadow_initSeg
[83, 1]
[131, 20]
rw [insert_erase (min'_mem _ _)]
case a.mpr.inl α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t : Finset α r : ℕ inst✝ : Fintype α hs : s.Nonempty cards' : (s.erase (s.min' hs)).card = (s.erase (s.min' hs)).card ⊢ s.card = (insert (s.min' hs) (s.erase (s.min' hs))).card ∧ (insert (s.min' hs) (s.erase (s.min' hs)) = s ∨ ∃ w ∈ s, w ∉ insert (s.min' hs) (s.erase (s.min' hs)) ∧ ∀ ⦃a : α⦄, w < a → (a ∈ insert (s.min' hs) (s.erase (s.min' hs)) ↔ a ∈ s))
case a.mpr.inl α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t : Finset α r : ℕ inst✝ : Fintype α hs : s.Nonempty cards' : (s.erase (s.min' hs)).card = (s.erase (s.min' hs)).card ⊢ s.card = s.card ∧ (s = s ∨ ∃ w ∈ s, w ∉ s ∧ ∀ ⦃a : α⦄, w < a → (a ∈ s ↔ a ∈ s))
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/KruskalKatona.lean
Finset.Colex.shadow_initSeg
[83, 1]
[131, 20]
exact ⟨rfl, Or.inl rfl⟩
case a.mpr.inl α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t : Finset α r : ℕ inst✝ : Fintype α hs : s.Nonempty cards' : (s.erase (s.min' hs)).card = (s.erase (s.min' hs)).card ⊢ s.card = s.card ∧ (s = s ∨ ∃ w ∈ s, w ∉ s ∧ ∀ ⦃a : α⦄, w < a → (a ∈ s ↔ a ∈ s))
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/KruskalKatona.lean
Finset.Colex.shadow_initSeg
[83, 1]
[131, 20]
rw [card_insert_of_not_mem ‹j ∉ t›, ← ‹_ = card t›, card_erase_add_one (min'_mem _ _)]
α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t✝ : Finset α r : ℕ inst✝ : Fintype α hs : s.Nonempty t : Finset α cards' : (s.erase (s.min' hs)).card = t.card k : α hks : k ∈ s.erase (s.min' hs) hkt : k ∉ t z : ∀ ⦃a : α⦄, k < a → (a ∈ t ↔ a ∈ s.erase (s.min' hs)) j : α := tᶜ.min' ⋯ hjk : j ≤ k this : j ∉ t ⊢ s.card = (insert j t).card
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/KruskalKatona.lean
Finset.Colex.shadow_initSeg
[83, 1]
[131, 20]
refine Or.inr ⟨k, mem_of_mem_erase ‹_›, fun hk ↦ hkt $ mem_of_mem_insert_of_ne hk hjk.ne', fun x hx ↦ ?_⟩
case a.mpr.inr.intro.intro.intro.inl α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t✝ : Finset α r : ℕ inst✝ : Fintype α hs : s.Nonempty t : Finset α cards' : (s.erase (s.min' hs)).card = t.card k : α hks : k ∈ s.erase (s.min' hs) hkt : k ∉ t z : ∀ ⦃a : α⦄, k < a → (a ∈ t ↔ a ∈ s.erase (s.min' hs)) j : α := tᶜ.min' ⋯ hjk✝ : j ≤ k this : j ∉ t hcard : s.card = (insert j t).card hjk : j < k ⊢ insert j t = s ∨ ∃ w ∈ s, w ∉ insert j t ∧ ∀ ⦃a : α⦄, w < a → (a ∈ insert j t ↔ a ∈ s)
case a.mpr.inr.intro.intro.intro.inl α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t✝ : Finset α r : ℕ inst✝ : Fintype α hs : s.Nonempty t : Finset α cards' : (s.erase (s.min' hs)).card = t.card k : α hks : k ∈ s.erase (s.min' hs) hkt : k ∉ t z : ∀ ⦃a : α⦄, k < a → (a ∈ t ↔ a ∈ s.erase (s.min' hs)) j : α := tᶜ.min' ⋯ hjk✝ : j ≤ k this : j ∉ t hcard : s.card = (insert j t).card hjk : j < k x : α hx : k < x ⊢ x ∈ insert j t ↔ x ∈ s
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/KruskalKatona.lean
Finset.Colex.shadow_initSeg
[83, 1]
[131, 20]
simpa only [mem_insert, z hx, (hjk.trans hx).ne', mem_erase, Ne, false_or_iff, and_iff_right_iff_imp] using fun _ ↦ ((min'_le _ _ $ mem_of_mem_erase hks).trans_lt hx).ne'
case a.mpr.inr.intro.intro.intro.inl α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t✝ : Finset α r : ℕ inst✝ : Fintype α hs : s.Nonempty t : Finset α cards' : (s.erase (s.min' hs)).card = t.card k : α hks : k ∈ s.erase (s.min' hs) hkt : k ∉ t z : ∀ ⦃a : α⦄, k < a → (a ∈ t ↔ a ∈ s.erase (s.min' hs)) j : α := tᶜ.min' ⋯ hjk✝ : j ≤ k this : j ∉ t hcard : s.card = (insert j t).card hjk : j < k x : α hx : k < x ⊢ x ∈ insert j t ↔ x ∈ s
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/KruskalKatona.lean
Finset.Colex.shadow_initSeg
[83, 1]
[131, 20]
apply mem_insert_of_mem
case a.mpr.inr.intro.intro.intro.inr.inl α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t✝ : Finset α r : ℕ inst✝ : Fintype α hs : s.Nonempty t : Finset α cards' : (s.erase (s.min' hs)).card = t.card k : α hks : k ∈ s.erase (s.min' hs) hkt : k ∉ t z : ∀ ⦃a : α⦄, k < a → (a ∈ t ↔ a ∈ s.erase (s.min' hs)) j : α := tᶜ.min' ⋯ hjk : j ≤ k this : j ∉ t hcard : s.card = (insert j t).card r₁ : j = k a : α ha : a ∈ s lt : k < a ⊢ a ∈ insert j t
case a.mpr.inr.intro.intro.intro.inr.inl.h α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t✝ : Finset α r : ℕ inst✝ : Fintype α hs : s.Nonempty t : Finset α cards' : (s.erase (s.min' hs)).card = t.card k : α hks : k ∈ s.erase (s.min' hs) hkt : k ∉ t z : ∀ ⦃a : α⦄, k < a → (a ∈ t ↔ a ∈ s.erase (s.min' hs)) j : α := tᶜ.min' ⋯ hjk : j ≤ k this : j ∉ t hcard : s.card = (insert j t).card r₁ : j = k a : α ha : a ∈ s lt : k < a ⊢ a ∈ t
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/KruskalKatona.lean
Finset.Colex.shadow_initSeg
[83, 1]
[131, 20]
rw [z lt]
case a.mpr.inr.intro.intro.intro.inr.inl.h α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t✝ : Finset α r : ℕ inst✝ : Fintype α hs : s.Nonempty t : Finset α cards' : (s.erase (s.min' hs)).card = t.card k : α hks : k ∈ s.erase (s.min' hs) hkt : k ∉ t z : ∀ ⦃a : α⦄, k < a → (a ∈ t ↔ a ∈ s.erase (s.min' hs)) j : α := tᶜ.min' ⋯ hjk : j ≤ k this : j ∉ t hcard : s.card = (insert j t).card r₁ : j = k a : α ha : a ∈ s lt : k < a ⊢ a ∈ t
case a.mpr.inr.intro.intro.intro.inr.inl.h α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t✝ : Finset α r : ℕ inst✝ : Fintype α hs : s.Nonempty t : Finset α cards' : (s.erase (s.min' hs)).card = t.card k : α hks : k ∈ s.erase (s.min' hs) hkt : k ∉ t z : ∀ ⦃a : α⦄, k < a → (a ∈ t ↔ a ∈ s.erase (s.min' hs)) j : α := tᶜ.min' ⋯ hjk : j ≤ k this : j ∉ t hcard : s.card = (insert j t).card r₁ : j = k a : α ha : a ∈ s lt : k < a ⊢ a ∈ s.erase (s.min' hs)
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/KruskalKatona.lean
Finset.Colex.shadow_initSeg
[83, 1]
[131, 20]
refine' mem_erase_of_ne_of_mem (lt_of_le_of_lt _ lt).ne' ha
case a.mpr.inr.intro.intro.intro.inr.inl.h α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t✝ : Finset α r : ℕ inst✝ : Fintype α hs : s.Nonempty t : Finset α cards' : (s.erase (s.min' hs)).card = t.card k : α hks : k ∈ s.erase (s.min' hs) hkt : k ∉ t z : ∀ ⦃a : α⦄, k < a → (a ∈ t ↔ a ∈ s.erase (s.min' hs)) j : α := tᶜ.min' ⋯ hjk : j ≤ k this : j ∉ t hcard : s.card = (insert j t).card r₁ : j = k a : α ha : a ∈ s lt : k < a ⊢ a ∈ s.erase (s.min' hs)
case a.mpr.inr.intro.intro.intro.inr.inl.h α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t✝ : Finset α r : ℕ inst✝ : Fintype α hs : s.Nonempty t : Finset α cards' : (s.erase (s.min' hs)).card = t.card k : α hks : k ∈ s.erase (s.min' hs) hkt : k ∉ t z : ∀ ⦃a : α⦄, k < a → (a ∈ t ↔ a ∈ s.erase (s.min' hs)) j : α := tᶜ.min' ⋯ hjk : j ≤ k this : j ∉ t hcard : s.card = (insert j t).card r₁ : j = k a : α ha : a ∈ s lt : k < a ⊢ s.min' hs ≤ k
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/KruskalKatona.lean
Finset.Colex.shadow_initSeg
[83, 1]
[131, 20]
apply min'_le _ _ (mem_of_mem_erase ‹_›)
case a.mpr.inr.intro.intro.intro.inr.inl.h α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t✝ : Finset α r : ℕ inst✝ : Fintype α hs : s.Nonempty t : Finset α cards' : (s.erase (s.min' hs)).card = t.card k : α hks : k ∈ s.erase (s.min' hs) hkt : k ∉ t z : ∀ ⦃a : α⦄, k < a → (a ∈ t ↔ a ∈ s.erase (s.min' hs)) j : α := tᶜ.min' ⋯ hjk : j ≤ k this : j ∉ t hcard : s.card = (insert j t).card r₁ : j = k a : α ha : a ∈ s lt : k < a ⊢ s.min' hs ≤ k
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/KruskalKatona.lean
Finset.Colex.shadow_initSeg
[83, 1]
[131, 20]
rw [r₁]
case a.mpr.inr.intro.intro.intro.inr.inr.inl α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t✝ : Finset α r : ℕ inst✝ : Fintype α hs : s.Nonempty t : Finset α cards' : (s.erase (s.min' hs)).card = t.card k : α hks : k ∈ s.erase (s.min' hs) hkt : k ∉ t z : ∀ ⦃a : α⦄, k < a → (a ∈ t ↔ a ∈ s.erase (s.min' hs)) j : α := tᶜ.min' ⋯ hjk : j ≤ k this : j ∉ t hcard : s.card = (insert j t).card r₁ : j = k ha : k ∈ s ⊢ k ∈ insert j t
case a.mpr.inr.intro.intro.intro.inr.inr.inl α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t✝ : Finset α r : ℕ inst✝ : Fintype α hs : s.Nonempty t : Finset α cards' : (s.erase (s.min' hs)).card = t.card k : α hks : k ∈ s.erase (s.min' hs) hkt : k ∉ t z : ∀ ⦃a : α⦄, k < a → (a ∈ t ↔ a ∈ s.erase (s.min' hs)) j : α := tᶜ.min' ⋯ hjk : j ≤ k this : j ∉ t hcard : s.card = (insert j t).card r₁ : j = k ha : k ∈ s ⊢ k ∈ insert k t
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/KruskalKatona.lean
Finset.Colex.shadow_initSeg
[83, 1]
[131, 20]
apply mem_insert_self
case a.mpr.inr.intro.intro.intro.inr.inr.inl α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t✝ : Finset α r : ℕ inst✝ : Fintype α hs : s.Nonempty t : Finset α cards' : (s.erase (s.min' hs)).card = t.card k : α hks : k ∈ s.erase (s.min' hs) hkt : k ∉ t z : ∀ ⦃a : α⦄, k < a → (a ∈ t ↔ a ∈ s.erase (s.min' hs)) j : α := tᶜ.min' ⋯ hjk : j ≤ k this : j ∉ t hcard : s.card = (insert j t).card r₁ : j = k ha : k ∈ s ⊢ k ∈ insert k t
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/KruskalKatona.lean
Finset.Colex.shadow_initSeg
[83, 1]
[131, 20]
apply mem_insert_of_mem
case a.mpr.inr.intro.intro.intro.inr.inr.inr α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t✝ : Finset α r : ℕ inst✝ : Fintype α hs : s.Nonempty t : Finset α cards' : (s.erase (s.min' hs)).card = t.card k : α hks : k ∈ s.erase (s.min' hs) hkt : k ∉ t z : ∀ ⦃a : α⦄, k < a → (a ∈ t ↔ a ∈ s.erase (s.min' hs)) j : α := tᶜ.min' ⋯ hjk : j ≤ k this : j ∉ t hcard : s.card = (insert j t).card r₁ : j = k a : α ha : a ∈ s gt : a < k ⊢ a ∈ insert j t
case a.mpr.inr.intro.intro.intro.inr.inr.inr.h α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t✝ : Finset α r : ℕ inst✝ : Fintype α hs : s.Nonempty t : Finset α cards' : (s.erase (s.min' hs)).card = t.card k : α hks : k ∈ s.erase (s.min' hs) hkt : k ∉ t z : ∀ ⦃a : α⦄, k < a → (a ∈ t ↔ a ∈ s.erase (s.min' hs)) j : α := tᶜ.min' ⋯ hjk : j ≤ k this : j ∉ t hcard : s.card = (insert j t).card r₁ : j = k a : α ha : a ∈ s gt : a < k ⊢ a ∈ t
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/KruskalKatona.lean
Finset.Colex.shadow_initSeg
[83, 1]
[131, 20]
rw [← r₁] at gt
case a.mpr.inr.intro.intro.intro.inr.inr.inr.h α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t✝ : Finset α r : ℕ inst✝ : Fintype α hs : s.Nonempty t : Finset α cards' : (s.erase (s.min' hs)).card = t.card k : α hks : k ∈ s.erase (s.min' hs) hkt : k ∉ t z : ∀ ⦃a : α⦄, k < a → (a ∈ t ↔ a ∈ s.erase (s.min' hs)) j : α := tᶜ.min' ⋯ hjk : j ≤ k this : j ∉ t hcard : s.card = (insert j t).card r₁ : j = k a : α ha : a ∈ s gt : a < k ⊢ a ∈ t
case a.mpr.inr.intro.intro.intro.inr.inr.inr.h α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t✝ : Finset α r : ℕ inst✝ : Fintype α hs : s.Nonempty t : Finset α cards' : (s.erase (s.min' hs)).card = t.card k : α hks : k ∈ s.erase (s.min' hs) hkt : k ∉ t z : ∀ ⦃a : α⦄, k < a → (a ∈ t ↔ a ∈ s.erase (s.min' hs)) j : α := tᶜ.min' ⋯ hjk : j ≤ k this : j ∉ t hcard : s.card = (insert j t).card r₁ : j = k a : α ha : a ∈ s gt : a < j ⊢ a ∈ t
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/KruskalKatona.lean
Finset.Colex.shadow_initSeg
[83, 1]
[131, 20]
by_contra
case a.mpr.inr.intro.intro.intro.inr.inr.inr.h α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t✝ : Finset α r : ℕ inst✝ : Fintype α hs : s.Nonempty t : Finset α cards' : (s.erase (s.min' hs)).card = t.card k : α hks : k ∈ s.erase (s.min' hs) hkt : k ∉ t z : ∀ ⦃a : α⦄, k < a → (a ∈ t ↔ a ∈ s.erase (s.min' hs)) j : α := tᶜ.min' ⋯ hjk : j ≤ k this : j ∉ t hcard : s.card = (insert j t).card r₁ : j = k a : α ha : a ∈ s gt : a < j ⊢ a ∈ t
case a.mpr.inr.intro.intro.intro.inr.inr.inr.h α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t✝ : Finset α r : ℕ inst✝ : Fintype α hs : s.Nonempty t : Finset α cards' : (s.erase (s.min' hs)).card = t.card k : α hks : k ∈ s.erase (s.min' hs) hkt : k ∉ t z : ∀ ⦃a : α⦄, k < a → (a ∈ t ↔ a ∈ s.erase (s.min' hs)) j : α := tᶜ.min' ⋯ hjk : j ≤ k this : j ∉ t hcard : s.card = (insert j t).card r₁ : j = k a : α ha : a ∈ s gt : a < j x✝ : a ∉ t ⊢ False
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/KruskalKatona.lean
Finset.Colex.shadow_initSeg
[83, 1]
[131, 20]
apply (min'_le tᶜ _ _).not_lt gt
case a.mpr.inr.intro.intro.intro.inr.inr.inr.h α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t✝ : Finset α r : ℕ inst✝ : Fintype α hs : s.Nonempty t : Finset α cards' : (s.erase (s.min' hs)).card = t.card k : α hks : k ∈ s.erase (s.min' hs) hkt : k ∉ t z : ∀ ⦃a : α⦄, k < a → (a ∈ t ↔ a ∈ s.erase (s.min' hs)) j : α := tᶜ.min' ⋯ hjk : j ≤ k this : j ∉ t hcard : s.card = (insert j t).card r₁ : j = k a : α ha : a ∈ s gt : a < j x✝ : a ∉ t ⊢ False
α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t✝ : Finset α r : ℕ inst✝ : Fintype α hs : s.Nonempty t : Finset α cards' : (s.erase (s.min' hs)).card = t.card k : α hks : k ∈ s.erase (s.min' hs) hkt : k ∉ t z : ∀ ⦃a : α⦄, k < a → (a ∈ t ↔ a ∈ s.erase (s.min' hs)) j : α := tᶜ.min' ⋯ hjk : j ≤ k this : j ∉ t hcard : s.card = (insert j t).card r₁ : j = k a : α ha : a ∈ s gt : a < j x✝ : a ∉ t ⊢ a ∈ tᶜ
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/KruskalKatona.lean
Finset.Colex.shadow_initSeg
[83, 1]
[131, 20]
rwa [mem_compl]
α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t✝ : Finset α r : ℕ inst✝ : Fintype α hs : s.Nonempty t : Finset α cards' : (s.erase (s.min' hs)).card = t.card k : α hks : k ∈ s.erase (s.min' hs) hkt : k ∉ t z : ∀ ⦃a : α⦄, k < a → (a ∈ t ↔ a ∈ s.erase (s.min' hs)) j : α := tᶜ.min' ⋯ hjk : j ≤ k this : j ∉ t hcard : s.card = (insert j t).card r₁ : j = k a : α ha : a ∈ s gt : a < j x✝ : a ∉ t ⊢ a ∈ tᶜ
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/KruskalKatona.lean
Finset.Colex.IsInitSeg.shadow
[133, 1]
[145, 26]
cases nonempty_fintype α
α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t : Finset α r : ℕ inst✝ : Finite α h₁ : IsInitSeg 𝒜 r ⊢ IsInitSeg (∂ 𝒜) (r - 1)
case intro α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t : Finset α r : ℕ inst✝ : Finite α h₁ : IsInitSeg 𝒜 r val✝ : Fintype α ⊢ IsInitSeg (∂ 𝒜) (r - 1)
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/KruskalKatona.lean
Finset.Colex.IsInitSeg.shadow
[133, 1]
[145, 26]
obtain rfl | hr := Nat.eq_zero_or_pos r
case intro α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t : Finset α r : ℕ inst✝ : Finite α h₁ : IsInitSeg 𝒜 r val✝ : Fintype α ⊢ IsInitSeg (∂ 𝒜) (r - 1)
case intro.inl α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t : Finset α inst✝ : Finite α val✝ : Fintype α h₁ : IsInitSeg 𝒜 0 ⊢ IsInitSeg (∂ 𝒜) (0 - 1) case intro.inr α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t : Finset α r : ℕ inst✝ : Finite α h₁ : IsInitSeg 𝒜 r val✝ : Fintype α hr : r > 0 ⊢ IsInitSeg (∂ 𝒜) (r - 1)
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/KruskalKatona.lean
Finset.Colex.IsInitSeg.shadow
[133, 1]
[145, 26]
obtain rfl | h𝒜 := 𝒜.eq_empty_or_nonempty
case intro.inr α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t : Finset α r : ℕ inst✝ : Finite α h₁ : IsInitSeg 𝒜 r val✝ : Fintype α hr : r > 0 ⊢ IsInitSeg (∂ 𝒜) (r - 1)
case intro.inr.inl α : Type u_1 inst✝¹ : LinearOrder α 𝒜₁ 𝒜₂ : Finset (Finset α) s t : Finset α r : ℕ inst✝ : Finite α val✝ : Fintype α hr : r > 0 h₁ : IsInitSeg ∅ r ⊢ IsInitSeg (∂ ∅) (r - 1) case intro.inr.inr α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t : Finset α r : ℕ inst✝ : Finite α h₁ : IsInitSeg 𝒜 r val✝ : Fintype α hr : r > 0 h𝒜 : 𝒜.Nonempty ⊢ IsInitSeg (∂ 𝒜) (r - 1)
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/KruskalKatona.lean
Finset.Colex.IsInitSeg.shadow
[133, 1]
[145, 26]
obtain ⟨s, rfl, rfl⟩ := h₁.exists_initSeg h𝒜
case intro.inr.inr α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t : Finset α r : ℕ inst✝ : Finite α h₁ : IsInitSeg 𝒜 r val✝ : Fintype α hr : r > 0 h𝒜 : 𝒜.Nonempty ⊢ IsInitSeg (∂ 𝒜) (r - 1)
case intro.inr.inr.intro.intro α : Type u_1 inst✝¹ : LinearOrder α 𝒜₁ 𝒜₂ : Finset (Finset α) s✝ t : Finset α inst✝ : Finite α val✝ : Fintype α s : Finset α hr : s.card > 0 h𝒜 : (initSeg s).Nonempty h₁ : IsInitSeg (initSeg s) s.card ⊢ IsInitSeg (∂ (initSeg s)) (s.card - 1)
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/KruskalKatona.lean
Finset.Colex.IsInitSeg.shadow
[133, 1]
[145, 26]
rw [shadow_initSeg (card_pos.1 hr), ← card_erase_of_mem (min'_mem _ _)]
case intro.inr.inr.intro.intro α : Type u_1 inst✝¹ : LinearOrder α 𝒜₁ 𝒜₂ : Finset (Finset α) s✝ t : Finset α inst✝ : Finite α val✝ : Fintype α s : Finset α hr : s.card > 0 h𝒜 : (initSeg s).Nonempty h₁ : IsInitSeg (initSeg s) s.card ⊢ IsInitSeg (∂ (initSeg s)) (s.card - 1)
case intro.inr.inr.intro.intro α : Type u_1 inst✝¹ : LinearOrder α 𝒜₁ 𝒜₂ : Finset (Finset α) s✝ t : Finset α inst✝ : Finite α val✝ : Fintype α s : Finset α hr : s.card > 0 h𝒜 : (initSeg s).Nonempty h₁ : IsInitSeg (initSeg s) s.card ⊢ IsInitSeg (initSeg (s.erase (s.min' ⋯))) (s.erase (s.min' ?m.16021)).card α : Type u_1 inst✝¹ : LinearOrder α 𝒜₁ 𝒜₂ : Finset (Finset α) s✝ t : Finset α inst✝ : Finite α val✝ : Fintype α s : Finset α hr : s.card > 0 h𝒜 : (initSeg s).Nonempty h₁ : IsInitSeg (initSeg s) s.card ⊢ s.Nonempty
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/KruskalKatona.lean
Finset.Colex.IsInitSeg.shadow
[133, 1]
[145, 26]
exact isInitSeg_initSeg
case intro.inr.inr.intro.intro α : Type u_1 inst✝¹ : LinearOrder α 𝒜₁ 𝒜₂ : Finset (Finset α) s✝ t : Finset α inst✝ : Finite α val✝ : Fintype α s : Finset α hr : s.card > 0 h𝒜 : (initSeg s).Nonempty h₁ : IsInitSeg (initSeg s) s.card ⊢ IsInitSeg (initSeg (s.erase (s.min' ⋯))) (s.erase (s.min' ?m.16021)).card α : Type u_1 inst✝¹ : LinearOrder α 𝒜₁ 𝒜₂ : Finset (Finset α) s✝ t : Finset α inst✝ : Finite α val✝ : Fintype α s : Finset α hr : s.card > 0 h𝒜 : (initSeg s).Nonempty h₁ : IsInitSeg (initSeg s) s.card ⊢ s.Nonempty
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/KruskalKatona.lean
Finset.Colex.IsInitSeg.shadow
[133, 1]
[145, 26]
have : 𝒜 ⊆ {∅} := fun s hs ↦ by rw [mem_singleton, ← Finset.card_eq_zero]; exact h₁.1 hs
case intro.inl α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t : Finset α inst✝ : Finite α val✝ : Fintype α h₁ : IsInitSeg 𝒜 0 ⊢ IsInitSeg (∂ 𝒜) (0 - 1)
case intro.inl α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t : Finset α inst✝ : Finite α val✝ : Fintype α h₁ : IsInitSeg 𝒜 0 this : 𝒜 ⊆ {∅} ⊢ IsInitSeg (∂ 𝒜) (0 - 1)
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/KruskalKatona.lean
Finset.Colex.IsInitSeg.shadow
[133, 1]
[145, 26]
have := shadow_monotone this
case intro.inl α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t : Finset α inst✝ : Finite α val✝ : Fintype α h₁ : IsInitSeg 𝒜 0 this : 𝒜 ⊆ {∅} ⊢ IsInitSeg (∂ 𝒜) (0 - 1)
case intro.inl α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t : Finset α inst✝ : Finite α val✝ : Fintype α h₁ : IsInitSeg 𝒜 0 this✝ : 𝒜 ⊆ {∅} this : ∂ 𝒜 ≤ ∂ {∅} ⊢ IsInitSeg (∂ 𝒜) (0 - 1)
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/KruskalKatona.lean
Finset.Colex.IsInitSeg.shadow
[133, 1]
[145, 26]
simp only [subset_empty, le_eq_subset, shadow_singleton_empty] at this
case intro.inl α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t : Finset α inst✝ : Finite α val✝ : Fintype α h₁ : IsInitSeg 𝒜 0 this✝ : 𝒜 ⊆ {∅} this : ∂ 𝒜 ≤ ∂ {∅} ⊢ IsInitSeg (∂ 𝒜) (0 - 1)
case intro.inl α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t : Finset α inst✝ : Finite α val✝ : Fintype α h₁ : IsInitSeg 𝒜 0 this✝ : 𝒜 ⊆ {∅} this : ∂ 𝒜 = ∅ ⊢ IsInitSeg (∂ 𝒜) (0 - 1)
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/KruskalKatona.lean
Finset.Colex.IsInitSeg.shadow
[133, 1]
[145, 26]
simp [this]
case intro.inl α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s t : Finset α inst✝ : Finite α val✝ : Fintype α h₁ : IsInitSeg 𝒜 0 this✝ : 𝒜 ⊆ {∅} this : ∂ 𝒜 = ∅ ⊢ IsInitSeg (∂ 𝒜) (0 - 1)
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/KruskalKatona.lean
Finset.Colex.IsInitSeg.shadow
[133, 1]
[145, 26]
rw [mem_singleton, ← Finset.card_eq_zero]
α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s✝ t : Finset α inst✝ : Finite α val✝ : Fintype α h₁ : IsInitSeg 𝒜 0 s : Finset α hs : s ∈ 𝒜 ⊢ s ∈ {∅}
α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s✝ t : Finset α inst✝ : Finite α val✝ : Fintype α h₁ : IsInitSeg 𝒜 0 s : Finset α hs : s ∈ 𝒜 ⊢ s.card = 0
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/KruskalKatona.lean
Finset.Colex.IsInitSeg.shadow
[133, 1]
[145, 26]
exact h₁.1 hs
α : Type u_1 inst✝¹ : LinearOrder α 𝒜 𝒜₁ 𝒜₂ : Finset (Finset α) s✝ t : Finset α inst✝ : Finite α val✝ : Fintype α h₁ : IsInitSeg 𝒜 0 s : Finset α hs : s ∈ 𝒜 ⊢ s.card = 0
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/KruskalKatona.lean
Finset.Colex.IsInitSeg.shadow
[133, 1]
[145, 26]
simp
case intro.inr.inl α : Type u_1 inst✝¹ : LinearOrder α 𝒜₁ 𝒜₂ : Finset (Finset α) s t : Finset α r : ℕ inst✝ : Finite α val✝ : Fintype α hr : r > 0 h₁ : IsInitSeg ∅ r ⊢ IsInitSeg (∂ ∅) (r - 1)
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/KruskalKatona.lean
Finset.UV.toColex_compress_lt_toColex
[156, 1]
[165, 26]
rw [compress, ite_ne_right_iff] at hA
α : Type u_1 inst✝ : LinearOrder α s U V : Finset α n : ℕ hU : U.Nonempty hV : V.Nonempty h : U.max' hU < V.max' hV hA : compress U V s ≠ s ⊢ { ofColex := compress U V s } < { ofColex := s }
α : Type u_1 inst✝ : LinearOrder α s U V : Finset α n : ℕ hU : U.Nonempty hV : V.Nonempty h : U.max' hU < V.max' hV hA : (Disjoint U s ∧ V ≤ s) ∧ (s ⊔ U) \ V ≠ s ⊢ { ofColex := compress U V s } < { ofColex := s }
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/KruskalKatona.lean
Finset.UV.toColex_compress_lt_toColex
[156, 1]
[165, 26]
rw [compress, if_pos hA.1, lt_iff_exists_forall_lt_mem_iff_mem]
α : Type u_1 inst✝ : LinearOrder α s U V : Finset α n : ℕ hU : U.Nonempty hV : V.Nonempty h : U.max' hU < V.max' hV hA : (Disjoint U s ∧ V ≤ s) ∧ (s ⊔ U) \ V ≠ s ⊢ { ofColex := compress U V s } < { ofColex := s }
α : Type u_1 inst✝ : LinearOrder α s U V : Finset α n : ℕ hU : U.Nonempty hV : V.Nonempty h : U.max' hU < V.max' hV hA : (Disjoint U s ∧ V ≤ s) ∧ (s ⊔ U) \ V ≠ s ⊢ ∃ w ∈ s, w ∉ (s ⊔ U) \ V ∧ ∀ ⦃a : α⦄, w < a → (a ∈ (s ⊔ U) \ V ↔ a ∈ s)
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/KruskalKatona.lean
Finset.UV.toColex_compress_lt_toColex
[156, 1]
[165, 26]
refine ⟨_, hA.1.2 $ max'_mem _ hV, not_mem_sdiff_of_mem_right $ max'_mem _ _, fun a ha ↦ ?_⟩
α : Type u_1 inst✝ : LinearOrder α s U V : Finset α n : ℕ hU : U.Nonempty hV : V.Nonempty h : U.max' hU < V.max' hV hA : (Disjoint U s ∧ V ≤ s) ∧ (s ⊔ U) \ V ≠ s ⊢ ∃ w ∈ s, w ∉ (s ⊔ U) \ V ∧ ∀ ⦃a : α⦄, w < a → (a ∈ (s ⊔ U) \ V ↔ a ∈ s)
α : Type u_1 inst✝ : LinearOrder α s U V : Finset α n : ℕ hU : U.Nonempty hV : V.Nonempty h : U.max' hU < V.max' hV hA : (Disjoint U s ∧ V ≤ s) ∧ (s ⊔ U) \ V ≠ s a : α ha : V.max' hV < a ⊢ a ∈ (s ⊔ U) \ V ↔ a ∈ s
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/KruskalKatona.lean
Finset.UV.toColex_compress_lt_toColex
[156, 1]
[165, 26]
have : a ∉ V := fun H ↦ ha.not_le (le_max' _ _ H)
α : Type u_1 inst✝ : LinearOrder α s U V : Finset α n : ℕ hU : U.Nonempty hV : V.Nonempty h : U.max' hU < V.max' hV hA : (Disjoint U s ∧ V ≤ s) ∧ (s ⊔ U) \ V ≠ s a : α ha : V.max' hV < a ⊢ a ∈ (s ⊔ U) \ V ↔ a ∈ s
α : Type u_1 inst✝ : LinearOrder α s U V : Finset α n : ℕ hU : U.Nonempty hV : V.Nonempty h : U.max' hU < V.max' hV hA : (Disjoint U s ∧ V ≤ s) ∧ (s ⊔ U) \ V ≠ s a : α ha : V.max' hV < a this : a ∉ V ⊢ a ∈ (s ⊔ U) \ V ↔ a ∈ s
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/KruskalKatona.lean
Finset.UV.toColex_compress_lt_toColex
[156, 1]
[165, 26]
have : a ∉ U := fun H ↦ ha.not_lt ((le_max' _ _ H).trans_lt h)
α : Type u_1 inst✝ : LinearOrder α s U V : Finset α n : ℕ hU : U.Nonempty hV : V.Nonempty h : U.max' hU < V.max' hV hA : (Disjoint U s ∧ V ≤ s) ∧ (s ⊔ U) \ V ≠ s a : α ha : V.max' hV < a this : a ∉ V ⊢ a ∈ (s ⊔ U) \ V ↔ a ∈ s
α : Type u_1 inst✝ : LinearOrder α s U V : Finset α n : ℕ hU : U.Nonempty hV : V.Nonempty h : U.max' hU < V.max' hV hA : (Disjoint U s ∧ V ≤ s) ∧ (s ⊔ U) \ V ≠ s a : α ha : V.max' hV < a this✝ : a ∉ V this : a ∉ U ⊢ a ∈ (s ⊔ U) \ V ↔ a ∈ s
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/KruskalKatona.lean
Finset.UV.toColex_compress_lt_toColex
[156, 1]
[165, 26]
simp [‹a ∉ U›, ‹a ∉ V›]
α : Type u_1 inst✝ : LinearOrder α s U V : Finset α n : ℕ hU : U.Nonempty hV : V.Nonempty h : U.max' hU < V.max' hV hA : (Disjoint U s ∧ V ≤ s) ∧ (s ⊔ U) \ V ≠ s a : α ha : V.max' hV < a this✝ : a ∉ V this : a ∉ U ⊢ a ∈ (s ⊔ U) \ V ↔ a ∈ s
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/KruskalKatona.lean
Finset.UV.compression_improved
[174, 1]
[195, 22]
obtain ⟨UVd, same_size, hU, hV, max_lt⟩ := h₁
α : Type u_1 inst✝ : LinearOrder α s U V : Finset α n : ℕ 𝒜 : Finset (Finset α) h₁ : Finset.UV.UsefulCompression U V h₂ : ∀ ⦃U₁ V₁ : Finset α⦄, Finset.UV.UsefulCompression U₁ V₁ → U₁.card < U.card → IsCompressed U₁ V₁ 𝒜 ⊢ (∂ (𝓒 U V 𝒜)).card ≤ (∂ 𝒜).card
case intro.intro.intro.intro α : Type u_1 inst✝ : LinearOrder α s U V : Finset α n : ℕ 𝒜 : Finset (Finset α) h₂ : ∀ ⦃U₁ V₁ : Finset α⦄, Finset.UV.UsefulCompression U₁ V₁ → U₁.card < U.card → IsCompressed U₁ V₁ 𝒜 UVd : Disjoint U V same_size : U.card = V.card hU : U.Nonempty hV : V.Nonempty max_lt : U.max' hU < V.max' hV ⊢ (∂ (𝓒 U V 𝒜)).card ≤ (∂ 𝒜).card
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/KruskalKatona.lean
Finset.UV.compression_improved
[174, 1]
[195, 22]
refine' card_shadow_compression_le _ _ fun x Hx ↦ ⟨min' V hV, min'_mem _ _, _⟩
case intro.intro.intro.intro α : Type u_1 inst✝ : LinearOrder α s U V : Finset α n : ℕ 𝒜 : Finset (Finset α) h₂ : ∀ ⦃U₁ V₁ : Finset α⦄, Finset.UV.UsefulCompression U₁ V₁ → U₁.card < U.card → IsCompressed U₁ V₁ 𝒜 UVd : Disjoint U V same_size : U.card = V.card hU : U.Nonempty hV : V.Nonempty max_lt : U.max' hU < V.max' hV ⊢ (∂ (𝓒 U V 𝒜)).card ≤ (∂ 𝒜).card
case intro.intro.intro.intro α : Type u_1 inst✝ : LinearOrder α s U V : Finset α n : ℕ 𝒜 : Finset (Finset α) h₂ : ∀ ⦃U₁ V₁ : Finset α⦄, Finset.UV.UsefulCompression U₁ V₁ → U₁.card < U.card → IsCompressed U₁ V₁ 𝒜 UVd : Disjoint U V same_size : U.card = V.card hU : U.Nonempty hV : V.Nonempty max_lt : U.max' hU < V.max' hV x : α Hx : x ∈ U ⊢ IsCompressed (U.erase x) (V.erase (V.min' hV)) 𝒜
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/KruskalKatona.lean
Finset.UV.compression_improved
[174, 1]
[195, 22]
obtain hU' | hU' := eq_or_lt_of_le (succ_le_iff.2 hU.card_pos)
case intro.intro.intro.intro α : Type u_1 inst✝ : LinearOrder α s U V : Finset α n : ℕ 𝒜 : Finset (Finset α) h₂ : ∀ ⦃U₁ V₁ : Finset α⦄, Finset.UV.UsefulCompression U₁ V₁ → U₁.card < U.card → IsCompressed U₁ V₁ 𝒜 UVd : Disjoint U V same_size : U.card = V.card hU : U.Nonempty hV : V.Nonempty max_lt : U.max' hU < V.max' hV x : α Hx : x ∈ U ⊢ IsCompressed (U.erase x) (V.erase (V.min' hV)) 𝒜
case intro.intro.intro.intro.inl α : Type u_1 inst✝ : LinearOrder α s U V : Finset α n : ℕ 𝒜 : Finset (Finset α) h₂ : ∀ ⦃U₁ V₁ : Finset α⦄, Finset.UV.UsefulCompression U₁ V₁ → U₁.card < U.card → IsCompressed U₁ V₁ 𝒜 UVd : Disjoint U V same_size : U.card = V.card hU : U.Nonempty hV : V.Nonempty max_lt : U.max' hU < V.max' hV x : α Hx : x ∈ U hU' : succ 0 = U.card ⊢ IsCompressed (U.erase x) (V.erase (V.min' hV)) 𝒜 case intro.intro.intro.intro.inr α : Type u_1 inst✝ : LinearOrder α s U V : Finset α n : ℕ 𝒜 : Finset (Finset α) h₂ : ∀ ⦃U₁ V₁ : Finset α⦄, Finset.UV.UsefulCompression U₁ V₁ → U₁.card < U.card → IsCompressed U₁ V₁ 𝒜 UVd : Disjoint U V same_size : U.card = V.card hU : U.Nonempty hV : V.Nonempty max_lt : U.max' hU < V.max' hV x : α Hx : x ∈ U hU' : succ 0 < U.card ⊢ IsCompressed (U.erase x) (V.erase (V.min' hV)) 𝒜
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/KruskalKatona.lean
Finset.UV.compression_improved
[174, 1]
[195, 22]
refine' h₂ ⟨UVd.mono (erase_subset _ _) (erase_subset _ _), _, _, _, _⟩ (card_erase_lt_of_mem Hx)
case intro.intro.intro.intro.inr α : Type u_1 inst✝ : LinearOrder α s U V : Finset α n : ℕ 𝒜 : Finset (Finset α) h₂ : ∀ ⦃U₁ V₁ : Finset α⦄, Finset.UV.UsefulCompression U₁ V₁ → U₁.card < U.card → IsCompressed U₁ V₁ 𝒜 UVd : Disjoint U V same_size : U.card = V.card hU : U.Nonempty hV : V.Nonempty max_lt : U.max' hU < V.max' hV x : α Hx : x ∈ U hU' : succ 0 < U.card ⊢ IsCompressed (U.erase x) (V.erase (V.min' hV)) 𝒜
case intro.intro.intro.intro.inr.refine'_1 α : Type u_1 inst✝ : LinearOrder α s U V : Finset α n : ℕ 𝒜 : Finset (Finset α) h₂ : ∀ ⦃U₁ V₁ : Finset α⦄, Finset.UV.UsefulCompression U₁ V₁ → U₁.card < U.card → IsCompressed U₁ V₁ 𝒜 UVd : Disjoint U V same_size : U.card = V.card hU : U.Nonempty hV : V.Nonempty max_lt : U.max' hU < V.max' hV x : α Hx : x ∈ U hU' : succ 0 < U.card ⊢ (U.erase x).card = (V.erase (V.min' hV)).card case intro.intro.intro.intro.inr.refine'_2 α : Type u_1 inst✝ : LinearOrder α s U V : Finset α n : ℕ 𝒜 : Finset (Finset α) h₂ : ∀ ⦃U₁ V₁ : Finset α⦄, Finset.UV.UsefulCompression U₁ V₁ → U₁.card < U.card → IsCompressed U₁ V₁ 𝒜 UVd : Disjoint U V same_size : U.card = V.card hU : U.Nonempty hV : V.Nonempty max_lt : U.max' hU < V.max' hV x : α Hx : x ∈ U hU' : succ 0 < U.card ⊢ (U.erase x).Nonempty case intro.intro.intro.intro.inr.refine'_3 α : Type u_1 inst✝ : LinearOrder α s U V : Finset α n : ℕ 𝒜 : Finset (Finset α) h₂ : ∀ ⦃U₁ V₁ : Finset α⦄, Finset.UV.UsefulCompression U₁ V₁ → U₁.card < U.card → IsCompressed U₁ V₁ 𝒜 UVd : Disjoint U V same_size : U.card = V.card hU : U.Nonempty hV : V.Nonempty max_lt : U.max' hU < V.max' hV x : α Hx : x ∈ U hU' : succ 0 < U.card ⊢ (V.erase (V.min' hV)).Nonempty case intro.intro.intro.intro.inr.refine'_4 α : Type u_1 inst✝ : LinearOrder α s U V : Finset α n : ℕ 𝒜 : Finset (Finset α) h₂ : ∀ ⦃U₁ V₁ : Finset α⦄, Finset.UV.UsefulCompression U₁ V₁ → U₁.card < U.card → IsCompressed U₁ V₁ 𝒜 UVd : Disjoint U V same_size : U.card = V.card hU : U.Nonempty hV : V.Nonempty max_lt : U.max' hU < V.max' hV x : α Hx : x ∈ U hU' : succ 0 < U.card ⊢ (U.erase x).max' ?intro.intro.intro.intro.inr.refine'_2 < (V.erase (V.min' hV)).max' ?intro.intro.intro.intro.inr.refine'_3
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/KruskalKatona.lean
Finset.UV.compression_improved
[174, 1]
[195, 22]
rw [← hU'] at same_size
case intro.intro.intro.intro.inl α : Type u_1 inst✝ : LinearOrder α s U V : Finset α n : ℕ 𝒜 : Finset (Finset α) h₂ : ∀ ⦃U₁ V₁ : Finset α⦄, Finset.UV.UsefulCompression U₁ V₁ → U₁.card < U.card → IsCompressed U₁ V₁ 𝒜 UVd : Disjoint U V same_size : U.card = V.card hU : U.Nonempty hV : V.Nonempty max_lt : U.max' hU < V.max' hV x : α Hx : x ∈ U hU' : succ 0 = U.card ⊢ IsCompressed (U.erase x) (V.erase (V.min' hV)) 𝒜
case intro.intro.intro.intro.inl α : Type u_1 inst✝ : LinearOrder α s U V : Finset α n : ℕ 𝒜 : Finset (Finset α) h₂ : ∀ ⦃U₁ V₁ : Finset α⦄, Finset.UV.UsefulCompression U₁ V₁ → U₁.card < U.card → IsCompressed U₁ V₁ 𝒜 UVd : Disjoint U V same_size : succ 0 = V.card hU : U.Nonempty hV : V.Nonempty max_lt : U.max' hU < V.max' hV x : α Hx : x ∈ U hU' : succ 0 = U.card ⊢ IsCompressed (U.erase x) (V.erase (V.min' hV)) 𝒜
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/KruskalKatona.lean
Finset.UV.compression_improved
[174, 1]
[195, 22]
have : erase U x = ∅ := by rw [← Finset.card_eq_zero, card_erase_of_mem Hx, ← hU']
case intro.intro.intro.intro.inl α : Type u_1 inst✝ : LinearOrder α s U V : Finset α n : ℕ 𝒜 : Finset (Finset α) h₂ : ∀ ⦃U₁ V₁ : Finset α⦄, Finset.UV.UsefulCompression U₁ V₁ → U₁.card < U.card → IsCompressed U₁ V₁ 𝒜 UVd : Disjoint U V same_size : succ 0 = V.card hU : U.Nonempty hV : V.Nonempty max_lt : U.max' hU < V.max' hV x : α Hx : x ∈ U hU' : succ 0 = U.card ⊢ IsCompressed (U.erase x) (V.erase (V.min' hV)) 𝒜
case intro.intro.intro.intro.inl α : Type u_1 inst✝ : LinearOrder α s U V : Finset α n : ℕ 𝒜 : Finset (Finset α) h₂ : ∀ ⦃U₁ V₁ : Finset α⦄, Finset.UV.UsefulCompression U₁ V₁ → U₁.card < U.card → IsCompressed U₁ V₁ 𝒜 UVd : Disjoint U V same_size : succ 0 = V.card hU : U.Nonempty hV : V.Nonempty max_lt : U.max' hU < V.max' hV x : α Hx : x ∈ U hU' : succ 0 = U.card this : U.erase x = ∅ ⊢ IsCompressed (U.erase x) (V.erase (V.min' hV)) 𝒜
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/KruskalKatona.lean
Finset.UV.compression_improved
[174, 1]
[195, 22]
have : erase V (min' V hV) = ∅ := by rw [← Finset.card_eq_zero, card_erase_of_mem (min'_mem _ _), ← same_size]
case intro.intro.intro.intro.inl α : Type u_1 inst✝ : LinearOrder α s U V : Finset α n : ℕ 𝒜 : Finset (Finset α) h₂ : ∀ ⦃U₁ V₁ : Finset α⦄, Finset.UV.UsefulCompression U₁ V₁ → U₁.card < U.card → IsCompressed U₁ V₁ 𝒜 UVd : Disjoint U V same_size : succ 0 = V.card hU : U.Nonempty hV : V.Nonempty max_lt : U.max' hU < V.max' hV x : α Hx : x ∈ U hU' : succ 0 = U.card this : U.erase x = ∅ ⊢ IsCompressed (U.erase x) (V.erase (V.min' hV)) 𝒜
case intro.intro.intro.intro.inl α : Type u_1 inst✝ : LinearOrder α s U V : Finset α n : ℕ 𝒜 : Finset (Finset α) h₂ : ∀ ⦃U₁ V₁ : Finset α⦄, Finset.UV.UsefulCompression U₁ V₁ → U₁.card < U.card → IsCompressed U₁ V₁ 𝒜 UVd : Disjoint U V same_size : succ 0 = V.card hU : U.Nonempty hV : V.Nonempty max_lt : U.max' hU < V.max' hV x : α Hx : x ∈ U hU' : succ 0 = U.card this✝ : U.erase x = ∅ this : V.erase (V.min' hV) = ∅ ⊢ IsCompressed (U.erase x) (V.erase (V.min' hV)) 𝒜
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/KruskalKatona.lean
Finset.UV.compression_improved
[174, 1]
[195, 22]
rw [‹erase U x = ∅›, ‹erase V (min' V hV) = ∅›]
case intro.intro.intro.intro.inl α : Type u_1 inst✝ : LinearOrder α s U V : Finset α n : ℕ 𝒜 : Finset (Finset α) h₂ : ∀ ⦃U₁ V₁ : Finset α⦄, Finset.UV.UsefulCompression U₁ V₁ → U₁.card < U.card → IsCompressed U₁ V₁ 𝒜 UVd : Disjoint U V same_size : succ 0 = V.card hU : U.Nonempty hV : V.Nonempty max_lt : U.max' hU < V.max' hV x : α Hx : x ∈ U hU' : succ 0 = U.card this✝ : U.erase x = ∅ this : V.erase (V.min' hV) = ∅ ⊢ IsCompressed (U.erase x) (V.erase (V.min' hV)) 𝒜
case intro.intro.intro.intro.inl α : Type u_1 inst✝ : LinearOrder α s U V : Finset α n : ℕ 𝒜 : Finset (Finset α) h₂ : ∀ ⦃U₁ V₁ : Finset α⦄, Finset.UV.UsefulCompression U₁ V₁ → U₁.card < U.card → IsCompressed U₁ V₁ 𝒜 UVd : Disjoint U V same_size : succ 0 = V.card hU : U.Nonempty hV : V.Nonempty max_lt : U.max' hU < V.max' hV x : α Hx : x ∈ U hU' : succ 0 = U.card this✝ : U.erase x = ∅ this : V.erase (V.min' hV) = ∅ ⊢ IsCompressed ∅ ∅ 𝒜
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/KruskalKatona.lean
Finset.UV.compression_improved
[174, 1]
[195, 22]
exact isCompressed_self _ _
case intro.intro.intro.intro.inl α : Type u_1 inst✝ : LinearOrder α s U V : Finset α n : ℕ 𝒜 : Finset (Finset α) h₂ : ∀ ⦃U₁ V₁ : Finset α⦄, Finset.UV.UsefulCompression U₁ V₁ → U₁.card < U.card → IsCompressed U₁ V₁ 𝒜 UVd : Disjoint U V same_size : succ 0 = V.card hU : U.Nonempty hV : V.Nonempty max_lt : U.max' hU < V.max' hV x : α Hx : x ∈ U hU' : succ 0 = U.card this✝ : U.erase x = ∅ this : V.erase (V.min' hV) = ∅ ⊢ IsCompressed ∅ ∅ 𝒜
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/KruskalKatona.lean
Finset.UV.compression_improved
[174, 1]
[195, 22]
rw [← Finset.card_eq_zero, card_erase_of_mem Hx, ← hU']
α : Type u_1 inst✝ : LinearOrder α s U V : Finset α n : ℕ 𝒜 : Finset (Finset α) h₂ : ∀ ⦃U₁ V₁ : Finset α⦄, Finset.UV.UsefulCompression U₁ V₁ → U₁.card < U.card → IsCompressed U₁ V₁ 𝒜 UVd : Disjoint U V same_size : succ 0 = V.card hU : U.Nonempty hV : V.Nonempty max_lt : U.max' hU < V.max' hV x : α Hx : x ∈ U hU' : succ 0 = U.card ⊢ U.erase x = ∅
no goals
https://github.com/YaelDillies/LeanCamCombi.git
034199694e3b91536d03bc4a8b0cdbd659cdf50f
LeanCamCombi/KruskalKatona.lean
Finset.UV.compression_improved
[174, 1]
[195, 22]
rw [← Finset.card_eq_zero, card_erase_of_mem (min'_mem _ _), ← same_size]
α : Type u_1 inst✝ : LinearOrder α s U V : Finset α n : ℕ 𝒜 : Finset (Finset α) h₂ : ∀ ⦃U₁ V₁ : Finset α⦄, Finset.UV.UsefulCompression U₁ V₁ → U₁.card < U.card → IsCompressed U₁ V₁ 𝒜 UVd : Disjoint U V same_size : succ 0 = V.card hU : U.Nonempty hV : V.Nonempty max_lt : U.max' hU < V.max' hV x : α Hx : x ∈ U hU' : succ 0 = U.card this : U.erase x = ∅ ⊢ V.erase (V.min' hV) = ∅
no goals