structure
Rel.Functional
{α : Type u_1}
{β : Type u_2}
(r : Rel α β)
extends r.Coinjective, r.Cosurjective :
Instances For
structure
Rel.Cofunctional
{α : Type u_1}
{β : Type u_2}
(r : Rel α β)
extends r.Injective, r.Surjective :
Instances For
structure
Rel.OneOne
{α : Type u_1}
{β : Type u_2}
(r : Rel α β)
extends r.Injective, r.Coinjective :
Instances For
structure
Rel.Bijective
{α : Type u_1}
{β : Type u_2}
(r : Rel α β)
extends r.Functional, r.Cofunctional :
Instances For
Instances For
theorem
Rel.CodomEqDom.mem_dom
{α : Type u_1}
{r : Rel α α}
(h : r.CodomEqDom)
{x y : α}
(hxy : r x y)
:
theorem
Rel.CodomEqDom.mem_codom
{α : Type u_1}
{r : Rel α α}
(h : r.CodomEqDom)
{x y : α}
(hxy : r x y)
:
An elementary description of the property CodomEqDom
.
@[simp]
@[simp]
@[simp]
@[simp]
@[simp]
@[simp]
theorem
Rel.Coinjective.comp
{α : Type u_1}
{β : Type u_2}
{γ : Type u_3}
{r : Rel α β}
{s : Rel β γ}
(hr : r.Coinjective)
(hs : s.Coinjective)
:
(r.comp s).Coinjective
theorem
Rel.Coinjective.mono
{α : Type u_1}
{β : Type u_2}
{r s : Rel α β}
(hs : s.Coinjective)
(h : r ≤ s)
:
An alternative spelling of Rel.graph
that is useful for proving inequalities of cardinals.
Equations
- r.graph' = Function.uncurry r
Instances For
theorem
Rel.sup_coinjective
{α : Type u_1}
{β : Type u_2}
{r s : Rel α β}
(hr : r.Coinjective)
(hs : s.Coinjective)
(h : Disjoint r.dom s.dom)
:
(r ⊔ s).Coinjective
theorem
Rel.sup_codomEqDom
{α : Type u_1}
{r s : Rel α α}
(hr : r.CodomEqDom)
(hs : s.CodomEqDom)
:
(r ⊔ s).CodomEqDom
theorem
Rel.sup_permutative
{α : Type u_1}
{r s : Rel α α}
(hr : r.Permutative)
(hs : s.Permutative)
(h : Disjoint r.dom s.dom)
:
(r ⊔ s).Permutative
theorem
Rel.iSup_coinjective_of_isChain
{α : Type u_2}
{β : Type u_3}
{T : Type u_1}
{r : T → Rel α β}
(h₁ : ∀ (t : T), (r t).Coinjective)
(h₂ : IsChain (fun (x1 x2 : Rel α β) => x1 ≤ x2) (Set.range r))
:
(⨆ (t : T), r t).Coinjective
theorem
Rel.iSup_codomEqDom_of_isChain
{α : Type u_2}
{T : Type u_1}
{r : T → Rel α α}
(h : ∀ (t : T), (r t).CodomEqDom)
:
(⨆ (t : T), r t).CodomEqDom
theorem
Rel.iSup_permutative_of_isChain
{α : Type u_2}
{T : Type u_1}
{r : T → Rel α α}
(h₁ : ∀ (t : T), (r t).Permutative)
(h₂ : IsChain (fun (x1 x2 : Rel α α) => x1 ≤ x2) (Set.range r))
:
(⨆ (t : T), r t).Permutative
theorem
Rel.biSup_permutative_of_isChain
{α : Type u_2}
{T : Type u_1}
{r : T → Rel α α}
{s : Set T}
(h₁ : ∀ t ∈ s, (r t).Permutative)
(h₂ : IsChain (fun (x1 x2 : Rel α α) => x1 ≤ x2) (r '' s))
:
(⨆ t ∈ s, r t).Permutative
noncomputable def
Rel.toFunction
{α : Type u_1}
{β : Type u_2}
(r : Rel α β)
(hr : r.Functional)
:
α → β
Equations
- r.toFunction hr a = ⋯.choose
Instances For
theorem
Rel.toFunction_rel
{α : Type u_1}
{β : Type u_2}
(r : Rel α β)
(hr : r.Functional)
(a : α)
:
r a (r.toFunction hr a)
theorem
Rel.toFunction_eq_iff
{α : Type u_1}
{β : Type u_2}
(r : Rel α β)
(hr : r.Functional)
(a : α)
(b : β)
:
Equations
- r.toEquiv hr = { toFun := r.toFunction ⋯, invFun := r.inv.toFunction ⋯, left_inv := ⋯, right_inv := ⋯ }
Instances For
theorem
Rel.toFunction_image
{α : Type u_1}
{β : Type u_2}
(r : Rel α β)
(hr : r.Functional)
(s : Set α)
: