Skip to content

Commit

Permalink
add some design documentation corresponding to issue #312. (Redo of b…
Browse files Browse the repository at this point in the history
…ad 957)
  • Loading branch information
JacquesCarette committed Mar 17, 2024
1 parent 995fdab commit 599744c
Showing 1 changed file with 17 additions and 0 deletions.
17 changes: 17 additions & 0 deletions doc/README/Design/Miscellany.agda
Original file line number Diff line number Diff line change
@@ -0,0 +1,17 @@
------------------------------------------------------------------------
-- The Agda standard library
--
-- Documentation describing some of the smaller choices in the library
------------------------------------------------------------------------

{-# OPTIONS --cubical-compatible --safe #-}

module README.Design.Miscellany where

-------------------------------------------------------------------------
-- Level polymorphism

-- `⊥` in `Data.Empty` and `⊤` in `Data.Unit` are not `Level`-polymorphic as that
-- tends to lead to unsolved metas (see discussion at issue #312). For that purpose,
-- there are now level-polymorphic version in `Data.Empty.Polymorphic` and
-- `Data.Unit.Polymorphic` respectively.

0 comments on commit 599744c

Please sign in to comment.