..
Bool
Add some algebra implementations
2020-07-17 08:25:20 -05:00
Fin
Add totality annotations to src
and libs/{prelude, base}
2021-06-12 21:06:08 -05:00
IOArray
Add totality annotations to src
and libs/{prelude, base}
2021-06-12 21:06:08 -05:00
List
[ base ] Some lacking implementations for Uninhabited
were added
2021-06-15 15:07:54 +03:00
Nat
Add totality annotations to src
and libs/{prelude, base}
2021-06-12 21:06:08 -05:00
Primitives
Add totality annotations to src
and libs/{prelude, base}
2021-06-12 21:06:08 -05:00
Vect
[ base ] Some lacking implementations for Uninhabited
were added
2021-06-15 15:07:54 +03:00
Bifoldable.idr
Add totality annotations to src
and libs/{prelude, base}
2021-06-12 21:06:08 -05:00
Bits.idr
Add Data.Bits to base ( #1033 )
2021-03-04 20:59:56 +00:00
Bool.idr
[ base ] Not (a == b)
implies not a == b
( #1315 )
2021-04-22 13:16:26 +01:00
Buffer.idr
Check sizes of buffers and strings in TTCs
2021-06-23 18:08:27 +01:00
Colist1.idr
Cleanup List1 ( #1091 )
2021-03-17 14:07:52 +00:00
Colist.idr
[ base ] Some lacking implementations for Uninhabited
were added
2021-06-15 15:07:54 +03:00
Contravariant.idr
Add totality annotations to src
and libs/{prelude, base}
2021-06-12 21:06:08 -05:00
DPair.idr
[ new ] Interface implementations for Subset
2021-03-09 11:25:03 +00:00
Either.idr
Add Bifunctor interface ( #701 )
2020-09-30 10:51:07 +01:00
Fin.idr
Merge pull request #1598 from gallais/show-void
2021-06-23 18:11:40 +01:00
Fuel.idr
[ new ] Proof search from 'Applications of Applicative Proof Search' ( #1093 )
2021-03-01 08:29:43 +00:00
Fun.idr
Some cleanup was done. Changed code is mosly equivalent to the former.
2021-02-16 19:05:33 +00:00
IOArray.idr
Add totality annotations to src
and libs/{prelude, base}
2021-06-12 21:06:08 -05:00
IORef.idr
Add totality annotations to src
and libs/{prelude, base}
2021-06-12 21:06:08 -05:00
List1.idr
Cut unneeded type specifications
2021-06-28 16:22:27 +01:00
List.idr
Merge pull request #1489 from buzden/some-uninhabiteds
2021-06-23 16:17:32 +01:00
Maybe.idr
Add totality annotations to src
and libs/{prelude, base}
2021-06-12 21:06:08 -05:00
Morphisms.idr
Simplify some lambdas ( #1561 )
2021-06-16 15:22:30 +01:00
Nat.idr
[ base ] Some lacking implementations for Uninhabited
were added
2021-06-15 15:07:54 +03:00
Ref.idr
Add totality annotations to src
and libs/{prelude, base}
2021-06-12 21:06:08 -05:00
Rel.idr
Add totality annotations to src
and libs/{prelude, base}
2021-06-12 21:06:08 -05:00
SnocList.idr
[ close #1384 ] built-in Snoc-lists [< 1, 2, 3 ] ( #1383 )
2021-05-20 12:56:25 +01:00
So.idr
[ fix #899 ] Be careful when generating an impossible LHS ( #1081 )
2021-02-22 09:53:30 +00:00
Stream.idr
[ fix #1581 ] public export Range functions and implementations ( #1602 )
2021-06-28 16:52:23 +01:00
String.idr
[ cleanup ] Test.Golden ( #1526 )
2021-06-21 17:30:11 +01:00
These.idr
[ new ] Add Bifoldable and Bitraversable interfaces to Prelude ( #1265 )
2021-04-08 17:25:37 +01:00
Vect.idr
include the other definition of drop because both are quite useful.
2021-06-14 11:44:38 +01:00
Zippable.idr
Make zip
infixr 6
2021-02-23 10:54:28 +00:00