mirror of
https://github.com/idris-lang/Idris2.git
synced 2024-11-28 19:13:02 +03:00
Add Control.Validation module to contrib package.
This commit is contained in:
parent
f3168d16aa
commit
67bab6b088
@ -58,6 +58,7 @@ data NotBothZero : (n, m : Nat) -> Type where
|
||||
LeftIsNotZero : NotBothZero (S n) m
|
||||
RightIsNotZero : NotBothZero n (S m)
|
||||
|
||||
export
|
||||
Uninhabited (NotBothZero 0 0) where
|
||||
uninhabited LeftIsNotZero impossible
|
||||
uninhabited RightIsNotZero impossible
|
||||
|
@ -12,6 +12,8 @@ modules = Control.ANSI,
|
||||
Control.Algebra.Laws,
|
||||
Control.Algebra.Implementations,
|
||||
|
||||
Control.Validation,
|
||||
|
||||
Data.Bool.Algebra,
|
||||
|
||||
Data.Linear.Array,
|
||||
|
Loading…
Reference in New Issue
Block a user