mirror of
https://github.com/idris-lang/Idris2.git
synced 2024-12-14 05:46:47 +03:00
13 lines
161 B
Idris
13 lines
161 B
Idris
|
import Language.Reflection
|
||
|
|
||
|
x : TTImp
|
||
|
x = `(with Prelude.Nil [])
|
||
|
|
||
|
%language ElabReflection
|
||
|
|
||
|
x' : Elab (List Nat)
|
||
|
x' = check x
|
||
|
|
||
|
l : List Nat
|
||
|
l = 1 :: %runElab x'
|