Skip to content

Commit c61b159

Browse files
Add missing Func record to Function.Bundles (#1353)
1 parent f06d7b6 commit c61b159

File tree

109 files changed

+318
-186
lines changed

Some content is hidden

Large Commits have some content hidden by default. Use the searchbox below for content that may be hidden.

109 files changed

+318
-186
lines changed

CHANGELOG.md

Lines changed: 19 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -285,3 +285,22 @@ Other minor additions
285285
```
286286

287287
* Added infix declarations to `Data.Product.∃-syntax` and `Data.Product.∄-syntax`.
288+
289+
* Added new definitions to `Function.Bundles`:
290+
```agda
291+
record Func : Set _
292+
_⟶_ : Set a → Set b → Set _
293+
mk⟶ : (A → B) → A ⟶ B
294+
```
295+
296+
* Added new proofs to `Function.Construct.Composition`:
297+
```agda
298+
function : Func R S → Func S T → Func R T
299+
_∘-⟶_ : (A ⟶ B) → (B ⟶ C) → (A ⟶ C)
300+
```
301+
302+
* Added new proofs to `Function.Construct.Identity`:
303+
```agda
304+
function : Func S S
305+
id-⟶ : A ⟶ A
306+
```

README/Case.agda

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -15,7 +15,7 @@ open import Data.Nat hiding (pred)
1515
open import Data.List
1616
open import Data.Sum
1717
open import Data.Product
18-
open import Function using (case_of_; case_return_of_)
18+
open import Function.Base using (case_of_; case_return_of_)
1919
open import Relation.Nullary
2020
open import Relation.Binary
2121
open import Relation.Binary.PropositionalEquality

README/Data/Nat/Induction.agda

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -10,7 +10,7 @@ module README.Data.Nat.Induction where
1010
open import Data.Nat
1111
open import Data.Nat.Induction
1212
open import Data.Product using (_,_)
13-
open import Function using (_∘_)
13+
open import Function.Base using (_∘_)
1414
open import Induction.WellFounded
1515
open import Relation.Binary.PropositionalEquality
1616

README/Data/Record.agda

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -13,7 +13,7 @@ module README.Data.Record where
1313

1414
open import Data.Product
1515
open import Data.String
16-
open import Function using (flip)
16+
open import Function.Base using (flip)
1717
open import Level
1818
open import Relation.Binary
1919

README/Data/Tree/AVL.agda

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -106,7 +106,7 @@ q₅′ = refl
106106
-- Partitioning a tree into the smallest element plus the rest, or the
107107
-- largest element plus the rest.
108108

109-
open import Function using (id)
109+
open import Function.Base using (id)
110110

111111
v₆ : headTail t₀ ≡ nothing
112112
v₆ = refl

README/Data/Trie/NonDependent.agda

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -60,7 +60,7 @@ open import Data.Product as Prod
6060
open import Data.String as String using (String)
6161
open import Data.These as These
6262

63-
open import Function using (case_of_; _$_; _∘′_; id; _on_)
63+
open import Function.Base using (case_of_; _$_; _∘′_; id; _on_)
6464
open import Relation.Nary
6565
open import Relation.Binary using (Rel)
6666
open import Relation.Nullary.Negation using (¬?)

notes/style-guide.md

Lines changed: 45 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -31,6 +31,51 @@ automate most of this.
3131
should always go at the end of the line rather than the beginning of the
3232
next line.
3333

34+
#### Empty lines
35+
36+
* All module headers and standard term definitions should have a single
37+
empty line after them.
38+
39+
* There should be _two_ empty lines between adjacent record or module definitions
40+
in order to better distinguish the end of the record or module, as they will
41+
already be using single empty lines between internal definitions.
42+
43+
* For example:
44+
```agda
45+
module Test1 where
46+
47+
def1 : ...
48+
def1 = ...
49+
50+
def2 : ...
51+
def2 = ...
52+
53+
54+
module Test2 where
55+
56+
record Record1 : Set where
57+
field
58+
field1 : ...
59+
60+
aux1 : ...
61+
aux1 = ...
62+
63+
aux2 : ...
64+
aux2 = ...
65+
66+
67+
record Record2 : Set where
68+
field
69+
field2 : ...
70+
71+
72+
record1 : Record1
73+
record1 = { field1 = ... }
74+
75+
record2 : Record2
76+
record2 = { field2 = ... }
77+
```
78+
3479
#### Modules
3580

3681
* As a rule of thumb there should only be one named module per file. Anonymous

src/Algebra/Construct/NaturalChoice/Min.agda

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -16,7 +16,7 @@ open import Algebra.Core
1616
open import Algebra.Bundles
1717
open import Data.Sum.Base using (inj₁; inj₂; [_,_])
1818
open import Data.Product using (_,_)
19-
open import Function using (id)
19+
open import Function.Base using (id)
2020

2121
open TotalOrder totalOrder renaming (Carrier to A)
2222
open import Algebra.Definitions _≈_

src/Algebra/Operations/CommutativeMonoid.agda

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -13,7 +13,7 @@ open import Algebra
1313
open import Data.List.Base as List using (List; []; _∷_; _++_)
1414
open import Data.Fin.Base using (Fin; zero)
1515
open import Data.Table.Base as Table using (Table)
16-
open import Function using (_∘_)
16+
open import Function.Base using (_∘_)
1717
open import Relation.Binary.PropositionalEquality as P using (_≡_)
1818

1919
module Algebra.Operations.CommutativeMonoid

src/Algebra/Operations/Semiring.agda

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -19,7 +19,7 @@ import Algebra.Operations.CommutativeMonoid as MonoidOperations
1919
open import Data.Nat.Base
2020
using (zero; suc; ℕ) renaming (_+_ to _ℕ+_; _*_ to _ℕ*_)
2121
open import Data.Product using (module Σ)
22-
open import Function using (_$_)
22+
open import Function.Base using (_$_)
2323
open import Relation.Binary
2424
open import Relation.Binary.PropositionalEquality as P using (_≡_)
2525

0 commit comments

Comments
 (0)