Extra facts about prod
This file defines prod.swap : α × β → β × α
and proves various simple lemmas about prod
.
@[simp]
@[simp]
@[simp]
theorem
prod.map_mk
{α : Type u_1}
{β : Type u_2}
{γ : Type u_3}
{δ : Type u_4}
(f : α → γ)
(g : β → δ)
(a : α)
(b : β) :
@[simp]
@[simp]
@[simp]
@[instance]
def
prod.lex.decidable
{α : Type u_1}
{β : Type u_2}
[decidable_eq α]
(r : α → α → Prop)
(s : β → β → Prop)
[decidable_rel r]
[decidable_rel s] :
decidable_rel (prod.lex r s)
Equations
- prod.lex.decidable r s = λ (p q : α × β), decidable_of_decidable_of_iff or.decidable _
theorem
function.injective.prod_map
{α : Type u_1}
{β : Type u_2}
{γ : Type u_3}
{δ : Type u_4}
{f : α → γ}
{g : β → δ} :
function.injective f → function.injective g → function.injective (prod.map f g)
theorem
function.surjective.prod_map
{α : Type u_1}
{β : Type u_2}
{γ : Type u_3}
{δ : Type u_4}
{f : α → γ}
{g : β → δ} :
function.surjective f → function.surjective g → function.surjective (prod.map f g)