Idris2/libs/base/base.ipkg
Edwin Brady 4726c32d94 Add --ignore-missing-ipkg flag
When bootstrapping, we're building things without packages being
available, so we can't expect to find them when looking for
dependencies. So, we find them another way, with an environment
variable. This flag is to tell Idris not to worry about missing
dependencies in this situation.

We also need to update the bootstrapping code, to deal with the new
version number format and new flag in the ipkg files for the libraries.
I think it's still safe to build from the previous version though - lets
see if CI agrees!
2021-02-27 19:39:47 +00:00

87 lines
2.1 KiB
Plaintext

package base
version = 0.3.0
opts = "--ignore-missing-ipkg"
modules = Control.App,
Control.App.Console,
Control.App.FileIO,
Control.Monad.Either,
Control.Monad.Error.Either,
Control.Monad.Error.Interface,
Control.Monad.Identity,
Control.Monad.Maybe,
Control.Monad.RWS,
Control.Monad.RWS.CPS,
Control.Monad.RWS.Interface,
Control.Monad.Reader,
Control.Monad.Reader.Interface,
Control.Monad.Reader.Reader,
Control.Monad.ST,
Control.Monad.State,
Control.Monad.State.Interface,
Control.Monad.State.State,
Control.Monad.Trans,
Control.Monad.Writer,
Control.Monad.Writer.CPS,
Control.Monad.Writer.Interface,
Control.WellFounded,
Data.Bool,
Data.Bool.Xor,
Data.Buffer,
Data.Colist,
Data.Colist1,
Data.DPair,
Data.Either,
Data.Fin,
Data.Fin.Order,
Data.Fuel,
Data.Fun,
Data.IOArray,
Data.IOArray.Prims,
Data.IORef,
Data.List,
Data.List.Elem,
Data.List.Views,
Data.List.Quantifiers,
Data.List1,
Data.Maybe,
Data.Morphisms,
Data.Nat,
Data.Nat.Order,
Data.Nat.Views,
Data.Primitives.Views,
Data.Ref,
Data.Rel,
Data.So,
Data.Stream,
Data.String,
Data.Strings,
Data.These,
Data.Vect,
Data.Vect.Elem,
Data.Vect.Quantifiers,
Data.Zippable,
Debug.Trace,
Decidable.Decidable,
Decidable.Equality,
Decidable.Equality.Core,
Decidable.Order,
Language.Reflection,
Language.Reflection.TT,
Language.Reflection.TTImp,
System,
System.Concurrency,
System.Clock,
System.Directory,
System.File,
System.FFI,
System.Info,
System.REPL