We read every piece of feedback, and take your input very seriously.
To see all available qualifiers, see our documentation.
Repr
Sym2
1 parent e242f1e commit 529a610Copy full SHA for 529a610
Mathlib/Data/Sym/Sym2.lean
@@ -765,4 +765,8 @@ instance [IsEmpty α] : IsEmpty (Sym2 α) :=
765
instance [Nontrivial α] : Nontrivial (Sym2 α) :=
766
diag_injective.nontrivial
767
768
+-- TODO: use a sort order if available, https://github.com/leanprover-community/mathlib/issues/18166
769
+unsafe instance [Repr α] : Repr (Sym2 α) where
770
+ reprPrec s _ := f!"s({repr s.unquot.1}, {repr s.unquot.2})"
771
+
772
end Sym2
0 commit comments