Skip to content

Commit

Permalink
Use instance of HAdd for +
Browse files Browse the repository at this point in the history
  • Loading branch information
IvanRenison committed Sep 18, 2024
1 parent 615909b commit 3d43f4c
Showing 1 changed file with 2 additions and 2 deletions.
4 changes: 2 additions & 2 deletions Mathlib/Combinatorics/SimpleGraph/Sum.lean
Original file line number Diff line number Diff line change
Expand Up @@ -39,8 +39,8 @@ protected def Sum (G : SimpleGraph α) (H : SimpleGraph β) : SimpleGraph (α
| Sum.inl _, Sum.inr _ | Sum.inr _, Sum.inl _ => id
loopless u := by cases u <;> simp

/-- Disjoint sum of `G` and `H`. -/
infixl:60 " + " => SimpleGraph.Sum
@[simps]
instance : HAdd (SimpleGraph α) (SimpleGraph β) (SimpleGraph (α ⊕ β)) := ⟨SimpleGraph.Sum

variable {G : SimpleGraph α} {H : SimpleGraph β}

Expand Down

0 comments on commit 3d43f4c

Please sign in to comment.