Skip to content

Commit 669a0ca

Browse files
committed
Add CHANGELOG and slightly simpler definition
1 parent 0a6680f commit 669a0ca

File tree

2 files changed

+7
-3
lines changed

2 files changed

+7
-3
lines changed

CHANGELOG.md

Lines changed: 5 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -71,6 +71,11 @@ Additions to existing modules
7171
++⁺ˡ : Reflexive R → ∀ zs → (_++ zs) Preserves (Pointwise R) ⟶ (Pointwise R)
7272
```
7373

74+
* In `Data.Maybe.Properties`:
75+
```agda
76+
maybe′-∘ : ∀ {b} (f : B → C) (g : A → B) → f ∘ (maybe′ g b) ≗ maybe′ (f ∘ g) (f b)
77+
```
78+
7479
* New lemmas in `Data.Nat.Properties`:
7580
```agda
7681
m≤n⇒m≤n*o : ∀ o .{{_ : NonZero o}} → m ≤ n → m ≤ n * o

src/Data/Maybe/Properties.agda

Lines changed: 2 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -97,9 +97,8 @@ maybe′-map : ∀ j (n : C) (f : A → B) ma →
9797
maybe′ j n (map f ma) ≡ maybe′ (j ∘′ f) n ma
9898
maybe′-map = maybe-map
9999

100-
maybe-∘ : {c x} (f : B C) (g : A B) f (maybe g c x) ≡ maybe (f ∘ g) (f c) x
101-
maybe-∘ {x = just _} _ _ = refl
102-
maybe-∘ {x = nothing} _ _ = refl
100+
maybe′-∘ : {b} (f : B C) (g : A B) f ∘ (maybe′ g b) ≗ maybe′ (f ∘ g) (f b)
101+
maybe′-∘ _ _ = maybe (λ _ refl) refl
103102

104103
------------------------------------------------------------------------
105104
-- _<∣>_

0 commit comments

Comments
 (0)