Skip to content

Algebraic structures with stable or decidable equality #1770

@Taneb

Description

@Taneb

In light of #1767, it might be useful to have copies of the algebraic hierarchy with stable equality, and with decidable equality

Here's a very rough sketch of what this could look like

record IsStableMagma {a ℓ} {A : Set a} (_≈_ : Rel A ℓ) (∙ : Op₂ A) : Set (a ⊔ ℓ) where
  field
    isMagma : IsMagma _≈_ ∙
    isStable :  x y  Stable (x ≈ y)

record IsDecidableMagma {a ℓ} {A : Set a} (_≈_ : Rel A ℓ) (∙ : Op₂ A) : Set (a ⊔ ℓ) where
  field
    isMagma : IsMagma _≈_ ∙
    isDecidable :  x y  Dec (x ≈ y)

  isStableMagma : IsStableMagma _≈_ ∙
  isStableMagma = record
    { isMagma = isMagma
    ; isStable = λ x y  decidable-stable (isDecidable x y)
    }

I've heard that many classical theorems, when you try to prove them constructively, depend on decidablility of equality.

I'm not sure how this interacts with the recently added Apartness things. I suspect that Apartness is weaker than Stable.

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