Idris2 icon indicating copy to clipboard operation
Idris2 copied to clipboard

A purely functional programming language with first class types

Results 306 Idris2 issues
Sort by recently updated
recently updated
newest added

**Issue by [nicolabotta](https://github.com/nicolabotta)** _Tuesday Oct 29, 2019 at 07:48 GMT_ _Originally opened as https://github.com/edwinb/Idris2-boot/issues/146_ ---- Is there a way of accessing these values in Idris 2? Something like `Numeric.IEEE`in Haskell?...

good first issue
Feature request
language: float

``` data Name : Type where UN : String -> Name -- user written name MN : String -> Int -> Name -- machine generated name data IsVar : Name...

status: confirmed bug
language: with

Seems like the compiler doesn't expand field projections of records unless they are explicitly deconstructed. # Minimal Example ``` public export record SimpleRecord where constructor MkSimpleRecord simpleField : Bool public...

Feature request
language: record
implem: eta

The compiler seems conflicted whether it would like linear arguments to be used in `with` clauses or not. ```idris pair : (1 _ : a) -> b -> (a, b)...

status: confirmed bug
language: quantity
language: with

I get a cryptic error message while lifting a `Preorder` relationship to `Maybe`. The type-checker is unable to unify identical types. # Steps to Reproduce Using the definition of `Preorder`...

error: bad message
status: confirmed bug
language: generalisation

Version: 0.2.0 OS: Windows using WSL Changed `PREFIX` to `/usr/local` and installed. Works fine while under `root`/`sudo` shell, or using `sudo idris2`, but shows `Uncaught error: (implicit):1:1--1:1:Prelude not found` on...

good first issue
Installation Issue
status: confirmed bug

# Steps to Reproduce ``` import Data.List.Elem %default total Subset : List a -> List a -> Type Subset xs ys = {0 x : a} -> Elem x xs...

status: confirmed bug
implem: scope

# Steps to Reproduce ``` data Thin : List a -> List a -> Type where Nil : Thin [] [] Skip : Thin xs ys -> Thin xs (y::ys)...

error: bad message
language: generalisation

Not a big deal, but the problem here is that `C` doesn't import `A`, so when it evals the `Elab` in `B`, (which returns an elab script that does reference...

enhancement
good first issue
language: reflection
error: reporting

I experiment with idris2 custom code generation backend, and it seems that the order `-p` arguments are important for the compilation result. ``` euler% idris2 -p contrib -p network -p...

status: confirmed bug
language: packaging
implem: scope
implem: import
implem: compilation