Documentation

Mathlib.Logic.Embedding.Set

Interactions between embeddings and sets. #

@[simp]
theorem Equiv.asEmbedding_range {α : Sort u_1} {β : Type u_2} {p : βProp} (e : α Subtype p) :
def Function.Embedding.optionElim {α : Type u_1} {β : Type u_2} (f : α β) (x : β) (h : xSet.range f) :
Option α β

Given an embedding f : α ↪ β and a point outside of Set.range f, construct an embedding Option α ↪ β.

Equations
@[simp]
theorem Function.Embedding.optionElim_apply {α : Type u_1} {β : Type u_2} (f : α β) (x : β) (h : xSet.range f) (a✝ : Option α) :
(f.optionElim x h) a✝ = Option.elim' x (⇑f) a✝
def Function.Embedding.optionEmbeddingEquiv (α : Type u_1) (β : Type u_2) :
(Option α β) (f : α β) × (Set.range f)

Equivalence between embeddings of Option α and a sigma type over the embeddings of α.

Equations
  • One or more equations did not get rendered due to their size.
@[simp]
theorem Function.Embedding.optionEmbeddingEquiv_symm_apply (α : Type u_1) (β : Type u_2) (f : (f : α β) × (Set.range f)) :
@[simp]
@[simp]
theorem Function.Embedding.optionEmbeddingEquiv_apply_snd_coe (α : Type u_1) (β : Type u_2) (f : Option α β) :
((optionEmbeddingEquiv α β) f).snd = f none
def Function.Embedding.codRestrict {α : Sort u_1} {β : Type u_2} (p : Set β) (f : α β) (H : ∀ (a : α), f a p) :
α p

Restrict the codomain of an embedding.

Equations
@[simp]
theorem Function.Embedding.codRestrict_apply {α : Sort u_1} {β : Type u_2} (p : Set β) (f : α β) (H : ∀ (a : α), f a p) (a : α) :
(codRestrict p f H) a = f a,
def Function.Embedding.image {α : Type u_1} {β : Type u_2} (f : α β) :
Set α Set β

Set.image as an embedding Set α ↪ Set β.

Equations
@[simp]
theorem Function.Embedding.image_apply {α : Type u_1} {β : Type u_2} (f : α β) (s : Set α) :
f.image s = f '' s
def Set.embeddingOfSubset {α : Type u_1} (s t : Set α) (h : s t) :
s t

The injection map is an embedding between subsets.

Equations
@[simp]
theorem Set.embeddingOfSubset_apply_coe {α : Type u_1} (s t : Set α) (h : s t) (x : s) :
((s.embeddingOfSubset t h) x) = x
def subtypeOrEquiv {α : Type u_1} (p q : αProp) [DecidablePred p] (h : Disjoint p q) :
{ x : α // p x q x } { x : α // p x } { x : α // q x }

A subtype {x // p x ∨ q x} over a disjunction of p q : α → Prop is equivalent to a sum of subtypes {x // p x} ⊕ {x // q x} such that ¬ p x is sent to the right, when Disjoint p q.

See also Equiv.sumCompl, for when IsCompl p q.

Equations
  • One or more equations did not get rendered due to their size.
@[simp]
theorem subtypeOrEquiv_apply {α : Type u_1} (p q : αProp) [DecidablePred p] (h : Disjoint p q) (a : { x : α // p x q x }) :
@[simp]
theorem subtypeOrEquiv_symm_inl {α : Type u_1} (p q : αProp) [DecidablePred p] (h : Disjoint p q) (x : { x : α // p x }) :
(subtypeOrEquiv p q h).symm (Sum.inl x) = x,
@[simp]
theorem subtypeOrEquiv_symm_inr {α : Type u_1} (p q : αProp) [DecidablePred p] (h : Disjoint p q) (x : { x : α // q x }) :
(subtypeOrEquiv p q h).symm (Sum.inr x) = x,
def Function.Embedding.sumSet {α : Type u_1} {s t : Set α} (h : Disjoint s t) :
s t α

For disjoint s t : Set α, the natural injection from ↑s ⊕ ↑t to α.

Equations
@[simp]
theorem Function.Embedding.sumSet_apply {α : Type u_1} {s t : Set α} (h : Disjoint s t) (a✝ : s t) :
@[simp]
theorem Function.Embedding.sumSet_preimage_inl {α : Type u_1} {s t r : Set α} (h : Disjoint s t) :
@[simp]
theorem Function.Embedding.sumSet_preimage_inr {α : Type u_1} {s t r : Set α} (h : Disjoint s t) :
@[simp]
theorem Function.Embedding.sumSet_range {α : Type u_1} {s t : Set α} (h : Disjoint s t) :
Set.range (sumSet h) = s t
def Function.Embedding.sigmaSet {α : Type u_1} {ι : Type u_2} {s : ιSet α} (h : Pairwise (onFun Disjoint s)) :
(i : ι) × (s i) α

For an indexed family s : ι → Set α of disjoint sets, the natural injection from the sigma-type (i : ι) × ↑(s i) to α.

Equations
@[simp]
theorem Function.Embedding.sigmaSet_apply {α : Type u_1} {ι : Type u_2} {s : ιSet α} (h : Pairwise (onFun Disjoint s)) (x : (i : ι) × (s i)) :
(sigmaSet h) x = x.snd
theorem Function.Embedding.coe_sigmaSet {α : Type u_1} {ι : Type u_2} {s : ιSet α} (h : Pairwise (onFun Disjoint s)) :
(sigmaSet h) = fun (x : (i : ι) × (s i)) => x.snd
@[simp]
theorem Function.Embedding.sigmaSet_preimage {α : Type u_1} {ι : Type u_2} {s : ιSet α} (h : Pairwise (onFun Disjoint s)) (i : ι) (r : Set α) :
@[simp]
theorem Function.Embedding.sigmaSet_range {α : Type u_1} {ι : Type u_2} {s : ιSet α} (h : Pairwise (onFun Disjoint s)) :
Set.range (sigmaSet h) = ⋃ (i : ι), s i