Skip to content
New issue

Have a question about this project? Sign up for a free GitHub account to open an issue and contact its maintainers and the community.

By clicking “Sign up for GitHub”, you agree to our terms of service and privacy statement. We’ll occasionally send you account related emails.

Already on GitHub? Sign in to your account

Port two Endomorphism submodules over to new Function hierarchy #2342

Merged
merged 22 commits into from
Jun 7, 2024
Merged
Show file tree
Hide file tree
Changes from 21 commits
Commits
Show all changes
22 commits
Select commit Hold shift + click to select a range
6619f11
port over two modules
JacquesCarette Apr 3, 2024
1af553e
and add to CHANGELOG
JacquesCarette Apr 3, 2024
81230ec
fix whitespace
JacquesCarette Apr 3, 2024
3305480
fix warning: it was pointing to a record that did not exist.
JacquesCarette Apr 4, 2024
e1e7c57
Merge branch 'FixWarning' into Endomorphism
JacquesCarette Apr 4, 2024
d1cae72
fix things as per Matthew's review - though this remains a breaking c…
JacquesCarette Apr 4, 2024
93e9e0f
take care of comments from James.
JacquesCarette Apr 9, 2024
35d3bb9
Merge branch 'master' into Endomorphism
JacquesCarette May 5, 2024
d258064
Merge branch 'master' into Endomorphism
JacquesCarette May 16, 2024
a2e3c26
adjust CHANGELOG for what will be implemented shortly
JacquesCarette May 16, 2024
e9fc145
Revert "take care of comments from James."
JacquesCarette May 16, 2024
9665443
Revert "fix things as per Matthew's review - though this remains a br…
JacquesCarette May 16, 2024
8cb04db
Revert "fix whitespace"
JacquesCarette May 16, 2024
154fb0e
Revert "port over two modules"
JacquesCarette May 16, 2024
d5d8113
rename these
JacquesCarette May 16, 2024
b04ab5d
fix tiny merge issue
JacquesCarette May 16, 2024
60ecbeb
get deprecations right (remove where not needed, make more global whe…
JacquesCarette May 22, 2024
08c8866
style guide - missing blank lines
JacquesCarette May 22, 2024
e7d4961
fix a bad merge
JacquesCarette May 22, 2024
b28f62d
fixed deprecations
jamesmckinna May 25, 2024
278547a
fix #2394
jamesmckinna Jun 5, 2024
c71cb83
minor tweaks
JacquesCarette Jun 7, 2024
File filter

Filter by extension

Filter by extension

Conversations
Failed to load comments.
Loading
Jump to
Jump to file
Failed to load files.
Loading
Diff view
Diff view
18 changes: 16 additions & 2 deletions CHANGELOG.md
Original file line number Diff line number Diff line change
Expand Up @@ -46,6 +46,11 @@ Deprecated modules
* `Data.List.Relation.Binary.Sublist.Propositional.Disjoint` deprecated in favour of
`Data.List.Relation.Binary.Sublist.Propositional.Slice`.

* The modules `Function.Endomorphism.Propositional` and
`Function.Endomorphism.Setoid` that use the old `Function`
hierarchy. Use `Function.Endo.Propositional` and
`Function.Endo.Setoid` instead.

Deprecated names
----------------

Expand Down Expand Up @@ -131,6 +136,11 @@ New modules
indexedSetoid : {A : Set a} → IndexedSetoid ℕ a _
```

* The modules `Function.Endo.Propositional` and
`Function.Endo.Setoid` are new but are actually proper ports of
`Function.Endomorphism.Propositional` and
`Function.Endomorphism.Setoid`.

* `Function.Relation.Binary.Equality`
```agda
setoid : Setoid a₁ a₂ → Setoid b₁ b₂ → Setoid _ _
Expand Down Expand Up @@ -235,13 +245,17 @@ Additions to existing modules
rawModule : RawModule R c ℓ
```

* In `Algebra.Morphism.Structures`
* In `Algebra.Morphism.Structures`:
```agda
module SuccessorSetMorphisms (N₁ : RawSuccessorSet a ℓ₁) (N₂ : RawSuccessorSet b ℓ₂) where
record IsSuccessorSetHomomorphism (⟦_⟧ : N₁.Carrier → N₂.Carrier) : Set _
record IsSuccessorSetMonomorphism (⟦_⟧ : N₁.Carrier → N₂.Carrier) : Set _
record IsSuccessorSetIsomorphism (⟦_⟧ : N₁.Carrier → N₂.Carrier) : Set _
record IsSuccessorSetIsomorphism (⟦_⟧ : N₁.Carrier → N₂.Carrier) : Set _

IsSemigroupHomomorphism : (A → B) → Set _
IsSemigroupMonomorphism : (A → B) → Set _
IsSemigroupIsomorphism : (A → B) → Set _
```
* In `Algebra.Properties.AbelianGroup`:
```
⁻¹-anti-homo‿- : (x - y) ⁻¹ ≈ y - x
Expand Down
121 changes: 121 additions & 0 deletions src/Function/Endo/Propositional.agda
Original file line number Diff line number Diff line change
@@ -0,0 +1,121 @@
------------------------------------------------------------------------
-- The Agda standard library
--
-- Endomorphisms on a Set
------------------------------------------------------------------------

{-# OPTIONS --cubical-compatible --safe #-}

module Function.Endo.Propositional {a} (A : Set a) where

open import Algebra using (Semigroup; Magma; RawMagma; Monoid; RawMonoid)
open import Algebra.Core
import Algebra.Definitions.RawMonoid as RawMonoidDefinitions
import Algebra.Properties.Monoid.Mult as MonoidMultProperties
open import Algebra.Structures using (IsMagma; IsSemigroup; IsMonoid)
open import Algebra.Morphism
using (module Definitions; IsMagmaHomomorphism; IsMonoidHomomorphism)
open Definitions using (Homomorphic₂)

open import Data.Nat.Base using (ℕ; zero; suc; _+_; +-rawMagma; +-0-rawMonoid)
open import Data.Nat.Properties using (+-0-monoid; +-semigroup)
open import Data.Product.Base using (_,_)

open import Function.Base using (id; _∘′_; _∋_; flip)
open import Function.Bundles using (Func; _⟶ₛ_; _⟨$⟩_)
open import Relation.Binary.Core using (_Preserves_⟶_)
open import Relation.Binary.PropositionalEquality.Core using (_≡_; refl; cong; cong₂)
import Relation.Binary.PropositionalEquality.Properties as ≡

import Function.Endo.Setoid (≡.setoid A) as Setoid

------------------------------------------------------------------------
-- Basic type and raw bundles

Endo : Set a
Endo = A → A

private

_∘_ : Op₂ Endo
_∘_ = _∘′_

∘-id-rawMonoid : RawMonoid a a
∘-id-rawMonoid = record { Carrier = Endo; _≈_ = _≡_ ; _∙_ = _∘_ ; ε = id }

open RawMonoid ∘-id-rawMonoid
using ()
renaming (rawMagma to ∘-rawMagma)


------------------------------------------------------------------------
-- Conversion back and forth with the Setoid-based notion of Endomorphism

fromSetoidEndo : Setoid.Endo → Endo
fromSetoidEndo = _⟨$⟩_

toSetoidEndo : Endo → Setoid.Endo
toSetoidEndo f = record
{ to = f
; cong = cong f
}

------------------------------------------------------------------------
-- Structures

∘-isMagma : IsMagma _≡_ _∘_
∘-isMagma = record
{ isEquivalence = ≡.isEquivalence
; ∙-cong = cong₂ _∘_
}

∘-magma : Magma _ _
∘-magma = record { isMagma = ∘-isMagma }

∘-isSemigroup : IsSemigroup _≡_ _∘_
∘-isSemigroup = record
{ isMagma = ∘-isMagma
; assoc = λ _ _ _ → refl
}

∘-semigroup : Semigroup _ _
∘-semigroup = record { isSemigroup = ∘-isSemigroup }

∘-id-isMonoid : IsMonoid _≡_ _∘_ id
∘-id-isMonoid = record
{ isSemigroup = ∘-isSemigroup
; identity = (λ _ → refl) , (λ _ → refl)
}

∘-id-monoid : Monoid _ _
∘-id-monoid = record { isMonoid = ∘-id-isMonoid }

------------------------------------------------------------------------
-- n-th iterated composition

infixr 8 _^_

_^_ : Endo → ℕ → Endo
_^_ = flip _×_ where open RawMonoidDefinitions ∘-id-rawMonoid

------------------------------------------------------------------------
-- Homomorphism

module _ (f : Endo) where

open MonoidMultProperties ∘-id-monoid

^-homo : Homomorphic₂ ℕ Endo _≡_ (f ^_) _+_ _∘_
^-homo = ×-homo-+ f

^-isMagmaHomomorphism : IsMagmaHomomorphism +-rawMagma ∘-rawMagma (f ^_)
^-isMagmaHomomorphism = record
{ isRelHomomorphism = record { cong = cong (f ^_) }
; homo = ^-homo
}

^-isMonoidHomomorphism : IsMonoidHomomorphism +-0-rawMonoid ∘-id-rawMonoid (f ^_)
^-isMonoidHomomorphism = record
{ isMagmaHomomorphism = ^-isMagmaHomomorphism
; ε-homo = refl
}
117 changes: 117 additions & 0 deletions src/Function/Endo/Setoid.agda
Original file line number Diff line number Diff line change
@@ -0,0 +1,117 @@
------------------------------------------------------------------------
-- The Agda standard library
--
-- Endomorphisms on a Setoid
------------------------------------------------------------------------

{-# OPTIONS --cubical-compatible --safe #-}

open import Relation.Binary.Bundles using (Setoid)

module Function.Endo.Setoid {c e} (S : Setoid c e) where

open import Agda.Builtin.Equality

open import Algebra using (Semigroup; Magma; RawMagma; Monoid; RawMonoid)
import Algebra.Definitions.RawMonoid as RawMonoidDefinitions
import Algebra.Properties.Monoid.Mult as MonoidMultProperties
open import Algebra.Structures using (IsMagma; IsSemigroup; IsMonoid)
open import Algebra.Morphism
using (module Definitions; IsMagmaHomomorphism; IsMonoidHomomorphism)
open Definitions using (Homomorphic₂)
open import Data.Nat.Base using (ℕ; zero; suc; _+_; +-rawMagma; +-0-rawMonoid)
open import Data.Nat.Properties using (+-semigroup; +-identityʳ)
open import Data.Product.Base using (_,_)
open import Function.Bundles using (Func; _⟶ₛ_; _⟨$⟩_)
open import Function.Construct.Identity using () renaming (function to identity)
open import Function.Construct.Composition using () renaming (function to _∘_)
open import Function.Relation.Binary.Setoid.Equality as Eq using (_⇨_)
open import Level using (Level; _⊔_)
open import Relation.Binary.Core using (_Preserves_⟶_)

private
open module E = Setoid (S ⇨ S) hiding (refl)
module S = Setoid S
open Func using (cong)


------------------------------------------------------------------------
JacquesCarette marked this conversation as resolved.
Show resolved Hide resolved
-- Basic type and raw bundles

Endo : Set _
Endo = S ⟶ₛ S

private
id : Endo
id = identity S

∘-id-rawMonoid : RawMonoid (c ⊔ e) (c ⊔ e)
∘-id-rawMonoid = record { Carrier = Endo; _≈_ = _≈_ ; _∙_ = _∘_ ; ε = id }

open RawMonoid ∘-id-rawMonoid
using ()
renaming (rawMagma to ∘-rawMagma)

--------------------------------------------------------------
-- Structures

∘-isMagma : IsMagma _≈_ _∘_
∘-isMagma = record
{ isEquivalence = isEquivalence
; ∙-cong = λ {_} {_} {_} {v} x≈y u≈v → S.trans u≈v (cong v x≈y)
}

∘-magma : Magma (c ⊔ e) (c ⊔ e)
∘-magma = record { isMagma = ∘-isMagma }

∘-isSemigroup : IsSemigroup _≈_ _∘_
∘-isSemigroup = record
{ isMagma = ∘-isMagma
; assoc = λ _ _ _ → S.refl
}

∘-semigroup : Semigroup (c ⊔ e) (c ⊔ e)
∘-semigroup = record { isSemigroup = ∘-isSemigroup }

∘-id-isMonoid : IsMonoid _≈_ _∘_ id
∘-id-isMonoid = record
{ isSemigroup = ∘-isSemigroup
; identity = (λ _ → S.refl) , (λ _ → S.refl)
}

∘-id-monoid : Monoid (c ⊔ e) (c ⊔ e)
∘-id-monoid = record { isMonoid = ∘-id-isMonoid }

------------------------------------------------------------------------
-- -- n-th iterated composition

infixr 8 _^_

_^_ : Endo → ℕ → Endo
f ^ n = n × f where open RawMonoidDefinitions ∘-id-rawMonoid

------------------------------------------------------------------------
-- Homomorphism

module _ (f : Endo) where

open MonoidMultProperties ∘-id-monoid

^-cong₂ : (f ^_) Preserves _≡_ ⟶ _≈_
^-cong₂ = ×-congˡ {f}

^-homo : Homomorphic₂ ℕ Endo _≈_ (f ^_) _+_ _∘_
^-homo = ×-homo-+ f

^-isMagmaHomomorphism : IsMagmaHomomorphism +-rawMagma ∘-rawMagma (f ^_)
^-isMagmaHomomorphism = record
{ isRelHomomorphism = record { cong = ^-cong₂ }
; homo = ^-homo
}

^-isMonoidHomomorphism : IsMonoidHomomorphism +-0-rawMonoid ∘-id-rawMonoid (f ^_)
^-isMonoidHomomorphism = record
{ isMagmaHomomorphism = ^-isMagmaHomomorphism
; ε-homo = S.refl
}

10 changes: 6 additions & 4 deletions src/Function/Endomorphism/Propositional.agda
Original file line number Diff line number Diff line change
@@ -1,16 +1,18 @@
------------------------------------------------------------------------
-- The Agda standard library
--
-- Endomorphisms on a Set
-- This module is DEPRECATED.
------------------------------------------------------------------------

{-# OPTIONS --cubical-compatible --safe #-}

-- Disabled to prevent warnings from deprecated names
{-# OPTIONS --warn=noUserWarning #-}

module Function.Endomorphism.Propositional {a} (A : Set a) where

{-# WARNING_ON_IMPORT
"Function.Endomorphism.Propositional was deprecated in v2.1.
Use Function.Endo.Propositional instead."
#-}

open import Algebra
open import Algebra.Morphism; open Definitions

Expand Down
10 changes: 6 additions & 4 deletions src/Function/Endomorphism/Setoid.agda
Original file line number Diff line number Diff line change
@@ -1,19 +1,21 @@
------------------------------------------------------------------------
-- The Agda standard library
--
-- Endomorphisms on a Setoid
-- This module is DEPRECATED.
------------------------------------------------------------------------

{-# OPTIONS --cubical-compatible --safe #-}

-- Disabled to prevent warnings from deprecated names
{-# OPTIONS --warn=noUserWarning #-}

open import Relation.Binary.Core using (_Preserves_⟶_)
open import Relation.Binary.Bundles using (Setoid)

module Function.Endomorphism.Setoid {c e} (S : Setoid c e) where

{-# WARNING_ON_IMPORT
"Function.Endomorphism.Setoid was deprecated in v2.1.
Use Function.Endo.Setoid instead."
#-}

open import Agda.Builtin.Equality

open import Algebra
Expand Down
1 change: 0 additions & 1 deletion src/Function/Equality.agda
Original file line number Diff line number Diff line change
Expand Up @@ -5,7 +5,6 @@
------------------------------------------------------------------------

{-# OPTIONS --cubical-compatible --safe #-}
{-# OPTIONS --warn=noUserWarning #-}

module Function.Equality where

Expand Down