Documentation

Mathlib.Combinatorics.SimpleGraph.DeleteEdges

Edge deletion #

This file defines operations deleting the edges of a simple graph and proves theorems in the finite case.

Main definitions #

def SimpleGraph.deleteEdges {V : Type u_1} (G : SimpleGraph V) (s : Set (Sym2 V)) :

Given a set of vertex pairs, remove all of the corresponding edges from the graph's edge set, if present.

See also: SimpleGraph.Subgraph.deleteEdges.

Equations
Instances For
    @[simp]
    theorem SimpleGraph.deleteEdges_adj {V : Type u_1} {v w : V} {G : SimpleGraph V} {s : Set (Sym2 V)} :
    (G.deleteEdges s).Adj v w G.Adj v w s(v, w)s
    @[simp]
    theorem SimpleGraph.deleteEdges_edgeSet {V : Type u_1} (G G' : SimpleGraph V) :
    @[simp]
    theorem SimpleGraph.deleteEdges_deleteEdges {V : Type u_1} {G : SimpleGraph V} (s s' : Set (Sym2 V)) :
    @[simp]
    theorem SimpleGraph.deleteEdges_le {V : Type u_1} {G : SimpleGraph V} (s : Set (Sym2 V)) :
    theorem SimpleGraph.deleteEdges_anti {V : Type u_1} {G : SimpleGraph V} {s₁ s₂ : Set (Sym2 V)} (h : s₁ s₂) :
    theorem SimpleGraph.deleteEdges_mono {V : Type u_1} {G H : SimpleGraph V} {s : Set (Sym2 V)} (h : G H) :
    @[simp]
    theorem SimpleGraph.deleteEdges_eq_self {V : Type u_1} {G : SimpleGraph V} {s : Set (Sym2 V)} :
    def SimpleGraph.DeleteFar {V : Type u_1} (G : SimpleGraph V) {𝕜 : Type u_2} [Ring 𝕜] [PartialOrder 𝕜] [Fintype G.edgeSet] (p : SimpleGraph VProp) (r : 𝕜) :

    A graph is r-delete-far from a property p if we must delete at least r edges from it to get a graph with the property p.

    Equations
    Instances For
      theorem SimpleGraph.deleteFar_iff {V : Type u_1} {G : SimpleGraph V} {𝕜 : Type u_2} [Ring 𝕜] [PartialOrder 𝕜] [Fintype G.edgeSet] {p : SimpleGraph VProp} {r : 𝕜} [Fintype (Sym2 V)] :
      G.DeleteFar p r ∀ ⦃H : SimpleGraph V⦄ [inst : DecidableRel H.Adj], H Gp Hr G.edgeFinset.card - H.edgeFinset.card
      theorem SimpleGraph.DeleteFar.le_card_sub_card {V : Type u_1} {G : SimpleGraph V} {𝕜 : Type u_2} [Ring 𝕜] [PartialOrder 𝕜] [Fintype G.edgeSet] {p : SimpleGraph VProp} {r : 𝕜} [Fintype (Sym2 V)] :
      G.DeleteFar p r∀ ⦃H : SimpleGraph V⦄ [inst : DecidableRel H.Adj], H Gp Hr G.edgeFinset.card - H.edgeFinset.card

      Alias of the forward direction of SimpleGraph.deleteFar_iff.

      theorem SimpleGraph.DeleteFar.mono {V : Type u_1} {G : SimpleGraph V} {𝕜 : Type u_2} [Ring 𝕜] [PartialOrder 𝕜] [Fintype G.edgeSet] {p : SimpleGraph VProp} {r₁ r₂ : 𝕜} (h : G.DeleteFar p r₂) (hr : r₁ r₂) :
      G.DeleteFar p r₁