-
Notifications
You must be signed in to change notification settings - Fork 257
Closed
Description
An IsOrderHomomorphism
agda-stdlib/src/Relation/Binary/Morphism/Structures.agda
Lines 60 to 66 in 54f5c38
record IsOrderHomomorphism (_≈₁_ : Rel A ℓ₁) (_≈₂_ : Rel B ℓ₂) | |
(_≲₁_ : Rel A ℓ₃) (_≲₂_ : Rel B ℓ₄) | |
(⟦_⟧ : A → B) : Set (a ⊔ ℓ₁ ⊔ ℓ₂ ⊔ ℓ₃ ⊔ ℓ₄) | |
where | |
field | |
cong : Homomorphic₂ _≈₁_ _≈₂_ ⟦_⟧ | |
mono : Homomorphic₂ _≲₁_ _≲₂_ ⟦_⟧ |
So: should we have a Relation.Binary.Morphism.Biased.Structures
definition to reflect that? How best (eg wrt parametrisation) to define it?
Metadata
Metadata
Assignees
Labels
No labels