mathlib documentation

data.nat.pairing

def nat.mkpair (a b : ) :

Pairing function for the natural numbers.

Equations
def nat.unpair (n : ) :

Unpairing function for the natural numbers.

Equations
@[simp]
theorem nat.mkpair_unpair (n : ) :

theorem nat.mkpair_unpair' {n a b : } (H : n.unpair = (a, b)) :
a.mkpair b = n

@[simp]
theorem nat.unpair_mkpair (a b : ) :
(a.mkpair b).unpair = (a, b)

theorem nat.unpair_lt {n : } (n1 : 1 n) :

theorem nat.unpair_le_left (n : ) :

theorem nat.le_mkpair_left (a b : ) :
a a.mkpair b

theorem nat.le_mkpair_right (a b : ) :
b a.mkpair b

theorem nat.unpair_le_right (n : ) :

theorem nat.mkpair_lt_mkpair_left {a₁ a₂ : } (b : ) (h : a₁ < a₂) :
a₁.mkpair b < a₂.mkpair b

theorem nat.mkpair_lt_mkpair_right (a : ) {b₁ b₂ : } (h : b₁ < b₂) :
a.mkpair b₁ < a.mkpair b₂