mathlib3 documentation

combinatorics.simple_graph.hasse

The Hasse diagram as a graph #

THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.

This file defines the Hasse diagram of an order (graph of covby, the covering relation) and the path graph on n vertices.

Main declarations #

def simple_graph.hasse (α : Type u_1) [preorder α] :

The Hasse diagram of an order as a simple graph. The graph of the covering relation.

Equations
@[simp]
theorem simple_graph.hasse_adj {α : Type u_1} [preorder α] {a b : α} :
(simple_graph.hasse α).adj a b a b b a

The path graph on n vertices.

Equations