mathlib documentation

data.​pequiv

data.​pequiv

structure pequiv  :
Type uType vType (max u v)

A pequiv is a partial equivalence, a representation of a bijection between a subset of α and a subset of β

@[instance]
def pequiv.​has_coe_to_fun {α : Type u} {β : Type v} :

Equations
@[simp]
theorem pequiv.​coe_mk_apply {α : Type u} {β : Type v} (f₁ : α → option β) (f₂ : β → option α) (h : ∀ (a : α) (b : β), a f₂ b b f₁ a) (x : α) :
{to_fun := f₁, inv_fun := f₂, inv := h} x = f₁ x

@[ext]
theorem pequiv.​ext {α : Type u} {β : Type v} {f g : α ≃. β} :
(∀ (x : α), f x = g x)f = g

theorem pequiv.​ext_iff {α : Type u} {β : Type v} {f g : α ≃. β} :
f = g ∀ (x : α), f x = g x

def pequiv.​refl (α : Type u_1) :
α ≃. α

Equations
def pequiv.​symm {α : Type u} {β : Type v} :
≃. β)β ≃. α

Equations
theorem pequiv.​mem_iff_mem {α : Type u} {β : Type v} (f : α ≃. β) {a : α} {b : β} :
a (f.symm) b b f a

theorem pequiv.​eq_some_iff {α : Type u} {β : Type v} (f : α ≃. β) {a : α} {b : β} :

def pequiv.​trans {α : Type u} {β : Type v} {γ : Type w} :
≃. β)≃. γ)α ≃. γ

Equations
@[simp]
theorem pequiv.​refl_apply {α : Type u} (a : α) :

@[simp]
theorem pequiv.​symm_refl {α : Type u} :

@[simp]
theorem pequiv.​symm_symm {α : Type u} {β : Type v} (f : α ≃. β) :
f.symm.symm = f

theorem pequiv.​symm_injective {α : Type u} {β : Type v} :

theorem pequiv.​trans_assoc {α : Type u} {β : Type v} {γ : Type w} {δ : Type x} (f : α ≃. β) (g : β ≃. γ) (h : γ ≃. δ) :
(f.trans g).trans h = f.trans (g.trans h)

theorem pequiv.​mem_trans {α : Type u} {β : Type v} {γ : Type w} (f : α ≃. β) (g : β ≃. γ) (a : α) (c : γ) :
c (f.trans g) a ∃ (b : β), b f a c g b

theorem pequiv.​trans_eq_some {α : Type u} {β : Type v} {γ : Type w} (f : α ≃. β) (g : β ≃. γ) (a : α) (c : γ) :
(f.trans g) a = option.some c ∃ (b : β), f a = option.some b g b = option.some c

theorem pequiv.​trans_eq_none {α : Type u} {β : Type v} {γ : Type w} (f : α ≃. β) (g : β ≃. γ) (a : α) :
(f.trans g) a = option.none ∀ (b : β) (c : γ), b f a c g b

@[simp]
theorem pequiv.​refl_trans {α : Type u} {β : Type v} (f : α ≃. β) :

@[simp]
theorem pequiv.​trans_refl {α : Type u} {β : Type v} (f : α ≃. β) :

theorem pequiv.​inj {α : Type u} {β : Type v} (f : α ≃. β) {a₁ a₂ : α} {b : β} :
b f a₁b f a₂a₁ = a₂

theorem pequiv.​injective_of_forall_ne_is_some {α : Type u} {β : Type v} (f : α ≃. β) (a₂ : α) :
(∀ (a₁ : α), a₁ a₂((f a₁).is_some))function.injective f

theorem pequiv.​injective_of_forall_is_some {α : Type u} {β : Type v} {f : α ≃. β} :
(∀ (a : α), ((f a).is_some))function.injective f

def pequiv.​of_set {α : Type u} (s : set α) [decidable_pred s] :
α ≃. α

Equations
theorem pequiv.​mem_of_set_self_iff {α : Type u} {s : set α} [decidable_pred s] {a : α} :

theorem pequiv.​mem_of_set_iff {α : Type u} {s : set α} [decidable_pred s] {a b : α} :
a (pequiv.of_set s) b a = b a s

@[simp]
theorem pequiv.​of_set_eq_some_iff {α : Type u} {s : set α} {h : decidable_pred s} {a b : α} :

@[simp]
theorem pequiv.​of_set_eq_some_self_iff {α : Type u} {s : set α} {h : decidable_pred s} {a : α} :

@[simp]
theorem pequiv.​of_set_symm {α : Type u} (s : set α) [decidable_pred s] :

@[simp]

@[simp]
theorem pequiv.​of_set_eq_refl {α : Type u} {s : set α} [decidable_pred s] :

theorem pequiv.​symm_trans_rev {α : Type u} {β : Type v} {γ : Type w} (f : α ≃. β) (g : β ≃. γ) :

theorem pequiv.​trans_symm {α : Type u} {β : Type v} (f : α ≃. β) :
f.trans f.symm = pequiv.of_set {a : α | ((f a).is_some)}

