Relations holding pairwise #
This file defines pairwise relations.
Main declarations #
Pairwise
:Pairwise r
states thatr i j
for alli ≠ j
.Set.Pairwise
:s.Pairwise r
states thatr i j
for alli ≠ j
withi, j ∈ s
.
Alias of the forward direction of Function.injective_iff_pairwise_ne
.
theorem
Pairwise.comp_of_injective
{α : Type u_1}
{β : Type u_2}
{r : α → α → Prop}
(hr : Pairwise r)
{f : β → α}
(hf : Function.Injective f)
:
Pairwise (Function.onFun r f)
theorem
Pairwise.of_comp_of_surjective
{α : Type u_1}
{β : Type u_2}
{r : α → α → Prop}
{f : β → α}
(hr : Pairwise (Function.onFun r f))
(hf : Function.Surjective f)
:
Pairwise r
theorem
Set.Pairwise.on_injective
{α : Type u_1}
{ι : Type u_3}
{r : α → α → Prop}
{f : ι → α}
{s : Set α}
(hs : s.Pairwise r)
(hf : Function.Injective f)
(hfs : ∀ (x : ι), f x ∈ s)
:
Pairwise (Function.onFun r f)