Documentation

Mathlib.Combinatorics.SimpleGraph.Connectivity.Represents

Representation of components by a set of vertices #

Main definition #

A set of vertices represents a set of components if it contains exactly one vertex from each component.

Equations
Instances For
    theorem SimpleGraph.ConnectedComponent.Represents.exists_inter_eq_singleton {V : Type u} {G : SimpleGraph V} {C : Set G.ConnectedComponent} {s : Set V} {c : G.ConnectedComponent} (hrep : Represents s C) (h : c C) :
    ∃ (x : V), s c.supp = {x}