Documentation

Mathlib.Algebra.PUnitInstances.Algebra

Instances on PUnit #

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
Equations
@[simp]
theorem PUnit.one_eq :
@[simp]
theorem PUnit.zero_eq :
theorem PUnit.mul_eq {x y : PUnit.{1}} :
x * y = unit
theorem PUnit.add_eq {x y : PUnit.{1}} :
x + y = unit
@[simp]
theorem PUnit.div_eq {x y : PUnit.{1}} :
x / y = unit
@[simp]
theorem PUnit.sub_eq {x y : PUnit.{1}} :
x - y = unit
@[simp]
@[simp]
theorem PUnit.neg_eq {x : PUnit.{1}} :