mirror of
https://github.com/idris-lang/Idris2.git
synced 2024-11-20 17:18:26 +03:00
Public export Decidable.Decidable.decision
This commit is contained in:
parent
7d33c0438a
commit
5f27842cbc
@ -186,6 +186,8 @@ This CHANGELOG describes the merged but unreleased changes. Please see [CHANGELO
|
||||
* Some pieces of `Data.Fin.Extra` from `contrib` were moved to `base` to modules
|
||||
`Data.Fin.Properties`, `Data.Fin.Arith` and `Data.Fin.Split`.
|
||||
|
||||
* `Decidable.Decidable.decison` is now `public export`.
|
||||
|
||||
#### Contrib
|
||||
|
||||
* `Data.List.Lazy` was moved from `contrib` to `base`.
|
||||
|
@ -51,5 +51,6 @@ interface Decidable k ts p where
|
||||
|
||||
||| Given a `Decidable` n-ary relation, provides a decision procedure for
|
||||
||| this relation.
|
||||
public export
|
||||
decision : (ts : Vect k Type) -> (p : Rel ts) -> Decidable k ts p => liftRel ts p Dec
|
||||
decision ts p = decide {ts} {p}
|
||||
|
Loading…
Reference in New Issue
Block a user