Zulip Chat Archive

Stream: graph theory

Topic: edge coloring


Matthew Ballard (May 08 2023 at 14:04):

@Utku Okur and Alec Helm worked on some results for edge colorings of graphs for a recent graduate class here. The repo is uofsc-spring-2023-math-768-001/project1. The current state of the repo might make your eyes bleed though.

Since @Yaël Dillies asked about this on another thread, I thought I should at least record here.

Kevin Buzzard (May 08 2023 at 14:10):

Is the repo public? Right now the hashtag isn't resolving to anything (for me)

Matthew Ballard (May 08 2023 at 14:16):

Thanks. Fixed.

Matthew Ballard (May 08 2023 at 14:18):

The goal was to do the two bounds in terms of maximal degree. We got

theorem maxDegree_le_edgeChromaticNumber [Fintype V] [DecidableRel G.Adj] [Fintype (edgeSet G)] :
    maxDegree G  edgeChromaticNumber G

But not the harder direction. I am not sure if Utku or Alec are planning on working on this.

Utku Okur (Dec 19 2024 at 23:50):

Would it be considered a constructive proof of Vizing's Theorem, if we use the assumptions:

variable {V : Type} {G : SimpleGraph V} [Fintype V] [CompleteLinearOrder V]

In other words, I assume that there is a linear order on the (finitely many) vertices of the graph and show that its edge chromatic number is bounded above by its maximum degree plus one? I thought that this would avoid "Classical.choose".

Mitchell Lee (Dec 20 2024 at 00:07):

It should be sufficient to have [Fintype G.edgeSet]. (Roughly, this hypothesis means that there is an explicit bijection between the edge set of GG and the set {1,,n}\{1, \ldots, n\}, for some nn.) Then, you may use induction (docs#Finset.induction_on) on G.edgeFinset (docs#SimpleGraph.edgeFinset). The hypotheses of [Fintype V] and [CompleteLinearOrder V] should not be necessary.

Mitchell Lee (Dec 20 2024 at 00:09):

You will likely need [DecidableEq V] as well, actually.

Mitchell Lee (Dec 20 2024 at 00:12):

Here is a reference for all the finiteness assumptions that one can make on simple graphs: https://leanprover-community.github.io/mathlib4_docs/Mathlib/Combinatorics/SimpleGraph/Finite.html


Last updated: May 02 2025 at 03:31 UTC