Commit 2022-12-23 16:03 d90ae095
View on Github →chore: move basic lemmas to basic files (#1109)
synchronize with https://github.com/leanprover-community/mathlib/pull/17882
Make
Removing disjoint_singleton
@[simp 1100]
because the linter complains it is not in simpNF (because of disjoint_singleton_left
and disjoint_singleton_right
).simp
of disjoint_singleton
, making disjoint_singleton_left
have a greater priority than disjoint_singleton_right
, then disjoint_singleton
can be proved by simp
.