File tree Expand file tree Collapse file tree 1 file changed +6
-0
lines changed
Mathlib/Combinatorics/SimpleGraph Expand file tree Collapse file tree 1 file changed +6
-0
lines changed Original file line number Diff line number Diff line change @@ -148,6 +148,9 @@ def edge : SimpleGraph V := fromEdgeSet {s(s, t)}
148148lemma edge_adj (v w : V) : (edge s t).Adj v w ↔ (v = s ∧ w = t ∨ v = t ∧ w = s) ∧ v ≠ w := by
149149 rw [edge, fromEdgeSet_adj, Set.mem_singleton_iff, Sym2.eq_iff]
150150
151+ lemma edge_comm : edge s t = edge t s := by
152+ rw [edge, edge, Sym2.eq_swap]
153+
151154variable [DecidableEq V] in
152155instance : DecidableRel (edge s t).Adj := fun _ _ ↦ by
153156 rw [edge_adj]; infer_instance
@@ -159,6 +162,9 @@ lemma edge_self_eq_bot : edge s s = ⊥ := by
159162lemma sup_edge_self : G ⊔ edge s s = G := by
160163 rw [edge_self_eq_bot, sup_of_le_left bot_le]
161164
165+ lemma lt_sup_edge (hne : s ≠ t) (hn : ¬ G.Adj s t) : G < G ⊔ edge s t :=
166+ left_lt_sup.2 fun h ↦ hn <| h <| (edge_adj ..).mpr ⟨Or.inl ⟨rfl, rfl⟩, hne⟩
167+
162168variable {s t}
163169
164170lemma edge_edgeSet_of_ne (h : s ≠ t) : (edge s t).edgeSet = {s(s, t)} := by
You can’t perform that action at this time.
0 commit comments