@@ -800,6 +800,14 @@ New modules
800
800
Algebra.Morphism.Construct.Identity
801
801
```
802
802
803
+ * Ordered algebraic structures (pomonoids, posemigroups, etc.)
804
+ ```
805
+ Algebra.Ordered
806
+ Algebra.Ordered.Bundles
807
+ Algebra.Ordered.Definitions
808
+ Algebra.Ordered.Structures
809
+ ```
810
+
803
811
* 'Optimised' tail-recursive exponentiation properties:
804
812
```
805
813
Algebra.Properties.Semiring.Exp.TailRecursiveOptimised
@@ -1549,10 +1557,18 @@ Other minor changes
1549
1557
1550
1558
* Added new proofs to ` Relation.Binary.Lattice.Properties.{Join,Meet}Semilattice ` :
1551
1559
``` agda
1560
+ isPosemigroup : IsPosemigroup _≈_ _≤_ _∨_
1561
+ posemigroup : Posemigroup c ℓ₁ ℓ₂
1552
1562
≈-dec⇒≤-dec : Decidable _≈_ → Decidable _≤_
1553
1563
≈-dec⇒isDecPartialOrder : Decidable _≈_ → IsDecPartialOrder _≈_ _≤_
1554
1564
```
1555
1565
1566
+ * Added new proofs to ` Relation.Binary.Lattice.Properties.Bounded{Join,Meet}Semilattice ` :
1567
+ ``` agda
1568
+ isCommutativePomonoid : IsCommutativePomonoid _≈_ _≤_ _∨_ ⊥
1569
+ commutativePomonoid : CommutativePomonoid c ℓ₁ ℓ₂
1570
+ ```
1571
+
1556
1572
* Added new proofs to ` Relation.Binary.Properties.Poset ` :
1557
1573
``` agda
1558
1574
≤-dec⇒≈-dec : Decidable _≤_ → Decidable _≈_
@@ -1666,6 +1682,9 @@ Other minor changes
1666
1682
sym⇒¬-sym : Symmetric _∼_ → Symmetric _≁_
1667
1683
cotrans⇒¬-trans : Cotransitive _∼_ → Transitive _≁_
1668
1684
irrefl⇒¬-refl : Reflexive _≈_ → Irreflexive _≈_ _∼_ → Reflexive _≁_
1685
+ mono₂⇒cong₂ : Symmetric ≈₁ → ≈₁ ⇒ ≤₁ → Antisymmetric ≈₂ ≤₂ → ∀ {f} →
1686
+ f Preserves₂ ≤₁ ⟶ ≤₁ ⟶ ≤₂ →
1687
+ f Preserves₂ ≈₁ ⟶ ≈₁ ⟶ ≈₂
1669
1688
```
1670
1689
1671
1690
* Added new operations in ` Relation.Binary.PropositionalEquality.Properties ` :
@@ -1945,4 +1964,4 @@ This is a full list of proofs that have changed form to use irrelevant instance
1945
1964
``` agda
1946
1965
Inverse⇒Injection : Inverse S T → Injection S T
1947
1966
↔⇒↣ : A ↔ B → A ↣ B
1948
- ```
1967
+ ```
0 commit comments