Lemmas about insertion, singleton, and pairs #
This file provides extra lemmas about insert
, singleton
, and pair
.
Tags #
insert, singleton
Set coercion to a type #
Lemmas about insert
#
insert α s
is the set {α} ∪ s
.
Inserting an element to a set is equivalent to the option type.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Lemmas about singletons #
Alias of the reverse direction of Set.singleton_subset_singleton
.
Equations
- Set.uniqueSingleton a = { default := ⟨a, ⋯⟩, uniq := ⋯ }
theorem
Set.eq_of_nonempty_of_subsingleton
{α : Type u_1}
[Subsingleton α]
(s t : Set α)
[Nonempty ↑s]
[Nonempty ↑t]
:
theorem
Set.eq_of_nonempty_of_subsingleton'
{α : Type u_1}
[Subsingleton α]
{s : Set α}
(t : Set α)
(hs : s.Nonempty)
[Nonempty ↑t]
:
Disjointness #
Lemmas about complement #
@[simp]
Lemmas about set difference #
Lemmas about pairs #
Powerset #
Lemmas about inclusion
, the injection of subtypes induced by ⊆
#
Decidability instances for sets #
Equations
- Set.decidableSingleton a b = inferInstanceAs (Decidable (a = b))