Skip to content

!-unique₂ takes implicit args in Terminal, whereas it takes explicit ones in Initial #366

@cxandru

Description

@cxandru

In Terminal, !-unique₂ : ∀ {A} {f g : A ⇒ ⊤} → f ≈ g takes f, g as implicit arguments, whereas in Initial, the arguments to the same function (!-unique₂ : ∀ {A} → (f g : ⊥ ⇒ A) → f ≈ g) are explicit.

This is probably an mistake and should be unified. I'm willing to fix this after I finish #362 .

Metadata

Metadata

Assignees

No one assigned

    Labels

    No labels
    No labels

    Type

    No type

    Projects

    No projects

    Milestone

    No milestone

    Relationships

    None yet

    Development

    No branches or pull requests

    Issue actions