Skip to content

Commit 9cbc30d

Browse files
committed
add: CHANGELOG
1 parent 6141208 commit 9cbc30d

File tree

1 file changed

+87
-0
lines changed

1 file changed

+87
-0
lines changed

CHANGELOG.md

Lines changed: 87 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -6,6 +6,11 @@ The library has been tested using Agda 2.7.0 and 2.7.0.1.
66
Highlights
77
----------
88

9+
* A major overhaul of the `Function` hierarchy sees the systematic development
10+
and use of theory of the left inverse to a given `Surjective` function `f`, in
11+
`Function.Consequences.Section`, up to and including full symmetry of `Bijection`, in
12+
`Function.Properties.Bijection`.
13+
914
Bug-fixes
1015
---------
1116

@@ -51,6 +56,32 @@ Deprecated names
5156
∣∣-trans ↦ ∥-trans
5257
```
5358

59+
* In `Function.Bundles.IsSurjection`:
60+
```agda
61+
to⁻ ↦ Function.Structures.IsSurjection.section
62+
to∘to⁻ ↦ Function.Structures.IsSurjection.strictlyInverseˡ
63+
```
64+
65+
* In `Function.Construct.Symmetry`:
66+
```agda
67+
injective ↦ Function.Consequences.Section.injective
68+
surjective ↦ Function.Consequences.Section.surjective
69+
bijective ↦ Function.Consequences.Section.bijective
70+
isBijection ↦ isBijectionWithoutCongruence
71+
isBijection-≡ ↦ isBijectionWithoutCongruence
72+
bijection-≡ ↦ bijectionWithoutCongruence
73+
```
74+
75+
* In `Function.Properties.Bijection`:
76+
```agda
77+
sym-≡ ↦ sym
78+
```
79+
80+
* In `Function.Properties.Surjection`:
81+
```agda
82+
injective⇒to⁻-cong ↦ Function.Construct.Symmetry.bijectionWithoutCongruence
83+
```
84+
5485
New modules
5586
-----------
5687

@@ -85,3 +116,59 @@ Additions to existing modules
85116
quasiring : Quasiring c ℓ → Quasiring (a ⊔ c) (a ⊔ ℓ)
86117
commutativeRing : CommutativeRing c ℓ → CommutativeRing (a ⊔ c) (a ⊔ ℓ)
87118
```
119+
120+
* In `Function.Bundles.Bijection`:
121+
```agda
122+
section : B → A
123+
inverseˡ : Inverseˡ _≈₁_ _≈₂_ to section
124+
strictlyInverseˡ : StrictlyInverseˡ _≈₂_ to section
125+
inverseʳ : Inverseʳ _≈₁_ _≈₂_ to section
126+
strictlyInverseʳ : StrictlyInverseʳ _≈₂_ section to
127+
```
128+
129+
* In `Function.Bundles.LeftInverse`:
130+
```agda
131+
surjective : Surjective _≈₁_ _≈₂_ to
132+
surjection : Surjection From To
133+
```
134+
135+
* In `Function.Bundles.RightInverse`:
136+
```agda
137+
isInjection : IsInjection to
138+
injective : Injective _≈₁_ _≈₂_ to
139+
injection : Injection From To
140+
```
141+
142+
* In `Function.Bundles.Surjection`:
143+
```agda
144+
section : B → A
145+
inverseˡ : Inverseˡ _≈₁_ _≈₂_ to section
146+
strictlyInverseˡ : StrictlyInverseˡ _≈₂_ to section
147+
```
148+
149+
* In `Function.Consequences`: the theory of the left inverse of a surjective function
150+
```agda
151+
module Section (surj : Surjective ≈₁ ≈₂ f)
152+
```
153+
154+
* In `Function.Properties.Bijection`:
155+
```agda
156+
sym : Bijection S T → Bijection T S
157+
```
158+
159+
* In `Function.Structures.IsBijection`:
160+
```agda
161+
section : B → A
162+
inverseˡ : Inverseˡ _≈₁_ _≈₂_ f section
163+
strictlyInverseˡ : StrictlyInverseˡ _≈₂_ f section
164+
inverseʳ : Inverseʳ _≈₁_ _≈₂_ f section
165+
strictlyInverseʳ : StrictlyInverseʳ _≈₂_ section f
166+
```
167+
168+
* In `Function.Structures.IsSurjection`:
169+
```agda
170+
section : B → A
171+
inverseˡ : Inverseˡ _≈₁_ _≈₂_ f section
172+
strictlyInverseˡ : StrictlyInverseˡ _≈₂_ f section
173+
```
174+

0 commit comments

Comments
 (0)