Functions over sets
Main definitions
Predicate
eq_on f₁ f₂ s
: functionsf₁
andf₂
are equal at every point ofs
;maps_to f s t
:f
sends every point ofs
to a point oft
;inj_on f s
: restriction off
tos
is injective;surj_on f s t
: every point ins
has a preimage ins
;bij_on f s t
:f
is a bijection betweens
andt
;left_inv_on f' f s
: for everyx ∈ s
we havef' (f x) = x
;right_inv_on f' f t
: for everyy ∈ t
we havef (f' y) = y
;inv_on f' f s t
:f'
is a two-side inverse off
ons
andt
, i.e. we haveleft_inv_on f' f s
andright_inv_on f' f t
.
Functions
restrict f s
: restrict the domain off
to the sets
;cod_restrict f s h
: givenh : ∀ x, f x ∈ s
, restrict the codomain off
to the sets
;maps_to.restrict f s t h
: givenh : maps_to f s t
, restrict the domain off
tos
and the codomain tot
.
Restrict
Restrict domain of a function f
to a set s
. Same as subtype.restrict
but this version
takes an argument ↥s
instead of subtype s
.
Equations
- set.restrict f s = λ (x : ↥s), f ↑x
Restrict codomain of a function f
to a set s
. Same as subtype.coind
but this version
has codomain ↥s
instead of subtype s
.
Equations
- set.cod_restrict f s h = λ (x : α), ⟨f x, _⟩
Equality on a set
maps to
maps_to f a b
means that the image of a
is contained in b
.
Equations
- set.maps_to f s t = ∀ ⦃x : α⦄, x ∈ s → f x ∈ t
Given a map f
sending s : set α
into t : set β
, restrict domain of f
to s
and the codomain to t
. Same as subtype.map
.
Equations
- set.maps_to.restrict f s t h = subtype.map f h
Injectivity on a set
f
is injective on a
if the restriction of f
to a
is injective.
Surjectivity on a set
f
is surjective from a
to b
if b
is contained in the image of a
.
Equations
- set.surj_on f s t = (t ⊆ f '' s)
Bijectivity
f
is bijective from s
to t
if f
is injective on s
and f '' s = t
.
Equations
- set.bij_on f s t = (set.maps_to f s t ∧ set.inj_on f s ∧ set.surj_on f s t)
left inverse
g
is a left inverse to f
on a
means that g (f x) = x
for all x ∈ a
.
Equations
- set.left_inv_on f' f s = ∀ ⦃x : α⦄, x ∈ s → f' (f x) = x
Right inverse
g
is a right inverse to f
on b
if f (g x) = x
for all x ∈ b
.
Equations
- set.right_inv_on f' f t = set.left_inv_on f f' t
Two-side inverses
g
is an inverse to f
viewed as a map from a
to b
Equations
- set.inv_on g f s t = (set.left_inv_on g f s ∧ set.right_inv_on g f t)