mirror of
https://github.com/idris-lang/Idris2.git
synced 2024-12-14 22:02:07 +03:00
22 lines
341 B
Idris
22 lines
341 B
Idris
|
module FailingTotality
|
||
|
|
||
|
%default total
|
||
|
|
||
|
failing "x is not covering."
|
||
|
|
||
|
x : Bool -> Nat
|
||
|
x True = 0
|
||
|
|
||
|
|
||
|
failing "x is not total, possibly not terminating due to recursive
|
||
|
path FailingTotality.x -> FailingTotality.x"
|
||
|
|
||
|
x : Bool
|
||
|
x = x
|
||
|
|
||
|
failing "D is not total, not strictly positive"
|
||
|
|
||
|
data D : Type where
|
||
|
Lam : (D -> D) -> D
|
||
|
|