Closed
Description
Do we have anywhere:
- the binary relation constructor
_<_ {A : Set a} (R : Rel A ℓ) : Rel (Maybe A) (a ⊔ ℓ)
(naming?) defined bynothing < just x
x R y → just x < just y
- proofs of its properties, incl. in particular
WellFounded R → WellFounded _<_
If not:
- where should it live?
- what should it be called?
- etc.
Elsewhere, this is the (_)⊥
lifting in (C)POs, but I don't seem to be able to find it.
Application: wellfoundedness of Strict
lexicographic ordering on List
, via uncons
, mimicking/extending the corresponding argument for Vec
.
Metadata
Metadata
Assignees
Labels
No labels