@[instance]
Restrict the domain of a relation to a subtype.
Equations
- r.restrict_domain s = λ (x : {x // x ∈ s}) (y : β), r x.val y
The graph of a function as a relation.
Equations
- function.graph f = λ (x : α) (y : β), f x = y
theorem
set.image_eq
{α : Type u_1}
{β : Type u_2}
(f : α → β)
(s : set α) :
f '' s = (function.graph f).image s
theorem
set.preimage_eq
{α : Type u_1}
{β : Type u_2}
(f : α → β)
(s : set β) :
f ⁻¹' s = (function.graph f).preimage s
theorem
set.preimage_eq_core
{α : Type u_1}
{β : Type u_2}
(f : α → β)
(s : set β) :
f ⁻¹' s = (function.graph f).core s