Skip to content

two names in "Algebra.Lattice.Properties.BooleanAlgebra" are confusing #2685

@onestruggler

Description

@onestruggler

Hi,

Two names at line 195 in "Algebra.Lattice.Properties.BooleanAlgebra" are confusing:

⊥≉⊤ : ¬ ⊥ ≈ ⊤
⊥≉⊤ = lemma ⊥ ⊤ (∧-identityʳ _) (∨-zeroʳ _)

⊤≉⊥ : ¬ ⊤ ≈ ⊥
⊤≉⊥ = lemma ⊤ ⊥ (∧-zeroʳ _) (∨-identityʳ _)

It seems better to use "¬⊥≈⊤" and "¬⊤≈⊥" instead.

Metadata

Metadata

Assignees

No one assigned

    Labels

    Type

    No type

    Projects

    No projects

    Milestone

    Relationships

    None yet

    Development

    No branches or pull requests

    Issue actions