Skip to content

Commit

Permalink
Public export Decidable.Decidable.decision
Browse files Browse the repository at this point in the history
  • Loading branch information
michaelmesser committed Jun 26, 2024
1 parent 7d33c04 commit 8dc0436
Show file tree
Hide file tree
Showing 2 changed files with 3 additions and 0 deletions.
2 changes: 2 additions & 0 deletions CHANGELOG_NEXT.md
Original file line number Diff line number Diff line change
Expand Up @@ -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`.
Expand Down
1 change: 1 addition & 0 deletions libs/base/Decidable/Decidable.idr
Original file line number Diff line number Diff line change
Expand Up @@ -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}

0 comments on commit 8dc0436

Please sign in to comment.