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 #
simple_graph.hasse
: Hasse diagram of an order.simple_graph.path_graph
: Path graph onn
vertices.
The Hasse diagram of an order as a simple graph. The graph of the covering relation.
@[simp]
αᵒᵈ
and α
have the same Hasse diagram.
Equations
- simple_graph.hasse_dual_iso = {to_equiv := {to_fun := order_dual.of_dual.to_fun, inv_fun := order_dual.of_dual.inv_fun, left_inv := _, right_inv := _}, map_rel_iff' := _}
@[simp]
@[simp]
@[simp]
theorem
simple_graph.hasse_prod
(α : Type u_1)
(β : Type u_2)
[partial_order α]
[partial_order β] :
simple_graph.hasse (α × β) = simple_graph.hasse α □ simple_graph.hasse β
theorem
simple_graph.hasse_preconnected_of_succ
(α : Type u_1)
[linear_order α]
[succ_order α]
[is_succ_archimedean α] :
theorem
simple_graph.hasse_preconnected_of_pred
(α : Type u_1)
[linear_order α]
[pred_order α]
[is_pred_archimedean α] :
The path graph on n
vertices.