-
Couldn't load subscription status.
- Fork 259
Open
Milestone
Description
Issue #2075 draws attention to the lack of a definition of StronglyNormalising (SN) of a relation R, defined by
StronglyNormalising (R : Rel A ℓ) = WellFounded (flip R)One fix might be to add such a definition to PR #2077...
... but a better one might be to add a new module Induction.Normalising defining both the above, and
data WeaklyNormalising (N : Pred A ℓ₁) (R : Rel A ℓ₂) : Pred A _ where
norm : ∀ {x} → N x → WeaklyNormalising N R x
step : ∀ {x y} → R x y → WeaklyNormalising N R y → WeaklyNormalising N R xsuch that ... suitable properties hold on the basis of suitable assumptions about N and R... (to be continued)
Ooops! I hadn't previously been aware of Relation.Binary.Rewriting!
Metadata
Metadata
Assignees
Labels
No labels