Idris2/idris2api.ipkg
Mathew Polzin fa06e9936b
Warn about unreachable default clauses (#1942)
* so much experimentation

* tests that show preliminary evidence the new stuff is working.

* small amount of cleanup

* more cleanup of various troubleshooting code.

* new test case added.

* only log unreachable indices if there are any.

* when traversing deeper simply skip over defaults since they have already been reviewed.

* Remove fallback clause that the changes in this PR correctly identified as unreachable.

* tidying up more.

* move some common functions to a new Core.Case.Util module.

* refer to case builder and case tree under new parent module.

* update imports to look for CaseTree in new submodule.

* update api ipkg

* remove unneeded application operators.

* remove or comment out unreachable default clauses caught by the changes in this PR.

* a bit of code documentation and renaming for clarity.

* bump previous version in CI.

* fix API usage of Util module.

* Add issue 1079 test cases.

* forgot to add new test cases file.

* remove commented-out lines by request of RefC author.

* Use a SortedSet instead of nubbing a list.

* update new case tree import.

* Update src/Core/Case/Util.idr

Co-authored-by: G. Allais <guillaume.allais@ens-lyon.org>

* remove function with nothing to offer above and beyond a differently named copy of the same code.

* replace a large tuple with a record; discover not all of the tuple's fields were needed.

* fix shadowing warning.

Co-authored-by: G. Allais <guillaume.allais@ens-lyon.org>
2021-10-02 12:55:21 +01:00

255 lines
5.5 KiB
Plaintext

package idris2
version = 0.5.1
modules =
Algebra,
Algebra.Preorder,
Algebra.Semiring,
Algebra.ZeroOneOmega,
Compiler.ANF,
Compiler.CaseOpts,
Compiler.Common,
Compiler.CompileExpr,
Compiler.Generated,
Compiler.Identity,
Compiler.Inline,
Compiler.LambdaLift,
Compiler.Opts.CSE,
Compiler.Separate,
Compiler.VMCode,
Compiler.ES.Ast,
Compiler.ES.Codegen,
Compiler.ES.Doc,
Compiler.ES.Javascript,
Compiler.ES.Node,
Compiler.ES.State,
Compiler.ES.TailRec,
Compiler.ES.ToAst,
Compiler.Interpreter.VMCode,
Compiler.RefC,
Compiler.RefC.CC,
Compiler.RefC.RefC,
Compiler.Scheme.Chez,
Compiler.Scheme.ChezSep,
Compiler.Scheme.Racket,
Compiler.Scheme.Gambit,
Compiler.Scheme.Common,
Core.AutoSearch,
Core.Binary,
Core.Binary.Prims,
Core.Case.CaseBuilder,
Core.Case.CaseTree,
Core.Case.Util,
Core.CompileExpr,
Core.Context,
Core.Context.Context,
Core.Context.Data,
Core.Context.Log,
Core.Core,
Core.Coverage,
Core.Directory,
Core.Env,
Core.FC,
Core.GetType,
Core.Hash,
Core.InitPrimitives,
Core.LinearCheck,
Core.Metadata,
Core.Name,
Core.Name.Namespace,
Core.Normalise,
Core.Normalise.Convert,
Core.Normalise.Eval,
Core.Normalise.Quote,
Core.Options,
Core.Options.Log,
Core.Ord,
Core.Primitives,
Core.Reflect,
Core.SchemeEval,
Core.Termination,
Core.Transform,
Core.TT,
Core.TTC,
Core.Unify,
Core.UnifyState,
Core.Value,
Core.SchemeEval.Builtins,
Core.SchemeEval.Compile,
Core.SchemeEval.Evaluate,
Core.SchemeEval.Quote,
Core.SchemeEval.ToScheme,
IdrisPaths,
Idris.CommandLine,
Idris.Desugar,
Idris.Desugar.Mutual,
Idris.Env,
Idris.Doc.HTML,
Idris.Doc.String,
Idris.Driver,
Idris.Error,
Idris.ModTree,
Idris.Package,
Idris.Package.Init,
Idris.Package.Types,
Idris.Parser,
Idris.Parser.Let,
Idris.Pretty,
Idris.Pretty.Render,
Idris.ProcessIdr,
Idris.REPL,
Idris.Resugar,
Idris.SetOptions,
Idris.Syntax,
Idris.Version,
Idris.Elab.Implementation,
Idris.Elab.Interface,
Idris.IDEMode.CaseSplit,
Idris.IDEMode.Commands,
Idris.IDEMode.Holes,
Idris.IDEMode.MakeClause,
Idris.IDEMode.Parser,
Idris.IDEMode.REPL,
Idris.IDEMode.SyntaxHighlight,
Idris.IDEMode.TokenLine,
Idris.REPL.Common,
Idris.REPL.Opts,
Idris.REPL.FuzzySearch,
Libraries.Control.ANSI,
Libraries.Control.ANSI.CSI,
Libraries.Control.ANSI.SGR,
Libraries.Control.Delayed,
Libraries.Data.ANameMap,
Libraries.Data.DList,
Libraries.Data.Fin,
Libraries.Data.Graph,
Libraries.Data.IMaybe,
Libraries.Data.IntMap,
Libraries.Data.IOArray,
Libraries.Data.IOMatrix,
Libraries.Data.LengthMatch,
Libraries.Data.List.Extra,
Libraries.Data.List.Lazy,
Libraries.Data.List1,
Libraries.Data.NameMap,
Libraries.Data.PosMap,
Libraries.Data.SortedMap,
Libraries.Data.SortedSet,
Libraries.Data.String.Extra,
Libraries.Data.String.Iterator,
Libraries.Data.StringMap,
Libraries.Data.StringTrie,
Libraries.Data.UserNameMap,
Libraries.Data.Version,
Libraries.System.Directory.Tree,
Libraries.Text.Bounded,
Libraries.Text.Distance.Levenshtein,
Libraries.Text.Lexer,
Libraries.Text.Lexer.Core,
Libraries.Text.Lexer.Tokenizer,
Libraries.Text.Literate,
Libraries.Text.Parser,
Libraries.Text.Parser.Core,
Libraries.Text.PrettyPrint.Prettyprinter,
Libraries.Text.PrettyPrint.Prettyprinter.Doc,
Libraries.Text.PrettyPrint.Prettyprinter.Render.HTML,
Libraries.Text.PrettyPrint.Prettyprinter.Render.String,
Libraries.Text.PrettyPrint.Prettyprinter.Render.Terminal,
Libraries.Text.PrettyPrint.Prettyprinter.SimpleDocTree,
Libraries.Text.PrettyPrint.Prettyprinter.Symbols,
Libraries.Text.PrettyPrint.Prettyprinter.Util,
Libraries.Text.Quantity,
Libraries.Text.Token,
Libraries.Utils.Binary,
Libraries.Utils.Hex,
Libraries.Utils.Octal,
Libraries.Utils.Path,
Libraries.Utils.Scheme,
Libraries.Utils.Shunting,
Libraries.Utils.String,
Libraries.Utils.Term,
Parser.Package,
Parser.Source,
Parser.Support,
Parser.Unlit,
Parser.Lexer.Common,
Parser.Lexer.Package,
Parser.Lexer.Source,
Parser.Rule.Package,
Parser.Rule.Source,
TTImp.BindImplicits,
TTImp.Elab,
TTImp.Impossible,
TTImp.Parser,
TTImp.PartialEval,
TTImp.ProcessBuiltin,
TTImp.ProcessData,
TTImp.ProcessDecls,
TTImp.ProcessDef,
TTImp.ProcessParams,
TTImp.ProcessRecord,
TTImp.ProcessRunElab,
TTImp.ProcessTransform,
TTImp.ProcessType,
TTImp.Reflect,
TTImp.TTImp,
TTImp.TTImp.Functor,
TTImp.Unelab,
TTImp.Utils,
TTImp.WithClause,
TTImp.Elab.Ambiguity,
TTImp.Elab.App,
TTImp.Elab.As,
TTImp.Elab.Binders,
TTImp.Elab.Case,
TTImp.Elab.Check,
TTImp.Elab.Delayed,
TTImp.Elab.Dot,
TTImp.Elab.Hole,
TTImp.Elab.ImplicitBind,
TTImp.Elab.Lazy,
TTImp.Elab.Local,
TTImp.Elab.Prim,
TTImp.Elab.Quote,
TTImp.Elab.Record,
TTImp.Elab.Rewrite,
TTImp.Elab.RunElab,
TTImp.Elab.Term,
TTImp.Elab.Utils,
TTImp.Interactive.CaseSplit,
TTImp.Interactive.ExprSearch,
TTImp.Interactive.GenerateDef,
TTImp.Interactive.MakeLemma,
Yaffle.Main,
Yaffle.REPL
depends = network
sourcedir = "src"