Skip to content

Commit 2ef5f87

Browse files
Improve pointers to README files and rename README.Dec (#975)
1 parent f12ca70 commit 2ef5f87

File tree

13 files changed

+49
-8
lines changed

13 files changed

+49
-8
lines changed

README.agda

Lines changed: 4 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -262,6 +262,10 @@ import IO
262262
-- More documentation
263263
------------------------------------------------------------------------
264264

265+
-- Examples of how decidability is handled in the library.
266+
267+
import README.Decidability
268+
265269
-- Some examples showing how the case expression can be used.
266270

267271
import README.Case

README/Dec.agda renamed to README/Decidability.agda

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -6,7 +6,7 @@
66

77
{-# OPTIONS --without-K --safe #-}
88

9-
module README.Dec where
9+
module README.Decidability where
1010

1111
-- Reflects and Dec are defined in Relation.Nullary, and operations on them can
1212
-- be found in Relation.Nullary.Reflects and Relation.Nullary.Decidable.

src/Data/AVL.agda

Lines changed: 2 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -9,6 +9,8 @@
99
-- The search tree invariant is specified using the technique
1010
-- described by Conor McBride in his talk "Pivotal pragmatism".
1111

12+
-- See README.Data.AVL for examples of how to use AVL trees.
13+
1214
{-# OPTIONS --without-K --safe #-}
1315

1416
open import Relation.Binary using (StrictTotalOrder)

src/Data/Integer.agda

Lines changed: 3 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -4,6 +4,9 @@
44
-- Integers
55
------------------------------------------------------------------------
66

7+
-- See README.Data.Integer for examples of how to use and reason about
8+
-- integers.
9+
710
{-# OPTIONS --without-K --safe #-}
811

912
module Data.Integer where

src/Data/Integer/Base.agda

Lines changed: 3 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -4,6 +4,9 @@
44
-- Integers, basic types and operations
55
------------------------------------------------------------------------
66

7+
-- See README.Data.Integer for examples of how to use and reason about
8+
-- integers.
9+
710
{-# OPTIONS --without-K --safe #-}
811

912
-- Disabled to prevent warnings from deprecated names

src/Data/List.agda

Lines changed: 3 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -4,6 +4,9 @@
44
-- Lists
55
------------------------------------------------------------------------
66

7+
-- See README.Data.List for examples of how to use and reason about
8+
-- lists.
9+
710
{-# OPTIONS --without-K --safe #-}
811

912
module Data.List where

src/Data/List/Base.agda

Lines changed: 3 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -4,6 +4,9 @@
44
-- Lists, basic types and operations
55
------------------------------------------------------------------------
66

7+
-- See README.Data.List for examples of how to use and reason about
8+
-- lists.
9+
710
{-# OPTIONS --without-K --safe #-}
811

912
module Data.List.Base where

src/Data/List/Fresh.agda

Lines changed: 3 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -6,6 +6,9 @@
66
-- Lambda-Calculus with Explicit Substitutions"
77
------------------------------------------------------------------------
88

9+
-- See README.Data.List.Fresh and README.Data.Trie.NonDependent for
10+
-- examples of how to use fresh lists.
11+
912
{-# OPTIONS --without-K --safe #-}
1013

1114
module Data.List.Fresh where

src/Data/Nat.agda

Lines changed: 3 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -4,6 +4,9 @@
44
-- Natural numbers
55
------------------------------------------------------------------------
66

7+
-- See README.Data.Nat for examples of how to use and reason about
8+
-- naturals.
9+
710
{-# OPTIONS --without-K --safe #-}
811

912
module Data.Nat where

src/Data/Nat/Base.agda

Lines changed: 3 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -4,6 +4,9 @@
44
-- Natural numbers, basic types and operations
55
------------------------------------------------------------------------
66

7+
-- See README.Data.Nat for examples of how to use and reason about
8+
-- naturals.
9+
710
{-# OPTIONS --without-K --safe #-}
811

912
module Data.Nat.Base where

0 commit comments

Comments
 (0)