ULift
instances for ring #
This file defines instances for ring, semiring and related structures on ULift
types.
(Recall ULift α
is just a "copy" of a type α
in a higher universe.)
We also provide ULift.ringEquiv : ULift R ≃+* R
.
Equations
- ULift.mulZeroClass = { mul := fun (x1 x2 : ULift.{?u.12, ?u.13} α) => x1 * x2, zero := 0, zero_mul := ⋯, mul_zero := ⋯ }
Equations
- ULift.distrib = { mul := fun (x1 x2 : ULift.{?u.14, ?u.15} α) => x1 * x2, add := fun (x1 x2 : ULift.{?u.14, ?u.15} α) => x1 + x2, left_distrib := ⋯, right_distrib := ⋯ }
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
The ring equivalence between ULift α
and α
.
Equations
- ULift.ringEquiv = { toFun := ULift.down, invFun := ULift.up, left_inv := ⋯, right_inv := ⋯, map_mul' := ⋯, map_add' := ⋯ }
Instances For
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
Equations
- ULift.commRing = { toRing := ULift.ring, mul_comm := ⋯ }