Idris2/libs/base/base.ipkg

131 lines
3.3 KiB
Plaintext

package base
version = 0.6.0
opts = "--ignore-missing-ipkg -Wno-shadowing"
modules = Control.App,
Control.App.Console,
Control.App.FileIO,
Control.Applicative.Const,
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,
Control.Function,
Control.Function.FunExt,
Control.Relation,
Control.Ord,
Control.Order,
Data.Bifoldable,
Data.Bits,
Data.Bool,
Data.Bool.Xor,
Data.Buffer,
Data.Colist,
Data.Colist1,
Data.Contravariant,
Data.DPair,
Data.Either,
Data.Fin,
Data.Fin.Order,
Data.Fuel,
Data.Fun,
Data.IOArray,
Data.IOArray.Prims,
Data.IORef,
Data.List,
Data.SnocList,
Data.SnocList.Elem,
Data.SnocList.Quantifiers,
Data.SnocList.Operations,
Data.List.Elem,
Data.List.HasLength,
Data.List.Views,
Data.List.Quantifiers,
Data.List1,
Data.List1.Elem,
Data.List1.Quantifiers,
Data.List1.Properties,
Data.Maybe,
Data.Morphisms,
Data.Nat,
Data.Nat.Order,
Data.Nat.Views,
Data.Primitives.Views,
Data.Ref,
Data.Rel,
Data.Singleton,
Data.So,
Data.SortedMap,
Data.SortedMap.Dependent,
Data.SortedSet,
Data.Stream,
Data.String,
Data.These,
Data.Vect,
Data.Vect.Elem,
Data.Vect.AtIndex,
Data.Vect.Quantifiers,
Data.Zippable,
Debug.Trace,
Deriving.Common,
Deriving.Foldable,
Deriving.Functor,
Deriving.Show,
Deriving.Traversable,
Decidable.Decidable,
Decidable.Equality,
Decidable.Equality.Core,
Language.Reflection,
Language.Reflection.TT,
Language.Reflection.TTImp,
Syntax.PreorderReasoning,
Syntax.PreorderReasoning.Generic,
System,
System.Clock,
System.Concurrency,
System.Directory,
System.Errno,
System.Escape,
System.FFI,
System.File,
System.File.Buffer,
System.File.Error,
System.File.Handle,
System.File.Meta,
System.File.Mode,
System.File.Permissions,
System.File.Process,
System.File.ReadWrite,
System.File.Support,
System.File.Types,
System.File.Virtual,
System.Info,
System.REPL,
System.Signal