A commutative semiring that is a domain whose polynomial semiring is not a domain #
NatMaxAdd
is the natural numbers equipped with the usual multiplication but with maximum as
addition. Under these operations it is a commutative semiring that is a domain, but
1 + 1 = 1 + 0 = 1
in this semiring so addition is not cancellative.
As a consequence, the polynomial semiring NatMaxAdd[X]
is not a domain,
even though it has no zero-divisors other than 0.
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.
NatMaxAdd
is isomorphic to ℕ
multiplicatively.
Equations
- NatMaxAdd.mulEquiv = { toEquiv := NatMaxAdd.mk.symm, map_mul' := NatMaxAdd.mulEquiv._proof_1 }
Instances For
Equations
- One or more equations did not get rendered due to their size.
theorem
not_isDomain_commSemiring_imp_isDomain_polynomial :
¬∀ (R : Type) [inst : CommSemiring R] [IsDomain R], IsDomain (Polynomial R)