mirror of
https://github.com/idris-lang/Idris2.git
synced 2024-12-17 16:21:46 +03:00
498421a236
This has caught a couple of things in the Idris 2 code base itself. Some tests needed partial annotations too.
18 lines
516 B
Idris
18 lines
516 B
Idris
partial
|
|
bar : (n : Nat) -> (m : Nat) -> n = m -> Nat
|
|
bar (S m) (S m) (Refl {x = S m}) = m
|
|
|
|
data Baz : Int -> Type where
|
|
AddThings : (x : Int) -> (y : Int) -> Baz (x + y)
|
|
|
|
addBaz : (x : Int) -> Baz x -> Int
|
|
addBaz (x + y) (AddThings x y) = x + y
|
|
|
|
-- Not allowed in Idris 2, we use unification rather than matching!
|
|
-- addBaz2 : (x : Int) -> Baz x -> Int
|
|
-- addBaz2 (_ + _) (AddThings x y) = x + y
|
|
|
|
-- Also not allowed in Idris 2!
|
|
-- addBaz3 : (x : Int) -> Baz x -> Int
|
|
-- addBaz3 (x + y) (AddThings _ _) = x + y
|