mathlib3 documentation

data.two_pointing

Two-pointings #

THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.

This file defines two_pointing α, the type of two pointings of α. A two-pointing is the data of two distinct terms.

This is morally a Type-valued nontrivial. Another type which is quite close in essence is sym2. Categorically speaking, prod is a cospan in the category of types. This forms the category of bipointed types. Two-pointed types form a full subcategory of those.

References #

@[protected, instance]
theorem two_pointing.ext {α : Type u_3} (x y : two_pointing α) (h : x.to_prod = y.to_prod) :
x = y
@[ext]
structure two_pointing (α : Type u_3) :
Type u_3

Two-pointing of a type. This is a Type-valued termed nontrivial.

Instances for two_pointing
theorem two_pointing.ext_iff {α : Type u_3} (x y : two_pointing α) :
@[simp]
theorem two_pointing.swap_to_prod {α : Type u_1} (p : two_pointing α) :
def two_pointing.swap {α : Type u_1} (p : two_pointing α) :

Swaps the two pointed elements.

Equations
theorem two_pointing.swap_fst {α : Type u_1} (p : two_pointing α) :
theorem two_pointing.swap_snd {α : Type u_1} (p : two_pointing α) :
@[simp]
theorem two_pointing.swap_swap {α : Type u_1} (p : two_pointing α) :
p.swap.swap = p
@[reducible]
theorem two_pointing.to_nontrivial {α : Type u_1} (p : two_pointing α) :
@[protected, instance]
def two_pointing.pi (α : Type u_1) {β : Type u_2} (q : two_pointing β) [nonempty α] :

The two-pointing of constant functions.

Equations
@[simp]
theorem two_pointing.pi_fst (α : Type u_1) {β : Type u_2} (q : two_pointing β) [nonempty α] :
@[simp]
theorem two_pointing.pi_snd (α : Type u_1) {β : Type u_2} (q : two_pointing β) [nonempty α] :
def two_pointing.prod {α : Type u_1} {β : Type u_2} (p : two_pointing α) (q : two_pointing β) :

The product of two two-pointings.

Equations
@[simp]
theorem two_pointing.prod_fst {α : Type u_1} {β : Type u_2} (p : two_pointing α) (q : two_pointing β) :
@[simp]
theorem two_pointing.prod_snd {α : Type u_1} {β : Type u_2} (p : two_pointing α) (q : two_pointing β) :
@[protected]
def two_pointing.sum {α : Type u_1} {β : Type u_2} (p : two_pointing α) (q : two_pointing β) :

The sum of two pointings. Keeps the first point from the left and the second point from the right.

Equations
@[simp]
theorem two_pointing.sum_fst {α : Type u_1} {β : Type u_2} (p : two_pointing α) (q : two_pointing β) :
@[simp]
theorem two_pointing.sum_snd {α : Type u_1} {β : Type u_2} (p : two_pointing α) (q : two_pointing β) :
@[protected]

The ff, tt two-pointing of bool.

Equations
@[protected]

The false, true two-pointing of Prop.

Equations