This CHANGELOG describes the history of already-released versions. Please see CHANGELOG_NEXT for changes merged into the main branch but not yet released.
- New magic constants
__LOC__
,__FILE__
,__LINE__
,__COL__
substituted at parsing time with a string corresponding to the location, filename, line or column number associated to the magic constant's position. - The termination checker is now a faithful implementation of the 2001 paper on size-change termination by Lee, Jones and Ben-Amram.
- New function option
%unsafe
to mark definitions that are escape hatches similar to the builtinsbelieve_me
,assert_total
, etc. - Elaborator scripts were made be able to record warnings.
- Rudimentary support for defining lazy functions (addressing issue #1066).
%hide
directives can now hide conflicting fixities from other modules.- Fixity declarations can now be kept private with export modifiers.
- Forward-declarations whose visibility differ from their actual definition now emit a warning, unless the definition has no specified visibility (addressing Issue #1236).
- New
fromTTImp
,fromName
, andfromDecls
names for customTTImp
,Name
, andDecls
literals. - Call to
%macro
-functions do not require theElabReflection
extension. - Default implicits are supported for named implementations.
- Elaborator scripts were made to be able to access project files, allowing the support for type providers and similar stuff.
- Elaborator scripts were made to be able to inspect which definitions are referred to by another definitions, and in which function currently elaborator is. These features together give an ability to inspect whether particular expressions are recursive (including mutual recursion).
- Adds documentation for unquotes
~( )
. - Adds documentation for laziness and codata primitives:
Lazy
,Inf
,Delay
, andForce
. - Adds
--no-cse
command-line option to disable common subexpression elimination for code generation debugging. - Fixes a confusion between data and type constructors in the
:di
command.
- Adds support for
CFLAGS
,CPPFLAGS
,LDFLAGS
andLDLIBS
to facilitate building on systems with non-standard installation locations of libraries (e.g. GMP). Versions of the flags with theIDRIS2_
prefix can also be used and take precedence.
- Non-recursive top-level constants are compiled to eagerly evaluated constants in Chez Scheme.
- FFI declarations can now specify which
require
to perform, i.e. which library to load before executing the FFI. The syntax isscheme,racket:my-function,my-library
.
- Generated JavaScript files now include a shebang when using the Node.js backend
- NodeJS now supports
popen
/pclose
for theRead
mode. getChar
is now supported on Node.js andputChar
is supported on both JavaScript backends.- Integer-indexed arrays are now supported.
-
If
IAlternative
expression withFirstSuccess
rule fails to typecheck, compiler now prints all tried alternatives, not only the last one. -
The elaboration of records has been changed so that the unbound implicits in the parameters' types become additional parameters e.g.
record HasLength (xs : List a) (n : Nat) where constructor MkHasLength 0 prf : length xs === n
is now correctly elaborated to
record HasLength {0 a : Type} (xs : List a) (n : Nat) where constructor MkHasLength 0 prf : length xs === n
instead of failing with a strange error about (a) vs (a .rec).
-
Elaboration of datatypes now respects the totality annotations: defining a
covering
orpartial
datatype in a%default total
file will not lead to a positivity error anymore. -
Fixed a bug in the positivity checker that meant
Lazy
could be used to hide negative occurrences. -
Made sure that the positivity checker now respects
assert_total
annotations. -
We now raise a warning for conflicting fixity declarations. They are dangerous as Idris will pick an arbitrary one and so the meaning of an expression can depend e.g. on the order in which modules are imported.
- Additionally some conflicting fixity declarations in the Idris 2 compiler and libraries have been removed.
-
Constructors mentioned on the left hand side of functions/case alternatives are now included in the
Refers to (runtime)
section of functions debug info. -
The Lifted IR Representation now has a
HasNamespaces
implementation inCompiler.Separate
so Compilation Units at that stage can be generated. -
Added the
compile.casetree.missing
log topic, along with its use inTTImp.ProcessDef.genRunTime
. This allows us to track when incompletecase
blocks get the runtime error added. -
Constant folding of trivial let statements and
believe_me
. -
Fixed a bug that caused holes to appear unexpectedly during quotation of dependent pairs.
-
Fixed a bug that caused
f
to sometimes be replaced byfx
after matchingfx = f x
. -
Fixed a bug in the totality checker that missed indirect references to partial data.
-
Refactor the idris2protocols package to depend on fewer Idris2 modules. We can now export the package independently. To avoid confusing tooling about which
.ipkg
to use, the package file is under the newly addedipkg
sub-directory. -
Added
Libraries.Data.WithDefault
to facilitate consistent use of a default-if-unspecified value, currently forprivate
visibility.
-
Improved performance of functions
isNL
,isSpace
, andisHexDigit
. -
Implements
Foldable
andTraversable
for pairs, right-biased asFunctor
. -
Added a constructor (
MkInterpolation
) toInterpolation
. -
Added an
Interpolation
implementation forVoid
. -
Added
Compose
instances forBifunctor
,Bifoldable
andBitraversable
.
-
Deprecates
setByte
andgetByte
fromData.Buffer
for removal in a future release. UsesetBits8
andgetBits8
instead (withcast
if you need to convert aBits8
to anInt
), as their values are limited, as opposed to the assumption insetByte
that the value is between 0 and 255. -
Adds RefC support for 16- and 32-bit access in
Data.Buffer
. -
Add
Show
instance toData.Vect.Quantifiers.All
and add a few helpers for listy computations on theAll
type. -
Add an alias for
HVect
toAll id
inData.Vect.Quantifiers.All
. This is the approach to getting a heterogeneousVect
of elements that is general preferred by the community vs. a standalone type as seen incontrib
. -
Add
Data.List.HasLength
from the compiler codebase slash contrib library but adopt the type signature from the compiler codebase and some of the naming from the contrib library. The type ended up beingHasLength n xs
rather thanHasLength xs n
. -
Moved
Data.SortedMap
andData.SortedSet
from contrib to base. -
Added missing buffer primitives (chezscheme only):
setInt8
,getInt8
,getInt16
,setInt64
,getInt64
-
Added new buffer (set/get) functions for built-in types
Bool
,Nat
,Integer
. -
Tightened the types of:
setInt16
(now takes anInt16
instead of anInt
),setInt32
(now takes anInt32
instead of anInt
),getInt32
(now returns anInt32
instead of anInt
) -
Adds left- and right-rotation for
FiniteBits
. -
Adds
Vect.permute
for applying permutations toVect
s. -
Adds
Vect.kSplits
andVect.nSplits
for splitting aVect
whose length is a known multiple of twoNat
s (k * n) into k vectors of length n (and vice-versa). -
Adds
Vect.allFins
for generating all theFin
elements as aVect
with matching length to the number of elements. -
Add
withRawMode
,enableRawMode
,resetRawMode
for character at a time input on stdin. -
Adds extraction functions to
Data.Singleton
. -
TTImp
reflection functions are nowpublic export
, enabling use at the type-level. -
Implemented
Eq
,Ord
,Semigroup
, andMonoid
forData.List.Quantifiers.All.All
andData.Vect.Quantifiers.All.All
. -
Generalized
imapProperty
inData.List.Quantifiers.All.All
andData.Vect.Quantifiers.All.All
. -
Add
zipPropertyWith
,traverseProperty
,traversePropertyRelevant
,mapPropertyRelevant
,(++)
,tabulate
andremember
toData.Vect.Quantifiers.All.All
. -
Add
anyToFin
toData.Vect.Quantifiers.Any
, converting theAny
witness to the index into the corresponding element. -
Implemented
Ord
forLanguage.Reflection.TT.Name
,Language.Reflection.TT.Namespace
andLanguage.Reflection.TT.UserName
. -
Adds
leftmost
andrightmost
toControl.Order
, a generalisation ofmin
andmax
. -
Adds
even
andodd
toData.Integral
. -
Eq
andOrd
implementations forFin n
now run in constant time. -
Adds
getTermCols
andgetTermLines
to the base library. They return the size of the terminal if either stdin or stdout is a tty. -
The
Data.List1
functionsfoldr1
andfoldr1By
are nowpublic export
. -
Added
uncons' : List a -> Maybe (a, List a)
tobase
. -
Adds
infixOfBy
andisInfixOfBy
intoData.List
. -
Adds
WithDefault
intoLanguage.Reflection.TTImp
, mirroring compiler addition. -
Adds updating functions to
SortedMap
andSortedDMap
. -
Adds
grouped
function toData.List
for splitting a list into equal-sized slices. -
Implements
Ord
forCount
fromLanguage.Reflection
. -
Implements
MonadState
forData.Ref
with a named implementation requiring a particular reference. -
Adds implementations of
Zippable
toEither
,Pair
,Maybe
,SortedMap
. -
Adds a
Compose
andFromApplicative
named implementations forZippable
. -
Adds
Semigroup
,Applicative
,Traversable
andZippable
forData.These
. -
Adds bindings for IEEE floating point constants NaN and (+/-) Inf, as well as machine epsilon and unit roundoff. Speeds vary depending on backend.
-
A more generalised way of applicative mapping of
TTImp
expression was added, calledmapATTImp
; the originalmapMTTimp
was implemented through the new one. -
Adds
Data.Vect.foldrImplGoLemma
. -
Ref
interface fromData.Ref
inheritsMonad
and was extended by a function for value modification implemented through reading and writing by default.
-
Changes
getNProcessors
to return the number of online processors rather than the number of configured processors. -
System
'sdie
now prints the error message on stderr rather than stdout -
Adds
popen2
to run a subprocess with bi-directional pipes. -
A function
popen2Wait
was added to wait for the process started withpopen2
function and clean up all system resources (to not to leave zombie processes in particular). -
Function
getStringAndFree
fromSystem.File.ReadWrite
was given an extra argument of typeFile
to return an empty string if no error happened.
-
Adds
Data.List.Sufficient
, a small library defining a structurally inductive view of lists. -
Remove
Data.List.HasLength
fromcontrib
library but add it to thebase
library with the type signature from the compiler codebase and some of the naming from thecontrib
library. The type ended up beingHasLength n xs
rather thanHasLength xs n
. -
Adds an implementation for
Functor Text.Lexer.Tokenizer.Tokenizer
. -
Adds
modFin
andstrengthenMod
toData.Fin.Extra
. These functions reason about the modulo operator's upper bound, which can be useful when working with indices (for example). -
Existing specialised variants of functions from the
Traversable
forLazyList
were made to be indeed lazy by the effect, but their requirements were strengthened fromApplicative
toMonad
. -
Implements
Sized
forData.Seq.Sized
andData.Seq.Unsized
.
-
In
Control.DivideAndConquer
: a port of the paper "A Type-Based Approach to Divide-And-Conquer Recursion in Coq" by Pedro Abreu, Benjamin Delaware, Alex Hubers, Christa Jenkins, J. Garret Morris, and Aaron Stump. https://doi.org/10.1145/3571196 -
Ports the first half of "Deferring the Details and Deriving Programs" by Liam O'Connor as
Data.ProofDelay
. https://doi.org/10.1145/3331554.3342605 http://liamoc.net/images/deferring.pdf
- The
data
subfolder of an installed or local dependency package is now automatically recognized as a "data" directory by Idris 2. See the documentation on Packages for details. - The compiler no longer installs its own C support library into
${PREFIX}/lib
. This folder's contents were always duplicates of files installed into${PREFIX}/idris2-${IDRIS2_VERSION}/lib
. If you need to adjust any tooling or scripts, point them to the latter location which still contains these installed library files. - Renamed
support-clean
Makefile target toclean-support
. This is in line with most of theinstall-<something>
andclean-<something>
naming. - Fixes an error in the
Makefile
where settingIDRIS2_PREFIX
caused bootstrapping to fail. - Updates the docs for
envvars
to match the changes introduced in #2649. - Both
make install
andidris2 --install...
now respectDESTDIR
which can be set to install into a staging directory for distro packaging. - Updates the docs for
envvars
to categorise when environment variables are used (runtime, build-time, or both). - Fixed build failure occuring when
make -j
is in effect. - Add
clean_names
function totestutils.sh
to normalise machine names
- New experimental Scheme based evaluator (only available if compiled via
Chez scheme or Racket). To access this at the REPL, set the evaluator mode to
the scheme based evaluator with
:set eval scheme
. - New option
evaltiming
to time how long an evaluation takes at the REPL, set with:set evaltiming
. - Renames
:lp/loadpackage
to:package
. - Adds
:import
, with the same functionality as:module
. - Adds the ability to request detailed help via
:help <replCmd>
, e.g.:help :help
or:help :let
. This also works with the:?
and:h
aliases.
-
There were two versions of record syntax used when updating records:
record { field = value } r
and
{ field := value } r
The former is now deprecated in favour of the latter syntax. The compiler will issue a warning when using the
record
keyword. -
Interpolated strings now make use of
concat
which is compiled intofastConcat
. The interpolated slices now make use of theInterpolation
interface available in the prelude. It has only one methodinterpolate
which is called for every expression that appears within an interpolation slice."hello \{world}"
is desugared into
concat [interpolate "hello ", interpolate world]
This allows you to write expressions within slices without having to call
show
but for this you need to implement theInterpolation
interface for each type that you intend to use within an interpolation slice. The reason for not reusingShow
is thatInterpolation
andShow
have conflicting semantics, typically this is the case forString
which adds double quotes around the string. -
Adds a
failing
block that requires its body to fail with a compile error. Optionally this block may contain a string which is checked to be contained in the error message. -
Bodies of
mutual
,failing
,using
andparameters
blocks are required to be indented comparing to the position of the keyword. -
%nomangle
has been deprecated in favour of%export
. -
Records now support DataOpts, i.e. we can write things like
record Wrap (phantom : Type) (a : Type) where [search a] -- this was previously not supported constructor MkWrap unWrap : a
-
Adds ability to forward-declare interface implementations, e.g.:
implementation IsOdd Nat -- forward declare for use in `IsEven` implementation IsEven Nat where isEven 0 = True isEven (S k) = not $ isOdd k implementation IsOdd Nat where isOdd 0 = False isOdd (S k) = not $ isEven k
-
Adds ability to forward-declare records, e.g.:
record B record A where b : B record B where a : A
- Removes deprecated support for
void
primitive. Nowvoid
is supported viaprim__void
. - Adds
%deprecate
pragma that can be used to warn when deprecated functions are used. - Package files now support a
langversion
field that can be used to specify what versions of Idris a package supports. As with dependency versions,>
,<
,>=
, and<=
can all be used.- For example,
langversion >= 0.5.1
.
- For example,
- Alternatives for primitive types of the
Core.TT.Constant
are moved out to a separate data typePrimTypes
. Signatures of functions that were working withConstant
are changed to usePrimTypes
when appropriate. - Codegens now take an additional
Ref Syn SyntaxInfo
argument. This empowers compiler writers to pretty print core terms e.g. to add comments with the original type annotations in the generated code. Refc.showcCleanStringChar
forgot some symbols which have now been added, ensuring the string is properly cleaned.- Constant-folds all casts and integral expressions (with the exception of type
Int
), leading to improved performance. - Increases accuracy of error reporting for keywords.
- Adds the
eval.stuck.outofscope
log topic in order to be able to spot when we get stuck due to a function being out of scope. - Improves the error reporting for syntactically incorrect records.
IPragma
now carries anFC
with it for better error reporting.- Adds the number of enum constructors to enum types during codegen, to allow
for trivial conversion to, e.g.,
Bits32
. - Adds constant-folding for
Nat
literals. - Fixes
CyclicMeta
inTTImp.ProcessDef
being considered a recoverable error.
-
The IDE protocol and its serialisation to S-Expressions are factored into a separate module hierarchy Protocol.{Hex, SExp, IDE}.
-
File context ranges sent in the IDE protocol follow the same convention as Bounds values in the parser:
- all offsets (line and column) are 0-based.
- Lines: start and end are within the bounds
- Column:
- start column is within the bounds;
- end column is after the bounds.
This changes behaviour from previous versions of the protocol. Matching PRs in the emacs modes:
-
The IDE protocol now supports specifying a socket and hostname via the
--ide-mode-socket
flag, allowing multiple IDE server instances to run on the same machine.
- Case-split no longer generates syntactically invalid Idris when splitting on auto-implicits.
- Case-split no longer shadows the function name when an internal named argument has the same name as the function.
- Case-split now avoids using upper-case names for pattern variables.
elemBy
andelem
are now defined for anyFoldable
structure. The specialised versions defined inData.(List/SnocList/Vect)
have been removed.filter
andmapMaybe
functions forList
were moved toprelude
frombase
.- Basic functions of
SnocList
((++)
,length
,filter
,mapMaybe
) and implementations ofEq
andOrd
were moved toprelude
frombase
. This may lead to a need to qualifying functions (e.g.List.filter
) due to possible ambiguity. - "Fish" and "chips" operators of
SnocList
were moved toPrelude.Types
fromPrelude.Basics
. - Adds
contra
for returning the opposite of a givenOrdering
. - Fix
pow
, using backend implementations. - Add
subtract
alias for(-)
- Adds
System.run
, which runs a shell command, and returns the stdout and return code of that run. - Adds escaped versions of
System.system
,Systen.File.popen
, andSystem.run
, which take a list of arguments, and escapes them. - Adds the
Injective
interface in moduleControl.Function
. - Changes
System.pclose
to return the return code of the closed process. - Deprecates
base
'sData.Nat.Order.decideLTE
in favor ofData.Nat.isLTE
. - Removes
base
's deprecatedSystem.Directory.dirEntry
. UsenextDirEntry
instead. - Removes
base
's deprecatedData.String.fastAppend
. UsefastConcat
instead. System.File.Buffer.writeBufferData
now returns the number of bytes that have been written when there is a write error.System.File.Buffer.readBufferData
now returns the number of bytes that have been read into the buffer.- Adds the
Data.List.Quantifiers.Interleaving
andData.List.Quantifiers.Split
datatypes, used for provably splitting a list into a list of proofs and a list of counter-proofs for a given property. - Properties of the
List1
type were moved fromData.List1
toData.List1.Properties
. Syntax.PreorderReasoning
was moved tobase
fromcontrib
.- Move the types and functions in
Data.Vect.Quantifiers
to their respective namespaces (All
for all-related things, andAny
for any-related things) to make the code consistent with the other quantifiers (List
andSnocList
). - Set the
all
andany
functions for proof-quantifiers topublic export
instead ofexport
, allowing them to be used with auto-implicitIsYes
. - Legacy duplicating type
Given
(with constructorAlways
) is removed from theDecidable.Decidable
. Use the typeIsYes
(with constructorItIsYes
) from the same module instead. - Adds
Data.List1.Elem
, ported fromData.List.Elem
. - Adds
Data.List1.Quantifiers
, ported fromData.List.Quantifiers
. - Changes the order of arguments in
RWST
transformer's runners functions (runRWST
.evalRWST
,execRWST
), now transformer argument is the last, as in the other standard transformers, likeReaderT
andStateT
. - Adds
Data.Fin.finToNatEqualityAsPointwise
, which takes a witness offinToNat k = finToNat l
and provesk ~~~ l
. - Drop first argument (path to the
node
executable) fromSystem.getArgs
on the Node.js backend to make it consistent with other backends. - Adds
Uninhabited
instances forFZ ~~~ FS k
andFS k ~~~ FZ
. - Change behavior of
channelPut
on the Racket backend to match the behavior on the Chez backend. fGetLine
has been marked ascovering
instead oftotal
.- Adds the ability to derive
Functor
andTraversable
using%runElab derive
in the implementation definition. - Fixes memory leaks in
currentDir
,fGetLine
, andfGetChars
. - Fixes
natToFinLT
being O(n) by proving thatSo (x < n)
impliesLT x n
, allowing the compiler to optimisenatToFinLT
away. - Fixes
SnocList.foldr
andSnocList.foldMap
to be performant and stack-safe. - Add
insertAt
,deleteAt
andreplaceAt
forList
- Add
scanr
,scanr1
andunsnoc
forVect
- Implement
DecEq
forSnocList
- Refactors
Test.Golden.runTest
to useSystem.Concurrency
from the base libraries instead ofSystem.Future
fromcontrib
. In addition to reducing the dependency oncontrib
in the core of Idris2, this also seems to provide a small performance improvement formake test
. - Splits
runner
intorunnerWith
for processing the options and configuring the test pools, and a newrunner
function for reading options from the command-line.
System.Random
support forInt
changed toInt32
; it already limited itself to 32 bits but now that is codified. JavaScript backends are now supported.- Removes
contrib
's deprecatedData.Num.Implementations
module. SeePrelude.Interfaces
instead. - Implements
Show tok => Show (ParsingError tok)
forText.Parser.Core
. Control.Linear.LIO
has been moved fromcontribs
tolinear
to guarantee that idris2 does not need to rely on contribs anymore.
Control.Linear.Network
now supportsconnect
in the linear environment, and can also access thesendBytes
,recvBytes
andrecvAllBytes
functions of the underlyingSocket
module.
-
Creates the
papers
andlinear
libraries to remove bits of type theory and pl propaganda fromcontrib
and instead clearly have them as implementations of their respective papers. -
Creates
Data.Linear.{Notation,LEither,LMaybe,LVect,Pow}
. -
Moves
Data.Container
, based on the papers "Categories of Containers" by Michael Abbott, Thorsten Altenkirch, and Neil Ghani, and "Derivatives of Containers" by Michael Abbott, Thorsten Altenkirch, Neil Ghani, and Conor McBride, topapers
. https://doi.org/10.1007/3-540-36576-1_2 https://doi.org/10.1007/3-540-44904-3_2 -
Moves the implementation of "Indexed induction-recursion" by Dybjer and Setzer to
papers
. https://doi.org/10.1016/j.jlap.2005.07.001 -
Ports "How to Take the Inverse of a Type" by Daniel Marshall and Dominic Orchard as
Data.Linear.{Communications,Diff,Inverse}
. https://doi.org/10.4230/LIPIcs.ECOOP.2022.5 -
Moves
Data.OpenUnion
, inspired by the paper "Freer monads, more extensible effects" by Oleg Kiselyov and Hiromi Ishii, topapers
. https://doi.org/10.1145/2887747.2804319 -
Moves
Data.Recursion.Free
, partially based on "Turing-Completeness Totally Free" by Conor McBride, topapers
. https://doi.org/10.1007/978-3-319-19797-5_13 -
Moves
Data.Tree.Perfect
topapers
. -
Moves
Data.Vect.Binary
, taken from the paper "Heterogeneous Binary Random-access Lists" by Wouter Swierstra, topapers
. https://doi.org/10.1017/S0956796820000064 -
Ports "Applications of Applicative Proof Search" by Liam O'Connor as
Search.{Generator,HDecidable,Negation,Properties,CTL,GCL}
. https://doi.org/10.1145/2976022.2976030 -
Implements "Dependent Tagless Final" by Nicolas Biri as
Language.Tagless
. https://doi.org/10.1145/3498886.3502201 -
Ports Todd Waugh Ambridge's Agda blog post series "Search over uniformly continuous decidable predicates on infinite collections of types" as
Search.Tychonoff
. https://www.cs.bham.ac.uk/~txw467/tychonoff/InfiniteSearch1.html -
Ports "Auto in Agda - Programming proof search using reflection" by Wen Kokke and Wouter Swierstra as
Search.Auto
. https://doi.org/10.1007/978-3-319-19797-5_14 -
Ports "Computing with Generic Trees in Agda" by Stephen Dolan as
Data.W
. https://doi.org/10.1145/3546196.3550165
- Adds docstrings for the lambda-lifted IR.
- Package files are now installed along-side build artifacts for installed
packages. This means all transitive dependencies of packages you specify with
the
depends
field are added automatically. - No longer builds
contrib
andpapers
during bootstrap, as these may rely on new features not yet present in the bootstrap version of Idris2.
- Missing methods in implementations now give a compile time error. This was always the intended behaviour, but until now had not been implemented!
- Records now work in
parameters
blocks andwhere
clauses. - Implementations of interfaces now work in
parameters
blocks andwhere
clauses - The syntax for Name reflection has changed, and now requires a single brace
instead of a double brace, e.g.
`{x}
- Raw string literals allows writing string while customising the escape
sequence. Start a string with
#"
in order to change the escape characters to\#
, close the string with"#
. Remains compatible with multiline string literals. - Interpolated strings allows inserting expressions within string literals
and avoid writing concatenation explicitly. Escape a left curly brace
\{
to start an interpolation slice and close it with a right curly brace}
to resume writing the string literal. The enclosed expression must be of typeString
. Interpolated strings are compatible with raw strings (the slices need to be escaped with\#{
instead) and multiline strings. - We now support ellipses (written
_
) on the left hand side of awith
clause. Ellipses are substituted for by the left hand side of the parent clause i.e.
filter : (p : a -> Bool) -> List a -> List a
filter p [] = []
filter p (x :: xs) with (p x)
_ | True = x :: filter p xs
_ | False = filter p xs
means
filter : (p : a -> Bool) -> List a -> List a
filter p [] = []
filter p (x :: xs) with (p x)
filter p (x :: xs) | True = x :: filter p xs
filter p (x :: xs) | False = filter p xs
- Added incremental compilation, using either the
--inc
flag or theIDRIS2_INC_CGS
environment variable, which compiles modules incrementally. In incremental mode, the final build step is much faster than in whole program mode (the default), at the cost of runtime performance being about half as good. The--whole-program
flag overrides incremental compilation, and reverts to whole program compilation. Incremental compilation is currently supported only by the Chez Scheme back end. This is currently supported only on Unix-like platforms (not yet Windows)- Note that you must set
IDRIS2_INC_CGS
when building and installing all libraries you plan to link with an incremental build. - Note also that this is experimental and not yet well tested!
- Note that you must set
- The type checker now tries a lot harder to avoid reducing expressions where it is not needed. This can give a huge performance improvement in programs that potentially do a lot of compile time evaluation. However, sometimes reducing expressions can help in totality and quantity checking, so this may cause some programs not to type check which previously did - in these cases, you will need to give the reduced expressions explicitly.
- Added
--list-packages
CLI option. - Added
--total
CLI option.
Changed
- Removed
Data.Strings
. UseData.String
instead.
- Reimplement the
Channels
primitive in the Chez-Scheme backend since it had some non-deterministic properties (see issue #1552). NOTE: Due to complications with race-conditions, Chez not having channels built-in, etc, the reimplementation changes the semantics slightly:channelPut
no longer blocks until the value has been received under thechez
backend, but instead only blocks if there is already a value in the channel that has not been received. With thanks to Alain Zscheile (@zseri) for help with understanding condition variables, and figuring out where the problems were and how to solve them.
- The old system of interfaces for defining order relations (to say,
for instance, that LTE is a partial order) is replaced with a new
system of interfaces. These interfaces defines properties of binary
relations (functions of type
ty -> ty -> Type
), and orders are defined simply as bundles of these properties.
- Added a new makefile target to install Idris 2 library documentation. After
make install
, typemake install-libdocs
to install it. After that, the index file can be found here:idris2 --libdir`/docs/index.html`.
- Desugar non-binding sequencing in do blocks to (
>>
) (#1095) - Multiline Strings with
"""
as delimiters (#1097) - Force strict indentation after usage of
with
keyword (#1107) - The syntax for parameter blocks has been updated. It now allows to declare implicit parameters and give multiplicities for parameters. The old syntax is still available for compatibility purposes but will be removed in the future.
- Add support for SnocList syntax:
[< 1, 2, 3]
desugars intoLin :< 1 :< 2 :< 3
and their semantic highlighting. - Underscores can be used as visual separators for digit grouping purposes in
integer literals:
10_000_000
is equivalent to10000000
and0b1111_0101_0000
is equivalent to0b111101010000
. This can aid readability of long literals, or literals whose value should clearly separate into parts, such as bytes or words in hexadecimal notation.
- Added more optimisations and transformations, particularly on case blocks, list-shaped types, and enumerations, so generated code will often be slightly faster.
- Added
--profile
flag, which generates profile data if supported by a back end. Currently supported by the Chez and Racket backends. - New
%builtin
pragma for compiling user defined natural numbers to primitiveInteger
s (see the docs) - The
version
field in.ipkg
files is now used. Packages are installed into a directory which includes its version number, and dependencies can have version number ranges using<=
,<
,>=
,>
,==
to express version constraints. Version numbers must be in the form of integers, separated by dots (e.g.1.0
,0.3.0
,3.1.4.1.5
etc) - Idris now looks in the current working directory, under a subdirectory
depends
for local installations of packages before looking globally. - Added an environment variable
IDRIS2_PACKAGE_PATH
for extending where to look for packages. - Added compiler warnings flags (
-W
prefix):-Wno-shadowing
: disable shadowing warnings.-Werror
: treat warnings as errors.
- Experimental flag (
-Xcheck-hashes
) to check hashes instead of filesystem times to determine if files should be recompiled. Should help with CI/CD caching.
- Added
:search
command, which searches for functions by type :load
/:l
and:cd
commands now only accept paths surrounded by double quotes- Added a timeout to "generate definition" and "proof search" commands,
defaulting to 1 second (1000 milliseconds) and configurable with
%search_timeout <time in milliseconds>
Added
Bifoldable
andBitraversable
interfaces.Foldable
addfoldlM
,foldMap
, andtoList
.Monad
interface>=>
,<=<
(Kleisli Arrows), and flipped bind (=<<
).Pair
Applicative and Monad implementations.SnocList
datatype (fliped cons of a linked list).(.:)
function "blackbird operator" (Composition of a two-argument function with a single-argument one.)on
function (Eg,((+) `on` f) x y = f x + f y
)
Changed
===
,~=~
, and<+>
operator precedence- Exctracted
Cast
interface and implementations fromPrelude.Types
toPrelude.Cast
- Renamed
Data.Strings
toData.String
Hidden
countFrom
Added
Control.Applicative.Const
.- New
Control.Monad
Monad Transformers types. Data.Bits
, an interface for bitwise operations.Data.Colist
andData.Colist1
.Data.Contravariant
interface for contravariant functors.Data.List
unzip
function.Data.List1
zip*
andunzip*
functions.Data.SnocList
.Data.Stream
unzipWith
andunzipWith3
fuctions.Data.Vect
unzipWith
andunzipWith3
functions.System.File
withFile
and total read functions.
Changed:
- Restructured Monad Transformers in
Control.Monad
zip
precedence
Added
Control.Validation
, a library for dependent types input validation.System.Console.GetOpt
, a library for specifying and parsing command line options.
- Moved
tests/Lib.idr
to package asTest/Golden.idr
. - Removed
contrib/Test/Golden.idr
which duplicated the test framework now in thetest
package.
- Now always uses
blodwen-sleep
instead ofidris2_sleep
in order to not block the Racket runtime whensleep
is called. - Redid condition variables in the Racket codegen based on page 5 of the
Microsoft Implementing CVs paper.
Previously, they were based on an implementation using semaphores and
asynchronous channels, which worked apart from
broadcast
. The rework fixesbroadcast
at the cost of losingwait-timeout
due to increased complexity of their internals and interactions between their associated functions.
- Now use
Number
to represent up to 32 bit precision signed and unsigned integers.Int32
still goes viaBigInt
for multiplication to avoid precision issues when getting results larger thanNumber.MAX_SAFE_INTEGER
.Bits32
goes viaBigInt
for multiplication for the same reason as well as for all bitops, sinceNumber
uses signed 32 bit integers for those. - Now use
Number
instead ofBigInt
to represent up to 32 bit fixed precision signed and unsigned integers. This should make interop with the FFI more straight forward, and might also improve performance.
- This code generator produces many Chez Scheme files and compiles them separately instead of producing one huge Scheme program. This significantly reduces the amount of memory needed to build large programs. Since this backend will skip calling the Chez compiler on modules that haven't changed, it also leads to shorter compilation times in large codebases where only some files have changed -- for example when developing Idris2 code generators. The codegen has a large parallelisation potential but at the moment, it is significantly slower for a full rebuild of a large codebase (the code generation stage takes about 3x longer).
- The API now exposes
Compiler.Separate.getCompilationUnits
, which can be used for separate code generation by any backend. - New fixed precision signed integer types
Int8
,Int16
,Int32
, andInt64
where added. In addition, all integral types now properly support all arithmetic and bitwise operations. - The compiler now provides primitive cast operations for all combinations
of primitives with the exception of going from
Double
toChar
and back, and going fromString
toChar
. - A new pragma
%doubleLit
to support overloaded floating point literals was added.
- Lots of small performance improvements, some of which may be especially noticeable in programs that do a lot of type level evaluation.
- Added HTML documentation generation, using the
--mkdoc
flag - Support for auto-completion in bash-like shells was added.
- Fixed case-splitting to respect any indentation there may be in the term being case-split and the surrounding symbols, instead of filtering out the whitespace and putting it back as indentation.
Library changes:
-
Overhaul of the concurrency primitives:
-
Renamed
System.Concurrency.Raw
toSystem.Concurrency
. -
Modified the implementation of
Prelude.IO.fork
in the Chez Scheme RTS, which now returns a semaphore instead of a thread object. This allows the main thread to wait for the child thread to finish (see next bullet). The Racket implementation already returned a thread descriptor, which could be used to wait for the thread to finish. -
Added
Prelude.IO.threadWait
which waits for a thread, identified by aThreadID
, to finish. This operation is supported by both the Chez Scheme and the Racket RTS'es. -
Added semaphores to
System.Concurrency
, supported by both the Chez Scheme and Racket RTS'es. -
Added barriers to
System.Concurrency
, supported by both the Chez Scheme and Racket RTS'es. -
Added synchronous channels to
System.Concurrency
, supported by both the Chez Scheme and Racket RTS'es. -
Fixed the support for mutexes in the Racket RTS. Formerly, they were implemented with semaphores, and calling
mutexRelease
multiple times would increment the internal counter multiple times, allowing multiple concurrentmutexAcquire
operations to succeed simultaneously. Currently,mutexRelease
fails when called on a mutex which isn't owned. (However,mutexRelease
does not check whether the mutex is in fact owned by the current thread, which may be a bug.) -
Modified the support for condition variables in the Racket RTS. Formerly, they were implemented using synchronous channels, meaning that: +
conditionSignal
was a blocking operation; and + callingconditionSignal
on a condition variable on which no thread was waiting would wake the next thread to callconditionWait
, whereas condition variables are supposed to be stateless, and only wake threads already in the queue. The implementation was replaced with an implementation based on asynchronous channels and mutexes, based on the following paper: Implementing Condition Variables with Semaphores by Andrew Birrell -
Removed
threadID
andblodwen-thisthread
. Formerly, in the Chez Scheme backend, this function returned "the thread ID of the current thread" as a value of typeThreadID
. However,fork
returned a "thread object" as a value of typeThreadID
. These are different kinds of values in Chez Scheme. As there was nothing one could do with a value of typeThreadID
, I chose to removethreadID
, as it allowed me to implementthreadWait
more easily. -
Renamed
blodwen-lock
andblodwen-unlock
toblodwen-mutex-acquire
andblodwen-mutex-release
for consistency, as these functions are referred to with acquire and release both in Chez Scheme and in the Idris2 concurrency module.
-
-
Added
Data.HVect
incontrib
, for heterogeneous vectors. -
Various other library functions added throughout
base
andcontrib
Command-line options changes:
- Added
--color
and--no-color
options for colored terminal output. Color is enabled by default. - Added
--console-width <auto|n>
option for printing margins. By default theauto
option is selected, the result is that the compiler detects the current terminal width and sets it as the option value, otherwise a user value can be provided. An explicit0
has the effect of simulating a terminal with unbounded width.
Language and compiler changes:
-
Removed multiplicity subtyping, as this is unsound and unfortunately causes more problems than it solves. This means you sometimes now need to write linear versions of functions as special cases. (Though note that the 1 multiplicity is still considered experimental, so hopefully this will change for the better in the future!)
-
Added new syntax for named applications of explicit arguments:
f {x [= t], x [= t], ...}
f {x [= t], x [= t], ..., _}
-
Added syntax for binding all explicit arguments (in the left hand side);
f {}
-
Added new syntax for record updates (without the need for the
record
keyword):{x := t, x $= t, ...}
-
Local implementations of interfaces (in
let
orwhere
blocks) now work, along with%hint
annotations on local definitions, meaning that local definitions can be searched in auto implicit search.- Note, though, that there are still some known limitations (with both local hints and local implementations) which will be resolved in the next version.
-
New experimental
refc
code generator, which generates C with reference counting. -
Added primitives to the parsing library used in the compiler to get more precise boundaries to the AST nodes
FC
.
REPL/IDE mode changes:
- Added
:color (on|off)
option for colored terminal output. - Added
:consolewidth (auto|n)
option for printing margins. Mirrors the command-line option.
Language changes:
Bits8
,Bits16
,Bits32
andBits64
primitive types added, with:Num
,Eq
,Ord
andShow
implementations.- Casts from
Integer
, for literals - Casts to
Int
(except forBits64
which might not fit),Integer
andString
- Passed to C FFI as
unsigned
- Primitives added in
Data.Buffer
- Elaborator reflection and quoting terms
- Requires extension
%language ElabReflection
- API defined in
Language.Reflection
, including functions for getting types of global names, constructors of data types, and adding new top level declarations - Implemented
%macro
function flag, to remove the syntactic noise of invoking elaborator scripts. This means the function must always be fully applied, and is run under%runElab
- Requires extension
- Add
import X as Y
- This imports the module
X
, adding aliases for the definitions in namespaceY
, so they can be referred to asY
.
- This imports the module
do
notation can now be qualified with a namespaceMyDo.do
opens ado
block where the>>=
operator used isMyDo.(>>=)
Library changes:
IO
operations in theprelude
andbase
libraries now use theHasIO
interface, rather than usingIO
directly.- Experimental
Data.Linear.Array
added tocontrib
, supporting mutable linear arrays with constant time read/write, convertible to immutable arrays with constant time read.- Anything in
Data.Linear
incontrib
, just like the rest ofcontrib
, should be considered experimental with the API able to change at any time! Further experiments inData.Linear
are welcome :).
- Anything in
- Experimental
Control.Linear.LIO
added tocontrib
, supporting computations which track the multiplicities of their return values, which allows linear resources to be tracked. - Added
Control.Monad.ST
, for update in-place viaSTRef
(which is likeIORef
, but can escape fromIO
). Also addedData.Ref
which provides an interface to bothIORef
andSTRef
. - Added
Control.ANSI
incontrib
, for usage of ANSI escape codes for text styling and cursor/screen control in terminals.
Command-line options changes:
- Removed
--ide-mode-socket-with
option.--ide-mode-socket
now accepts an optionalhost:port
argument. - Added options to override source directory, build directory and output
directory:
--source-dir
,--build-dir
,--output-dir
.- These options are also available as fields in the package description:
sourcedir
,builddir
,outputdir
.
- These options are also available as fields in the package description:
Compiler changes:
- It is now possible to create new backends with minimal overhead.
Idris.Driver
exposes the functionmainWithCodegens
that takes a list of codegens. The feature in documented here. - New code generators
node
andjavascript
.
REPL/IDE mode changes:
- Implemented
:module
command, to load a module during a REPL session. - Implemented
:doc
, which displays documentation for a name. - Implemented
:browse
, which lists the names exported by a namespace. - Added
:psnext
, which continues the previous proof search, looking for the next type correct expression- Correspondingly, added the IDE mode command
proof-search-next
(which takes no arguments)
- Correspondingly, added the IDE mode command
- Added
:gdnext
, which continues the previous program search, looking for the next type correct implementation- Correspondingly, added the IDE mode command
generate-def-next
(which takes no arguments)
- Correspondingly, added the IDE mode command
- Improved program search to allow deconstructing intermediate values, and in simple cases, the result of recursive calls.
The implementation is now self-hosted. To initialise the build, either use
the bootstrapping version of Idris2
or build from the generated Scheme, using make bootstrap
.
Language changes:
total
,covering
andpartial
flags on functions now have an effect.%default <totality status>
has been implemented. By default, functions must be at leastcovering
- That is,
%default covering
is the default status.
- That is,
- Fields of records can be accessed (and updated) using the dot syntax,
such as
r.field1.field2
orrecord { field1.field2 = 42 }
. For details, see the "records" entry in the user manual - New function flag
%tcinline
which means that the function should be inlined for the purposes of totality checking (but otherwise not inlined). This can be used as a hint for totality checking, to make the checker look inside functions that it otherwise might not. - %transform directive, for declaring transformation rules on runtime expressions. Transformation rules are automatically added for top level implementations of interfaces.
- A %spec flag on functions which allows arguments to be marked for partial evaluation, following the rules from "Scrapping Your Inefficient Engine" (ICFP 2010, Brady & Hammond)
- To improve error messages, one can use
with NS.name <term>
orwith [NS.name1, NS.name2, ...] <term>
to disable disambiguation for the given names in<term>
. Example:with MyNS.(>>=) do ...
.
Library additions:
- Additional file management operations in
base
- New module in
base
for time (System.Clock
) - New modules in
contrib
for JSON (Language.JSON.*
); random numbers (System.Random
)
Compiler updates:
- Data types with a single constructor, with a single unerased arguments,
are translated to just that argument, to save repeated packing and unpacking.
(c.f.
newtype
in Haskell)- A data type can opt out of this behaviour by specifying
noNewtype
in its options list.noNewtype
allows code generators to apply special handling to the generated constructor/deconstructor, for a newtype-like data type, that would otherwise be optimised away.
- A data type can opt out of this behaviour by specifying
- 0-multiplicity constructor arguments are now properly erased, not just given a placeholder null value.
Other improvements:
- Various performance improvements in the typechecker:
- Noting which metavariables are blocking unification constraints, so that they only get retried if those metavariables make progress.
- Evaluating
fromInteger
at compile time.
- Extend Idris2's literate mode to support reading Markdown and OrgMode files. For more details see: "literate" in the user manual.
Everything :). For full details, see: updates