Skip to content

Commit

Permalink
Merge branch 'master' into issue2458
Browse files Browse the repository at this point in the history
  • Loading branch information
jamesmckinna authored Sep 3, 2024
2 parents f04ff44 + 4972983 commit f7bb1d6
Show file tree
Hide file tree
Showing 4 changed files with 41 additions and 8 deletions.
11 changes: 11 additions & 0 deletions CHANGELOG.md
Original file line number Diff line number Diff line change
Expand Up @@ -29,6 +29,12 @@ Deprecated names
homo ↦ ∙-homo
```

* In `Algebra.Properties.CommutativeMagma.Divisibility`:
```agda
∣-factors ↦ x|xy∧y|xy
∣-factors-≈ ↦ xy≈z⇒x|z∧y|z
```

* In `Data.Vec.Properties`:
```agda
++-assoc _ ↦ ++-assoc-eqFree
Expand Down Expand Up @@ -76,6 +82,11 @@ Additions to existing modules
++⁺ˡ : Reflexive R → ∀ zs → (_++ zs) Preserves (Pointwise R) ⟶ (Pointwise R)
```

* In `Data.Maybe.Properties`:
```agda
maybe′-∘ : ∀ f g → f ∘ (maybe′ g b) ≗ maybe′ (f ∘ g) (f b)
```

* New lemmas in `Data.Nat.Properties`:
```agda
m≤n⇒m≤n*o : ∀ o .{{_ : NonZero o}} → m ≤ n → m ≤ n * o
Expand Down
33 changes: 26 additions & 7 deletions src/Algebra/Properties/CommutativeMagma/Divisibility.agda
Original file line number Diff line number Diff line change
Expand Up @@ -7,15 +7,14 @@
{-# OPTIONS --cubical-compatible --safe #-}

open import Algebra using (CommutativeMagma)
open import Data.Product.Base using (_×_; _,_; map)

module Algebra.Properties.CommutativeMagma.Divisibility
{a ℓ} (CM : CommutativeMagma a ℓ)
where

open CommutativeMagma CM
open import Data.Product.Base using (_×_; _,_)

open import Relation.Binary.Reasoning.Setoid setoid
open CommutativeMagma CM using (magma; _≈_; _∙_; comm)

------------------------------------------------------------------------
-- Re-export the contents of magmas
Expand All @@ -31,8 +30,28 @@ x∣xy x y = y , comm y x
xy≈z⇒x∣z : x y {z} x ∙ y ≈ z x ∣ z
xy≈z⇒x∣z x y xy≈z = ∣-respʳ xy≈z (x∣xy x y)

∣-factors : x y (x ∣ x ∙ y) × (y ∣ x ∙ y)
∣-factors x y = x∣xy x y , x∣yx y x
x|xy∧y|xy : x y (x ∣ x ∙ y) × (y ∣ x ∙ y)
x|xy∧y|xy x y = x∣xy x y , x∣yx y x

∣-factors-≈ : x y {z} x ∙ y ≈ z x ∣ z × y ∣ z
∣-factors-≈ x y xy≈z = xy≈z⇒x∣z x y xy≈z , xy≈z⇒y∣z x y xy≈z
xy≈z⇒x|z∧y|z : x y {z} x ∙ y ≈ z x ∣ z × y ∣ z
xy≈z⇒x|z∧y|z x y xy≈z = xy≈z⇒x∣z x y xy≈z , xy≈z⇒y∣z x y xy≈z


------------------------------------------------------------------------
-- DEPRECATED NAMES
------------------------------------------------------------------------
-- Please use the new names as continuing support for the old names is
-- not guaranteed.

-- Version 2.2

∣-factors = x|xy∧y|xy
{-# WARNING_ON_USAGE ∣-factors
"Warning: ∣-factors was deprecated in v2.2.
Please use x|xy∧y|xy instead. "
#-}
∣-factors-≈ = xy≈z⇒x|z∧y|z
{-# WARNING_ON_USAGE ∣-factors-≈
"Warning: ∣-factors-≈ was deprecated in v2.2.
Please use xy≈z⇒x|z∧y|z instead. "
#-}
2 changes: 1 addition & 1 deletion src/Data/List/Relation/Unary/All.agda
Original file line number Diff line number Diff line change
Expand Up @@ -115,7 +115,7 @@ zip = zipWith id
unzip : All (P ∩ Q) ⊆ All P ∩ All Q
unzip = unzipWith id

module _(S : Setoid a ℓ) {P : Pred (Setoid.Carrier S) p} where
module _ (S : Setoid a ℓ) {P : Pred (Setoid.Carrier S) p} where
open Setoid S renaming (refl to ≈-refl)
open SetoidMembership S

Expand Down
3 changes: 3 additions & 0 deletions src/Data/Maybe/Properties.agda
Original file line number Diff line number Diff line change
Expand Up @@ -97,6 +97,9 @@ maybe′-map : ∀ j (n : C) (f : A → B) ma →
maybe′ j n (map f ma) ≡ maybe′ (j ∘′ f) n ma
maybe′-map = maybe-map

maybe′-∘ : {b} (f : B C) (g : A B) f ∘ (maybe′ g b) ≗ maybe′ (f ∘ g) (f b)
maybe′-∘ _ _ = maybe (λ _ refl) refl

------------------------------------------------------------------------
-- _<∣>_

Expand Down

0 comments on commit f7bb1d6

Please sign in to comment.