Skip to content

Commit 594f239

Browse files
committed
[ fix #1694 ] Add ordered algebraic structures.
1 parent 650e05f commit 594f239

File tree

10 files changed

+801
-3
lines changed

10 files changed

+801
-3
lines changed

CHANGELOG.md

Lines changed: 20 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -800,6 +800,14 @@ New modules
800800
Algebra.Morphism.Construct.Identity
801801
```
802802

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+
803811
* 'Optimised' tail-recursive exponentiation properties:
804812
```
805813
Algebra.Properties.Semiring.Exp.TailRecursiveOptimised
@@ -1549,10 +1557,18 @@ Other minor changes
15491557

15501558
* Added new proofs to `Relation.Binary.Lattice.Properties.{Join,Meet}Semilattice`:
15511559
```agda
1560+
isPosemigroup : IsPosemigroup _≈_ _≤_ _∨_
1561+
posemigroup : Posemigroup c ℓ₁ ℓ₂
15521562
≈-dec⇒≤-dec : Decidable _≈_ → Decidable _≤_
15531563
≈-dec⇒isDecPartialOrder : Decidable _≈_ → IsDecPartialOrder _≈_ _≤_
15541564
```
15551565

1566+
* Added new proofs to `Relation.Binary.Lattice.Properties.Bounded{Join,Meet}Semilattice`:
1567+
```agda
1568+
isCommutativePomonoid : IsCommutativePomonoid _≈_ _≤_ _∨_ ⊥
1569+
commutativePomonoid : CommutativePomonoid c ℓ₁ ℓ₂
1570+
```
1571+
15561572
* Added new proofs to `Relation.Binary.Properties.Poset`:
15571573
```agda
15581574
≤-dec⇒≈-dec : Decidable _≤_ → Decidable _≈_
@@ -1666,6 +1682,9 @@ Other minor changes
16661682
sym⇒¬-sym : Symmetric _∼_ → Symmetric _≁_
16671683
cotrans⇒¬-trans : Cotransitive _∼_ → Transitive _≁_
16681684
irrefl⇒¬-refl : Reflexive _≈_ → Irreflexive _≈_ _∼_ → Reflexive _≁_
1685+
mono₂⇒cong₂ : Symmetric ≈₁ → ≈₁ ⇒ ≤₁ → Antisymmetric ≈₂ ≤₂ → ∀ {f} →
1686+
f Preserves₂ ≤₁ ⟶ ≤₁ ⟶ ≤₂ →
1687+
f Preserves₂ ≈₁ ⟶ ≈₁ ⟶ ≈₂
16691688
```
16701689

16711690
* 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
19451964
```agda
19461965
Inverse⇒Injection : Inverse S T → Injection S T
19471966
↔⇒↣ : A ↔ B → A ↣ B
1948-
```
1967+
```

src/Algebra/Ordered.agda

Lines changed: 15 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -0,0 +1,15 @@
1+
------------------------------------------------------------------------
2+
-- The Agda standard library
3+
--
4+
-- Definitions of ordered algebraic structures like promonoids and
5+
-- posemigroups (packed in records together with sets, orders,
6+
-- operations, etc.)
7+
------------------------------------------------------------------------
8+
9+
{-# OPTIONS --without-K --safe #-}
10+
11+
module Algebra.Ordered where
12+
13+
open import Algebra.Ordered.Definitions public
14+
open import Algebra.Ordered.Structures public
15+
open import Algebra.Ordered.Bundles public

0 commit comments

Comments
 (0)