@@ -621,7 +621,7 @@ Non-backwards compatible changes
621621 raw bundles to ` Data.X.Base ` , this definition can now be made directly. Knock-on
622622 consequences include the need to retain the old constructor name, now introduced
623623 as a pattern synonym, and introduction of (a function equivalent to) the former
624- field name/projection function ` proof ` as ` ≤″-proof ` in ` Data.Nat.Properties ` .
624+ field name/projection function ` proof ` as ` ≤″-proof ` in ` Data.Nat.Properties ` .
625625
626626* Accordingly, the definition has been changed to:
627627 ``` agda
@@ -842,7 +842,6 @@ Non-backwards compatible changes
842842 IO.Effectful
843843 IO.Instances
844844 ```
845-
846845### (Issue #2096 ) Introduction of flipped relation symbol for ` Relation.Binary.Bundles.Preorder `
847846
848847* Previously, the relation symbol ` _∼_ ` was (notationally) symmetric, so that its
@@ -856,9 +855,25 @@ Non-backwards compatible changes
856855 Therefore, only _ declarations_ of ` PartialOrder ` records will need their field names
857856 updating.
858857
859- * NB (issues #1214 #2098 ) the corresponding situation regarding the ` flip ` ped
860- relation symbols ` _≥_ ` , ` _>_ ` (and their negated versions!) has not (yet)
861- been addressed.
858+ ### (Issue #1214 ) Reorganisation of the introduction of negated relation symbols under ` Relation.Binary `
859+
860+ * Previously, negated relation symbols ` _≰_ ` (for ` Poset ` ) and ` _≮_ ` (` TotalOrder ` )
861+ were introduced in the corresponding ` Relation.Binary.Properties ` modules, for re-export.
862+
863+ * Now they are introduced as definitions in the corresponding ` Relation.Binary.Bundles ` ,
864+ together with, for uniformity's sake, an additional negated symbol ` _⋦_ ` for ` Preorder ` ,
865+ with their (obvious) intended semantics:
866+ ``` agda
867+ infix 4 _⋦_ _≰_ _≮_
868+ Preorder._⋦_ : Rel Carrier _
869+ StrictPartialOrder._≮_ : Rel Carrier _
870+ ```
871+ Additionally, ` Poset._≰_ ` is defined by renaming public export of ` Preorder._⋦_ `
872+
873+ * Backwards compatibility has been maintained, with deprecated definitions in the
874+ corresponding ` Relation.Binary.Properties ` modules, and the corresponding client
875+ client module ` import ` s being adjusted accordingly.
876+
862877
863878### Standardisation of ` insertAt ` /` updateAt ` /` removeAt `
864879
@@ -879,12 +894,12 @@ Non-backwards compatible changes
879894 ```
880895 _─_ ↦ removeAt
881896 ```
882-
897+
883898* In ` Data.Vec.Base ` :
884899 ``` agda
885900 insert ↦ insertAt
886901 remove ↦ removeAt
887-
902+
888903 updateAt : Fin n → (A → A) → Vec A n → Vec A n
889904 ↦
890905 updateAt : Vec A n → Fin n → (A → A) → Vec A n
@@ -895,12 +910,12 @@ Non-backwards compatible changes
895910 remove : Fin (suc n) → Vector A (suc n) → Vector A n
896911 ↦
897912 removeAt : Vector A (suc n) → Fin (suc n) → Vector A n
898-
913+
899914 updateAt : Fin n → (A → A) → Vector A n → Vector A n
900915 ↦
901916 updateAt : Vector A n → Fin n → (A → A) → Vector A n
902917 ```
903-
918+
904919* The old names (and the names of all proofs about these functions) have been deprecated appropriately.
905920
906921### Changes to triple reasoning interface
@@ -1659,7 +1674,7 @@ Deprecated names
16591674 take-drop-id ↦ take++drop≡id
16601675
16611676 map-insert ↦ map-insertAt
1662-
1677+
16631678 insert-lookup ↦ insertAt-lookup
16641679 insert-punchIn ↦ insertAt-punchIn
16651680 remove-PunchOut ↦ removeAt-punchOut
@@ -1685,7 +1700,7 @@ Deprecated names
16851700 updateAt-cong-relative ↦ updateAt-cong-local
16861701
16871702 map-updateAt ↦ map-updateAt-local
1688-
1703+
16891704 insert-lookup ↦ insertAt-lookup
16901705 insert-punchIn ↦ insertAt-punchIn
16911706 remove-punchOut ↦ removeAt-punchOut
@@ -1743,11 +1758,6 @@ Deprecated names
17431758 fromForeign ↦ Foreign.Haskell.Coerce.coerce
17441759 ```
17451760
1746- * In ` Relation.Binary.Bundles.Preorder ` :
1747- ```
1748- _∼_ ↦ _≲_
1749- ```
1750-
17511761* In ` Relation.Binary.Indexed.Heterogeneous.Bundles.Preorder ` :
17521762 ```
17531763 _∼_ ↦ _≲_
@@ -1759,6 +1769,15 @@ Deprecated names
17591769 invPreorder ↦ converse-preorder
17601770 ```
17611771
1772+ * Moved negated relation symbol from ` Relation.Binary.Properties.Poset ` :
1773+ ```
1774+ _≰_ ↦ Relation.Binary.Bundles.Poset._≰_
1775+ ```
1776+
1777+ * Moved negated relation symbol from ` Relation.Binary.Properties.TotalOrder ` :
1778+ ```
1779+ _≮_ ↦ Relation.Binary.Bundles.StrictPartialOrder._≮_
1780+
17621781* In `Relation.Nullary.Decidable.Core`:
17631782 ```
17641783 excluded-middle ↦ ¬¬-excluded-middle
@@ -3301,9 +3320,9 @@ Additions to existing modules
33013320
33023321* Added new proofs to ` Relation.Binary.Consequences ` :
33033322 ```
3304- sym⇒¬-sym : Symmetric _∼_ → Symmetric _≁_
3305- cotrans⇒¬-trans : Cotransitive _∼_ → Transitive _≁_
3306- irrefl⇒¬-refl : Reflexive _≈_ → Irreflexive _≈_ _∼_ → Reflexive _≁_
3323+ sym⇒¬-sym : Symmetric _∼_ → Symmetric (¬_ ∘₂ _∼_)
3324+ cotrans⇒¬-trans : Cotransitive _∼_ → Transitive (¬_ ∘₂ _∼_)
3325+ irrefl⇒¬-refl : Reflexive _≈_ → Irreflexive _≈_ _∼_ → Reflexive (¬_ ∘₂ _∼_)
33073326 mono₂⇒cong₂ : Symmetric ≈₁ → ≈₁ ⇒ ≤₁ → Antisymmetric ≈₂ ≤₂ → ∀ {f} →
33083327 f Preserves₂ ≤₁ ⟶ ≤₁ ⟶ ≤₂ →
33093328 f Preserves₂ ≈₁ ⟶ ≈₁ ⟶ ≈₂
0 commit comments