Require all definitions to be total in tests/typedd-book/chapter11/ArithCmdDo.idr

This commit is contained in:
Kamil Shakirov 2020-10-21 13:54:24 +06:00 committed by G. Allais
parent 71a638ef28
commit 127db79a6b

View File

@ -2,7 +2,7 @@ import Data.Primitives.Views
import Data.Strings
import System
-- %default total
%default total
export
data Command : Type -> Type where