Zulip Chat Archive

Stream: graph theory

Topic: G.chromaticNumber ≤ n → G.Colorable n


Iván Renison (Dec 07 2023 at 17:30):

Hello, I'm trying to prove this:

theorem chromaticNumber_le_then_colorable {G : SimpleGraph α} {n : } (hc : G.chromaticNumber  n) :
    G.Colorable n := by sorry

But I'm not being able to
There is a theorem that says (hc : G.Colorable m) → G.Colorable G.chromaticNumber but I'm not being able to us it because what I have is different
How could I do?

Yaël Dillies (Dec 07 2023 at 17:31):

docs#SimpleGraph.Colorable.mono

Iván Renison (Dec 07 2023 at 17:34):

I'm not able to get that G is colorable with some number, so I don't no how to get the hc parameter for Colorable.mono

Mauricio Collares (Dec 07 2023 at 17:38):

Do you have any other hypotheses which imply the graph can be coloured with finitely many colours?

Yaël Dillies (Dec 07 2023 at 17:39):

If not, then the theorem is wrong as it could be that G.chromaticNumber = 0.

Iván Renison (Dec 07 2023 at 17:40):

I can add that α is not empty

Iván Renison (Dec 07 2023 at 17:41):

So with that I think that G.chromaticNumber > 0

Iván Renison (Dec 07 2023 at 17:43):

I can also add that α is finite, but the I think that the theorem should be valid with α infinity, it's correct that?

Mauricio Collares (Dec 07 2023 at 17:44):

If G is an infinite complete graph and n is any positive integer, then the theorem is false

Kyle Miller (Dec 07 2023 at 17:44):

If G is not colorable with finitely many colors, then you'd have G.chromaticNumber = 0 but not G.Colorable n.

Kyle Miller (Dec 07 2023 at 17:45):

I've been meaning to get around to upgrading this API by making chromaticNumber be a docs#ENat

Kyle Miller (Dec 07 2023 at 17:46):

Another solution would be to have a G.chromaticNumberLE n style of predicate, but that's more limited than an ENat I think

Iván Renison (Dec 07 2023 at 17:47):

Okey, I didn't had in mind that "If G isn't colorable with finitely many colors, this will be 0."

Iván Renison (Dec 07 2023 at 17:47):

I will add that α is finite

Iván Renison (Dec 07 2023 at 17:47):

Thank you vary much

Kyle Miller (Dec 07 2023 at 17:47):

One way the library works right now is to include the assumption that the chromatic number is positive, or to include the assumption that there exists some n' such that G.colorable n'

Kyle Miller (Dec 07 2023 at 17:47):

This can be useful for you: docs#SimpleGraph.colorable_of_chromaticNumber_pos

Iván Renison (Dec 07 2023 at 17:48):

Yes, it seems good idea

Iván Renison (Dec 07 2023 at 17:49):

Thanks

Kyle Miller (Dec 07 2023 at 22:44):

If anyone wants to help clean this up (or maybe finish it -- I haven't checked if mathlib builds completely), #8883 refactors chromaticNumber to be ENat-valued.


Last updated: Dec 20 2023 at 11:08 UTC