Fix bootstrap

This was broken in #425, because Idris2-boot hasn't implemented the
fix for #116
This commit is contained in:
Niklas Larsson 2020-07-08 22:33:37 +02:00
parent b955d2e50c
commit 1d7378778a

View File

@ -460,11 +460,12 @@ runRepl : {auto c : Ref Ctxt Defs} ->
runRepl fname = do
u <- newRef UST initUState
m <- newRef MD initMetadata
case fname of
Nothing => pure ()
Just fn => do
errs <- loadMainFile fn
displayErrors errs
the (Core ()) $
case fname of
Nothing => pure ()
Just fn => do
errs <- loadMainFile fn
displayErrors errs
repl {u} {s}