Documentation

Counterexamples.LinearOrderWithPosMulPosEqZero

An example of a LinearOrderedCommMonoidWithZero in which the product of two positive elements vanishes.

This is the monoid with 3 elements 0, ε, 1 where ε ^ 2 = 0 and everything else is forced. The order is 0 < ε < 1. Since ε ^ 2 = 0, the product of strictly positive elements can vanish.

Relevant Zulip chat: https://leanprover.zulipchat.com/#narrow/stream/116395-maths/topic/mul_pos

The three element monoid.

Instances For
    Equations

    The order on Foo is the one induced by the natural order on the image of aux1.

    Equations
    Instances For

      A tactic to prove facts by cases.

      Equations
      Instances For

        Multiplication on Foo: the only external input is that ε ^ 2 = 0.

        Equations
        Instances For
          Equations
          • One or more equations did not get rendered due to their size.
          theorem Counterexample.Foo.not_mul_pos :
          ¬∀ {M : Type} [inst : LinearOrderedCommMonoidWithZero M] (a b : M), 0 < a0 < b0 < a * b