Add documentation for Not.

This commit is contained in:
Marshall Abrams 2023-08-14 22:44:07 -05:00
parent badf1e98c8
commit bdb6531b86

View File

@ -6,6 +6,10 @@ import Prelude.Ops
%default total
||| `Not x` is an alias for `x -> Void`, indicating that any term of type `x`
||| leads to a contradiction. It can be used in conjunction with `void` or
||| `absurd`.
public export
Not : Type -> Type
Not x = x -> Void