Documentation

Counterexamples.MonicNonRegular

Monic does not necessarily imply IsRegular in a Semiring with no opposites #

This counterexample shows that the hypothesis Ring R cannot be changed to Semiring R in Polynomial.Monic.isRegular.

The example is very simple.

The coefficient Semiring is the Semiring N₃ of the natural numbers {0, 1, 2, 3} where the standard addition and standard multiplication are truncated at 3.

The products (X + 2) * (X + 2) and (X + 2) * (X + 3) are equal to X ^ 2 + 4 * X + 4 and X ^ 2 + 5 * X + 6 respectively.

By truncation, 4, 5, 6 all mean 3 in N. It follows that multiplication by (X + 2) is not injective.

N₃ is going to be a CommSemiring where addition and multiplication are truncated at 3.

Instances For

    Truncated addition on N₃.

    Equations
    • One or more equations did not get rendered due to their size.

    Truncated multiplication on N₃.

    Equations
    • One or more equations did not get rendered due to their size.
    theorem Counterexample.NonRegular.N₃.X_add_two_mul_X_add_two :
    (Polynomial.X + Polynomial.C 2) * (Polynomial.X + Polynomial.C 2) = (Polynomial.X + Polynomial.C 2) * (Polynomial.X + Polynomial.C 3)

    The main example: multiplication by the polynomial X + 2 is not injective, yet the polynomial is monic.

    theorem Counterexample.NonRegular.N₃.monic_X_add_two :
    (Polynomial.X + Polynomial.C 2).Monic

    The statement of the counterexample: not all monic polynomials over semirings are regular.