diff --git a/CHANGELOG.md b/CHANGELOG.md index 22732ed359..80ce0dda32 100644 --- a/CHANGELOG.md +++ b/CHANGELOG.md @@ -888,6 +888,24 @@ Deprecated names raise ↦ _↑ʳ_ ``` + Issue #1726: the relation `_≺_` and its single constructor `_≻toℕ_` + have been deprecated in favour of their extensional equivalent `_<_` + but omitting the inversion principle which pattern matching on `_≻toℕ_` + would achieve; this instead is proxied by the property `Data.Fin.Properties.toℕ<`. + +* In `Data.Fin.Induction`: + ``` + ≺-Rec + ≺-wellFounded + ≺-recBuilder + ≺-rec + ``` + + As with Issue #1726 above: the deprecation of relation `_≺_` means that these definitions + associated with wf-recursion are deprecated in favour of their `_<_` counterparts. + But it's not quite sensible to say that these definiton should be *renamed* to *anything*, + least of all those counterparts... the type confusion would be intolerable. + * In `Data.Fin.Properties`: ``` toℕ-raise ↦ toℕ-↑ʳ @@ -898,6 +916,9 @@ Deprecated names eq? ↦ inj⇒≟ ``` + Likewise under issue #1726: the properties `≺⇒<′` and `<′⇒≺` have been deprecated + in favour of their proxy counterparts `<⇒<′` and `<′⇒<`. + * In `Data.Fin.Permutation.Components`: ``` reverse ↦ Data.Fin.Base.opposite diff --git a/src/Data/Fin/Base.agda b/src/Data/Fin/Base.agda index 06c4581337..93ea438156 100644 --- a/src/Data/Fin/Base.agda +++ b/src/Data/Fin/Base.agda @@ -290,9 +290,6 @@ _>_ : IRel Fin 0ℓ i > j = toℕ i ℕ.> toℕ j -data _≺_ : ℕ → ℕ → Set where - _≻toℕ_ : ∀ n (i : Fin n) → toℕ i ≺ n - ------------------------------------------------------------------------ -- An ordering view. @@ -335,3 +332,15 @@ NB argument order has been flipped: the left-hand argument is the Fin m the right-hand is the Nat index increment." #-} + +data _≺_ : ℕ → ℕ → Set where + _≻toℕ_ : ∀ n (i : Fin n) → toℕ i ≺ n + +{-# WARNING_ON_USAGE _≺_ +"Warning: _≺_ was deprecated in v2.0. +Please use equivalent relation _<_ instead." +#-} +{-# WARNING_ON_USAGE _≻toℕ_ +"Warning: _≻toℕ_ was deprecated in v2.0. +Please use toℕ