Skip to content

Commit 6563fa2

Browse files
committed
feat: the graph made of all non-diag edges is complete (#31443)
1 parent afa82c7 commit 6563fa2

File tree

1 file changed

+2
-0
lines changed

1 file changed

+2
-0
lines changed

Mathlib/Combinatorics/SimpleGraph/Basic.lean

Lines changed: 2 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -602,6 +602,8 @@ theorem fromEdgeSet_empty : fromEdgeSet (∅ : Set (Sym2 V)) = ⊥ := by
602602
ext v w
603603
simp only [fromEdgeSet_adj, Set.mem_empty_iff_false, false_and, bot_adj]
604604

605+
@[simp] lemma fromEdgeSet_not_isDiag : fromEdgeSet {e : Sym2 V | ¬ e.IsDiag} = ⊤ := by ext; simp
606+
605607
@[simp]
606608
theorem fromEdgeSet_univ : fromEdgeSet (Set.univ : Set (Sym2 V)) = ⊤ := by
607609
ext v w

0 commit comments

Comments
 (0)