theorem pequiv.​symm_trans {α : Type u} {β : Type v} (f : α ≃. β) :
f.symm.trans f = pequiv.of_set {b : β | (((f.symm) b).is_some)}

theorem pequiv.​trans_symm_eq_iff_forall_is_some {α : Type u} {β : Type v} {f : α ≃. β} :
f.trans f.symm = pequiv.refl α ∀ (a : α), ((f a).is_some)

@[instance]
def pequiv.​has_bot {α : Type u} {β : Type v} :
has_bot ≃. β)

Equations
@[simp]
theorem pequiv.​bot_apply {α : Type u} {β : Type v} (a : α) :

@[simp]
theorem pequiv.​symm_bot {α : Type u} {β : Type v} :

@[simp]
theorem pequiv.​trans_bot {α : Type u} {β : Type v} {γ : Type w} (f : α ≃. β) :

@[simp]
theorem pequiv.​bot_trans {α : Type u} {β : Type v} {γ : Type w} (f : β ≃. γ) :

theorem pequiv.​is_some_symm_get {α : Type u} {β : Type v} (f : α ≃. β) {a : α} (h : ((f a).is_some)) :

def pequiv.​single {α : Type u} {β : Type v} [decidable_eq α] [decidable_eq β] :
α → β → α ≃. β

Equations
theorem pequiv.​mem_single {α : Type u} {β : Type v} [decidable_eq α] [decidable_eq β] (a : α) (b : β) :

theorem pequiv.​mem_single_iff {α : Type u} {β : Type v} [decidable_eq α] [decidable_eq β] (a₁ a₂ : α) (b₁ b₂ : β) :
b₁ (pequiv.single a₂ b₂) a₁ a₁ = a₂ b₁ = b₂

@[simp]
theorem pequiv.​symm_single {α : Type u} {β : Type v} [decidable_eq α] [decidable_eq β] (a : α) (b : β) :

@[simp]
theorem pequiv.​single_apply {α : Type u} {β : Type v} [decidable_eq α] [decidable_eq β] (a : α) (b : β) :

theorem pequiv.​single_apply_of_ne {α : Type u} {β : Type v} [decidable_eq α] [decidable_eq β] {a₁ a₂ : α} (h : a₁ a₂) (b : β) :

theorem pequiv.​single_trans_of_mem {α : Type u} {β : Type v} {γ : Type w} [decidable_eq α] [decidable_eq β] [decidable_eq γ] (a : α) {b : β} {c : γ} {f : β ≃. γ} :
c f b(pequiv.single a b).trans f = pequiv.single a c

theorem pequiv.​trans_single_of_mem {α : Type u} {β : Type v} {γ : Type w} [decidable_eq α] [decidable_eq β] [decidable_eq γ] {a : α} {b : β} (c : γ) {f : α ≃. β} :
b f af.trans (pequiv.single b c) = pequiv.single a c

@[simp]
theorem pequiv.​single_trans_single {α : Type u} {β : Type v} {γ : Type w} [decidable_eq α] [decidable_eq β] [decidable_eq γ] (a : α) (b : β) (c : γ) :

@[simp]
theorem pequiv.​single_subsingleton_eq_refl {α : Type u} [decidable_eq α] [subsingleton α] (a b : α) :

theorem pequiv.​trans_single_of_eq_none {β : Type v} {γ : Type w} {δ : Type x} [decidable_eq β] [decidable_eq γ] {b : β} (c : γ) {f : δ ≃. β} :

theorem pequiv.​single_trans_of_eq_none {α : Type u} {β : Type v} {δ : Type x} [decidable_eq α] [decidable_eq β] (a : α) {b : β} {f : β ≃. δ} :

theorem pequiv.​single_trans_single_of_ne {α : Type u} {β : Type v} {γ : Type w} [decidable_eq α] [decidable_eq β] [decidable_eq γ] {b₁ b₂ : β} (h : b₁ b₂) (a : α) (c : γ) :

@[instance]
def pequiv.​partial_order {α : Type u} {β : Type v} :

Equations
theorem pequiv.​le_def {α : Type u} {β : Type v} {f g : α ≃. β} :
f g ∀ (a : α) (b : β), b f ab g a

@[instance]
def pequiv.​order_bot {α : Type u} {β : Type v} :
order_bot ≃. β)

Equations
@[instance]
def pequiv.​semilattice_inf_bot {α : Type u} {β : Type v} [decidable_eq α] [decidable_eq β] :

Equations
def equiv.​to_pequiv {α : Type u_1} {β : Type u_2} :
α βα ≃. β

Equations
@[simp]
theorem equiv.​to_pequiv_refl {α : Type u_1} :

theorem equiv.​to_pequiv_trans {α : Type u_1} {β : Type u_2} {γ : Type u_3} (f : α β) (g : β γ) :

theorem equiv.​to_pequiv_symm {α : Type u_1} {β : Type u_2} (f : α β) :

theorem equiv.​to_pequiv_apply {α : Type u_1} {β : Type u_2} (f : α β) (x : α) :