Skip to content

A Question on Apartness definitions -- particularly irrefl #2594

Closed
@bsaul

Description

@bsaul

I have an observation/question about the apartness/inequality definitions (sorry if this is not a particularly well formed yet). As I read about apartness in constructive math texts, it's generally defined on top of a notion of inequality (though perhaps inequivalence is a better term). For example, in A Course in Constructive Algebra by Mines, Richman, and Ruitenberg on p.8 (1988 ed): "We regard the relation of inequality as conventional and not necessarily the denial of equality. ... A consistent [which is what they call irreflexive], symmetric, cotranstive inequality is called an apartness." On the surface, this all well and good and the definition of apartness seems to match what's in the stdlib (at least of v2.2 without looking back in history).

But after reading Apartness and Uniformity by Bridges and Vîţă, I began to wonder if the stdlib has the relation between inequivalence and equivalence correct. Here's how Bridges and Vîţă (p. 8) define inequality:

Image

Note the condition that $\neq$ (which translates to _#_ in stdlib notation) implies the negation of equality (i.e. the "denial inequality" in the sense of Hines et al). Currently we have have an an ApartnessRelation is Irreflexive _≈_ _#_, which translates to ∀ {x y} → x ≈ y → ¬ (x # y), but this is the opposite of the Bridges definition, as I understand. Is the stdlib definition incorrect? or what am I missing here?

This is tangentially related to #2588 and Heyting algebra stuff more generally as that's were apartness starts to show up in the Algebra modules.

Metadata

Metadata

Assignees

No one assigned

    Type

    No type

    Projects

    No projects

    Milestone

    No milestone

    Relationships

    None yet

    Development

    No branches or pull requests

    Issue actions