Documentation

Mathlib.Combinatorics.SimpleGraph.LapMatrix

Laplacian Matrix #

This module defines the Laplacian matrix of a graph, and proves some of its elementary properties.

Main definitions & Results #

def SimpleGraph.degMatrix {V : Type u_1} (R : Type u_2) [Fintype V] [DecidableEq V] (G : SimpleGraph V) [DecidableRel G.Adj] [AddMonoidWithOne R] :
Matrix V V R

The diagonal matrix consisting of the degrees of the vertices in the graph.

Equations
Instances For
    def SimpleGraph.lapMatrix {V : Type u_1} (R : Type u_2) [Fintype V] [DecidableEq V] (G : SimpleGraph V) [DecidableRel G.Adj] [AddGroupWithOne R] :
    Matrix V V R

    The Laplacian matrix lapMatrix G R of a graph G is the matrix L = D - A where D is the degree and A the adjacency matrix of G.

    Equations
    Instances For
      theorem SimpleGraph.degMatrix_mulVec_apply {V : Type u_1} {R : Type u_2} [Fintype V] [DecidableEq V] (G : SimpleGraph V) [DecidableRel G.Adj] [NonAssocSemiring R] (v : V) (vec : VR) :
      (SimpleGraph.degMatrix R G).mulVec vec v = (G.degree v) * vec v
      theorem SimpleGraph.lapMatrix_mulVec_apply {V : Type u_1} {R : Type u_2} [Fintype V] [DecidableEq V] (G : SimpleGraph V) [DecidableRel G.Adj] [NonAssocRing R] (v : V) (vec : VR) :
      (SimpleGraph.lapMatrix R G).mulVec vec v = (G.degree v) * vec v - uG.neighborFinset v, vec u
      theorem SimpleGraph.lapMatrix_mulVec_const_eq_zero {V : Type u_1} {R : Type u_2} [Fintype V] [DecidableEq V] (G : SimpleGraph V) [DecidableRel G.Adj] [Ring R] :
      ((SimpleGraph.lapMatrix R G).mulVec fun (x : V) => 1) = 0
      theorem SimpleGraph.dotProduct_mulVec_degMatrix {V : Type u_1} {R : Type u_2} [Fintype V] [DecidableEq V] (G : SimpleGraph V) [DecidableRel G.Adj] [CommRing R] (x : VR) :
      Matrix.dotProduct x ((SimpleGraph.degMatrix R G).mulVec x) = i : V, (G.degree i) * x i * x i
      theorem SimpleGraph.degree_eq_sum_if_adj {V : Type u_1} (R : Type u_2) [Fintype V] (G : SimpleGraph V) [DecidableRel G.Adj] [AddCommMonoidWithOne R] (i : V) :
      (G.degree i) = j : V, if G.Adj i j then 1 else 0
      theorem SimpleGraph.lapMatrix_toLinearMap₂' {V : Type u_1} (R : Type u_2) [Fintype V] [DecidableEq V] (G : SimpleGraph V) [DecidableRel G.Adj] [Field R] [CharZero R] (x : VR) :
      ((Matrix.toLinearMap₂' (SimpleGraph.lapMatrix R G)) x) x = (i : V, j : V, if G.Adj i j then (x i - x j) ^ 2 else 0) / 2

      Let $L$ be the graph Laplacian and let $x \in \mathbb{R}$, then $$x^{\top} L x = \sum_{i \sim j} (x_{i}-x_{j})^{2}$$, where $\sim$ denotes the adjacency relation

      The Laplacian matrix is positive semidefinite

      theorem SimpleGraph.lapMatrix_toLinearMap₂'_apply'_eq_zero_iff_forall_adj {V : Type u_1} (R : Type u_2) [Fintype V] [DecidableEq V] (G : SimpleGraph V) [DecidableRel G.Adj] [LinearOrderedField R] (x : VR) :
      ((Matrix.toLinearMap₂' (SimpleGraph.lapMatrix R G)) x) x = 0 ∀ (i j : V), G.Adj i jx i = x j
      theorem SimpleGraph.lapMatrix_toLin'_apply_eq_zero_iff_forall_adj {V : Type u_1} [Fintype V] [DecidableEq V] (G : SimpleGraph V) [DecidableRel G.Adj] (x : V) :
      (Matrix.toLin' (SimpleGraph.lapMatrix G)) x = 0 ∀ (i j : V), G.Adj i jx i = x j
      theorem SimpleGraph.lapMatrix_toLinearMap₂'_apply'_eq_zero_iff_forall_reachable {V : Type u_1} [Fintype V] [DecidableEq V] (G : SimpleGraph V) [DecidableRel G.Adj] (x : V) :
      ((Matrix.toLinearMap₂' (SimpleGraph.lapMatrix G)) x) x = 0 ∀ (i j : V), G.Reachable i jx i = x j
      theorem SimpleGraph.lapMatrix_toLin'_apply_eq_zero_iff_forall_reachable {V : Type u_1} [Fintype V] [DecidableEq V] (G : SimpleGraph V) [DecidableRel G.Adj] (x : V) :
      (Matrix.toLin' (SimpleGraph.lapMatrix G)) x = 0 ∀ (i j : V), G.Reachable i jx i = x j
      theorem SimpleGraph.mem_ker_toLin'_lapMatrix_of_connectedComponent {V : Type u_1} [Fintype V] [DecidableEq V] {G : SimpleGraph V} [DecidableRel G.Adj] [DecidableEq G.ConnectedComponent] (c : G.ConnectedComponent) :
      (fun (i : V) => if G.connectedComponentMk i = c then 1 else 0) LinearMap.ker (Matrix.toLin' (SimpleGraph.lapMatrix G))
      def SimpleGraph.lapMatrix_ker_basis_aux {V : Type u_1} [Fintype V] [DecidableEq V] (G : SimpleGraph V) [DecidableRel G.Adj] [DecidableEq G.ConnectedComponent] (c : G.ConnectedComponent) :
      (LinearMap.ker (Matrix.toLin' (SimpleGraph.lapMatrix G)))

      Given a connected component c of a graph G, lapMatrix_ker_basis_aux c is the map V → ℝ which is 1 on the vertices in c and 0 elsewhere. The family of these maps indexed by the connected components of G proves to be a basis of the kernel of lapMatrix G R

      Equations
      • G.lapMatrix_ker_basis_aux c = fun (i : V) => if G.connectedComponentMk i = c then 1 else 0,
      Instances For
        theorem SimpleGraph.linearIndependent_lapMatrix_ker_basis_aux {V : Type u_1} [Fintype V] [DecidableEq V] (G : SimpleGraph V) [DecidableRel G.Adj] [DecidableEq G.ConnectedComponent] :
        LinearIndependent G.lapMatrix_ker_basis_aux
        theorem SimpleGraph.top_le_span_range_lapMatrix_ker_basis_aux {V : Type u_1} [Fintype V] [DecidableEq V] (G : SimpleGraph V) [DecidableRel G.Adj] [DecidableEq G.ConnectedComponent] :
        Submodule.span (Set.range G.lapMatrix_ker_basis_aux)
        noncomputable def SimpleGraph.lapMatrix_ker_basis {V : Type u_1} [Fintype V] [DecidableEq V] (G : SimpleGraph V) [DecidableRel G.Adj] [DecidableEq G.ConnectedComponent] :
        Basis G.ConnectedComponent (LinearMap.ker (Matrix.toLin' (SimpleGraph.lapMatrix G)))

        lapMatrix_ker_basis G is a basis of the nullspace indexed by its connected components, the basis is made up of the functions V → ℝ which are 1 on the vertices of the given connected component and 0 elsewhere.

        Equations
        Instances For

          The number of connected components in G is the dimension of the nullspace its Laplacian.