mirror of
https://github.com/idris-lang/Idris2.git
synced 2024-12-01 09:49:24 +03:00
a972778eab
They don't all pass yet, for minor reasons. Coming shortly... Unfortunately the startup overhead for chez is really noticeable here!
21 lines
336 B
Idris
21 lines
336 B
Idris
import Data.Fin
|
|
|
|
data NNat = NZ | NS NNat
|
|
|
|
zsym : (x : NNat) -> x = NZ -> NZ = x
|
|
zsym NZ Refl = Refl
|
|
zsym (NS _) Refl impossible
|
|
|
|
zsym' : (x : NNat) -> x = NZ -> NZ = x
|
|
zsym' NZ Refl = Refl
|
|
|
|
foo : Nat -> String
|
|
foo 0 = "zero"
|
|
foo 1 = "one"
|
|
foo x = "something else"
|
|
|
|
bar : Fin (S (S (S Z))) -> String
|
|
bar 0 = "a"
|
|
bar 1 = "b"
|
|
bar 2 = "c"
|