File tree Expand file tree Collapse file tree 1 file changed +4
-4
lines changed
Mathlib/Combinatorics/SimpleGraph/Connectivity Expand file tree Collapse file tree 1 file changed +4
-4
lines changed Original file line number Diff line number Diff line change @@ -332,10 +332,10 @@ namespace ConnectedComponent
332332instance inhabited [Inhabited V] : Inhabited G.ConnectedComponent :=
333333 ⟨G.connectedComponentMk default⟩
334334
335- instance isEmpty [IsEmpty V] : IsEmpty ( ConnectedComponent G) := by
336- by_contra! hc
337- obtain ⟨v, _⟩ := hc.some.exists_rep
338- exact IsEmpty. false v
335+ instance isEmpty [IsEmpty V] : IsEmpty G. ConnectedComponent := Quot.instIsEmpty
336+ instance [Subsingleton V] : Subsingleton G.ConnectedComponent := Quot.Subsingleton
337+ instance [Unique V] : Unique G.ConnectedComponent := Quot.instUnique
338+ instance [Nonempty V] : Nonempty G.ConnectedComponent := Nonempty.map G.connectedComponentMk ‹_›
339339
340340@[elab_as_elim]
341341protected theorem ind {β : G.ConnectedComponent → Prop }
You can’t perform that action at this time.
0 commit comments