Documentation

Mathlib.Algebra.Group.PUnit

PUnit is a commutative group #

This file collects facts about algebraic structures on the one-element type, e.g. that it is a commutative ring.

Equations
Equations
Equations
Equations
Equations
Equations
Equations
@[simp]
theorem PUnit.one_eq :
@[simp]
theorem PUnit.zero_eq :
theorem PUnit.mul_eq (x y : PUnit) :
x * y = unit
theorem PUnit.add_eq (x y : PUnit) :
x + y = unit
@[simp]
theorem PUnit.div_eq (x y : PUnit) :
x / y = unit
@[simp]
theorem PUnit.sub_eq (x y : PUnit) :
x - y = unit
@[simp]
theorem PUnit.inv_eq (x : PUnit) :
@[simp]
theorem PUnit.neg_eq (x : PUnit) :