Ends #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
This file contains a definition of the ends of a simple graph, as sections of the inverse system assigning, to each finite set of vertices, the connected components of its complement.
The components outside a given set of vertices K
Equations
The connected component of v
in G.induce Kᶜ
.
Equations
- G.component_compl_mk vK = (simple_graph.induce Kᶜ G).connected_component_mk ⟨v, vK⟩
The set of vertices of G
making up the connected component C
Equations
A component_compl
specialization of quot.lift
, where soundness has to be proved only
for adjacent vertices.
Equations
- simple_graph.component_compl.lift f h = simple_graph.connected_component.lift (λ (vv : ↥Kᶜ), f _) _
The induced graph on the vertices C
.
Equations
- C.coe_graph = simple_graph.induce ↑C G
Any vertex adjacent to a vertex of C
and not lying in K
must lie in C
.
Assuming G
is preconnected and K
not empty, given any connected component C
outside of K
,
there exists a vertex k ∈ K
adjacent to a vertex v ∈ C
.
If K ⊆ L
, the components outside of L
are all contained in a single component outside of K
.
The functor assigning, to a finite set in V
, the set of connected components in its complement.
Equations
- G.component_compl_functor = {obj := λ (K : (finset V)ᵒᵖ), G.component_compl ↑(opposite.unop K), map := λ (_x _x_1 : (finset V)ᵒᵖ) (f : _x ⟶ _x_1), simple_graph.component_compl.hom _, map_id' := _, map_comp' := _}
The end of a graph, defined as the sections of the functor component_compl_functor
.