Skip to content

Commit

Permalink
colorable_zero_iff
Browse files Browse the repository at this point in the history
  • Loading branch information
jt496 committed Jan 28, 2025
1 parent 7fb23e3 commit 90f348a
Showing 1 changed file with 4 additions and 0 deletions.
4 changes: 4 additions & 0 deletions Mathlib/Combinatorics/SimpleGraph/Coloring.lean
Original file line number Diff line number Diff line change
Expand Up @@ -137,6 +137,10 @@ theorem isEmpty_of_colorable_zero (h : G.Colorable 0) : IsEmpty V := by
obtain ⟨i, hi⟩ := h.some v
exact Nat.not_lt_zero _ hi

@[simp]
lemma colorable_zero_iff : G.Colorable 0 ↔ IsEmpty V :=
fun h => G.isEmpty_of_colorable_zero h, fun _ => G.colorable_of_isEmpty 0

/-- The "tautological" coloring of a graph, using the vertices of the graph as colors. -/
def selfColoring : G.Coloring V := Coloring.mk id fun {_ _} => G.ne_of_adj

Expand Down

0 comments on commit 90f348a

Please sign in to comment.