mirror of
https://github.com/idris-lang/Idris2.git
synced 2024-12-20 18:21:47 +03:00
52 lines
911 B
Idris
52 lines
911 B
Idris
|
module RefDefsDeep
|
||
|
|
||
|
import Language.Reflection
|
||
|
|
||
|
import RefDefs
|
||
|
|
||
|
%default total
|
||
|
|
||
|
%language ElabReflection
|
||
|
|
||
|
logCurrFn : Elab ()
|
||
|
logCurrFn = do
|
||
|
currFn <- getCurrentFn
|
||
|
logMsg "elab" 0 "=== current fn: \{show currFn} ==="
|
||
|
|
||
|
%runElab logCurrFn
|
||
|
|
||
|
f : Nat -> Nat
|
||
|
f x = case %runElab logCurrFn of () => x + 4
|
||
|
|
||
|
f' : Nat -> Nat
|
||
|
f' x = x + case %runElab logCurrFn of () => 4
|
||
|
|
||
|
f'' : Nat -> Nat
|
||
|
f'' Z = 4
|
||
|
f'' (S x) = f $ case %runElab logCurrFn of () => x
|
||
|
|
||
|
f''' : Nat -> Nat
|
||
|
f''' x = case x of
|
||
|
Z => 4
|
||
|
S x => f $ case %runElab logCurrFn of () => x
|
||
|
|
||
|
n : Nat -> Nat
|
||
|
n x = x + f x where
|
||
|
f : Nat -> Nat
|
||
|
f x = case %runElab logCurrFn of () => x + 4
|
||
|
|
||
|
w : Nat -> Nat
|
||
|
w x with (x + 5)
|
||
|
_ | Z = x + case %runElab logCurrFn of () => 4
|
||
|
_ | S n = f $ case %runElab logCurrFn of () => n
|
||
|
|
||
|
%runElab
|
||
|
traverse_ printRefDefs
|
||
|
[ `{f}
|
||
|
, `{f'}
|
||
|
, `{f''}
|
||
|
, `{f'''}
|
||
|
, `{n}
|
||
|
, `{w}
|
||
|
]
|