Skip to content

Inconsistencies between Relation.Binary.Definitions and Relation.Unary and Relation.Nullary #2091

Closed
@jamesmckinna

Description

@jamesmckinna

Maybe it's worth considering reconciling all the relational hierarchy at each arity wrt definitions of:

  • Irrelevant
    Recomputable
    Stable
    WeaklyDecidable
    Decidable
    Satisfiable
    Empty
    Universal
    etc. (the list may grow...)

because otherwise, we have a lot of redundant repetition on the one hand, but with 'gaps' on the other. There's some overlap/degeneracy at arity 0 for eg Satisfiable/Universal (the identity) and Empty (negation), but I think that is harmless...

Maybe there are good reasons to do with dependencies (eg. Relation.Nullary.Decidable.Core.recompute can't be typed with a Nullary definition of Recomputable... unless we bite the bullet and lift it out into a Relation.Nullary.Definitions etc. But maybe that's not such a bad idea, either? See also #2243 for my current approach to this particular predicate...

UPDATED: partial fix in #2259 (and largely orthogonal to #2243 )

Activity

added this to the v2.1 milestone on Sep 26, 2023
added a commit that references this issue on Jan 17, 2024
0b3e5cd
added a commit that references this issue on Feb 5, 2024
f70be79
jamesmckinna

jamesmckinna commented on Feb 5, 2024

@jamesmckinna
ContributorAuthor

Reconsidering whether to keep this open, I think on balance after the merge of #2259 that this one can be considered closed by that PR... the other cases being a little too non-uniform to be worth pursuing?

added a commit that references this issue on Jul 10, 2024
7c7c030
added a commit that references this issue on Sep 7, 2024
4144346
Sign up for free to join this conversation on GitHub. Already have an account? Sign in to comment

Metadata

Metadata

Assignees

No one assigned

    Labels

    No labels
    No labels

    Type

    No type

    Projects

    No projects

    Relationships

    None yet

      Development

      No branches or pull requests

        Participants

        @jamesmckinna

        Issue actions

          Inconsistencies between `Relation.Binary.Definitions` and `Relation.Unary` and `Relation.Nullary` · Issue #2091 · agda/agda-stdlib