Injective functions
- to_fun : α → β
- inj' : function.injective c.to_fun
α ↪ β
is a bundled injective function.
Equations
- function.has_coe_to_fun = {F := λ (x : α ↪ β), α → β, coe := function.embedding.to_fun β}
Convert an α ≃ β
to α ↪ β
.
Equations
- function.embedding.congr e₁ e₂ f = e₁.symm.to_embedding.trans (f.trans e₂.to_embedding)
A right inverse surj_inv
of a surjective function as an embedding
.
Equations
- function.embedding.of_surjective f hf = {to_fun := function.surj_inv hf, inj' := _}
Convert a surjective embedding
to an equiv
Equations
- f.equiv_of_surjective hf = equiv.of_bijective ⇑f _
Change the value of an embedding f
at one point. If the prescribed image
is already occupied by some f a'
, then swap the values at these two points.
Embedding into option
Equations
- function.embedding.some = {to_fun := option.some α, inj' := _}
Embedding of a subtype
.
Equations
- function.embedding.subtype p = {to_fun := coe coe_to_lift, inj' := _}
Fixing an element b : β
gives an embedding α ↪ α × β
.
Equations
- function.embedding.sectl α b = {to_fun := λ (a : α), (a, b), inj' := _}
Fixing an element a : α
gives an embedding β ↪ α × β
.
Equations
- function.embedding.sectr a β = {to_fun := λ (b : β), (a, b), inj' := _}
The embedding of α
into the sum α ⊕ β
.
The embedding of β
into the sum α ⊕ β
.
sigma.mk
as an function.embedding
.
If f : α ↪ α'
is an embedding and g : Π a, β α ↪ β' (f α)
is a family
of embeddings, then sigma.map f g
is an embedding.
Equations
- e.arrow_congr_left = function.embedding.Pi_congr_right (λ (_x : γ), e)
Equations
- e.arrow_congr_right = let f' : (α → γ) → β → γ := λ (f : α → γ) (b : β), dite (∃ (c : α), ⇑e c = b) (λ (h : ∃ (c : α), ⇑e c = b), f (classical.some h)) (λ (h : ¬∃ (c : α), ⇑e c = b), inhabited.default γ) in {to_fun := f', inj' := _}
Equations
- f.subtype_map h = {to_fun := subtype.map ⇑f h, inj' := _}
The embedding of a left cancellative semigroup into itself by left multiplication by a fixed element.
The embedding of a left cancellative additive semigroup into itself by left translation by a fixed element.
The embedding of a right cancellative additive semigroup into itself by right translation by a fixed element.
The embedding of a right cancellative semigroup into itself by right multiplication by a fixed element.