Skip to content

Commit 108169d

Browse files
committed
chore: clean up FiveWheelLike (#31813)
Restores lemmas in Mathlib.Combinatorics.SimpleGraph.FiveWheelLike that had been commented out during nightly testing, but which now build again (unmodified).
1 parent 7ce4a4b commit 108169d

File tree

1 file changed

+2
-14
lines changed

1 file changed

+2
-14
lines changed

Mathlib/Combinatorics/SimpleGraph/FiveWheelLike.lean

Lines changed: 2 additions & 14 deletions
Original file line numberDiff line numberDiff line change
@@ -346,13 +346,6 @@ lemma exists_isFiveWheelLike_succ_of_not_adj_le_two (hW : ∀ ⦃y⦄, y ∈ s
346346
notMem_mono inter_subset_left hbs, erase_eq_of_notMem <| notMem_mono inter_subset_right hat,
347347
card_insert_of_notMem (fun h ↦ G.irrefl (hW h)), hw.card_inter]
348348

349-
#adaptation_note
350-
/--
351-
Due to a change in `grind` between `nightly-2025-10-31` and `nightly-2025-11-02`,
352-
this proof is no longer working. I've temporarily commented it out to get a build of
353-
`nightly-testing`.
354-
-/
355-
/-
356349
/--
357350
If `G` is a `Kᵣ₊₂`-free graph with `n` vertices containing a `Wᵣ,ₖ` but no `Wᵣ,ₖ₊₁`
358351
then `G.minDegree ≤ (2 * r + k) * n / (2 * r + k + 3)`
@@ -415,16 +408,11 @@ lemma minDegree_le_of_cliqueFree_fiveWheelLikeFree_succ [Fintype α]
415408
rw [hap, ← add_mul, card_add_card_compl, mul_comm, two_mul, ← add_assoc]
416409
gcongr
417410
cutsat
418-
-/
411+
419412
end IsFiveWheelLike
420413

421414
variable [DecidableEq α]
422415

423-
#adaptation_note
424-
/--
425-
I've temporarily commented it out to get a build of `nightly-testing`. See the note above.
426-
-/
427-
/-
428416
/-- **Andrasfái-Erdős-Sós** theorem
429417
430418
If `G` is a `Kᵣ₊₁`-free graph with `n` vertices and `(3 * r - 4) * n / (3 * r - 1) < G.minDegree`
@@ -459,6 +447,6 @@ theorem colorable_of_cliqueFree_lt_minDegree [Fintype α] [DecidableRel G.Adj]
459447
apply (Nat.mul_le_mul_right _ (Nat.div_mul_le_self ..)).trans
460448
nlinarith
461449
exact (hd.trans_le <| minDegree_le_minDegree hle).not_ge <| hD.trans <| this
462-
-/
450+
463451
end AES
464452
end SimpleGraph

0 commit comments

Comments
 (0)