├── .editorconfig ├── .gitattributes ├── .github ├── ISSUE_TEMPLATE │ ├── feature-requests-and-proposals.md │ ├── installation-problem.md │ └── language-problem.md ├── linters │ ├── .chktexrc │ ├── .ecrc │ ├── .markdown-lint.yml │ ├── .stylelintrc.json │ └── .textlintrc.yml ├── pull_request_template.md ├── scripts │ └── katla.sh └── workflows │ ├── ci-bootstrap.yml │ ├── ci-idris2-and-libs.yml │ ├── ci-lint.yml │ ├── ci-sphinx.yml │ └── ci-super-linter.yml ├── .gitignore ├── .readthedocs.yaml ├── CHANGELOG.md ├── CHANGELOG_NEXT.md ├── CITATION.cff ├── CONTRIBUTING.md ├── CONTRIBUTORS ├── INSTALL.md ├── LICENSE ├── Makefile ├── README.md ├── Release ├── CHECKLIST └── mkdist.sh ├── benchmark ├── bench.sh ├── benchmarks │ ├── mergeInt │ │ ├── mergeInt.idr │ │ ├── mergeInt.in │ │ └── mergeInt_fast.in │ ├── mergeStr │ │ ├── mergeStr.idr │ │ ├── mergeStr.in │ │ ├── mergeStr_fast.in │ │ └── words │ ├── spellcheck │ │ ├── input │ │ ├── input_large │ │ ├── input_small │ │ ├── spellcheck.idr │ │ ├── spellcheck.in │ │ ├── spellcheck_fast.in │ │ └── words │ ├── treeInt │ │ ├── BTree.idr │ │ ├── treeInt.idr │ │ ├── treeInt.in │ │ └── treeInt_fast.in │ └── triples │ │ ├── triples.idr │ │ ├── triples.in │ │ └── triples_fast.in └── readme.md ├── bootstrap-stage1-chez.sh ├── bootstrap-stage1-racket.sh ├── bootstrap-stage2.sh ├── bootstrap ├── compile.ss ├── idris2-boot.sh ├── idris2-rktboot.sh └── idris2_app │ ├── idris2.rkt │ └── idris2.ss ├── config.mk ├── default.nix ├── docs ├── .python-version ├── LICENSE ├── Makefile ├── README.md ├── make.bat ├── pyproject.toml ├── requirements.txt ├── source │ ├── _static │ │ └── .gitkeep │ ├── app │ │ ├── exceptionsstate.rst │ │ ├── index.rst │ │ ├── interfaces.rst │ │ ├── introapp.rst │ │ └── linear.rst │ ├── backends │ │ ├── backend-cookbook.rst │ │ ├── chez.rst │ │ ├── custom.rst │ │ ├── gambit.rst │ │ ├── incremental.rst │ │ ├── index.rst │ │ ├── javascript.rst │ │ ├── libraries.rst │ │ ├── racket.rst │ │ └── refc.rst │ ├── conf.py │ ├── cookbook │ │ ├── Calculator.idr │ │ ├── LambdaCalculus.idr │ │ ├── index.rst │ │ └── parsing.rst │ ├── faq │ │ └── faq.rst │ ├── ffi │ │ ├── ffi.rst │ │ ├── index.rst │ │ └── readline.rst │ ├── image │ │ └── login.png │ ├── implementation │ │ ├── ide-protocol.rst │ │ ├── index.rst │ │ └── overview.rst │ ├── index.rst │ ├── libraries │ │ └── index.rst │ ├── listing │ │ ├── idris-prompt-helloworld.txt │ │ ├── idris-prompt-interp.txt │ │ └── idris-prompt-start.txt │ ├── proofs │ │ ├── definitional.rst │ │ ├── index.rst │ │ ├── inductive.rst │ │ ├── patterns.rst │ │ ├── pluscomm.rst │ │ └── propositional.rst │ ├── reference │ │ ├── builtins.rst │ │ ├── debugging.rst │ │ ├── documenting.rst │ │ ├── envvars.rst │ │ ├── failing.rst │ │ ├── index.rst │ │ ├── literate.rst │ │ ├── operators.rst │ │ ├── overloadedlit.rst │ │ ├── packages.rst │ │ ├── pragmas.rst │ │ ├── records.rst │ │ └── strings.rst │ ├── tutorial │ │ ├── conclusions.rst │ │ ├── index.rst │ │ ├── interactive.rst │ │ ├── interfaces.rst │ │ ├── interp.rst │ │ ├── introduction.rst │ │ ├── miscellany.rst │ │ ├── modules.rst │ │ ├── multiplicities.rst │ │ ├── packages.rst │ │ ├── starting.rst │ │ ├── theorems.rst │ │ ├── typesfuns.rst │ │ ├── views.rst │ │ └── windows.rst │ ├── typedd │ │ └── typedd.rst │ └── updates │ │ └── updates.rst └── uv.lock ├── flake.lock ├── flake.nix ├── icons ├── idris-128x128.png ├── idris-256x256.png ├── idris-48x48.png ├── idris-512x512.png ├── idris-64x64.png ├── idris.ico ├── idris_icon.rc ├── text-x-idris.svg ├── x-idris-bytecode.xml ├── x-idris-literate.xml └── x-idris.xml ├── idris2.ipkg ├── idris2api.ipkg ├── ipkg └── idris2protocols.ipkg ├── libs ├── base │ ├── Control │ │ ├── App.idr │ │ ├── App │ │ │ ├── Console.idr │ │ │ └── FileIO.idr │ │ ├── Applicative │ │ │ └── Const.idr │ │ ├── Function.idr │ │ ├── Function │ │ │ └── FunExt.idr │ │ ├── Monad │ │ │ ├── Either.idr │ │ │ ├── Error │ │ │ │ ├── Either.idr │ │ │ │ └── Interface.idr │ │ │ ├── Identity.idr │ │ │ ├── Maybe.idr │ │ │ ├── Partial.idr │ │ │ ├── RWS.idr │ │ │ ├── RWS │ │ │ │ ├── CPS.idr │ │ │ │ └── Interface.idr │ │ │ ├── Reader.idr │ │ │ ├── Reader │ │ │ │ ├── Interface.idr │ │ │ │ └── Reader.idr │ │ │ ├── ST.idr │ │ │ ├── State.idr │ │ │ ├── State │ │ │ │ ├── Interface.idr │ │ │ │ └── State.idr │ │ │ ├── Trans.idr │ │ │ ├── Writer.idr │ │ │ └── Writer │ │ │ │ ├── CPS.idr │ │ │ │ └── Interface.idr │ │ ├── Ord.idr │ │ ├── Order.idr │ │ ├── Relation.idr │ │ ├── Relation │ │ │ └── Closure.idr │ │ └── WellFounded.idr │ ├── Data │ │ ├── Bifoldable.idr │ │ ├── Bits.idr │ │ ├── Bool.idr │ │ ├── Bool │ │ │ ├── Decidable.idr │ │ │ └── Xor.idr │ │ ├── Buffer.idr │ │ ├── Colist.idr │ │ ├── Colist1.idr │ │ ├── Contravariant.idr │ │ ├── DPair.idr │ │ ├── Double.idr │ │ ├── Either.idr │ │ ├── Fin.idr │ │ ├── Fin │ │ │ ├── Arith.idr │ │ │ ├── Order.idr │ │ │ ├── Properties.idr │ │ │ └── Split.idr │ │ ├── Fuel.idr │ │ ├── Fun.idr │ │ ├── IOArray.idr │ │ ├── IOArray │ │ │ └── Prims.idr │ │ ├── IORef.idr │ │ ├── Integral.idr │ │ ├── List.idr │ │ ├── List │ │ │ ├── AtIndex.idr │ │ │ ├── Elem.idr │ │ │ ├── HasLength.idr │ │ │ ├── Lazy.idr │ │ │ ├── Lazy │ │ │ │ └── Quantifiers.idr │ │ │ ├── Quantifiers.idr │ │ │ └── Views.idr │ │ ├── List1.idr │ │ ├── List1 │ │ │ ├── Elem.idr │ │ │ ├── Properties.idr │ │ │ └── Quantifiers.idr │ │ ├── Maybe.idr │ │ ├── Morphisms.idr │ │ ├── Nat.idr │ │ ├── Nat │ │ │ ├── Order.idr │ │ │ ├── Order │ │ │ │ └── Properties.idr │ │ │ └── Views.idr │ │ ├── OpenUnion.idr │ │ ├── Primitives │ │ │ ├── Interpolation.idr │ │ │ └── Views.idr │ │ ├── Ref.idr │ │ ├── Rel.idr │ │ ├── Singleton.idr │ │ ├── SnocList.idr │ │ ├── SnocList │ │ │ ├── Elem.idr │ │ │ ├── HasLength.idr │ │ │ ├── Operations.idr │ │ │ └── Quantifiers.idr │ │ ├── So.idr │ │ ├── SortedMap.idr │ │ ├── SortedMap │ │ │ └── Dependent.idr │ │ ├── SortedSet.idr │ │ ├── Stream.idr │ │ ├── String.idr │ │ ├── These.idr │ │ ├── Vect.idr │ │ ├── Vect │ │ │ ├── AtIndex.idr │ │ │ ├── Elem.idr │ │ │ ├── Quantifiers.idr │ │ │ └── Views.idr │ │ ├── Void.idr │ │ └── Zippable.idr │ ├── Debug │ │ └── Trace.idr │ ├── Decidable │ │ ├── Decidable.idr │ │ ├── Equality.idr │ │ └── Equality │ │ │ └── Core.idr │ ├── Deriving │ │ ├── Common.idr │ │ ├── Foldable.idr │ │ ├── Functor.idr │ │ ├── Show.idr │ │ └── Traversable.idr │ ├── Language │ │ ├── Reflection.idr │ │ └── Reflection │ │ │ ├── TT.idr │ │ │ └── TTImp.idr │ ├── Makefile │ ├── Syntax │ │ ├── PreorderReasoning.idr │ │ ├── PreorderReasoning │ │ │ ├── Generic.idr │ │ │ └── Ops.idr │ │ └── WithProof.idr │ ├── System.idr │ ├── System │ │ ├── Clock.idr │ │ ├── Concurrency.idr │ │ ├── Directory.idr │ │ ├── Errno.idr │ │ ├── Escape.idr │ │ ├── FFI.idr │ │ ├── File.idr │ │ ├── File │ │ │ ├── Buffer.idr │ │ │ ├── Error.idr │ │ │ ├── Handle.idr │ │ │ ├── Meta.idr │ │ │ ├── Mode.idr │ │ │ ├── Permissions.idr │ │ │ ├── Process.idr │ │ │ ├── ReadWrite.idr │ │ │ ├── Support.idr │ │ │ ├── Types.idr │ │ │ └── Virtual.idr │ │ ├── Info.idr │ │ ├── REPL.idr │ │ ├── Signal.idr │ │ └── Term.idr │ └── base.ipkg ├── contrib │ ├── Control │ │ ├── ANSI.idr │ │ ├── ANSI │ │ │ ├── CSI.idr │ │ │ └── SGR.idr │ │ ├── Arrow.idr │ │ ├── Category.idr │ │ ├── Delayed.idr │ │ └── Validation.idr │ ├── Data │ │ ├── Binary.idr │ │ ├── Binary │ │ │ └── Digit.idr │ │ ├── Fin │ │ │ └── Extra.idr │ │ ├── Fun │ │ │ ├── Extra.idr │ │ │ └── Graph.idr │ │ ├── IMaybe.idr │ │ ├── IOMatrix.idr │ │ ├── Int │ │ │ └── Order.idr │ │ ├── Late.idr │ │ ├── Linear │ │ │ └── Array.idr │ │ ├── List │ │ │ ├── Alternating.idr │ │ │ ├── Elem │ │ │ │ └── Extra.idr │ │ │ ├── Equalities.idr │ │ │ ├── Extra.idr │ │ │ ├── Palindrome.idr │ │ │ ├── Reverse.idr │ │ │ ├── Sufficient.idr │ │ │ ├── TailRec.idr │ │ │ └── Views │ │ │ │ └── Extra.idr │ │ ├── Logic │ │ │ └── Propositional.idr │ │ ├── Monoid │ │ │ └── Exponentiation.idr │ │ ├── Nat │ │ │ ├── Ack.idr │ │ │ ├── Division.idr │ │ │ ├── Equational.idr │ │ │ ├── Exponentiation.idr │ │ │ ├── Fact.idr │ │ │ ├── Factor.idr │ │ │ ├── Fib.idr │ │ │ ├── Order │ │ │ │ ├── Relation.idr │ │ │ │ └── Strict.idr │ │ │ └── Properties.idr │ │ ├── Order.idr │ │ ├── Path.idr │ │ ├── Rel │ │ │ └── Complement.idr │ │ ├── Seq │ │ │ ├── Internal.idr │ │ │ ├── Sized.idr │ │ │ └── Unsized.idr │ │ ├── Stream │ │ │ └── Extra.idr │ │ ├── String │ │ │ ├── Extra.idr │ │ │ ├── Interpolation.idr │ │ │ ├── Iterator.idr │ │ │ ├── Parser.idr │ │ │ ├── Parser │ │ │ │ └── Expression.idr │ │ │ └── Position.idr │ │ ├── Telescope.idr │ │ ├── Telescope │ │ │ ├── Congruence.idr │ │ │ ├── Fun.idr │ │ │ ├── Segment.idr │ │ │ ├── SimpleFun.idr │ │ │ └── Telescope.idr │ │ ├── Validated.idr │ │ └── Vect │ │ │ ├── Extra.idr │ │ │ ├── Properties.idr │ │ │ ├── Properties │ │ │ ├── Fin.idr │ │ │ ├── Foldr.idr │ │ │ ├── Index.idr │ │ │ ├── Map.idr │ │ │ └── Tabulate.idr │ │ │ └── Sort.idr │ ├── Debug │ │ └── Buffer.idr │ ├── Decidable │ │ ├── Decidable │ │ │ └── Extra.idr │ │ ├── Finite │ │ │ └── Fin.idr │ │ └── Order │ │ │ └── Strict.idr │ ├── Language │ │ ├── JSON.idr │ │ └── JSON │ │ │ ├── Data.idr │ │ │ ├── Lexer.idr │ │ │ ├── Parser.idr │ │ │ ├── String.idr │ │ │ ├── String │ │ │ ├── Lexer.idr │ │ │ ├── Parser.idr │ │ │ └── Tokens.idr │ │ │ └── Tokens.idr │ ├── Makefile │ ├── System │ │ ├── Console │ │ │ └── GetOpt.idr │ │ ├── Directory │ │ │ └── Tree.idr │ │ ├── Future.idr │ │ ├── Path.idr │ │ └── Random.idr │ ├── Test │ │ └── REDIRECT.md │ ├── Text │ │ ├── Bounded.idr │ │ ├── Distance │ │ │ └── Levenshtein.idr │ │ ├── Lexer.idr │ │ ├── Lexer │ │ │ ├── Core.idr │ │ │ └── Tokenizer.idr │ │ ├── Literate.idr │ │ ├── Parser.idr │ │ ├── Parser │ │ │ ├── Core.idr │ │ │ └── Expression.idr │ │ ├── PrettyPrint │ │ │ ├── Prettyprinter.idr │ │ │ └── Prettyprinter │ │ │ │ ├── Doc.idr │ │ │ │ ├── Render │ │ │ │ ├── HTML.idr │ │ │ │ ├── String.idr │ │ │ │ └── Terminal.idr │ │ │ │ ├── SimpleDocTree.idr │ │ │ │ ├── Symbols.idr │ │ │ │ └── Util.idr │ │ ├── Quantity.idr │ │ └── Token.idr │ └── contrib.ipkg ├── linear │ ├── Control │ │ └── Linear │ │ │ └── LIO.idr │ ├── Data │ │ ├── Linear.idr │ │ └── Linear │ │ │ ├── Bifunctor.idr │ │ │ ├── Copies.idr │ │ │ ├── Interface.idr │ │ │ ├── LEither.idr │ │ │ ├── LList.idr │ │ │ ├── LMaybe.idr │ │ │ ├── LNat.idr │ │ │ ├── LVect.idr │ │ │ ├── List │ │ │ └── LQuantifiers.idr │ │ │ └── Notation.idr │ ├── Makefile │ ├── System │ │ └── Concurrency │ │ │ ├── Linear.idr │ │ │ └── Session.idr │ └── linear.ipkg ├── network │ ├── .gitignore │ ├── Control │ │ └── Linear │ │ │ └── Network.idr │ ├── Makefile │ ├── Network │ │ ├── FFI.idr │ │ ├── Socket.idr │ │ └── Socket │ │ │ ├── Data.idr │ │ │ └── Raw.idr │ └── network.ipkg ├── papers │ ├── Control │ │ └── DivideAndConquer.idr │ ├── Data │ │ ├── Container.idr │ │ ├── Description │ │ │ ├── Indexed.idr │ │ │ └── Regular.idr │ │ ├── Enumerate.idr │ │ ├── Enumerate │ │ │ ├── Common.idr │ │ │ └── Indexed.idr │ │ ├── INTEGER.idr │ │ ├── InductionRecursion │ │ │ └── DybjerSetzer.idr │ │ ├── Linear │ │ │ ├── Communications.idr │ │ │ ├── Diff.idr │ │ │ └── Inverse.idr │ │ ├── ProofDelay.idr │ │ ├── Recursion │ │ │ └── Free.idr │ │ ├── Tree │ │ │ └── Perfect.idr │ │ ├── Vect │ │ │ └── Binary.idr │ │ └── W.idr │ ├── Language │ │ ├── IntrinsicScoping │ │ │ ├── TypeTheory.idr │ │ │ └── Variables.idr │ │ ├── IntrinsicTyping │ │ │ ├── ABT.idr │ │ │ ├── Krivine.idr │ │ │ ├── SECD.idr │ │ │ └── STLCR.idr │ │ ├── Tagless.idr │ │ └── TypeTheory.idr │ ├── Makefile │ ├── Search │ │ ├── Auto.idr │ │ ├── CTL.idr │ │ ├── GCL.idr │ │ ├── Generator.idr │ │ ├── HDecidable.idr │ │ ├── Negation.idr │ │ ├── Properties.idr │ │ └── Tychonoff │ │ │ └── PartI.idr │ └── papers.ipkg ├── prelude │ ├── Builtin.idr │ ├── Makefile │ ├── Prelude.idr │ ├── Prelude │ │ ├── Basics.idr │ │ ├── Cast.idr │ │ ├── EqOrd.idr │ │ ├── IO.idr │ │ ├── Interfaces.idr │ │ ├── Interpolation.idr │ │ ├── Num.idr │ │ ├── Ops.idr │ │ ├── Show.idr │ │ ├── Types.idr │ │ └── Uninhabited.idr │ ├── PrimIO.idr │ └── prelude.ipkg └── test │ ├── Makefile │ ├── README.md │ ├── Test │ └── Golden.idr │ └── test.ipkg ├── lint └── lint.py ├── nix ├── buildIdris.nix ├── idris2Api.nix ├── init.el ├── lib.nix ├── package.nix ├── support.nix ├── templates │ ├── pkg │ │ ├── Foo.idr │ │ ├── default.nix │ │ ├── flake.nix │ │ └── mypkg.ipkg │ └── pkgWithDeps │ │ ├── Bar.idr │ │ ├── default.nix │ │ ├── flake.nix │ │ └── pkgWithDeps.ipkg ├── test.nix └── text-editor.nix ├── samples ├── BTree.idr ├── FFI-readline │ ├── Test │ │ ├── ReadHistory.idr │ │ ├── ReadTab.idr │ │ └── test.ipkg │ ├── readline.ipkg │ ├── readline_glue │ │ ├── .gitignore │ │ ├── Makefile │ │ ├── idris_readline.c │ │ └── idris_readline.h │ └── src │ │ └── Text │ │ └── Readline.idr ├── Interp.idr ├── InterpE.idr ├── MyOrd.idr ├── NamedSemi.idr ├── Prims.idr ├── Proofs.idr ├── Vect.idr ├── Void.idr ├── With.idr ├── bmain.idr ├── deprec.idr ├── dummy.ipkg ├── fctypes.idr ├── ffi │ ├── Small.idr │ ├── Struct.idr │ ├── args.idr │ ├── dummy.ipkg │ └── smallc.c ├── holes.idr ├── io.idr ├── listcomp.idr ├── multiplicity.idr ├── params.idr ├── proofs │ ├── induction.idr │ ├── pluscomm.idr │ ├── plusprops.idr │ ├── prfintro.idr │ └── proof.ipkg └── wheres.idr ├── src ├── Algebra.idr ├── Algebra │ ├── Preorder.idr │ ├── Semiring.idr │ ├── SizeChange.idr │ └── ZeroOneOmega.idr ├── Compiler │ ├── ANF.idr │ ├── CaseOpts.idr │ ├── Common.idr │ ├── CompileExpr.idr │ ├── ES │ │ ├── Ast.idr │ │ ├── Codegen.idr │ │ ├── Doc.idr │ │ ├── Javascript.idr │ │ ├── Node.idr │ │ ├── State.idr │ │ ├── TailRec.idr │ │ └── ToAst.idr │ ├── Generated.idr │ ├── Inline.idr │ ├── Interpreter │ │ └── VMCode.idr │ ├── LambdaLift.idr │ ├── NoMangle.idr │ ├── Opts │ │ ├── CSE.idr │ │ ├── ConstantFold.idr │ │ ├── Constructor.idr │ │ ├── Identity.idr │ │ ├── InlineHeuristics.idr │ │ └── ToplevelConstants.idr │ ├── RefC.idr │ ├── RefC │ │ ├── CC.idr │ │ └── RefC.idr │ ├── Scheme │ │ ├── Chez.idr │ │ ├── ChezSep.idr │ │ ├── Common.idr │ │ ├── Gambit.idr │ │ └── Racket.idr │ ├── Separate.idr │ └── VMCode.idr ├── Core │ ├── AutoSearch.idr │ ├── Binary.idr │ ├── Binary │ │ └── Prims.idr │ ├── Case │ │ ├── CaseBuilder.idr │ │ ├── CaseTree.idr │ │ ├── CaseTree │ │ │ └── Pretty.idr │ │ └── Util.idr │ ├── CompileExpr.idr │ ├── CompileExpr │ │ └── Pretty.idr │ ├── Context.idr │ ├── Context │ │ ├── Context.idr │ │ ├── Data.idr │ │ ├── Log.idr │ │ ├── Pretty.idr │ │ └── TTC.idr │ ├── Core.idr │ ├── Coverage.idr │ ├── Directory.idr │ ├── Env.idr │ ├── FC.idr │ ├── GetType.idr │ ├── Hash.idr │ ├── InitPrimitives.idr │ ├── LinearCheck.idr │ ├── Metadata.idr │ ├── Name.idr │ ├── Name │ │ ├── CompatibleVars.idr │ │ ├── Namespace.idr │ │ └── Scoped.idr │ ├── Normalise.idr │ ├── Normalise │ │ ├── Convert.idr │ │ ├── Eval.idr │ │ └── Quote.idr │ ├── Options.idr │ ├── Options │ │ └── Log.idr │ ├── Ord.idr │ ├── Primitives.idr │ ├── Reflect.idr │ ├── SchemeEval.idr │ ├── SchemeEval │ │ ├── Builtins.idr │ │ ├── Compile.idr │ │ ├── Evaluate.idr │ │ ├── Quote.idr │ │ └── ToScheme.idr │ ├── TT.idr │ ├── TT │ │ ├── Binder.idr │ │ ├── Primitive.idr │ │ ├── Subst.idr │ │ ├── Term.idr │ │ ├── Term │ │ │ └── Subst.idr │ │ ├── Traversals.idr │ │ ├── Var.idr │ │ └── Views.idr │ ├── TTC.idr │ ├── Termination.idr │ ├── Termination │ │ ├── CallGraph.idr │ │ ├── Positivity.idr │ │ ├── References.idr │ │ └── SizeChange.idr │ ├── Transform.idr │ ├── Unify.idr │ ├── UnifyState.idr │ ├── Value.idr │ └── WithData.idr ├── Idris │ ├── CommandLine.idr │ ├── Desugar.idr │ ├── Desugar │ │ └── Mutual.idr │ ├── Doc │ │ ├── Annotations.idr │ │ ├── Brackets.idr │ │ ├── Display.idr │ │ ├── HTML.idr │ │ ├── Keywords.idr │ │ └── String.idr │ ├── Driver.idr │ ├── Elab │ │ ├── Implementation.idr │ │ └── Interface.idr │ ├── Env.idr │ ├── Error.idr │ ├── IDEMode │ │ ├── CaseSplit.idr │ │ ├── Commands.idr │ │ ├── Holes.idr │ │ ├── MakeClause.idr │ │ ├── Parser.idr │ │ ├── Pretty.idr │ │ ├── REPL.idr │ │ ├── SyntaxHighlight.idr │ │ └── TokenLine.idr │ ├── Main.idr │ ├── ModTree.idr │ ├── Package.idr │ ├── Package │ │ ├── Init.idr │ │ ├── ToJson.idr │ │ └── Types.idr │ ├── Parser.idr │ ├── Parser │ │ └── Let.idr │ ├── Pretty.idr │ ├── Pretty │ │ ├── Annotations.idr │ │ └── Render.idr │ ├── ProcessIdr.idr │ ├── REPL.idr │ ├── REPL │ │ ├── Common.idr │ │ ├── FuzzySearch.idr │ │ └── Opts.idr │ ├── Resugar.idr │ ├── SetOptions.idr │ ├── Syntax.idr │ ├── Syntax │ │ ├── Builtin.idr │ │ ├── Pragmas.idr │ │ ├── TTC.idr │ │ ├── Traversals.idr │ │ └── Views.idr │ └── Version.idr ├── Libraries │ ├── Control │ │ ├── ANSI.idr │ │ ├── ANSI │ │ │ ├── CSI.idr │ │ │ └── SGR.idr │ │ └── Delayed.idr │ ├── Data │ │ ├── ANameMap.idr │ │ ├── DList.idr │ │ ├── Erased.idr │ │ ├── Graph.idr │ │ ├── IMaybe.idr │ │ ├── IOMatrix.idr │ │ ├── IntMap.idr │ │ ├── List │ │ │ ├── Extra.idr │ │ │ ├── HasLength.idr │ │ │ ├── LengthMatch.idr │ │ │ ├── Quantifiers │ │ │ │ └── Extra.idr │ │ │ ├── SizeOf.idr │ │ │ └── Thin.idr │ │ ├── List01.idr │ │ ├── List01 │ │ │ └── Quantifiers.idr │ │ ├── NameMap.idr │ │ ├── NameMap │ │ │ └── Traversable.idr │ │ ├── NatSet.idr │ │ ├── Ordering │ │ │ └── Extra.idr │ │ ├── PosMap.idr │ │ ├── Record.idr │ │ ├── SnocList │ │ │ ├── Extra.idr │ │ │ ├── HasLength.idr │ │ │ ├── LengthMatch.idr │ │ │ └── SizeOf.idr │ │ ├── Span.idr │ │ ├── SparseMatrix.idr │ │ ├── String.idr │ │ ├── String │ │ │ ├── Builder.idr │ │ │ ├── Extra.idr │ │ │ └── Iterator.idr │ │ ├── StringMap.idr │ │ ├── StringTrie.idr │ │ ├── Tap.idr │ │ ├── UserNameMap.idr │ │ ├── VarSet.idr │ │ ├── VarSet │ │ │ └── Core.idr │ │ ├── Version.idr │ │ ├── WithData.idr │ │ └── WithDefault.idr │ ├── System │ │ └── Directory │ │ │ └── Tree.idr │ ├── Text │ │ ├── Bounded.idr │ │ ├── Distance │ │ │ └── Levenshtein.idr │ │ ├── Lexer.idr │ │ ├── Lexer │ │ │ ├── Core.idr │ │ │ └── Tokenizer.idr │ │ ├── Literate.idr │ │ ├── Parser.idr │ │ ├── Parser │ │ │ └── Core.idr │ │ ├── PrettyPrint │ │ │ ├── Prettyprinter.idr │ │ │ └── Prettyprinter │ │ │ │ ├── Doc.idr │ │ │ │ ├── Render │ │ │ │ ├── HTML.idr │ │ │ │ ├── String.idr │ │ │ │ └── Terminal.idr │ │ │ │ ├── SimpleDocTree.idr │ │ │ │ ├── Symbols.idr │ │ │ │ └── Util.idr │ │ ├── Quantity.idr │ │ └── Token.idr │ └── Utils │ │ ├── Binary.idr │ │ ├── Octal.idr │ │ ├── Path.idr │ │ ├── Scheme.idr │ │ ├── Shunting.idr │ │ └── String.idr ├── Parser │ ├── Lexer │ │ ├── Common.idr │ │ ├── Package.idr │ │ └── Source.idr │ ├── Package.idr │ ├── Rule │ │ ├── Package.idr │ │ └── Source.idr │ ├── Source.idr │ ├── Support.idr │ ├── Support │ │ └── Escaping.idr │ └── Unlit.idr ├── Protocol │ ├── Hex.idr │ ├── IDE.idr │ ├── IDE │ │ ├── Command.idr │ │ ├── Decoration.idr │ │ ├── FileContext.idr │ │ ├── Formatting.idr │ │ ├── Highlight.idr │ │ ├── Holes.idr │ │ └── Result.idr │ ├── SExp.idr │ └── SExp │ │ └── Parser.idr ├── TTImp │ ├── BindImplicits.idr │ ├── Elab.idr │ ├── Elab │ │ ├── Ambiguity.idr │ │ ├── App.idr │ │ ├── As.idr │ │ ├── Binders.idr │ │ ├── Case.idr │ │ ├── Check.idr │ │ ├── Delayed.idr │ │ ├── Dot.idr │ │ ├── Hole.idr │ │ ├── ImplicitBind.idr │ │ ├── Lazy.idr │ │ ├── Local.idr │ │ ├── Prim.idr │ │ ├── Quote.idr │ │ ├── Record.idr │ │ ├── Rewrite.idr │ │ ├── RunElab.idr │ │ ├── Term.idr │ │ └── Utils.idr │ ├── Impossible.idr │ ├── Interactive │ │ ├── CaseSplit.idr │ │ ├── Completion.idr │ │ ├── ExprSearch.idr │ │ ├── GenerateDef.idr │ │ ├── Intro.idr │ │ └── MakeLemma.idr │ ├── Parser.idr │ ├── PartialEval.idr │ ├── ProcessBuiltin.idr │ ├── ProcessData.idr │ ├── ProcessDecls.idr │ ├── ProcessDecls │ │ └── Totality.idr │ ├── ProcessDef.idr │ ├── ProcessFnOpt.idr │ ├── ProcessParams.idr │ ├── ProcessRecord.idr │ ├── ProcessRunElab.idr │ ├── ProcessTransform.idr │ ├── ProcessType.idr │ ├── Reflect.idr │ ├── TTImp.idr │ ├── TTImp │ │ ├── Functor.idr │ │ ├── TTC.idr │ │ └── Traversals.idr │ ├── Unelab.idr │ ├── Utils.idr │ └── WithClause.idr └── Yaffle │ ├── Main.idr │ └── REPL.idr ├── support ├── Makefile ├── c │ ├── .gitignore │ ├── Makefile │ ├── getline.c │ ├── getline.h │ ├── idris_directory.c │ ├── idris_directory.h │ ├── idris_file.c │ ├── idris_file.h │ ├── idris_memory.c │ ├── idris_memory.h │ ├── idris_net.c │ ├── idris_net.h │ ├── idris_signal.c │ ├── idris_signal.h │ ├── idris_support.c │ ├── idris_support.h │ ├── idris_system.c │ ├── idris_system.h │ ├── idris_term.c │ ├── idris_term.h │ ├── idris_util.c │ ├── idris_util.h │ └── windows │ │ ├── win_hack.c │ │ ├── win_utils.c │ │ └── win_utils.h ├── chez │ ├── .gitignore │ ├── Makefile │ ├── ct-support.ss │ └── support.ss ├── docs │ ├── alternative.css │ ├── blackandwhite.css │ ├── default.css │ └── index.html ├── gambit │ ├── foreign.scm │ └── support.scm ├── js │ ├── support.js │ ├── support_system.js │ ├── support_system_clock.js │ ├── support_system_directory.js │ ├── support_system_file.js │ └── support_system_signal.js ├── racket │ ├── ct-support.rkt │ └── support.rkt └── refc │ ├── Makefile │ ├── _datatypes.h │ ├── buffer.c │ ├── buffer.h │ ├── cBackend.h │ ├── casts.c │ ├── casts.h │ ├── clock.c │ ├── clock.h │ ├── mathFunctions.c │ ├── mathFunctions.h │ ├── memoryManagement.c │ ├── memoryManagement.h │ ├── prim.c │ ├── prim.h │ ├── refc_util.c │ ├── refc_util.h │ ├── runtime.c │ ├── runtime.h │ ├── stringOps.c │ ├── stringOps.h │ ├── threads.c │ └── threads.h ├── tests ├── Main.idr ├── Makefile ├── README.md ├── allbackends │ ├── basic048 │ │ ├── Module'.idr │ │ ├── expected │ │ ├── input │ │ ├── input-ed │ │ └── run │ ├── evaluator004 │ │ ├── Issue735.idr │ │ ├── expected │ │ ├── input │ │ └── run │ ├── evaluator005 │ │ ├── Issue1200.idr │ │ ├── expected │ │ └── run │ ├── issue2362 │ │ ├── Issue2362.idr │ │ ├── expected │ │ └── run │ ├── perf006 │ │ ├── Issue775.idr │ │ ├── expected │ │ └── run │ └── popen2 │ │ ├── Test.idr │ │ ├── expected │ │ └── run ├── allschemes │ ├── channels001 │ │ ├── Main.idr │ │ ├── expected │ │ └── run │ ├── channels002 │ │ ├── Main.idr │ │ ├── expected │ │ └── run │ ├── channels003 │ │ ├── Main.idr │ │ ├── expected │ │ └── run │ ├── channels004 │ │ ├── Main.idr │ │ ├── expected │ │ └── run │ ├── channels005 │ │ ├── Main.idr │ │ ├── expected │ │ └── run │ ├── channels006 │ │ ├── Main.idr │ │ ├── expected │ │ └── run │ ├── double001 │ │ ├── URandEpsilon.idr │ │ ├── expected │ │ ├── input │ │ └── run │ ├── double002 │ │ ├── NaN.idr │ │ ├── expected │ │ ├── input │ │ └── run │ ├── double003 │ │ ├── Inf.idr │ │ ├── expected │ │ ├── input │ │ └── run │ ├── ffi001 │ │ ├── Struct.idr │ │ ├── expected │ │ └── run │ ├── memo001 │ │ ├── Memo.idr │ │ ├── expected │ │ └── run │ ├── memo002 │ │ ├── Memo.idr │ │ ├── expected │ │ └── run │ ├── memo003 │ │ ├── Memo.idr │ │ ├── expected │ │ └── run │ ├── memo004 │ │ ├── Memo.idr │ │ ├── expected │ │ ├── run │ │ └── test.ipkg │ ├── memo005 │ │ ├── Memo.idr │ │ ├── expected │ │ ├── run │ │ └── test.ipkg │ ├── scheme001 │ │ ├── CastStringDouble.idr │ │ ├── expected │ │ └── run │ └── scheme002 │ │ ├── TermSize.idr │ │ ├── expected │ │ └── run ├── base │ ├── control_app001 │ │ ├── TestException.idr │ │ ├── expected │ │ └── run │ ├── control_monad_instances │ │ ├── SearchReader.idr │ │ ├── SearchState.idr │ │ ├── SearchWriter.idr │ │ ├── expected │ │ └── run │ ├── data_bits001 │ │ ├── BitOps.idr │ │ ├── expected │ │ └── run │ ├── data_bits002 │ │ ├── BitRotate.idr │ │ ├── expected │ │ └── run │ ├── data_fin │ │ ├── Num.idr │ │ ├── expected │ │ ├── fromInteger.idr │ │ ├── performance.idr │ │ └── run │ ├── data_integral │ │ ├── Integral.idr │ │ ├── expected │ │ └── run │ ├── data_list001 │ │ ├── List.idr │ │ ├── expected │ │ └── run │ ├── data_list002 │ │ ├── Prefix.idr │ │ ├── expected │ │ └── run │ ├── data_list003 │ │ ├── Elem.idr │ │ ├── expected │ │ └── run │ ├── data_listone001 │ │ ├── Elem.idr │ │ ├── expected │ │ └── run │ ├── data_nat │ │ ├── Properties.idr │ │ ├── expected │ │ └── run │ ├── data_ref_monadstate │ │ ├── RefMonadState.idr │ │ ├── a-test.ipkg │ │ ├── expected │ │ └── run │ ├── data_singleton │ │ ├── RLE.idr │ │ ├── expected │ │ └── run │ ├── data_snoclist001 │ │ ├── SL.idr │ │ ├── expected │ │ └── run │ ├── data_snoclist002 │ │ ├── Elem.idr │ │ ├── expected │ │ └── run │ ├── data_string │ │ ├── StringReduce.idr │ │ ├── expected │ │ └── run │ ├── data_string_lines001 │ │ ├── Lines.idr │ │ ├── expected │ │ └── run │ ├── data_string_parse_proof │ │ ├── StringParse.idr │ │ ├── expected │ │ └── run │ ├── data_string_unlines001 │ │ ├── Unlines.idr │ │ ├── expected │ │ └── run │ ├── data_vect001 │ │ ├── Vect.idr │ │ ├── expected │ │ └── run │ ├── data_vect002 │ │ ├── Elem.idr │ │ ├── expected │ │ └── run │ ├── deriving_foldable │ │ ├── DeriveFoldable.idr │ │ ├── expected │ │ └── run │ ├── deriving_functor │ │ ├── DeriveFunctor.idr │ │ ├── Search.idr │ │ ├── expected │ │ └── run │ ├── deriving_show │ │ ├── DeriveShow.idr │ │ ├── Search.idr │ │ ├── expected │ │ ├── input │ │ └── run │ ├── deriving_traversable │ │ ├── DeriveTraversable.idr │ │ ├── expected │ │ └── run │ ├── sortedmap_001 │ │ ├── SortedMapTest.idr │ │ ├── expected │ │ └── run │ ├── system_directory │ │ ├── ReadDir.idr │ │ ├── dir │ │ │ └── a │ │ ├── expected │ │ └── run │ ├── system_env │ │ ├── Test.idr │ │ ├── expected │ │ └── run │ ├── system_errno │ │ ├── Test.idr │ │ ├── expected │ │ └── run │ ├── system_file001 │ │ ├── ReadFilePage.idr │ │ ├── expected │ │ ├── run │ │ └── test.txt │ ├── system_fileError │ │ ├── FileErrors.idr │ │ ├── expected │ │ ├── read_only.txt │ │ └── run │ ├── system_file_copyFile │ │ ├── CopyFile.idr │ │ ├── expected │ │ ├── run │ │ └── source.bin │ ├── system_file_fGetChars │ │ ├── ReadFile.idr │ │ ├── big.txt │ │ ├── empty.txt │ │ ├── expected │ │ ├── run │ │ └── small.txt │ ├── system_file_fRead │ │ ├── ReadFile.idr │ │ ├── expected │ │ ├── run │ │ └── sampleFile.txt │ ├── system_file_popen │ │ ├── Popen.idr │ │ ├── expected │ │ └── run │ ├── system_file_remove │ │ ├── Test.idr │ │ ├── expected │ │ └── run │ ├── system_get_environment │ │ ├── Test.idr │ │ ├── expected │ │ └── run │ ├── system_info001 │ │ ├── .gitignore │ │ ├── NumProcessors.idr │ │ └── run │ ├── system_info_os001 │ │ ├── Os.idr │ │ ├── expected │ │ └── run │ ├── system_run │ │ ├── Run.idr │ │ ├── expected │ │ └── run │ ├── system_signal001 │ │ ├── IgnoreSignal.idr │ │ ├── expected │ │ └── run │ ├── system_signal002 │ │ ├── HandleSignal.idr │ │ ├── expected │ │ └── run │ ├── system_signal003 │ │ ├── DefaultSignal.idr │ │ ├── expected │ │ └── run │ ├── system_signal004 │ │ ├── HandleManySignals.idr │ │ ├── expected │ │ └── run │ ├── system_system │ │ ├── Test.idr │ │ ├── expected │ │ ├── run │ │ ├── seventeen.sh │ │ └── zero.sh │ ├── system_time001 │ │ ├── Time.idr │ │ ├── expected │ │ └── run │ ├── ttimp_show001 │ │ ├── expected │ │ ├── input │ │ └── run │ └── void_error │ │ ├── Main.idr │ │ ├── expected │ │ └── run ├── chez │ ├── barrier001 │ │ ├── Main.idr │ │ ├── expected │ │ ├── input │ │ └── run │ ├── bitops │ │ ├── BitOps.idr │ │ ├── expected │ │ └── run │ ├── buffer001 │ │ ├── Main.idr │ │ ├── expected │ │ └── run │ ├── casts │ │ ├── Casts.idr │ │ ├── expected │ │ └── run │ ├── channels007 │ │ ├── Main.idr │ │ ├── expected │ │ └── run │ ├── channels008 │ │ ├── Main.idr │ │ ├── expected │ │ └── run │ ├── channels009 │ │ ├── Main.idr │ │ ├── expected │ │ └── run │ ├── chez001 │ │ ├── Total.idr │ │ ├── expected │ │ └── run │ ├── chez002 │ │ ├── Pythag.idr │ │ ├── expected │ │ ├── input │ │ └── run │ ├── chez003 │ │ ├── IORef.idr │ │ ├── expected │ │ └── run │ ├── chez004 │ │ ├── Buffer.idr │ │ ├── expected │ │ └── run │ ├── chez005 │ │ ├── Filter.idr │ │ ├── expected │ │ ├── input │ │ └── run │ ├── chez006 │ │ ├── TypeCase.idr │ │ ├── TypeCase2.idr │ │ ├── expected │ │ ├── input │ │ └── run │ ├── chez007 │ │ ├── TypeCase.idr │ │ ├── expected │ │ └── run │ ├── chez008 │ │ ├── Nat.idr │ │ ├── expected │ │ └── run │ ├── chez009 │ │ ├── expected │ │ ├── run │ │ └── uni.idr │ ├── chez010 │ │ ├── .gitignore │ │ ├── CB.idr │ │ ├── Makefile │ │ ├── cblib.c │ │ ├── expected │ │ └── run │ ├── chez011 │ │ ├── bangs.idr │ │ ├── expected │ │ ├── input │ │ └── run │ ├── chez012 │ │ ├── array.idr │ │ ├── expected │ │ └── run │ ├── chez013 │ │ ├── .gitignore │ │ ├── Makefile │ │ ├── Struct.idr │ │ ├── expected │ │ ├── run │ │ ├── struct.c │ │ └── struct.h │ ├── chez014 │ │ ├── Echo.idr │ │ ├── expected │ │ └── run │ ├── chez015 │ │ ├── Numbers.idr │ │ ├── expected │ │ └── run │ ├── chez016 │ │ ├── expected │ │ ├── folder with spaces │ │ │ └── Main.idr │ │ └── run │ ├── chez017 │ │ ├── dir.idr │ │ ├── expected │ │ └── run │ ├── chez018 │ │ ├── File.idr │ │ ├── expected │ │ ├── run │ │ └── test.txt │ ├── chez019 │ │ ├── expected │ │ ├── input │ │ ├── partial.idr │ │ └── run │ ├── chez020 │ │ ├── Popen.idr │ │ ├── expected │ │ └── run │ ├── chez021 │ │ ├── Bits.idr │ │ ├── expected │ │ ├── input │ │ └── run │ ├── chez022 │ │ ├── Makefile │ │ ├── expected │ │ ├── mkalloc.c │ │ ├── run │ │ └── usealloc.idr │ ├── chez023 │ │ ├── File.idr │ │ ├── expected │ │ └── run │ ├── chez024 │ │ ├── Envy.idr │ │ ├── expected │ │ └── run │ ├── chez025 │ │ ├── expected │ │ ├── input │ │ ├── run │ │ └── runst.idr │ ├── chez026 │ │ ├── Dummy.idr │ │ ├── dummy.ipkg │ │ ├── expected │ │ └── run │ ├── chez027 │ │ ├── StringParser.idr │ │ ├── expected │ │ └── run │ ├── chez028 │ │ ├── ExpressionParser.idr │ │ ├── expected │ │ └── run │ ├── chez029 │ │ ├── BitCasts.idr │ │ ├── expected │ │ └── run │ ├── chez030 │ │ ├── ExtraRuntime.idr │ │ ├── expected │ │ ├── extensions.scm │ │ └── run │ ├── chez031 │ │ ├── Specifiers.idr │ │ ├── expected │ │ ├── input │ │ └── run │ ├── chez032 │ │ ├── BitOps.idr │ │ ├── expected │ │ └── run │ ├── chez033 │ │ ├── Main.idr │ │ ├── Mod.idr │ │ ├── expected │ │ └── run │ ├── chez034 │ │ ├── ThreadData.idr │ │ ├── expected │ │ └── run │ ├── chez035 │ │ ├── Mod1.idr │ │ ├── Mod2.idr │ │ ├── expected │ │ ├── input │ │ └── run │ ├── chez036 │ │ ├── Crash.idr │ │ ├── Crash2.idr │ │ ├── Crash3.idr │ │ ├── expected │ │ └── run │ ├── chez037 │ │ ├── Hello.idr │ │ ├── expected │ │ └── run │ ├── chez038 │ │ ├── ThreadId.idr │ │ ├── expected │ │ └── run │ ├── constfold │ │ ├── Check.idr │ │ ├── Fold.idr │ │ ├── expected │ │ └── run │ ├── constfold2 │ │ ├── Check.idr │ │ ├── Fold.idr │ │ ├── expected │ │ └── run │ ├── constfold3 │ │ ├── Check.idr │ │ ├── Fold.idr │ │ ├── expected │ │ └── run │ ├── forkjoin001 │ │ ├── Main.idr │ │ ├── expected │ │ └── run │ ├── futures001 │ │ ├── Futures.idr │ │ ├── expected │ │ └── run │ ├── futures002 │ │ ├── Futures.idr │ │ ├── expected │ │ └── run │ ├── inlineiobind │ │ ├── Check.idr │ │ ├── Main.idr │ │ ├── expected │ │ └── run │ ├── integers │ │ ├── TestIntegers.idr │ │ ├── expected │ │ └── run │ ├── nat2fin │ │ ├── Check.idr │ │ ├── Test.idr │ │ ├── expected │ │ └── run │ ├── newints │ │ ├── IntOps.idr │ │ ├── expected │ │ └── run │ ├── perf001 │ │ ├── Fact.idr │ │ ├── expected │ │ └── run │ ├── reg001 │ │ ├── expected │ │ ├── numbers.idr │ │ └── run │ ├── reg002 │ │ ├── Main.idr │ │ ├── expected │ │ └── run │ ├── semaphores001 │ │ ├── Main.idr │ │ ├── expected │ │ └── run │ └── semaphores002 │ │ ├── Main.idr │ │ ├── expected │ │ └── run ├── cli │ ├── exec001 │ │ ├── expected │ │ ├── issue3398.idr │ │ └── run │ ├── exec002 │ │ ├── expected │ │ └── run │ ├── exec003 │ │ ├── expected │ │ └── run │ ├── exec004 │ │ ├── expected │ │ └── run │ └── optional001 │ │ ├── expected │ │ ├── run │ │ └── test.ipkg ├── codegen │ ├── .gitignore │ ├── builtin001 │ │ ├── Main.idr │ │ ├── expected │ │ └── run │ ├── con001 │ │ ├── Main.idr │ │ ├── expected │ │ └── run │ ├── enum │ │ ├── Check.idr │ │ ├── Enum.idr │ │ ├── expected │ │ └── run │ ├── fix3375 │ │ ├── Prog.idr │ │ ├── expected │ │ └── run │ └── fix3515 │ │ ├── Main.idr │ │ ├── expected │ │ └── run ├── contrib │ ├── getOpt001 │ │ ├── UseGetOpt.idr │ │ ├── expected │ │ ├── run │ │ └── test.ipkg │ ├── json_001 │ │ ├── CharEncoding.idr │ │ ├── expected │ │ └── run │ ├── json_002 │ │ ├── ShowJSON.idr │ │ ├── expected │ │ └── run │ ├── json_003 │ │ ├── CastJSON.idr │ │ ├── expected │ │ └── run │ ├── json_004 │ │ ├── JSON.idr │ │ ├── expected │ │ └── run │ ├── lexer │ │ ├── Test.idr │ │ ├── expected │ │ └── run │ ├── list_alternating │ │ ├── AlternatingList.idr │ │ ├── expected │ │ └── run │ ├── perf001 │ │ ├── GCDPerf.idr │ │ ├── expected │ │ └── run │ └── system_directory_tree_copyDir │ │ ├── CopyDir.idr │ │ ├── expected │ │ ├── run │ │ └── templateDir │ │ ├── nestedDir │ │ └── anotherFile.txt │ │ └── source.bin ├── gambit │ └── bitops001 │ │ ├── BitOps.idr │ │ ├── expected │ │ └── run ├── ideMode │ ├── ideMode001 │ │ ├── LocType.idr │ │ ├── dummy.ipkg │ │ ├── expected │ │ ├── input │ │ ├── input2 │ │ └── run │ ├── ideMode002 │ │ ├── .gitignore │ │ ├── expected.in │ │ ├── gen_expected.sh │ │ ├── input │ │ └── run │ ├── ideMode003 │ │ ├── LocType.idr │ │ ├── dummy.ipkg │ │ ├── expected │ │ ├── input │ │ └── run │ ├── ideMode004 │ │ ├── expected │ │ ├── input │ │ └── run │ ├── ideMode006 │ │ ├── Unsafe.idr │ │ ├── dummy.ipkg │ │ ├── expected │ │ ├── input │ │ └── run │ ├── ideMode007 │ │ ├── Syntax.idr │ │ ├── dummy.ipkg │ │ ├── expected │ │ ├── input │ │ └── run │ ├── ideMode008 │ │ ├── Interface.idr │ │ ├── dummy.ipkg │ │ ├── expected │ │ ├── input │ │ └── run │ ├── ideMode009 │ │ ├── Ambiguity.idr │ │ ├── expected │ │ ├── input │ │ └── run │ ├── ideMode010 │ │ ├── Rainbow.idr │ │ ├── dummy.ipkg │ │ ├── expected │ │ ├── input │ │ └── run │ ├── ideMode011 │ │ ├── Implementation.idr │ │ ├── dummy.ipkg │ │ ├── expected │ │ ├── input │ │ └── run │ ├── ideMode012 │ │ ├── Case.idr │ │ ├── dummy.ipkg │ │ ├── expected │ │ ├── input │ │ └── run │ ├── ideMode013 │ │ ├── RecordUpdate.idr │ │ ├── dummy.ipkg │ │ ├── expected │ │ ├── input │ │ └── run │ ├── ideMode014 │ │ ├── With.idr │ │ ├── dummy.ipkg │ │ ├── expected │ │ ├── input │ │ └── run │ ├── ideMode015 │ │ ├── Ranges.idr │ │ ├── dummy.ipkg │ │ ├── expected │ │ ├── input │ │ └── run │ ├── ideMode016 │ │ ├── StringLiterals.idr │ │ ├── dummy.ipkg │ │ ├── expected │ │ ├── input │ │ └── run │ ├── ideMode017 │ │ ├── WithApp.idr │ │ ├── dummy.ipkg │ │ ├── expected │ │ ├── input │ │ └── run │ ├── ideMode018 │ │ ├── Rewrite.idr │ │ ├── dummy.ipkg │ │ ├── expected │ │ ├── input │ │ └── run │ ├── ideMode019 │ │ ├── RecordProjections.idr │ │ ├── dummy.ipkg │ │ ├── expected │ │ ├── input │ │ └── run │ ├── ideMode020 │ │ ├── Tuples.idr │ │ ├── dummy.ipkg │ │ ├── expected │ │ ├── input │ │ └── run │ ├── ideMode021 │ │ ├── LetBinders.idr │ │ ├── dummy.ipkg │ │ ├── expected │ │ ├── input │ │ └── run │ ├── ideMode022 │ │ ├── SnocRainbow.idr │ │ ├── dummy.ipkg │ │ ├── expected │ │ ├── input │ │ └── run │ ├── ideMode023 │ │ ├── Fail.idr │ │ ├── dummy.ipkg │ │ ├── expected │ │ ├── input │ │ └── run │ └── ideMode024 │ │ ├── Holes.idr │ │ ├── dummy.ipkg │ │ ├── expected │ │ ├── input │ │ └── run ├── idris2 │ ├── api │ │ ├── README │ │ └── api001 │ │ │ ├── Hello.idr │ │ │ ├── LazyCodegen.idr │ │ │ ├── expected │ │ │ └── run │ ├── basic │ │ ├── basic001 │ │ │ ├── Vect.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── basic002 │ │ │ ├── Do.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── basic003 │ │ │ ├── Ambig1.idr │ │ │ ├── Ambig2.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── basic004 │ │ │ ├── Stuff.idr │ │ │ ├── Wheres.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── basic005 │ │ │ ├── NoInfer.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── basic006 │ │ │ ├── PMLet.idr │ │ │ ├── Stuff.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── basic007 │ │ │ ├── DoLocal.idr │ │ │ ├── Stuff.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── basic008 │ │ │ ├── If.idr │ │ │ ├── Stuff.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── basic009 │ │ │ ├── LetCase.idr │ │ │ ├── Stuff.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── basic010 │ │ │ ├── Comp.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── basic011 │ │ │ ├── Dots1.idr │ │ │ ├── Dots2.idr │ │ │ ├── Dots3.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── basic012 │ │ │ ├── VIndex.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── basic013 │ │ │ ├── Implicits.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── basic014 │ │ │ ├── Rewrite.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── basic015 │ │ │ ├── George.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── basic016 │ │ │ ├── Eta.idr │ │ │ ├── Eta2.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── basic017 │ │ │ ├── CaseInf.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── basic018 │ │ │ ├── Fin.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── basic019 │ │ │ ├── CaseBlock.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── basic020 │ │ │ ├── Mut.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── basic021 │ │ │ ├── CaseDep.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── basic022 │ │ │ ├── Erase.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── basic023 │ │ │ ├── Params.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── basic024 │ │ │ ├── PatLam.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── basic025 │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── basic026 │ │ │ ├── Erl.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── basic027 │ │ │ ├── Temp.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── basic028 │ │ │ ├── Do.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── basic029 │ │ │ ├── Params.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── basic030 │ │ │ ├── arity.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── basic031 │ │ │ ├── erased.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── basic032 │ │ │ ├── Idiom.idr │ │ │ ├── Idiom2.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── basic033 │ │ │ ├── expected │ │ │ ├── run │ │ │ └── unboundimps.idr │ │ ├── basic034 │ │ │ ├── expected │ │ │ ├── lets.idr │ │ │ └── run │ │ ├── basic035 │ │ │ ├── expected │ │ │ ├── input │ │ │ ├── run │ │ │ └── using.idr │ │ ├── basic036 │ │ │ ├── defimp.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── basic037 │ │ │ ├── Comments.idr │ │ │ ├── Issue279.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── basic038 │ │ │ ├── Resugar.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── basic039 │ │ │ ├── Main.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── basic040 │ │ │ ├── Default.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── basic041 │ │ │ ├── QDo.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── basic042 │ │ │ ├── LiteralsInteger.idr │ │ │ ├── LiteralsString.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ ├── input2 │ │ │ └── run │ │ ├── basic043 │ │ │ ├── BitCasts.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── basic044 │ │ │ ├── Term.idr │ │ │ ├── Vec.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── basic045 │ │ │ ├── Main.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── basic046 │ │ │ ├── TupleSections.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── basic047 │ │ │ ├── InterleavingLets.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── basic049 │ │ │ ├── Fld.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── basic050 │ │ │ ├── Ilc.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── basic051 │ │ │ ├── Issue833.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── basic052 │ │ │ ├── DoubleClBrace.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── basic053 │ │ │ ├── UnderscoredIntegerLiterals.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── basic054 │ │ │ ├── Issue1023.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── basic055 │ │ │ ├── BitOps.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── basic056 │ │ │ ├── DoubleLit.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── basic057 │ │ │ ├── LetIn.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── basic058 │ │ │ ├── DataTypeOp.idr │ │ │ ├── DataTypeProj.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── basic059 │ │ │ ├── MultiClaim.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── basic060 │ │ │ ├── Snoc.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── basic061 │ │ │ ├── IgnoreDo.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── basic062 │ │ │ ├── Issue1943.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── basic063 │ │ │ ├── NoDeclaration.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── basic064 │ │ │ ├── Issue2072.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── basic065 │ │ │ ├── Issue215.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── basic066 │ │ │ ├── comment.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── basic067 │ │ │ ├── expected │ │ │ ├── input │ │ │ ├── run │ │ │ ├── unclosed1.idr │ │ │ ├── unclosed2.idr │ │ │ └── unclosed3.idr │ │ ├── basic068 │ │ │ ├── Issue2138.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── basic069 │ │ │ ├── DebugInfo.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── basic070 │ │ │ ├── Issue2592.idr │ │ │ ├── Issue2593.idr │ │ │ ├── Issue2782.idr │ │ │ ├── Issue3016.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── basic071 │ │ │ ├── A.idr │ │ │ ├── B.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── basic072 │ │ │ ├── Issue3327.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── basic073 │ │ │ ├── DefaultHole.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── basic074 │ │ │ ├── erased.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── basic075 │ │ │ ├── Issue2128.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── basic076 │ │ │ ├── Issue3670.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── case001 │ │ │ ├── InlineCase.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── case002 │ │ │ ├── WhereData.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── dotted001 │ │ │ ├── Issue2726.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── dotted002 │ │ │ ├── DottedType.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── idiom001 │ │ │ ├── Main.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── interpolation001 │ │ │ ├── IfThenElse.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── interpolation002 │ │ │ ├── StringLiteral.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── interpolation003 │ │ │ ├── Test.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── interpolation004 │ │ │ ├── StringLiteral.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── literals001 │ │ │ ├── Test.idr │ │ │ ├── expected │ │ │ └── run │ │ └── rewrite001 │ │ │ ├── Issue2573.idr │ │ │ ├── expected │ │ │ └── run │ ├── builtin │ │ ├── builtin001 │ │ │ ├── Test.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── builtin002 │ │ │ ├── Test.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── builtin003 │ │ │ ├── Test.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── builtin004 │ │ │ ├── Test.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── builtin005 │ │ │ ├── Test.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── builtin006 │ │ │ ├── Test.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── builtin007 │ │ │ ├── Test.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── builtin008 │ │ │ ├── Test.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── builtin009 │ │ │ ├── Test.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── builtin010 │ │ │ ├── Test.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── builtin011 │ │ │ ├── Test.idr │ │ │ ├── expected │ │ │ └── run │ │ └── builtin012 │ │ │ ├── Issue1799.idr │ │ │ ├── expected │ │ │ └── run │ ├── casetree │ │ ├── casetree001 │ │ │ ├── IsS.idr │ │ │ ├── Issue762.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── casetree002 │ │ │ ├── DefaultCases.idr │ │ │ ├── Issue1079.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── casetree003 │ │ │ ├── ForcedPats.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── casetree004 │ │ │ ├── LocalArgs.idr │ │ │ ├── PiMatch.idr │ │ │ ├── expected │ │ │ └── run │ │ └── heuristics001 │ │ │ ├── Main.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ ├── coverage │ │ ├── coverage001 │ │ │ ├── Vect.idr │ │ │ ├── Vect2.idr │ │ │ ├── Vect3.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── coverage002 │ │ │ ├── Vect.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── coverage003 │ │ │ ├── Cover.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── coverage004 │ │ │ ├── Cover.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── coverage005 │ │ │ ├── Cover.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── coverage006 │ │ │ ├── expected │ │ │ ├── foobar.idr │ │ │ ├── input │ │ │ └── run │ │ ├── coverage007 │ │ │ ├── eq.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── coverage008 │ │ │ ├── expected │ │ │ ├── input │ │ │ ├── run │ │ │ └── wcov.idr │ │ ├── coverage009 │ │ │ ├── expected │ │ │ ├── run │ │ │ └── unreachable.idr │ │ ├── coverage010 │ │ │ ├── casetot.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── coverage011 │ │ │ ├── Sing.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── coverage012 │ │ │ ├── Issue484.idr │ │ │ ├── Issue899.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── coverage013 │ │ │ ├── Issue1022-Refl.idr │ │ │ ├── Issue1022.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── coverage014 │ │ │ ├── Issue794.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── coverage015 │ │ │ ├── Issue1169.idr │ │ │ ├── Issue1366.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── coverage016 │ │ │ ├── Issue633-2.idr │ │ │ ├── Issue633.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── coverage017 │ │ │ ├── Issue1421.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── coverage018 │ │ │ ├── Issue1831_1.idr │ │ │ ├── Issue1831_2.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── coverage019 │ │ │ ├── Issue1632.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── coverage020 │ │ │ ├── Issue3143.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── coverage021 │ │ │ ├── Head.idr │ │ │ ├── Issue2250a.idr │ │ │ ├── Issue2250b.idr │ │ │ ├── Issue2250c.idr │ │ │ ├── Issue3276.idr │ │ │ ├── Visibility.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── coverage022 │ │ │ ├── Issue3477.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── coverage023 │ │ │ ├── Main.idr │ │ │ ├── X.idr │ │ │ ├── Y.idr │ │ │ ├── expected │ │ │ └── run │ │ └── impossible001 │ │ │ ├── DottedTypeImpossible.idr │ │ │ ├── expected │ │ │ └── run │ ├── data │ │ ├── data001 │ │ │ ├── Test.idr │ │ │ ├── TestImpl.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── data002 │ │ │ ├── Test.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── data003 │ │ │ ├── Issue3457.idr │ │ │ ├── OopsDef.idr │ │ │ ├── OopsRef.idr │ │ │ ├── Positivity.idr │ │ │ ├── Test.idr │ │ │ ├── Test2.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── data004 │ │ │ ├── EmptySearch.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── data005 │ │ │ ├── Issue1204.idr │ │ │ ├── Issue586.idr │ │ │ ├── Issue586b.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── data006 │ │ │ ├── ConvertPiInfo.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── record001 │ │ │ ├── Record.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── record002 │ │ │ ├── Record.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── record003 │ │ │ ├── Record.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── record004 │ │ │ ├── Main.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── record005 │ │ │ ├── Fld.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── record006 │ │ │ ├── Fld.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── record007 │ │ │ ├── Bond.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── record008 │ │ │ ├── Postfix.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── record009 │ │ │ ├── expected │ │ │ ├── input │ │ │ ├── record.idr │ │ │ └── run │ │ ├── record010 │ │ │ ├── expected │ │ │ ├── record.idr │ │ │ └── run │ │ ├── record011 │ │ │ ├── Issue2095.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── record012 │ │ │ ├── Issue2065.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── record013 │ │ │ ├── Issue1945.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── record014 │ │ │ ├── Issue1404.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── record015 │ │ │ ├── Issue2176.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── record016 │ │ │ ├── HoleRecord.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── record017 │ │ │ ├── RecordOptions.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── record018 │ │ │ ├── expected │ │ │ ├── mut.idr │ │ │ └── run │ │ ├── record019 │ │ │ ├── BindParams.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── record020 │ │ │ ├── RecordImplicit.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── record021 │ │ │ ├── Issue3501.idr │ │ │ ├── RecordParam.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── record022 │ │ │ ├── EmptySearch.idr │ │ │ ├── expected │ │ │ └── run │ │ └── record023 │ │ │ ├── Broken.idr │ │ │ ├── Main.idr │ │ │ ├── expected │ │ │ └── run │ ├── debug │ │ └── debug001 │ │ │ ├── TypePat.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ ├── error │ │ ├── error001 │ │ │ ├── Error.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── error002 │ │ │ ├── Error.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── error003 │ │ │ ├── Error.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── error004 │ │ │ ├── Error1.idr │ │ │ ├── Error2.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── error005 │ │ │ ├── IfErr.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── error006 │ │ │ ├── IfErr.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── error007 │ │ │ ├── CongErr.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── error008 │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── error009 │ │ │ ├── Exists.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── error010 │ │ │ ├── Loop.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── error011 │ │ │ ├── ConstructorDuplicate.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── error012 │ │ │ ├── expected │ │ │ └── run │ │ ├── error013 │ │ │ ├── Issue361.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── error014 │ │ │ ├── Issue735.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── error015 │ │ │ ├── Issue110.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── error016 │ │ │ ├── Issue1230.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── error017 │ │ │ ├── Issue962-case.idr │ │ │ ├── Issue962.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── error018 │ │ │ ├── Issue1031-2.idr │ │ │ ├── Issue1031-3.idr │ │ │ ├── Issue1031-4.idr │ │ │ ├── Issue1031.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── error019 │ │ │ ├── Error.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── error020 │ │ │ ├── Error.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── error021 │ │ │ ├── DeepAmbig.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── error022 │ │ │ ├── UpdateLoc.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── error023 │ │ │ ├── Error1.idr │ │ │ ├── Error2.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── error024 │ │ │ ├── Error1.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── error025 │ │ │ ├── IAlternativePrints.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── error026 │ │ │ ├── DoBlockFC.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── error027 │ │ │ ├── Issue2950.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── error028 │ │ │ ├── Issue3313.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── error029 │ │ │ ├── Issue34.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── error030 │ │ │ ├── Issue1236-2.idr │ │ │ ├── Issue1236.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── error032 │ │ │ ├── expected │ │ │ └── run │ │ ├── error033 │ │ │ ├── Examples.idr │ │ │ ├── UnifyPiInfo.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── perror001 │ │ │ ├── PError.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── perror002 │ │ │ ├── PError.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── perror003 │ │ │ ├── PError.idr │ │ │ ├── PError2.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── perror004 │ │ │ ├── PError.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── perror005 │ │ │ ├── PError.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── perror006 │ │ │ ├── PError.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── perror007 │ │ │ ├── StrError1.idr │ │ │ ├── StrError10.idr │ │ │ ├── StrError11.idr │ │ │ ├── StrError12.idr │ │ │ ├── StrError2.idr │ │ │ ├── StrError3.idr │ │ │ ├── StrError4.idr │ │ │ ├── StrError5.idr │ │ │ ├── StrError6.idr │ │ │ ├── StrError7.idr │ │ │ ├── StrError8.idr │ │ │ ├── StrError9.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── perror008 │ │ │ ├── Issue1224a.idr │ │ │ ├── Issue1224b.idr │ │ │ ├── Issue710a.idr │ │ │ ├── Issue710b.idr │ │ │ ├── Issue710c.idr │ │ │ ├── Issue710d.idr │ │ │ ├── Issue710e.idr │ │ │ ├── Issue710f.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── perror009 │ │ │ ├── Error1.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── perror010 │ │ │ ├── NamedReturn1.idr │ │ │ ├── NamedReturn2.idr │ │ │ ├── NamedReturn3.idr │ │ │ ├── NamedReturn4.idr │ │ │ ├── TrailingLam.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── perror011 │ │ │ ├── Issue1345.idr │ │ │ ├── Issue1496-1.idr │ │ │ ├── Issue1496-2.idr │ │ │ ├── Main.idr │ │ │ ├── Pretty.idr │ │ │ ├── expected │ │ │ ├── foo.ipkg │ │ │ └── run │ │ ├── perror012 │ │ │ ├── CaseParseError.idr │ │ │ ├── LamParseError.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── perror013 │ │ │ ├── EmptyFailing.idr │ │ │ ├── EmptyMutual.idr │ │ │ ├── EmptyParameters.idr │ │ │ ├── EmptyUsing.idr │ │ │ ├── expected │ │ │ ├── run │ │ │ └── x.ipkg │ │ ├── perror014 │ │ │ ├── ParseList.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── perror015 │ │ │ ├── ParseWith.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── perror016 │ │ │ ├── ParseIf.idr │ │ │ ├── ParseIf2.idr │ │ │ ├── ParseIf3.idr │ │ │ ├── ParseIf4.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── perror017 │ │ │ ├── ParseImpl.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── perror018 │ │ │ ├── ParseRecord.idr │ │ │ ├── ParseRecord2.idr │ │ │ ├── ParseRecord3.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── perror019 │ │ │ ├── ImplError.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── perror020 │ │ │ ├── Issue2769.idr │ │ │ ├── Issue2769b.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── perror021 │ │ │ ├── Implicit.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── perror022 │ │ │ ├── Indent.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── perror023 │ │ │ ├── ParseError.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── perror024 │ │ │ ├── ParseError.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── perror025 │ │ │ ├── DataWhere.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── perror026 │ │ │ ├── Micro.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── perror027 │ │ │ ├── Outdent.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── perror028 │ │ │ ├── LetInDo.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── perror029 │ │ │ ├── DelayParse.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── perror030 │ │ │ ├── LoggingParse.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── perror031 │ │ │ ├── Issue3251.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── perror032 │ │ │ ├── LambdaImpossible.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── perror033 │ │ │ ├── DeclIndent.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── perror034 │ │ │ ├── Error.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── perror035 │ │ │ ├── ParseError.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── perror036 │ │ │ ├── Issue3594.idr │ │ │ ├── Main.idr │ │ │ ├── expected │ │ │ └── run │ │ └── withMatches │ │ │ ├── WithMatch.idr │ │ │ ├── expected │ │ │ └── run │ ├── evaluator │ │ ├── evaluator001 │ │ │ ├── Issue650.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── evaluator002 │ │ │ ├── Lib.idr │ │ │ ├── Main.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── evaluator003 │ │ │ ├── Issue705.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── evaluator004 │ │ │ ├── Issue1282.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── evaluator005 │ │ │ ├── TypeCase.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── interpreter001 │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── interpreter002 │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── interpreter003 │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── interpreter004 │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── interpreter005 │ │ │ ├── Issue37.idr │ │ │ ├── Issue37.lidr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── interpreter006 │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── interpreter007 │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── interpreter008 │ │ │ ├── Issue2041.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ └── spec001 │ │ │ ├── Desc.idr │ │ │ ├── Desc2.idr │ │ │ ├── Identity.idr │ │ │ ├── Mult3.idr │ │ │ ├── expected │ │ │ └── run │ ├── failing │ │ ├── failing001 │ │ │ ├── Fail.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── failing002 │ │ │ ├── FailingBug.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── failing003 │ │ │ ├── FailingTotality.idr │ │ │ ├── expected │ │ │ └── run │ │ └── failing004 │ │ │ ├── Issue2821.idr │ │ │ ├── expected │ │ │ └── run │ ├── interactive │ │ ├── interactive001 │ │ │ ├── LocType.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── interactive002 │ │ │ ├── IEdit.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── interactive003 │ │ │ ├── IEdit.idr │ │ │ ├── IEdit2.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ ├── input2 │ │ │ └── run │ │ ├── interactive004 │ │ │ ├── IEdit.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── interactive005 │ │ │ ├── IEdit.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── interactive006 │ │ │ ├── IEdit.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── interactive007 │ │ │ ├── IEdit.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── interactive008 │ │ │ ├── IEdit.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── interactive009 │ │ │ ├── Door.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── interactive010 │ │ │ ├── IEdit.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── interactive011 │ │ │ ├── IEdit.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── interactive012 │ │ │ ├── WithLift.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── interactive013 │ │ │ ├── Spacing.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── interactive014 │ │ │ ├── case.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── interactive015 │ │ │ ├── IEdit.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── interactive016 │ │ │ ├── Cont.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── interactive017 │ │ │ ├── RLE.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── interactive018 │ │ │ ├── PlusPrf.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── interactive019 │ │ │ ├── TypeSearch.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── interactive020 │ │ │ ├── Issue835.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── interactive021 │ │ │ ├── TypeAtDoNotation.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── interactive022 │ │ │ ├── TypeAtBangSyntax.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── interactive023 │ │ │ ├── TypeAtLambda.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── interactive024 │ │ │ ├── TypeAtAsPatterns.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── interactive025 │ │ │ ├── TypeAtInterfaces.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── interactive026 │ │ │ ├── TypeAtRecords.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── interactive027 │ │ │ ├── TypeAtLocalVars.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── interactive028 │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── interactive029 │ │ │ ├── Issue834.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── interactive030 │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── interactive031 │ │ │ ├── Signatures.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── interactive032 │ │ │ ├── Uninh.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── interactive033 │ │ │ ├── UninhIndent.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── interactive034 │ │ │ ├── expected │ │ │ ├── input │ │ │ ├── run │ │ │ └── timeout.idr │ │ ├── interactive035 │ │ │ ├── expected │ │ │ ├── input │ │ │ ├── run │ │ │ └── unify.idr │ │ ├── interactive036 │ │ │ ├── casefn.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── interactive037 │ │ │ ├── Holes.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── interactive038 │ │ │ ├── IEdit.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── interactive039 │ │ │ ├── CS_Syntax.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── interactive040 │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── interactive041 │ │ │ ├── Issue1741.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── interactive042 │ │ │ ├── Issue35-2.idr │ │ │ ├── Issue35.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── interactive043 │ │ │ ├── ImplicitSplits.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── interactive044 │ │ │ ├── SplitShadow.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── interactive045 │ │ │ ├── Issue1742.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── interactive046 │ │ │ ├── Issue2712.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── interactive047 │ │ │ ├── Missing.idr │ │ │ ├── expected │ │ │ └── run │ │ └── interactive048 │ │ │ ├── Issue3487.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ ├── interface │ │ ├── interface001 │ │ │ ├── IFace.idr │ │ │ ├── IFace1.idr │ │ │ ├── Stuff.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ ├── input1 │ │ │ └── run │ │ ├── interface002 │ │ │ ├── Functor.idr │ │ │ ├── Stuff.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── interface003 │ │ │ ├── Do.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── interface004 │ │ │ ├── Do.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── interface005 │ │ │ ├── Deps.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── interface006 │ │ │ ├── Apply.idr │ │ │ ├── Biapplicative.idr │ │ │ ├── Bimonad.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── interface007 │ │ │ ├── A.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── interface008 │ │ │ ├── Deps.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── interface009 │ │ │ ├── Odd.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── interface010 │ │ │ ├── Dep.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── interface011 │ │ │ ├── FuncImpl.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── interface012 │ │ │ ├── Defmeth.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── interface013 │ │ │ ├── TypeInt.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── interface014 │ │ │ ├── DepInt.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── interface015 │ │ │ ├── expected │ │ │ ├── gnu.idr │ │ │ └── run │ │ ├── interface016 │ │ │ ├── TwoNum.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── interface017 │ │ │ ├── Tricho.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── interface018 │ │ │ ├── Sized.idr │ │ │ ├── Sized2.idr │ │ │ ├── Sized3.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── interface019 │ │ │ ├── LocalHints.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── interface020 │ │ │ ├── LocalInterface.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── interface021 │ │ │ ├── LocalHint.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── interface022 │ │ │ ├── DotMethod.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── interface023 │ │ │ ├── AppComp.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── interface024 │ │ │ ├── EH.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── interface025 │ │ │ ├── AutoSearchHide1.idr │ │ │ ├── AutoSearchHide2.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── interface026 │ │ │ ├── UninhabitedRec.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── interface027 │ │ │ ├── expected │ │ │ ├── input │ │ │ ├── params.idr │ │ │ └── run │ │ ├── interface028 │ │ │ ├── InterfaceArgs.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── interface029 │ │ │ ├── ForwardImpl1.idr │ │ │ ├── ForwardImpl2.idr │ │ │ ├── ForwardImpl3.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── interface030 │ │ │ ├── DefaultImplicitsInImpls.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── interface031 │ │ │ ├── DefaulthintWithDep.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── interface032 │ │ │ ├── DefaulthintInterfaceBug.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── interface033 │ │ │ ├── PairErroneouslyFound.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── interface034 │ │ │ ├── Main.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── interface035 │ │ │ ├── Issue3448.idr │ │ │ ├── NoUnbound.idr │ │ │ ├── expected │ │ │ └── run │ │ └── interface036 │ │ │ ├── Issue3474.idr │ │ │ ├── expected │ │ │ └── run │ ├── linear │ │ ├── linear001 │ │ │ ├── Door.idr │ │ │ ├── Stuff.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── linear002 │ │ │ ├── Door.idr │ │ │ ├── Stuff.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── linear003 │ │ │ ├── Linear.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── linear005 │ │ │ ├── Door.idr │ │ │ ├── Linear.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── linear006 │ │ │ ├── ZFun.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── linear007 │ │ │ ├── LCase.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── linear008 │ │ │ ├── Door.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── linear009 │ │ │ ├── expected │ │ │ ├── input │ │ │ ├── qtt.idr │ │ │ └── run │ │ ├── linear010 │ │ │ ├── Door.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── linear011 │ │ │ ├── Network.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── linear012 │ │ │ ├── expected │ │ │ ├── input │ │ │ ├── linholes.idr │ │ │ └── run │ │ ├── linear013 │ │ │ ├── Issue758.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── linear014 │ │ │ ├── Issue55.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── linear015 │ │ │ ├── Issue1861.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── linear016 │ │ │ ├── Issue2895.idr │ │ │ ├── Issue2895_2.idr │ │ │ ├── expected │ │ │ └── run │ │ └── linear017 │ │ │ ├── As.idr │ │ │ ├── expected │ │ │ └── run │ ├── literate │ │ ├── literate001 │ │ │ ├── IEdit.lidr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── literate002 │ │ │ ├── IEdit.lidr │ │ │ ├── IEdit2.lidr │ │ │ ├── expected │ │ │ ├── input │ │ │ ├── input2 │ │ │ └── run │ │ ├── literate003 │ │ │ ├── IEdit.lidr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── literate004 │ │ │ ├── IEdit.lidr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── literate005 │ │ │ ├── IEdit.lidr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── literate006 │ │ │ ├── Door.lidr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── literate007 │ │ │ ├── IEdit.lidr │ │ │ ├── IEdit.org │ │ │ ├── IEditOrg.org │ │ │ ├── expected │ │ │ ├── input │ │ │ ├── input2 │ │ │ └── run │ │ ├── literate008 │ │ │ ├── IEdit.lidr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── literate009 │ │ │ ├── WithLift.lidr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── literate010 │ │ │ ├── MyFirstIdrisProgram.org │ │ │ ├── expected │ │ │ └── run │ │ ├── literate011 │ │ │ ├── IEdit.md │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── literate012 │ │ │ ├── IEdit.org │ │ │ ├── IEdit2.org │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── literate013 │ │ │ ├── Lit.lidr │ │ │ ├── LitTeX.tex │ │ │ ├── expected │ │ │ └── run │ │ ├── literate014 │ │ │ ├── expected │ │ │ ├── input │ │ │ ├── run │ │ │ └── with.lidr │ │ ├── literate015 │ │ │ ├── case.lidr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── literate016 │ │ │ ├── IEdit.org │ │ │ ├── IEdit2.org │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── literate017 │ │ │ ├── .gitignore │ │ │ ├── expected │ │ │ ├── input │ │ │ ├── project-expected.ipkg │ │ │ ├── run │ │ │ └── src │ │ │ │ ├── A │ │ │ │ ├── A.org │ │ │ │ └── AB.lidr │ │ │ │ ├── B │ │ │ │ ├── B.md │ │ │ │ └── BA.markdown │ │ │ │ └── Main.idr │ │ ├── literate018 │ │ │ ├── Test.lidr.md │ │ │ ├── expected │ │ │ └── run │ │ ├── literate019 │ │ │ ├── Test1.typ │ │ │ ├── Test2.idr.typ │ │ │ ├── expected │ │ │ └── run │ │ └── literate020 │ │ │ ├── IEdit.dj │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ ├── misc │ │ ├── docs001 │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── docs002 │ │ │ ├── Doc.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── docs003 │ │ │ ├── RecordDoc.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── docs004 │ │ │ ├── DocImpl.idr │ │ │ ├── List.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ ├── input2 │ │ │ └── run │ │ ├── docs005 │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── eta001 │ │ │ ├── Issue1370.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── golden001 │ │ │ ├── 000-hello │ │ │ │ ├── expected │ │ │ │ └── run │ │ │ ├── Main.idr │ │ │ ├── Test.idr │ │ │ ├── expected │ │ │ ├── hello.ipkg │ │ │ ├── run │ │ │ └── test.ipkg │ │ ├── import001 │ │ │ ├── Mult.idr │ │ │ ├── Nat.idr │ │ │ ├── Test.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── import002 │ │ │ ├── Mult.idr │ │ │ ├── Nat.idr │ │ │ ├── Test.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── import003 │ │ │ ├── A.idr │ │ │ ├── B.idr │ │ │ ├── C.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── import004 │ │ │ ├── Cycle1.idr │ │ │ ├── Cycle2.idr │ │ │ ├── Loop.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── import005 │ │ │ ├── As.idr │ │ │ ├── Test.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── import006 │ │ │ ├── A │ │ │ │ ├── B.idr │ │ │ │ └── C.idr │ │ │ ├── cyclic.ipkg │ │ │ ├── expected │ │ │ └── run │ │ ├── import007 │ │ │ ├── Mod.idr │ │ │ ├── Mod1.idr │ │ │ ├── Mod2.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── import008 │ │ │ ├── Exe │ │ │ │ ├── Mod.idr │ │ │ │ └── exe.ipkg │ │ │ ├── Lib │ │ │ │ ├── Conf.idr │ │ │ │ └── lib.ipkg │ │ │ ├── expected │ │ │ └── run │ │ ├── import009 │ │ │ ├── Import.idr │ │ │ ├── Infix.idr │ │ │ ├── Prefix.idr │ │ │ ├── Resugar.idr │ │ │ ├── Test.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── inlining001 │ │ │ ├── Inlining.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── lazy001 │ │ │ ├── Lazy.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── lazy002 │ │ │ ├── LazyFoldlM.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── lazy003 │ │ │ ├── DelayLam.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── lazy004 │ │ │ ├── LazyFor.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── lazy005 │ │ │ ├── LiftedBot.idr │ │ │ ├── LiftedTrace.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── namespace001 │ │ │ ├── Dup.idr │ │ │ ├── Scope.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── namespace002 │ │ │ ├── Issue1313.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── namespace003 │ │ │ ├── Test.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── namespace004 │ │ │ ├── Export.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── namespace005 │ │ │ ├── Lib1.idr │ │ │ ├── Lib2.idr │ │ │ ├── LibPre1.idr │ │ │ ├── LibPre2.idr │ │ │ ├── Main0.idr │ │ │ ├── Main1.idr │ │ │ ├── Main3.idr │ │ │ ├── MainConflict.idr │ │ │ ├── MainFail.idr │ │ │ ├── MainPre0.idr │ │ │ ├── MainPre1.idr │ │ │ ├── NonConflict1.idr │ │ │ ├── NonConflict2.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── params001 │ │ │ ├── expected │ │ │ ├── param.idr │ │ │ ├── parambad.idr │ │ │ └── run │ │ ├── params002 │ │ │ ├── ParamsPrint.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── params003 │ │ │ ├── casesplit.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── params004 │ │ │ ├── Issue2331.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── pretty001 │ │ │ ├── Issue1328A.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── pretty002 │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── primloop │ │ │ ├── PrimLoop.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── quantifiers001 │ │ │ ├── TestQuantifiers.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── real001 │ │ │ ├── Channel.idr │ │ │ ├── Linear.idr │ │ │ ├── MakeChans.idr │ │ │ ├── TestProto.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── real002 │ │ │ ├── Store.idr │ │ │ ├── StoreL.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── unification001 │ │ │ ├── Issue647.idr │ │ │ ├── expected │ │ │ └── run │ │ └── with003 │ │ │ ├── Main.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ ├── mkdoc │ │ └── mkdoc001 │ │ │ ├── Test1.idr │ │ │ ├── Test2.idr │ │ │ ├── Test3.idr │ │ │ ├── Test4.idr │ │ │ ├── expected │ │ │ ├── run │ │ │ └── test.ipkg │ ├── operators │ │ ├── operators001 │ │ │ ├── Test.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── operators002 │ │ │ ├── Error2.idr │ │ │ ├── Errors.idr │ │ │ ├── Errors2.idr │ │ │ ├── Errors3.idr │ │ │ ├── Errors4.idr │ │ │ ├── Errors5.idr │ │ │ ├── Lin.idr │ │ │ ├── LinImport.idr │ │ │ ├── Test.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── operators003 │ │ │ ├── Error1.idr │ │ │ ├── Error2.idr │ │ │ ├── Error3.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── operators004 │ │ │ ├── Test.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── operators005 │ │ │ ├── Test.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── operators006 │ │ │ ├── Test.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── operators007 │ │ │ ├── Test.idr │ │ │ ├── Test2.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── operators008 │ │ │ ├── Test.idr │ │ │ ├── Test2.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── operators009 │ │ │ ├── Test.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── operators010 │ │ │ ├── Test.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── operators011 │ │ │ ├── Module.idr │ │ │ ├── Test.idr │ │ │ ├── Test1.idr │ │ │ ├── Test2.idr │ │ │ ├── Test3.idr │ │ │ ├── Test4.idr │ │ │ ├── expected │ │ │ └── run │ │ └── operators012 │ │ │ ├── Y.idr │ │ │ ├── expected │ │ │ └── run │ ├── perf │ │ ├── perf001 │ │ │ ├── Big.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── perf002 │ │ │ ├── Big.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── perf003 │ │ │ ├── Auto.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── perf004 │ │ │ ├── bigdpair.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── perf005 │ │ │ ├── Bad1.idr │ │ │ ├── Bad2.idr │ │ │ ├── Bad3.idr │ │ │ ├── Lambda.idr │ │ │ ├── NoRegression.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── perf007 │ │ │ ├── Slooow.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── perf008 │ │ │ ├── FinPerf.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── perf009 │ │ │ ├── A.idr │ │ │ ├── B.idr │ │ │ ├── C.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── perf010 │ │ │ ├── Printf.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── perf011 │ │ │ ├── A.idr │ │ │ ├── B.idr │ │ │ ├── C.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── perf012 │ │ │ ├── Main.idr │ │ │ ├── expected │ │ │ └── run │ │ └── perf2202 │ │ │ ├── Church.idr │ │ │ ├── expected │ │ │ ├── many10000.idr │ │ │ └── run │ ├── pkg │ │ ├── multiline-comments │ │ │ ├── Main.idr │ │ │ ├── expected │ │ │ ├── run │ │ │ └── test.ipkg │ │ ├── pkg001 │ │ │ ├── Dummy.idr │ │ │ ├── dummy.ipkg │ │ │ ├── expected │ │ │ └── run │ │ ├── pkg002 │ │ │ ├── dummy.ipkg │ │ │ ├── expected │ │ │ ├── run │ │ │ └── src │ │ │ │ └── Top │ │ │ │ └── Dummy.idr │ │ ├── pkg003 │ │ │ ├── Main.idr │ │ │ ├── expected │ │ │ ├── run │ │ │ └── testpkg.ipkg │ │ ├── pkg004 │ │ │ ├── Dummy.idr │ │ │ ├── dummy.ipkg │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── pkg005 │ │ │ ├── Foo.idr │ │ │ ├── expected │ │ │ ├── foo.ipkg │ │ │ ├── input │ │ │ └── run │ │ ├── pkg006 │ │ │ ├── depends │ │ │ │ ├── bar-1.0.1 │ │ │ │ │ └── bar.ipkg │ │ │ │ ├── bar-baz │ │ │ │ │ └── bar-baz.ipkg │ │ │ │ ├── foo-0.5 │ │ │ │ │ └── foo.ipkg │ │ │ │ ├── foo-bar-1.3.1 │ │ │ │ │ └── foo-bar.ipkg │ │ │ │ └── quux │ │ │ │ │ └── quux.ipkg │ │ │ ├── expected │ │ │ ├── run │ │ │ ├── test1.ipkg │ │ │ ├── test2.ipkg │ │ │ ├── test3.ipkg │ │ │ ├── test4.ipkg │ │ │ └── test5.ipkg │ │ ├── pkg007 │ │ │ ├── A │ │ │ │ └── Path │ │ │ │ │ └── Of │ │ │ │ │ └── Dires │ │ │ │ │ ├── First.idr │ │ │ │ │ └── Second.idr │ │ │ ├── Another │ │ │ │ ├── Fourth.idr │ │ │ │ └── One │ │ │ │ │ └── Third.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ ├── input2 │ │ │ ├── run │ │ │ └── src │ │ │ │ ├── And │ │ │ │ └── A │ │ │ │ │ └── Proof.idr │ │ │ │ └── Yet │ │ │ │ └── Another │ │ │ │ └── Path.idr │ │ ├── pkg008 │ │ │ ├── Bar.idr │ │ │ ├── Foo.idr │ │ │ ├── bar.ipkg │ │ │ ├── expected │ │ │ ├── foo.ipkg │ │ │ └── run │ │ ├── pkg009 │ │ │ ├── expected │ │ │ ├── run │ │ │ └── testpkg │ │ │ │ ├── Main.idr │ │ │ │ └── testpkg.ipkg │ │ ├── pkg010 │ │ │ ├── Main.idr │ │ │ ├── expected │ │ │ ├── run │ │ │ └── testpkg.ipkg │ │ ├── pkg011 │ │ │ ├── dot-slash-dot │ │ │ │ ├── Main.idr │ │ │ │ └── testpkg.ipkg │ │ │ ├── dot-slash-name-slash │ │ │ │ ├── src │ │ │ │ │ └── Main.idr │ │ │ │ └── testpkg.ipkg │ │ │ ├── dot-slash │ │ │ │ ├── Main.idr │ │ │ │ └── testpkg.ipkg │ │ │ ├── dot │ │ │ │ ├── Main.idr │ │ │ │ └── testpkg.ipkg │ │ │ ├── expected │ │ │ ├── run │ │ │ └── sibling │ │ │ │ ├── pkg │ │ │ │ └── testpkg.ipkg │ │ │ │ └── src │ │ │ │ └── Main.idr │ │ ├── pkg012 │ │ │ ├── Main.idr │ │ │ ├── expected │ │ │ ├── run │ │ │ └── testpkg.ipkg │ │ ├── pkg013 │ │ │ ├── depends │ │ │ │ ├── bar-0.7.2 │ │ │ │ │ └── bar.ipkg │ │ │ │ └── foo-0.1.0 │ │ │ │ │ └── foo.ipkg │ │ │ ├── expected │ │ │ ├── run │ │ │ └── test.ipkg │ │ ├── pkg014 │ │ │ ├── depends │ │ │ │ ├── bar-0.1.0 │ │ │ │ │ └── bar.ipkg │ │ │ │ ├── bar-0.1.1 │ │ │ │ │ └── bar.ipkg │ │ │ │ ├── baz-0.1.0 │ │ │ │ │ └── baz.ipkg │ │ │ │ ├── baz-0.2.0 │ │ │ │ │ └── baz.ipkg │ │ │ │ ├── baz-0.3.0 │ │ │ │ │ └── baz.ipkg │ │ │ │ ├── foo-0.1.0 │ │ │ │ │ └── foo.ipkg │ │ │ │ ├── foo-0.2.0 │ │ │ │ │ └── foo.ipkg │ │ │ │ └── foo-0.3.0 │ │ │ │ │ └── foo.ipkg │ │ │ ├── expected │ │ │ ├── run │ │ │ └── test.ipkg │ │ ├── pkg015 │ │ │ ├── depends │ │ │ │ ├── bar-0.1.0 │ │ │ │ │ └── bar.ipkg │ │ │ │ ├── bar-0.1.1 │ │ │ │ │ └── bar.ipkg │ │ │ │ ├── baz-0.1.0 │ │ │ │ │ └── baz.ipkg │ │ │ │ ├── baz-0.2.0 │ │ │ │ │ └── baz.ipkg │ │ │ │ ├── baz-0.3.0 │ │ │ │ │ └── baz.ipkg │ │ │ │ ├── foo-0.1.0 │ │ │ │ │ └── foo.ipkg │ │ │ │ ├── foo-0.2.0 │ │ │ │ │ └── foo.ipkg │ │ │ │ ├── foo-0.3.0 │ │ │ │ │ └── foo.ipkg │ │ │ │ └── prz-0.1.0 │ │ │ │ │ └── prz.ipkg │ │ │ ├── expected │ │ │ ├── run │ │ │ └── test.ipkg │ │ ├── pkg016 │ │ │ ├── bar.ipkg │ │ │ ├── bar │ │ │ │ └── Bar.idr │ │ │ ├── baz.ipkg │ │ │ ├── baz │ │ │ │ └── Baz.idr │ │ │ ├── expected │ │ │ ├── foo.ipkg │ │ │ ├── foo │ │ │ │ └── Foo.idr │ │ │ ├── run │ │ │ ├── src │ │ │ │ └── Test.idr │ │ │ └── test.ipkg │ │ ├── pkg017 │ │ │ ├── a1 │ │ │ │ ├── A.idr │ │ │ │ └── a1.ipkg │ │ │ ├── a2 │ │ │ │ ├── A.idr │ │ │ │ └── a2.ipkg │ │ │ ├── b1 │ │ │ │ ├── b1.ipkg │ │ │ │ └── src │ │ │ │ │ └── B1.idr │ │ │ ├── b2 │ │ │ │ ├── b2.ipkg │ │ │ │ └── src │ │ │ │ │ └── B2.idr │ │ │ ├── expected │ │ │ ├── input1 │ │ │ ├── input2 │ │ │ └── run │ │ ├── pkg018 │ │ │ ├── bad.ipkg │ │ │ ├── bad2.ipkg │ │ │ ├── expected │ │ │ └── run │ │ ├── pkg019 │ │ │ ├── expected │ │ │ ├── run │ │ │ ├── src │ │ │ │ ├── And │ │ │ │ │ └── A │ │ │ │ │ │ └── Proof.idr │ │ │ │ ├── Main.idr │ │ │ │ └── Yet │ │ │ │ │ └── Another │ │ │ │ │ └── Path.idr │ │ │ └── test.ipkg │ │ ├── pkg020 │ │ │ ├── expected │ │ │ ├── run │ │ │ ├── src │ │ │ │ └── Stuff.idr │ │ │ └── test.ipkg │ │ ├── pkg021 │ │ │ ├── expected │ │ │ ├── input │ │ │ ├── run │ │ │ ├── src │ │ │ │ └── Stuff.idr │ │ │ └── test.ipkg │ │ └── pkg022 │ │ │ ├── Capitalised-With-Dashes.ipkg │ │ │ ├── Main.idr │ │ │ ├── expected │ │ │ └── run │ ├── reflection │ │ ├── bindvar_mn │ │ │ ├── Id.idr │ │ │ ├── Plus.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── reflection001 │ │ │ ├── expected │ │ │ ├── input │ │ │ ├── quote.idr │ │ │ └── run │ │ ├── reflection002 │ │ │ ├── expected │ │ │ ├── input │ │ │ ├── power.idr │ │ │ └── run │ │ ├── reflection003 │ │ │ ├── expected │ │ │ ├── refprims.idr │ │ │ └── run │ │ ├── reflection004 │ │ │ ├── expected │ │ │ ├── input │ │ │ ├── refdecl.idr │ │ │ └── run │ │ ├── reflection005 │ │ │ ├── expected │ │ │ ├── input │ │ │ ├── refdecl.idr │ │ │ └── run │ │ ├── reflection006 │ │ │ ├── expected │ │ │ ├── input │ │ │ ├── refleq.idr │ │ │ └── run │ │ ├── reflection007 │ │ │ ├── NatExpr.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── reflection008 │ │ │ ├── Interp.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── reflection009 │ │ │ ├── expected │ │ │ ├── perf.idr │ │ │ └── run │ │ ├── reflection010 │ │ │ ├── Name.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── reflection011 │ │ │ ├── expected │ │ │ ├── input │ │ │ ├── run │ │ │ └── tryref.idr │ │ ├── reflection012 │ │ │ ├── expected │ │ │ ├── input │ │ │ ├── nameinfo.idr │ │ │ └── run │ │ ├── reflection013 │ │ │ ├── WithUnambig.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── reflection014 │ │ │ ├── expected │ │ │ ├── refdecl.idr │ │ │ └── run │ │ ├── reflection015 │ │ │ ├── MacroRetFunc.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── reflection016 │ │ │ ├── BindElabScBug.idr │ │ │ ├── Eta.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── reflection017 │ │ │ ├── CanElabType.idr │ │ │ ├── StillCantEscape.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── reflection018 │ │ │ ├── AtTypeLevel.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── reflection019 │ │ │ ├── ElabScriptWarning.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ ├── run │ │ │ └── test.ipkg │ │ ├── reflection020 │ │ │ ├── FromDecls.idr │ │ │ ├── FromName.idr │ │ │ ├── FromTTImp.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── reflection021 │ │ │ ├── QuoteSearch.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── reflection022 │ │ │ ├── BadElabScript.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── reflection023 │ │ │ ├── DeclMacro.idr │ │ │ ├── UseMacroWithoutExtension.idr │ │ │ ├── expected │ │ │ ├── run │ │ │ └── test.ipkg │ │ ├── reflection024 │ │ │ ├── .gitignore │ │ │ ├── expected │ │ │ ├── run │ │ │ ├── src │ │ │ │ ├── Inside │ │ │ │ │ └── PrintDirs.idr │ │ │ │ ├── LessSimpleRW.idr │ │ │ │ ├── SimpleRW.idr │ │ │ │ ├── TypeProviders.idr │ │ │ │ ├── existentToRead │ │ │ │ ├── existentToWrite │ │ │ │ └── fancy-record.txt │ │ │ └── test.ipkg │ │ ├── reflection025 │ │ │ ├── CurrFn.idr │ │ │ ├── InspectRec.idr │ │ │ ├── RefDefs.idr │ │ │ ├── RefDefsDeep.idr │ │ │ ├── expected │ │ │ ├── run │ │ │ └── test.ipkg │ │ ├── reflection026 │ │ │ ├── Issue3168.idr │ │ │ ├── expected │ │ │ ├── run │ │ │ └── test.ipkg │ │ ├── reflection027 │ │ │ ├── TraverseWithConst.idr │ │ │ ├── expected │ │ │ ├── run │ │ │ └── test.ipkg │ │ ├── reflection028 │ │ │ ├── GetVis.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ ├── run │ │ │ └── test.ipkg │ │ ├── reflection030 │ │ │ ├── SearchZero.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── reflection031 │ │ │ ├── WithFC.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── reflection032 │ │ │ ├── DeterminingData.idr │ │ │ ├── DeterminingRecord.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── reflection033 │ │ │ ├── QuotingShadowed.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── reflection034 │ │ │ ├── ResugarTerm.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── reflection034_2 │ │ │ ├── LocalVars.idr │ │ │ ├── expected │ │ │ └── run │ │ └── reflection035 │ │ │ ├── Broken.idr │ │ │ ├── Main.idr │ │ │ ├── expected │ │ │ └── run │ ├── reg │ │ ├── reg001 │ │ │ ├── D.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── reg002 │ │ │ ├── expected │ │ │ ├── linm.idr │ │ │ └── run │ │ ├── reg003 │ │ │ ├── Holes.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── reg004 │ │ │ ├── ambig.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── reg005 │ │ │ ├── expected │ │ │ ├── iftype.idr │ │ │ └── run │ │ ├── reg006 │ │ │ ├── Cmd.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── reg007 │ │ │ ├── Main.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── reg008 │ │ │ ├── Vending.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── reg009 │ │ │ ├── Case.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── reg010 │ │ │ ├── Recordname.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── reg011 │ │ │ ├── expected │ │ │ ├── mut.idr │ │ │ └── run │ │ ├── reg012 │ │ │ ├── Foo.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── reg013 │ │ │ ├── UnboundImplicits.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── reg014 │ │ │ ├── casecase.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── reg015 │ │ │ ├── anyfail.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── reg016 │ │ │ ├── Using.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── reg017 │ │ │ ├── expected │ │ │ ├── lammult.idr │ │ │ └── run │ │ ├── reg018 │ │ │ ├── cycle.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── reg019 │ │ │ ├── expected │ │ │ ├── lazybug.idr │ │ │ └── run │ │ ├── reg020 │ │ │ ├── expected │ │ │ ├── input │ │ │ ├── matchlits.idr │ │ │ └── run │ │ ├── reg021 │ │ │ ├── case.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── reg022 │ │ │ ├── case.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── reg023 │ │ │ ├── boom.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── reg024 │ │ │ ├── expected │ │ │ ├── input │ │ │ ├── run │ │ │ └── split.idr │ │ ├── reg025 │ │ │ ├── expected │ │ │ ├── input │ │ │ ├── lift.idr │ │ │ └── run │ │ ├── reg026 │ │ │ ├── Meh.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── reg027 │ │ │ ├── expected │ │ │ ├── pwhere.idr │ │ │ └── run │ │ ├── reg028 │ │ │ ├── Test.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── reg029 │ │ │ ├── expected │ │ │ ├── lqueue.idr │ │ │ └── run │ │ ├── reg030 │ │ │ ├── A.idr │ │ │ ├── B.idr │ │ │ ├── C.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── reg031 │ │ │ ├── dpair.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── reg032 │ │ │ ├── expected │ │ │ ├── recupdate.idr │ │ │ └── run │ │ ├── reg033 │ │ │ ├── DerivingEq.idr │ │ │ ├── expected │ │ │ ├── run │ │ │ └── test.idr │ │ ├── reg034 │ │ │ ├── expected │ │ │ ├── run │ │ │ └── void.idr │ │ ├── reg035 │ │ │ ├── Implicit.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── reg036 │ │ │ ├── Test.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── reg037 │ │ │ ├── Test.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── reg038 │ │ │ ├── Test1.idr │ │ │ ├── Test2.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── reg039 │ │ │ ├── dupdup.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── reg040 │ │ │ ├── CoverBug.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── reg041 │ │ │ ├── expected │ │ │ ├── run │ │ │ └── tuple.idr │ │ ├── reg042 │ │ │ ├── NatOpts.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── reg043 │ │ │ ├── NotFake.idr │ │ │ ├── TestFake.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── reg044 │ │ │ ├── Methods.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── reg045 │ │ │ ├── expected │ │ │ ├── run │ │ │ └── withparams.idr │ │ ├── reg046 │ │ │ ├── Postpone.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── reg047 │ │ │ ├── QualifiedDoBang.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── reg048 │ │ │ ├── expected │ │ │ ├── inferror.idr │ │ │ └── run │ │ ├── reg049 │ │ │ ├── expected │ │ │ ├── lettype.idr │ │ │ └── run │ │ ├── reg050 │ │ │ ├── expected │ │ │ ├── loopy.idr │ │ │ └── run │ │ ├── reg051 │ │ │ ├── BigFins.idr │ │ │ ├── expected │ │ │ ├── run │ │ │ └── test.ipkg │ │ ├── reg052 │ │ │ ├── DPairQuote.idr │ │ │ ├── expected │ │ │ ├── run │ │ │ └── test.ipkg │ │ ├── reg053 │ │ │ ├── ImplicitParam.idr │ │ │ ├── Issue2444.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── reg054 │ │ │ ├── Issue3354.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── reg055 │ │ │ ├── Module01.idr │ │ │ ├── Module02.idr │ │ │ ├── Module03.idr │ │ │ ├── Module04.idr │ │ │ ├── Module05.idr │ │ │ ├── Module06.idr │ │ │ ├── Module07.idr │ │ │ ├── Module08.idr │ │ │ ├── Module09.idr │ │ │ ├── Module10.idr │ │ │ ├── Module11.idr │ │ │ ├── Module12.idr │ │ │ ├── Module13.idr │ │ │ ├── Module14.idr │ │ │ ├── Module15.idr │ │ │ ├── Module16.idr │ │ │ ├── Module17.idr │ │ │ ├── Module18.idr │ │ │ ├── Module19.idr │ │ │ ├── Module20.idr │ │ │ ├── Module21.idr │ │ │ ├── Module22.idr │ │ │ ├── Module23.idr │ │ │ ├── Module24.idr │ │ │ ├── Module25.idr │ │ │ ├── Module26.idr │ │ │ ├── Module27.idr │ │ │ ├── Module28.idr │ │ │ ├── Module29.idr │ │ │ ├── Module30.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── reg056 │ │ │ ├── WithUnambigNamesTTC.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── reg057 │ │ │ ├── Issue3623.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── reg058 │ │ │ ├── Issue3654.idr │ │ │ ├── expected │ │ │ └── run │ │ └── reg059 │ │ │ ├── Issue3669.idr │ │ │ ├── expected │ │ │ └── run │ ├── repl │ │ ├── repl001 │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── repl002 │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── repl003 │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── repl004 │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── repl005 │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── repl006 │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ └── repl007 │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ ├── schemeeval │ │ ├── schemeeval001 │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── schemeeval002 │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── schemeeval003 │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── schemeeval004 │ │ │ ├── expected │ │ │ ├── input │ │ │ ├── list.idr │ │ │ └── run │ │ ├── schemeeval005 │ │ │ ├── Printf.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ └── schemeeval006 │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ ├── termination │ │ └── termination001 │ │ │ ├── AgdaIssue6059.idr │ │ │ ├── expected │ │ │ └── run │ ├── total │ │ ├── positivity001 │ │ │ ├── Issue660.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── positivity002 │ │ │ ├── Issue660.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── positivity003 │ │ │ ├── Issue660.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── positivity004 │ │ │ ├── Issue1771-1.idr │ │ │ ├── Issue1771-2.idr │ │ │ ├── Issue1771-3.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── positivity005 │ │ │ ├── Issue2548.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── total001 │ │ │ ├── Total.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── total002 │ │ │ ├── Total.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── total003 │ │ │ ├── Total.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── total004 │ │ │ ├── Total.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── total005 │ │ │ ├── Total.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── total006 │ │ │ ├── Total.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── total007 │ │ │ ├── expected │ │ │ ├── partial.idr │ │ │ └── run │ │ ├── total008 │ │ │ ├── expected │ │ │ ├── partial.idr │ │ │ └── run │ │ ├── total009 │ │ │ ├── expected │ │ │ ├── run │ │ │ └── tree.idr │ │ ├── total010 │ │ │ ├── PartialWith.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── total011 │ │ │ ├── Issue1460.idr │ │ │ ├── Issue1782.idr │ │ │ ├── Issue1828.idr │ │ │ ├── Issue1859-2.idr │ │ │ ├── Issue1859.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── total012 │ │ │ ├── Issue1828.idr │ │ │ ├── TotallyTotal.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── total013 │ │ │ ├── Issue1404.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── total014 │ │ │ ├── FunCompTC.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── total015 │ │ │ ├── CoveringData.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── total016 │ │ │ ├── AssertPositivity.idr │ │ │ ├── LazyPositivityCheck.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── total017 │ │ │ ├── Paper.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── total018 │ │ │ ├── Issue2448.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── total019 │ │ │ ├── Check.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── total020 │ │ │ ├── Check.idr │ │ │ ├── expected │ │ │ ├── run │ │ │ └── test.ipkg │ │ ├── total021 │ │ │ ├── Issue-3030.idr │ │ │ ├── Issue-3030b.idr │ │ │ ├── Issue-524.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── total022 │ │ │ ├── Dot.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── total023 │ │ │ ├── Abel2002.idr │ │ │ ├── expected │ │ │ ├── input │ │ │ └── run │ │ ├── total024 │ │ │ ├── Issue1988.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── total025 │ │ │ ├── Issue3317.idr │ │ │ ├── Issue3353.idr │ │ │ ├── Pragma.idr │ │ │ ├── Totality.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── total026 │ │ │ ├── compilerOption.idr │ │ │ ├── doubleTotal.idr │ │ │ ├── duplicates.idr │ │ │ ├── expected │ │ │ ├── implementation.idr │ │ │ ├── implementationOverride.idr │ │ │ ├── interface.idr │ │ │ ├── issue3437.idr │ │ │ ├── noOverrideDefault.idr │ │ │ ├── overrideDefault.idr │ │ │ ├── run │ │ │ └── sameAsDefault.idr │ │ ├── total027 │ │ │ ├── dataDifferentTotality.idr │ │ │ ├── dataSameTotality.idr │ │ │ ├── dataTotalityOnlyDeclaration.idr │ │ │ ├── dataTotalityOnlyDefinition.idr │ │ │ ├── expected │ │ │ ├── recordDifferentTotality.idr │ │ │ ├── recordSameTotality.idr │ │ │ ├── recordTotalityOnlyDeclaration.idr │ │ │ ├── recordTotalityOnlyDefinition.idr │ │ │ └── run │ │ ├── total028 │ │ │ ├── Main.idr │ │ │ ├── expected │ │ │ └── run │ │ └── total029 │ │ │ ├── Issue806.idr │ │ │ ├── expected │ │ │ └── run │ ├── warning │ │ ├── warning001 │ │ │ ├── Holes.idr │ │ │ ├── Issue1401.idr │ │ │ ├── Issue539.idr │ │ │ ├── Issue621.idr │ │ │ ├── PR1407.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── warning002 │ │ │ ├── Foo.idr │ │ │ ├── Main.idr │ │ │ ├── deprecated.ipkg │ │ │ ├── expected │ │ │ └── run │ │ ├── warning003 │ │ │ ├── Main.idr │ │ │ ├── deprecated.ipkg │ │ │ ├── expected │ │ │ └── run │ │ ├── warning004 │ │ │ ├── Lib1.idr │ │ │ ├── Lib2.idr │ │ │ ├── Main1.idr │ │ │ ├── expected │ │ │ └── run │ │ ├── warning005 │ │ │ ├── Main.idr │ │ │ ├── expected │ │ │ └── run │ │ └── warning006 │ │ │ ├── Issue2325.idr │ │ │ ├── Main.idr │ │ │ ├── expected │ │ │ └── run │ └── with │ │ ├── with001 │ │ ├── Temp.idr │ │ ├── expected │ │ └── run │ │ ├── with002 │ │ ├── Temp.idr │ │ ├── expected │ │ └── run │ │ ├── with004 │ │ ├── Issue637-2.idr │ │ ├── Issue637-3.idr │ │ ├── Issue637.idr │ │ ├── expected │ │ ├── input │ │ └── run │ │ ├── with005 │ │ ├── Issue893.idr │ │ ├── WithProof.idr │ │ ├── expected │ │ └── run │ │ ├── with006 │ │ ├── SparseWith.idr │ │ ├── expected │ │ └── run │ │ ├── with007 │ │ ├── With0.idr │ │ ├── expected │ │ └── run │ │ ├── with008 │ │ ├── WithClause.idr │ │ ├── expected │ │ └── run │ │ ├── with009 │ │ ├── WithClause.idr │ │ ├── expected │ │ └── run │ │ ├── with010 │ │ ├── NestedWith.idr │ │ ├── expected │ │ └── run │ │ ├── with011 │ │ ├── WithImplicits.idr │ │ ├── expected │ │ └── run │ │ └── with012 │ │ ├── WithProof0.idr │ │ ├── WithProof0ElabFail.idr │ │ ├── WithProof0Fail.idr │ │ ├── WithProof1.idr │ │ ├── WithProof1Fail.idr │ │ ├── expected │ │ └── run ├── linear │ └── system_concurrency_session │ │ ├── Main.idr │ │ ├── expected │ │ └── run ├── node │ ├── args │ │ ├── TestArgs.idr │ │ ├── expected │ │ └── run │ ├── bitops │ │ ├── BitOps.idr │ │ ├── expected │ │ └── run │ ├── casts │ │ ├── Casts.idr │ │ ├── expected │ │ └── run │ ├── double001 │ │ ├── URandEpsilon.idr │ │ ├── expected │ │ ├── input │ │ └── run │ ├── double002 │ │ ├── NaN.idr │ │ ├── expected │ │ ├── input │ │ └── run │ ├── double003 │ │ ├── Inf.idr │ │ ├── expected │ │ ├── input │ │ └── run │ ├── doubles │ │ ├── Doubles.idr │ │ ├── expected │ │ └── run │ ├── executable │ │ ├── TestExecutable.idr │ │ ├── expected │ │ └── run │ ├── fastConcat │ │ ├── FastConcat.idr │ │ ├── expected │ │ └── run │ ├── ffi001 │ │ ├── Foreign.idr │ │ ├── expected │ │ └── run │ ├── fix1839 │ │ ├── OS.idr │ │ ├── expected │ │ └── run │ ├── idiom001 │ │ ├── Main.idr │ │ ├── expected │ │ └── run │ ├── integer_array │ │ ├── array.idr │ │ ├── expected │ │ └── run │ ├── integers │ │ ├── TestIntegers.idr │ │ ├── expected │ │ └── run │ ├── memo │ │ ├── Memo.idr │ │ ├── expected │ │ └── run │ ├── newints │ │ ├── IntOps.idr │ │ ├── expected │ │ └── run │ ├── node001 │ │ ├── Total.idr │ │ ├── expected │ │ └── run │ ├── node002 │ │ ├── Pythag.idr │ │ ├── expected │ │ ├── input │ │ └── run │ ├── node003 │ │ ├── IORef.idr │ │ ├── expected │ │ └── run │ ├── node004 │ │ ├── .gitignore │ │ ├── Buffer.idr │ │ ├── expected │ │ └── run │ ├── node005 │ │ ├── Filter.idr │ │ ├── expected │ │ ├── input │ │ └── run │ ├── node006 │ │ ├── TypeCase.idr │ │ ├── TypeCase2.idr │ │ ├── expected │ │ ├── input │ │ └── run │ ├── node007 │ │ ├── TypeCase.idr │ │ ├── expected │ │ └── run │ ├── node008 │ │ ├── Nat.idr │ │ ├── expected │ │ └── run │ ├── node009 │ │ ├── expected │ │ ├── run │ │ └── uni.idr │ ├── node011 │ │ ├── bangs.idr │ │ ├── expected │ │ ├── input │ │ └── run │ ├── node012 │ │ ├── array.idr │ │ ├── expected │ │ └── run │ ├── node015 │ │ ├── Numbers.idr │ │ ├── expected │ │ └── run │ ├── node017 │ │ ├── .gitignore │ │ ├── dir.idr │ │ ├── expected │ │ └── run │ ├── node018 │ │ ├── .gitignore │ │ ├── File.idr │ │ ├── expected │ │ ├── run │ │ └── test.txt │ ├── node019 │ │ ├── expected │ │ ├── input │ │ ├── partial.idr │ │ └── run │ ├── node020 │ │ ├── Popen.idr │ │ ├── expected │ │ └── run │ ├── node021 │ │ ├── Bits.idr │ │ ├── expected │ │ ├── input │ │ └── run │ ├── node022 │ │ ├── BitCasts.idr │ │ ├── expected │ │ └── run │ ├── node023 │ │ ├── Casts.idr │ │ ├── expected │ │ └── run │ ├── node024 │ │ ├── BitOps.idr │ │ ├── expected │ │ └── run │ ├── node025 │ │ ├── Fix1037.idr │ │ ├── expected │ │ └── run │ ├── node026 │ │ ├── Fix1795.idr │ │ ├── expected │ │ └── run │ ├── node027 │ │ ├── PID.idr │ │ ├── expected │ │ └── run │ ├── node028 │ │ ├── HelloWorld.idr │ │ ├── LazyIsStillThere.idr │ │ ├── expected │ │ └── run │ ├── nomangle001 │ │ ├── expected │ │ ├── nomangle.idr │ │ └── run │ ├── nomangle002 │ │ ├── expected │ │ ├── nomangle1.idr │ │ ├── nomangle2.idr │ │ └── run │ ├── perf001 │ │ ├── Span.idr │ │ ├── expected │ │ └── run │ ├── reg001 │ │ ├── expected │ │ ├── numbers.idr │ │ └── run │ ├── reg002 │ │ ├── Issue1843.idr │ │ ├── expected │ │ └── run │ ├── stringcast │ │ ├── StringCast.idr │ │ ├── expected │ │ └── run │ ├── syntax001 │ │ ├── caseBlock.idr │ │ ├── expected │ │ └── run │ ├── tailrec001 │ │ ├── expected │ │ ├── run │ │ └── tailrec.idr │ ├── tailrec002 │ │ ├── EvenOdd.idr │ │ ├── Main.idr │ │ ├── expected │ │ └── run │ └── tailrec_libs │ │ ├── expected │ │ ├── run │ │ └── tailrec.idr ├── prelude │ ├── bind001 │ │ ├── bind.idr │ │ ├── expected │ │ └── run │ ├── char001 │ │ ├── chars.idr │ │ ├── expected │ │ └── run │ ├── double001 │ │ ├── Types.idr │ │ ├── expected │ │ └── run │ ├── nat001 │ │ ├── expected │ │ ├── nats.idr │ │ └── run │ ├── operators001 │ │ ├── Test.idr │ │ ├── expected │ │ └── run │ ├── reg001 │ │ ├── expected │ │ ├── fixity.idr │ │ └── run │ └── unpack │ │ ├── expected │ │ ├── run │ │ └── unpack.idr ├── racket │ ├── barrier001 │ │ ├── Main.idr │ │ ├── expected │ │ ├── input │ │ └── run │ ├── conditions001 │ │ ├── Main.idr │ │ ├── expected │ │ └── run │ ├── conditions002 │ │ ├── Main.idr │ │ ├── expected │ │ └── run │ ├── conditions003 │ │ ├── Main.idr │ │ ├── expected │ │ └── run │ ├── conditions004 │ │ ├── Main.idr │ │ ├── expected │ │ └── run │ ├── conditions005 │ │ ├── Main.idr │ │ ├── expected │ │ └── run │ ├── conditions006 │ │ ├── Main.idr │ │ ├── expected │ │ └── run │ ├── conditions007 │ │ ├── Main.idr │ │ ├── expected │ │ └── run │ ├── ffi001 │ │ ├── RacketLib.idr │ │ ├── expected │ │ └── run │ ├── forkjoin001 │ │ ├── Main.idr │ │ ├── expected │ │ └── run │ ├── futures001 │ │ ├── Futures.idr │ │ ├── expected │ │ └── run │ ├── futures002 │ │ ├── Futures.idr │ │ ├── expected │ │ └── run │ ├── mutex001 │ │ ├── Main.idr │ │ ├── expected │ │ └── run │ ├── mutex002 │ │ ├── Main.idr │ │ ├── expected │ │ └── run │ ├── mutex003 │ │ ├── Main.idr │ │ ├── expected │ │ └── run │ ├── mutex004 │ │ ├── Main.idr │ │ ├── expected │ │ └── run │ ├── mutex005 │ │ ├── Main.idr │ │ ├── expected │ │ └── run │ ├── semaphores001 │ │ ├── Main.idr │ │ ├── expected │ │ └── run │ └── semaphores002 │ │ ├── Main.idr │ │ ├── expected │ │ └── run ├── refc │ ├── args │ │ ├── TestArgs.idr │ │ ├── expected │ │ └── run │ ├── basicpatternmatch │ │ ├── Main.idr │ │ ├── expected │ │ └── run │ ├── buffer │ │ ├── TestBuffer.idr │ │ ├── expected │ │ ├── run │ │ └── testRead.buf │ ├── callingConvention │ │ ├── Main.idr │ │ ├── expected │ │ └── run │ ├── ccompilerArgs │ │ ├── Main.idr │ │ ├── expected │ │ ├── library │ │ │ ├── Makefile │ │ │ ├── externalc.c │ │ │ └── externalc.h │ │ └── run │ ├── clock │ │ ├── TestClock.idr │ │ ├── expected │ │ └── run │ ├── doubles │ │ ├── TestDoubles.idr │ │ ├── expected │ │ └── run │ ├── garbageCollect │ │ ├── TestGarbageCollect.idr │ │ ├── expected │ │ └── run │ ├── integers │ │ ├── TestIntegers.idr │ │ ├── expected │ │ └── run │ ├── issue1778 │ │ ├── Reverse.idr │ │ ├── expected │ │ └── run │ ├── issue2424 │ │ ├── ControlAppMonadTest.idr │ │ ├── expected │ │ └── run │ ├── issue2452 │ │ ├── BitsCase.idr │ │ ├── expected │ │ └── run │ ├── piTypecase001 │ │ ├── Test.idr │ │ ├── expected │ │ └── run │ ├── prims │ │ ├── Test.idr │ │ ├── expected │ │ └── run │ ├── refc001 │ │ ├── Tail.idr │ │ ├── expected │ │ └── run │ ├── refc002 │ │ ├── RecordProjection.idr │ │ ├── expected │ │ └── run │ ├── refc003 │ │ ├── Issue1191.idr │ │ ├── expected │ │ └── run │ ├── reg001 │ │ ├── Issue1843.idr │ │ ├── expected │ │ └── run │ ├── reuse │ │ ├── Main.idr │ │ ├── expected │ │ └── run │ └── strings │ │ ├── TestStrings.idr │ │ ├── expected │ │ └── run ├── templates │ ├── simple-test │ │ ├── Test.idr │ │ ├── expected │ │ ├── input │ │ ├── notes.md │ │ └── run │ ├── ttimp │ │ ├── Interp.yaff │ │ ├── expected │ │ ├── input │ │ ├── notes.md │ │ └── run │ └── with-ipkg │ │ ├── Dummy.idr │ │ ├── dummy.ipkg │ │ ├── expected │ │ ├── notes.md │ │ └── run ├── tests.ipkg ├── testutils.sh ├── ttimp │ ├── basic001 │ │ ├── Interp.yaff │ │ ├── expected │ │ ├── input │ │ └── run │ ├── basic002 │ │ ├── Adder.yaff │ │ ├── expected │ │ ├── input │ │ └── run │ ├── basic003 │ │ ├── Hole.yaff │ │ ├── expected │ │ ├── input │ │ └── run │ ├── basic004 │ │ ├── AsPat.yaff │ │ ├── expected │ │ ├── input │ │ └── run │ ├── basic005 │ │ ├── Ambig.yaff │ │ ├── expected │ │ ├── input │ │ └── run │ ├── basic006 │ │ ├── Ambig.yaff │ │ ├── expected │ │ ├── input │ │ └── run │ ├── coverage002 │ │ ├── Vect.yaff │ │ ├── expected │ │ ├── input │ │ └── run │ ├── dot001 │ │ ├── Dot.yaff │ │ ├── Dot2.yaff │ │ ├── Dot3.yaff │ │ ├── Dot4.yaff │ │ ├── expected │ │ └── run │ ├── eta001 │ │ ├── Eta.yaff │ │ ├── expected │ │ ├── input │ │ └── run │ ├── lazy001 │ │ ├── Lazy.yaff │ │ ├── LazyInf.yaff │ │ ├── expected │ │ ├── input │ │ └── run │ ├── nest001 │ │ ├── Let.yaff │ │ ├── expected │ │ ├── input │ │ └── run │ ├── nest002 │ │ ├── Case.yaff │ │ ├── expected │ │ ├── input │ │ └── run │ ├── perf001 │ │ ├── bigsuc.yaff │ │ ├── expected │ │ └── run │ ├── perf002 │ │ ├── BigVect.yaff │ │ ├── expected │ │ ├── input │ │ └── run │ ├── perf003 │ │ ├── Id.yaff │ │ ├── expected │ │ ├── input │ │ └── run │ ├── qtt001 │ │ ├── QTT.yaff │ │ ├── expected │ │ ├── input │ │ └── run │ ├── qtt003 │ │ ├── QTTEq.yaff │ │ ├── expected │ │ ├── input │ │ └── run │ ├── record001 │ │ ├── Record.yaff │ │ ├── expected │ │ ├── input │ │ └── run │ ├── record002 │ │ ├── Record.yaff │ │ ├── expected │ │ ├── input │ │ └── run │ ├── record003 │ │ ├── Record.yaff │ │ ├── expected │ │ ├── input │ │ └── run │ ├── record004 │ │ ├── Record.yaff │ │ ├── expected │ │ ├── input │ │ └── run │ ├── total001 │ │ ├── Vect.yaff │ │ ├── expected │ │ ├── input │ │ └── run │ ├── total002 │ │ ├── Total.yaff │ │ ├── expected │ │ ├── input │ │ └── run │ ├── total003 │ │ ├── Bad.yaff │ │ ├── expected │ │ ├── input │ │ └── run │ └── total004 │ │ ├── expected │ │ ├── input │ │ ├── issue3437.yaff │ │ └── run ├── typedd-book │ ├── chapter01 │ │ ├── All.idr │ │ ├── FCTypes.idr │ │ ├── Hello.idr │ │ ├── HelloHole.idr │ │ ├── HoleFix.idr │ │ ├── expected │ │ ├── input │ │ └── run │ ├── chapter02 │ │ ├── All.idr │ │ ├── AveMain.idr │ │ ├── Average.idr │ │ ├── Double.idr │ │ ├── Generic.idr │ │ ├── HOF.idr │ │ ├── Let_Where.idr │ │ ├── Partial.idr │ │ ├── Reverse.idr │ │ ├── expected │ │ └── run │ ├── chapter03 │ │ ├── All.idr │ │ ├── IsEven.idr │ │ ├── Matrix.idr │ │ ├── VecSort.idr │ │ ├── Vectors.idr │ │ ├── WordLength.idr │ │ ├── WordLength_vec.idr │ │ ├── XOR.idr │ │ ├── expected │ │ └── run │ ├── chapter04 │ │ ├── All.idr │ │ ├── BSTree.idr │ │ ├── DataStore.idr │ │ ├── Direction.idr │ │ ├── Generic.idr │ │ ├── Picture.idr │ │ ├── Shape.idr │ │ ├── SumInputs.idr │ │ ├── Tree.idr │ │ ├── TryIndex.idr │ │ ├── Vect.idr │ │ ├── Vehicle.idr │ │ ├── expected │ │ └── run │ ├── chapter05 │ │ ├── All.idr │ │ ├── DepPairs.idr │ │ ├── Do.idr │ │ ├── Hello.idr │ │ ├── Loops.idr │ │ ├── PrintLength.idr │ │ ├── ReadNum.idr │ │ ├── ReadVect.idr │ │ ├── expected │ │ └── run │ ├── chapter06 │ │ ├── Adder.idr │ │ ├── All.idr │ │ ├── DataStore.idr │ │ ├── DataStoreHoles.idr │ │ ├── Maybe.idr │ │ ├── Printf.idr │ │ ├── TypeFuns.idr │ │ ├── TypeSynonyms.idr │ │ ├── expected │ │ └── run │ ├── chapter07 │ │ ├── Album.idr │ │ ├── All.idr │ │ ├── Eq.idr │ │ ├── Expr.idr │ │ ├── Fold.idr │ │ ├── Tree.idr │ │ ├── expected │ │ └── run │ ├── chapter08 │ │ ├── All.idr │ │ ├── AppendVec.idr │ │ ├── CheckEqDec.idr │ │ ├── CheckEqMaybe.idr │ │ ├── EqNat.idr │ │ ├── ExactLength.idr │ │ ├── ExactLengthDec.idr │ │ ├── ReverseVec.idr │ │ ├── TCVects.idr │ │ ├── Void.idr │ │ ├── expected │ │ └── run │ ├── chapter09 │ │ ├── All.idr │ │ ├── Elem.idr │ │ ├── ElemBool.idr │ │ ├── ElemType.idr │ │ ├── Hangman.idr │ │ ├── RemoveElem.idr │ │ ├── expected │ │ └── run │ ├── chapter10 │ │ ├── All.idr │ │ ├── DLFail.idr │ │ ├── DataStore.idr │ │ ├── DescribeList.idr │ │ ├── DescribeList2.idr │ │ ├── IsSuffix.idr │ │ ├── MergeSort.idr │ │ ├── MergeSortView.idr │ │ ├── Reverse.idr │ │ ├── ReverseSnoc.idr │ │ ├── Shape.idr │ │ ├── Shape_abs.idr │ │ ├── SnocList.idr │ │ ├── TestStore.idr │ │ ├── expected │ │ └── run │ ├── chapter11 │ │ ├── All.idr │ │ ├── Arith.idr │ │ ├── ArithCmd.idr │ │ ├── ArithCmdDo.idr │ │ ├── ArithTotal.idr │ │ ├── Greet.idr │ │ ├── InfIO.idr │ │ ├── InfList.idr │ │ ├── Label.idr │ │ ├── RunIO.idr │ │ ├── StreamFail.idr │ │ ├── Streams.idr │ │ ├── expected │ │ └── run │ ├── chapter12 │ │ ├── All.idr │ │ ├── ArithState.idr │ │ ├── DataStore.idr │ │ ├── Record.idr │ │ ├── State.idr │ │ ├── StateMonad.idr │ │ ├── Traverse.idr │ │ ├── TreeLabel.idr │ │ ├── TreeLabelState.idr │ │ ├── TreeLabelType.idr │ │ ├── expected │ │ └── run │ ├── chapter13 │ │ ├── All.idr │ │ ├── Door.idr │ │ ├── Stack.idr │ │ ├── StackIO.idr │ │ ├── Vending.idr │ │ ├── expected │ │ └── run │ └── chapter14 │ │ ├── ATM.idr │ │ ├── All.idr │ │ ├── DoorJam.idr │ │ ├── Hangman.idr │ │ ├── expected │ │ └── run └── vmcode │ └── basic001 │ ├── Test.idr │ ├── expected │ └── run └── www ├── README.md ├── katla.sh └── source ├── idris-logo-base.png └── index.md /.editorconfig: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/.editorconfig -------------------------------------------------------------------------------- /.gitattributes: -------------------------------------------------------------------------------- 1 | bootstrap/idris2_app/* linguist-generated 2 | -------------------------------------------------------------------------------- /.github/linters/.chktexrc: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/.github/linters/.chktexrc -------------------------------------------------------------------------------- /.github/linters/.ecrc: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/.github/linters/.ecrc -------------------------------------------------------------------------------- /.github/scripts/katla.sh: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/.github/scripts/katla.sh -------------------------------------------------------------------------------- /.gitignore: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/.gitignore -------------------------------------------------------------------------------- /.readthedocs.yaml: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/.readthedocs.yaml -------------------------------------------------------------------------------- /CHANGELOG.md: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/CHANGELOG.md -------------------------------------------------------------------------------- /CHANGELOG_NEXT.md: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/CHANGELOG_NEXT.md -------------------------------------------------------------------------------- /CITATION.cff: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/CITATION.cff -------------------------------------------------------------------------------- /CONTRIBUTING.md: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/CONTRIBUTING.md -------------------------------------------------------------------------------- /CONTRIBUTORS: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/CONTRIBUTORS -------------------------------------------------------------------------------- /INSTALL.md: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/INSTALL.md -------------------------------------------------------------------------------- /LICENSE: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/LICENSE -------------------------------------------------------------------------------- /Makefile: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/Makefile -------------------------------------------------------------------------------- /README.md: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/README.md -------------------------------------------------------------------------------- /Release/CHECKLIST: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/Release/CHECKLIST -------------------------------------------------------------------------------- /Release/mkdist.sh: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/Release/mkdist.sh -------------------------------------------------------------------------------- /benchmark/bench.sh: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/benchmark/bench.sh -------------------------------------------------------------------------------- /benchmark/benchmarks/mergeInt/mergeInt.in: -------------------------------------------------------------------------------- 1 | 1000 -------------------------------------------------------------------------------- /benchmark/benchmarks/mergeInt/mergeInt_fast.in: -------------------------------------------------------------------------------- 1 | 200 -------------------------------------------------------------------------------- /benchmark/benchmarks/mergeStr/mergeStr.in: -------------------------------------------------------------------------------- 1 | 30 -------------------------------------------------------------------------------- /benchmark/benchmarks/mergeStr/mergeStr_fast.in: -------------------------------------------------------------------------------- 1 | 6 -------------------------------------------------------------------------------- /benchmark/benchmarks/spellcheck/spellcheck.in: -------------------------------------------------------------------------------- 1 | input -------------------------------------------------------------------------------- /benchmark/benchmarks/spellcheck/spellcheck_fast.in: -------------------------------------------------------------------------------- 1 | input_small -------------------------------------------------------------------------------- /benchmark/benchmarks/treeInt/treeInt.in: -------------------------------------------------------------------------------- 1 | 350 -------------------------------------------------------------------------------- /benchmark/benchmarks/treeInt/treeInt_fast.in: -------------------------------------------------------------------------------- 1 | 80 -------------------------------------------------------------------------------- /benchmark/benchmarks/triples/triples.in: -------------------------------------------------------------------------------- 1 | 600 -------------------------------------------------------------------------------- /benchmark/benchmarks/triples/triples_fast.in: -------------------------------------------------------------------------------- 1 | 450 -------------------------------------------------------------------------------- /benchmark/readme.md: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/benchmark/readme.md -------------------------------------------------------------------------------- /bootstrap-stage1-chez.sh: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/bootstrap-stage1-chez.sh -------------------------------------------------------------------------------- /bootstrap-stage1-racket.sh: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/bootstrap-stage1-racket.sh -------------------------------------------------------------------------------- /bootstrap-stage2.sh: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/bootstrap-stage2.sh -------------------------------------------------------------------------------- /bootstrap/compile.ss: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/bootstrap/compile.ss -------------------------------------------------------------------------------- /bootstrap/idris2-boot.sh: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/bootstrap/idris2-boot.sh -------------------------------------------------------------------------------- /bootstrap/idris2-rktboot.sh: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/bootstrap/idris2-rktboot.sh -------------------------------------------------------------------------------- /config.mk: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/config.mk -------------------------------------------------------------------------------- /default.nix: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/default.nix -------------------------------------------------------------------------------- /docs/.python-version: -------------------------------------------------------------------------------- 1 | 3.10 2 | -------------------------------------------------------------------------------- /docs/LICENSE: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/docs/LICENSE -------------------------------------------------------------------------------- /docs/Makefile: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/docs/Makefile -------------------------------------------------------------------------------- /docs/README.md: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/docs/README.md -------------------------------------------------------------------------------- /docs/make.bat: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/docs/make.bat -------------------------------------------------------------------------------- /docs/pyproject.toml: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/docs/pyproject.toml -------------------------------------------------------------------------------- /docs/requirements.txt: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/docs/requirements.txt -------------------------------------------------------------------------------- /docs/source/_static/.gitkeep: -------------------------------------------------------------------------------- 1 | -------------------------------------------------------------------------------- /docs/source/app/index.rst: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/docs/source/app/index.rst -------------------------------------------------------------------------------- /docs/source/app/linear.rst: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/docs/source/app/linear.rst -------------------------------------------------------------------------------- /docs/source/conf.py: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/docs/source/conf.py -------------------------------------------------------------------------------- /docs/source/faq/faq.rst: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/docs/source/faq/faq.rst -------------------------------------------------------------------------------- /docs/source/ffi/ffi.rst: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/docs/source/ffi/ffi.rst -------------------------------------------------------------------------------- /docs/source/ffi/index.rst: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/docs/source/ffi/index.rst -------------------------------------------------------------------------------- /docs/source/image/login.png: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/docs/source/image/login.png -------------------------------------------------------------------------------- /docs/source/index.rst: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/docs/source/index.rst -------------------------------------------------------------------------------- /docs/uv.lock: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/docs/uv.lock -------------------------------------------------------------------------------- /flake.lock: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/flake.lock -------------------------------------------------------------------------------- /flake.nix: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/flake.nix -------------------------------------------------------------------------------- /icons/idris-128x128.png: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/icons/idris-128x128.png -------------------------------------------------------------------------------- /icons/idris-256x256.png: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/icons/idris-256x256.png -------------------------------------------------------------------------------- /icons/idris-48x48.png: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/icons/idris-48x48.png -------------------------------------------------------------------------------- /icons/idris-512x512.png: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/icons/idris-512x512.png -------------------------------------------------------------------------------- /icons/idris-64x64.png: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/icons/idris-64x64.png -------------------------------------------------------------------------------- /icons/idris.ico: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/icons/idris.ico -------------------------------------------------------------------------------- /icons/idris_icon.rc: -------------------------------------------------------------------------------- 1 | 0 ICON "idris.ico" 2 | -------------------------------------------------------------------------------- /icons/text-x-idris.svg: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/icons/text-x-idris.svg -------------------------------------------------------------------------------- /icons/x-idris-bytecode.xml: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/icons/x-idris-bytecode.xml -------------------------------------------------------------------------------- /icons/x-idris.xml: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/icons/x-idris.xml -------------------------------------------------------------------------------- /idris2.ipkg: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/idris2.ipkg -------------------------------------------------------------------------------- /idris2api.ipkg: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/idris2api.ipkg -------------------------------------------------------------------------------- /ipkg/idris2protocols.ipkg: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/ipkg/idris2protocols.ipkg -------------------------------------------------------------------------------- /libs/base/Control/App.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/libs/base/Control/App.idr -------------------------------------------------------------------------------- /libs/base/Control/Ord.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/libs/base/Control/Ord.idr -------------------------------------------------------------------------------- /libs/base/Data/Bits.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/libs/base/Data/Bits.idr -------------------------------------------------------------------------------- /libs/base/Data/Bool.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/libs/base/Data/Bool.idr -------------------------------------------------------------------------------- /libs/base/Data/Buffer.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/libs/base/Data/Buffer.idr -------------------------------------------------------------------------------- /libs/base/Data/Colist.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/libs/base/Data/Colist.idr -------------------------------------------------------------------------------- /libs/base/Data/DPair.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/libs/base/Data/DPair.idr -------------------------------------------------------------------------------- /libs/base/Data/Double.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/libs/base/Data/Double.idr -------------------------------------------------------------------------------- /libs/base/Data/Either.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/libs/base/Data/Either.idr -------------------------------------------------------------------------------- /libs/base/Data/Fin.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/libs/base/Data/Fin.idr -------------------------------------------------------------------------------- /libs/base/Data/Fuel.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/libs/base/Data/Fuel.idr -------------------------------------------------------------------------------- /libs/base/Data/Fun.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/libs/base/Data/Fun.idr -------------------------------------------------------------------------------- /libs/base/Data/IORef.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/libs/base/Data/IORef.idr -------------------------------------------------------------------------------- /libs/base/Data/List.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/libs/base/Data/List.idr -------------------------------------------------------------------------------- /libs/base/Data/List1.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/libs/base/Data/List1.idr -------------------------------------------------------------------------------- /libs/base/Data/Maybe.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/libs/base/Data/Maybe.idr -------------------------------------------------------------------------------- /libs/base/Data/Nat.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/libs/base/Data/Nat.idr -------------------------------------------------------------------------------- /libs/base/Data/Ref.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/libs/base/Data/Ref.idr -------------------------------------------------------------------------------- /libs/base/Data/Rel.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/libs/base/Data/Rel.idr -------------------------------------------------------------------------------- /libs/base/Data/So.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/libs/base/Data/So.idr -------------------------------------------------------------------------------- /libs/base/Data/Stream.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/libs/base/Data/Stream.idr -------------------------------------------------------------------------------- /libs/base/Data/String.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/libs/base/Data/String.idr -------------------------------------------------------------------------------- /libs/base/Data/These.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/libs/base/Data/These.idr -------------------------------------------------------------------------------- /libs/base/Data/Vect.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/libs/base/Data/Vect.idr -------------------------------------------------------------------------------- /libs/base/Data/Void.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/libs/base/Data/Void.idr -------------------------------------------------------------------------------- /libs/base/Debug/Trace.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/libs/base/Debug/Trace.idr -------------------------------------------------------------------------------- /libs/base/Makefile: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/libs/base/Makefile -------------------------------------------------------------------------------- /libs/base/System.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/libs/base/System.idr -------------------------------------------------------------------------------- /libs/base/System/FFI.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/libs/base/System/FFI.idr -------------------------------------------------------------------------------- /libs/base/System/File.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/libs/base/System/File.idr -------------------------------------------------------------------------------- /libs/base/System/Info.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/libs/base/System/Info.idr -------------------------------------------------------------------------------- /libs/base/System/REPL.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/libs/base/System/REPL.idr -------------------------------------------------------------------------------- /libs/base/System/Term.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/libs/base/System/Term.idr -------------------------------------------------------------------------------- /libs/base/base.ipkg: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/libs/base/base.ipkg -------------------------------------------------------------------------------- /libs/contrib/Makefile: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/libs/contrib/Makefile -------------------------------------------------------------------------------- /libs/contrib/contrib.ipkg: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/libs/contrib/contrib.ipkg -------------------------------------------------------------------------------- /libs/linear/Makefile: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/libs/linear/Makefile -------------------------------------------------------------------------------- /libs/linear/linear.ipkg: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/libs/linear/linear.ipkg -------------------------------------------------------------------------------- /libs/network/.gitignore: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/libs/network/.gitignore -------------------------------------------------------------------------------- /libs/network/Makefile: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/libs/network/Makefile -------------------------------------------------------------------------------- /libs/network/network.ipkg: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/libs/network/network.ipkg -------------------------------------------------------------------------------- /libs/papers/Data/W.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/libs/papers/Data/W.idr -------------------------------------------------------------------------------- /libs/papers/Makefile: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/libs/papers/Makefile -------------------------------------------------------------------------------- /libs/papers/papers.ipkg: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/libs/papers/papers.ipkg -------------------------------------------------------------------------------- /libs/prelude/Builtin.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/libs/prelude/Builtin.idr -------------------------------------------------------------------------------- /libs/prelude/Makefile: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/libs/prelude/Makefile -------------------------------------------------------------------------------- /libs/prelude/Prelude.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/libs/prelude/Prelude.idr -------------------------------------------------------------------------------- /libs/prelude/PrimIO.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/libs/prelude/PrimIO.idr -------------------------------------------------------------------------------- /libs/prelude/prelude.ipkg: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/libs/prelude/prelude.ipkg -------------------------------------------------------------------------------- /libs/test/Makefile: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/libs/test/Makefile -------------------------------------------------------------------------------- /libs/test/README.md: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/libs/test/README.md -------------------------------------------------------------------------------- /libs/test/Test/Golden.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/libs/test/Test/Golden.idr -------------------------------------------------------------------------------- /libs/test/test.ipkg: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/libs/test/test.ipkg -------------------------------------------------------------------------------- /lint/lint.py: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/lint/lint.py -------------------------------------------------------------------------------- /nix/buildIdris.nix: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/nix/buildIdris.nix -------------------------------------------------------------------------------- /nix/idris2Api.nix: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/nix/idris2Api.nix -------------------------------------------------------------------------------- /nix/init.el: -------------------------------------------------------------------------------- 1 | (require 'idris2-mode) 2 | -------------------------------------------------------------------------------- /nix/lib.nix: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/nix/lib.nix -------------------------------------------------------------------------------- /nix/package.nix: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/nix/package.nix -------------------------------------------------------------------------------- /nix/support.nix: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/nix/support.nix -------------------------------------------------------------------------------- /nix/templates/pkg/Foo.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/nix/templates/pkg/Foo.idr -------------------------------------------------------------------------------- /nix/test.nix: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/nix/test.nix -------------------------------------------------------------------------------- /nix/text-editor.nix: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/nix/text-editor.nix -------------------------------------------------------------------------------- /samples/BTree.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/samples/BTree.idr -------------------------------------------------------------------------------- /samples/FFI-readline/Test/test.ipkg: -------------------------------------------------------------------------------- 1 | package test 2 | 3 | opts = "-p readline" 4 | -------------------------------------------------------------------------------- /samples/Interp.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/samples/Interp.idr -------------------------------------------------------------------------------- /samples/InterpE.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/samples/InterpE.idr -------------------------------------------------------------------------------- /samples/MyOrd.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/samples/MyOrd.idr -------------------------------------------------------------------------------- /samples/NamedSemi.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/samples/NamedSemi.idr -------------------------------------------------------------------------------- /samples/Prims.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/samples/Prims.idr -------------------------------------------------------------------------------- /samples/Proofs.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/samples/Proofs.idr -------------------------------------------------------------------------------- /samples/Vect.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/samples/Vect.idr -------------------------------------------------------------------------------- /samples/Void.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/samples/Void.idr -------------------------------------------------------------------------------- /samples/With.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/samples/With.idr -------------------------------------------------------------------------------- /samples/bmain.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/samples/bmain.idr -------------------------------------------------------------------------------- /samples/deprec.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/samples/deprec.idr -------------------------------------------------------------------------------- /samples/dummy.ipkg: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/samples/dummy.ipkg -------------------------------------------------------------------------------- /samples/fctypes.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/samples/fctypes.idr -------------------------------------------------------------------------------- /samples/ffi/Small.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/samples/ffi/Small.idr -------------------------------------------------------------------------------- /samples/ffi/Struct.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/samples/ffi/Struct.idr -------------------------------------------------------------------------------- /samples/ffi/args.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/samples/ffi/args.idr -------------------------------------------------------------------------------- /samples/ffi/dummy.ipkg: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/samples/ffi/dummy.ipkg -------------------------------------------------------------------------------- /samples/ffi/smallc.c: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/samples/ffi/smallc.c -------------------------------------------------------------------------------- /samples/holes.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/samples/holes.idr -------------------------------------------------------------------------------- /samples/io.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/samples/io.idr -------------------------------------------------------------------------------- /samples/listcomp.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/samples/listcomp.idr -------------------------------------------------------------------------------- /samples/multiplicity.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/samples/multiplicity.idr -------------------------------------------------------------------------------- /samples/params.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/samples/params.idr -------------------------------------------------------------------------------- /samples/proofs/proof.ipkg: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/samples/proofs/proof.ipkg -------------------------------------------------------------------------------- /samples/wheres.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/samples/wheres.idr -------------------------------------------------------------------------------- /src/Algebra.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Algebra.idr -------------------------------------------------------------------------------- /src/Algebra/Preorder.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Algebra/Preorder.idr -------------------------------------------------------------------------------- /src/Algebra/Semiring.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Algebra/Semiring.idr -------------------------------------------------------------------------------- /src/Compiler/ANF.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Compiler/ANF.idr -------------------------------------------------------------------------------- /src/Compiler/CaseOpts.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Compiler/CaseOpts.idr -------------------------------------------------------------------------------- /src/Compiler/Common.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Compiler/Common.idr -------------------------------------------------------------------------------- /src/Compiler/ES/Ast.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Compiler/ES/Ast.idr -------------------------------------------------------------------------------- /src/Compiler/ES/Doc.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Compiler/ES/Doc.idr -------------------------------------------------------------------------------- /src/Compiler/ES/Node.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Compiler/ES/Node.idr -------------------------------------------------------------------------------- /src/Compiler/ES/State.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Compiler/ES/State.idr -------------------------------------------------------------------------------- /src/Compiler/ES/ToAst.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Compiler/ES/ToAst.idr -------------------------------------------------------------------------------- /src/Compiler/Inline.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Compiler/Inline.idr -------------------------------------------------------------------------------- /src/Compiler/NoMangle.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Compiler/NoMangle.idr -------------------------------------------------------------------------------- /src/Compiler/Opts/CSE.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Compiler/Opts/CSE.idr -------------------------------------------------------------------------------- /src/Compiler/RefC.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Compiler/RefC.idr -------------------------------------------------------------------------------- /src/Compiler/RefC/CC.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Compiler/RefC/CC.idr -------------------------------------------------------------------------------- /src/Compiler/Separate.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Compiler/Separate.idr -------------------------------------------------------------------------------- /src/Compiler/VMCode.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Compiler/VMCode.idr -------------------------------------------------------------------------------- /src/Core/AutoSearch.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Core/AutoSearch.idr -------------------------------------------------------------------------------- /src/Core/Binary.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Core/Binary.idr -------------------------------------------------------------------------------- /src/Core/Binary/Prims.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Core/Binary/Prims.idr -------------------------------------------------------------------------------- /src/Core/Case/Util.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Core/Case/Util.idr -------------------------------------------------------------------------------- /src/Core/CompileExpr.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Core/CompileExpr.idr -------------------------------------------------------------------------------- /src/Core/Context.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Core/Context.idr -------------------------------------------------------------------------------- /src/Core/Context/Data.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Core/Context/Data.idr -------------------------------------------------------------------------------- /src/Core/Context/Log.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Core/Context/Log.idr -------------------------------------------------------------------------------- /src/Core/Context/TTC.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Core/Context/TTC.idr -------------------------------------------------------------------------------- /src/Core/Core.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Core/Core.idr -------------------------------------------------------------------------------- /src/Core/Coverage.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Core/Coverage.idr -------------------------------------------------------------------------------- /src/Core/Directory.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Core/Directory.idr -------------------------------------------------------------------------------- /src/Core/Env.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Core/Env.idr -------------------------------------------------------------------------------- /src/Core/FC.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Core/FC.idr -------------------------------------------------------------------------------- /src/Core/GetType.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Core/GetType.idr -------------------------------------------------------------------------------- /src/Core/Hash.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Core/Hash.idr -------------------------------------------------------------------------------- /src/Core/LinearCheck.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Core/LinearCheck.idr -------------------------------------------------------------------------------- /src/Core/Metadata.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Core/Metadata.idr -------------------------------------------------------------------------------- /src/Core/Name.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Core/Name.idr -------------------------------------------------------------------------------- /src/Core/Name/Scoped.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Core/Name/Scoped.idr -------------------------------------------------------------------------------- /src/Core/Normalise.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Core/Normalise.idr -------------------------------------------------------------------------------- /src/Core/Options.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Core/Options.idr -------------------------------------------------------------------------------- /src/Core/Options/Log.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Core/Options/Log.idr -------------------------------------------------------------------------------- /src/Core/Ord.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Core/Ord.idr -------------------------------------------------------------------------------- /src/Core/Primitives.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Core/Primitives.idr -------------------------------------------------------------------------------- /src/Core/Reflect.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Core/Reflect.idr -------------------------------------------------------------------------------- /src/Core/SchemeEval.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Core/SchemeEval.idr -------------------------------------------------------------------------------- /src/Core/TT.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Core/TT.idr -------------------------------------------------------------------------------- /src/Core/TT/Binder.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Core/TT/Binder.idr -------------------------------------------------------------------------------- /src/Core/TT/Primitive.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Core/TT/Primitive.idr -------------------------------------------------------------------------------- /src/Core/TT/Subst.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Core/TT/Subst.idr -------------------------------------------------------------------------------- /src/Core/TT/Term.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Core/TT/Term.idr -------------------------------------------------------------------------------- /src/Core/TT/Var.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Core/TT/Var.idr -------------------------------------------------------------------------------- /src/Core/TT/Views.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Core/TT/Views.idr -------------------------------------------------------------------------------- /src/Core/TTC.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Core/TTC.idr -------------------------------------------------------------------------------- /src/Core/Termination.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Core/Termination.idr -------------------------------------------------------------------------------- /src/Core/Transform.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Core/Transform.idr -------------------------------------------------------------------------------- /src/Core/Unify.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Core/Unify.idr -------------------------------------------------------------------------------- /src/Core/UnifyState.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Core/UnifyState.idr -------------------------------------------------------------------------------- /src/Core/Value.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Core/Value.idr -------------------------------------------------------------------------------- /src/Core/WithData.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Core/WithData.idr -------------------------------------------------------------------------------- /src/Idris/CommandLine.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Idris/CommandLine.idr -------------------------------------------------------------------------------- /src/Idris/Desugar.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Idris/Desugar.idr -------------------------------------------------------------------------------- /src/Idris/Doc/Display.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Idris/Doc/Display.idr -------------------------------------------------------------------------------- /src/Idris/Doc/HTML.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Idris/Doc/HTML.idr -------------------------------------------------------------------------------- /src/Idris/Doc/String.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Idris/Doc/String.idr -------------------------------------------------------------------------------- /src/Idris/Driver.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Idris/Driver.idr -------------------------------------------------------------------------------- /src/Idris/Env.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Idris/Env.idr -------------------------------------------------------------------------------- /src/Idris/Error.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Idris/Error.idr -------------------------------------------------------------------------------- /src/Idris/Main.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Idris/Main.idr -------------------------------------------------------------------------------- /src/Idris/ModTree.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Idris/ModTree.idr -------------------------------------------------------------------------------- /src/Idris/Package.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Idris/Package.idr -------------------------------------------------------------------------------- /src/Idris/Parser.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Idris/Parser.idr -------------------------------------------------------------------------------- /src/Idris/Parser/Let.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Idris/Parser/Let.idr -------------------------------------------------------------------------------- /src/Idris/Pretty.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Idris/Pretty.idr -------------------------------------------------------------------------------- /src/Idris/ProcessIdr.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Idris/ProcessIdr.idr -------------------------------------------------------------------------------- /src/Idris/REPL.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Idris/REPL.idr -------------------------------------------------------------------------------- /src/Idris/REPL/Common.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Idris/REPL/Common.idr -------------------------------------------------------------------------------- /src/Idris/REPL/Opts.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Idris/REPL/Opts.idr -------------------------------------------------------------------------------- /src/Idris/Resugar.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Idris/Resugar.idr -------------------------------------------------------------------------------- /src/Idris/SetOptions.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Idris/SetOptions.idr -------------------------------------------------------------------------------- /src/Idris/Syntax.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Idris/Syntax.idr -------------------------------------------------------------------------------- /src/Idris/Syntax/TTC.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Idris/Syntax/TTC.idr -------------------------------------------------------------------------------- /src/Idris/Version.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Idris/Version.idr -------------------------------------------------------------------------------- /src/Parser/Package.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Parser/Package.idr -------------------------------------------------------------------------------- /src/Parser/Source.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Parser/Source.idr -------------------------------------------------------------------------------- /src/Parser/Support.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Parser/Support.idr -------------------------------------------------------------------------------- /src/Parser/Unlit.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Parser/Unlit.idr -------------------------------------------------------------------------------- /src/Protocol/Hex.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Protocol/Hex.idr -------------------------------------------------------------------------------- /src/Protocol/IDE.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Protocol/IDE.idr -------------------------------------------------------------------------------- /src/Protocol/SExp.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Protocol/SExp.idr -------------------------------------------------------------------------------- /src/TTImp/Elab.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/TTImp/Elab.idr -------------------------------------------------------------------------------- /src/TTImp/Elab/App.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/TTImp/Elab/App.idr -------------------------------------------------------------------------------- /src/TTImp/Elab/As.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/TTImp/Elab/As.idr -------------------------------------------------------------------------------- /src/TTImp/Elab/Case.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/TTImp/Elab/Case.idr -------------------------------------------------------------------------------- /src/TTImp/Elab/Check.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/TTImp/Elab/Check.idr -------------------------------------------------------------------------------- /src/TTImp/Elab/Dot.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/TTImp/Elab/Dot.idr -------------------------------------------------------------------------------- /src/TTImp/Elab/Hole.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/TTImp/Elab/Hole.idr -------------------------------------------------------------------------------- /src/TTImp/Elab/Lazy.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/TTImp/Elab/Lazy.idr -------------------------------------------------------------------------------- /src/TTImp/Elab/Local.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/TTImp/Elab/Local.idr -------------------------------------------------------------------------------- /src/TTImp/Elab/Prim.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/TTImp/Elab/Prim.idr -------------------------------------------------------------------------------- /src/TTImp/Elab/Quote.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/TTImp/Elab/Quote.idr -------------------------------------------------------------------------------- /src/TTImp/Elab/Record.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/TTImp/Elab/Record.idr -------------------------------------------------------------------------------- /src/TTImp/Elab/Term.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/TTImp/Elab/Term.idr -------------------------------------------------------------------------------- /src/TTImp/Elab/Utils.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/TTImp/Elab/Utils.idr -------------------------------------------------------------------------------- /src/TTImp/Impossible.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/TTImp/Impossible.idr -------------------------------------------------------------------------------- /src/TTImp/Parser.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/TTImp/Parser.idr -------------------------------------------------------------------------------- /src/TTImp/PartialEval.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/TTImp/PartialEval.idr -------------------------------------------------------------------------------- /src/TTImp/ProcessData.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/TTImp/ProcessData.idr -------------------------------------------------------------------------------- /src/TTImp/ProcessDef.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/TTImp/ProcessDef.idr -------------------------------------------------------------------------------- /src/TTImp/ProcessType.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/TTImp/ProcessType.idr -------------------------------------------------------------------------------- /src/TTImp/Reflect.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/TTImp/Reflect.idr -------------------------------------------------------------------------------- /src/TTImp/TTImp.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/TTImp/TTImp.idr -------------------------------------------------------------------------------- /src/TTImp/TTImp/TTC.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/TTImp/TTImp/TTC.idr -------------------------------------------------------------------------------- /src/TTImp/Unelab.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/TTImp/Unelab.idr -------------------------------------------------------------------------------- /src/TTImp/Utils.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/TTImp/Utils.idr -------------------------------------------------------------------------------- /src/TTImp/WithClause.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/TTImp/WithClause.idr -------------------------------------------------------------------------------- /src/Yaffle/Main.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Yaffle/Main.idr -------------------------------------------------------------------------------- /src/Yaffle/REPL.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/src/Yaffle/REPL.idr -------------------------------------------------------------------------------- /support/Makefile: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/support/Makefile -------------------------------------------------------------------------------- /support/c/.gitignore: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/support/c/.gitignore -------------------------------------------------------------------------------- /support/c/Makefile: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/support/c/Makefile -------------------------------------------------------------------------------- /support/c/getline.c: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/support/c/getline.c -------------------------------------------------------------------------------- /support/c/getline.h: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/support/c/getline.h -------------------------------------------------------------------------------- /support/c/idris_file.c: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/support/c/idris_file.c -------------------------------------------------------------------------------- /support/c/idris_file.h: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/support/c/idris_file.h -------------------------------------------------------------------------------- /support/c/idris_memory.c: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/support/c/idris_memory.c -------------------------------------------------------------------------------- /support/c/idris_memory.h: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/support/c/idris_memory.h -------------------------------------------------------------------------------- /support/c/idris_net.c: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/support/c/idris_net.c -------------------------------------------------------------------------------- /support/c/idris_net.h: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/support/c/idris_net.h -------------------------------------------------------------------------------- /support/c/idris_signal.c: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/support/c/idris_signal.c -------------------------------------------------------------------------------- /support/c/idris_signal.h: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/support/c/idris_signal.h -------------------------------------------------------------------------------- /support/c/idris_support.c: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/support/c/idris_support.c -------------------------------------------------------------------------------- /support/c/idris_support.h: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/support/c/idris_support.h -------------------------------------------------------------------------------- /support/c/idris_system.c: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/support/c/idris_system.c -------------------------------------------------------------------------------- /support/c/idris_system.h: -------------------------------------------------------------------------------- 1 | #pragma once 2 | 3 | int idris2_system(const char *command); 4 | -------------------------------------------------------------------------------- /support/c/idris_term.c: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/support/c/idris_term.c -------------------------------------------------------------------------------- /support/c/idris_term.h: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/support/c/idris_term.h -------------------------------------------------------------------------------- /support/c/idris_util.c: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/support/c/idris_util.c -------------------------------------------------------------------------------- /support/c/idris_util.h: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/support/c/idris_util.h -------------------------------------------------------------------------------- /support/c/windows/win_hack.c: -------------------------------------------------------------------------------- 1 | int chmod(char **str, int perm) { return 0; } 2 | -------------------------------------------------------------------------------- /support/chez/.gitignore: -------------------------------------------------------------------------------- 1 | support-sep.ss 2 | -------------------------------------------------------------------------------- /support/chez/Makefile: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/support/chez/Makefile -------------------------------------------------------------------------------- /support/chez/support.ss: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/support/chez/support.ss -------------------------------------------------------------------------------- /support/docs/default.css: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/support/docs/default.css -------------------------------------------------------------------------------- /support/docs/index.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/support/docs/index.html -------------------------------------------------------------------------------- /support/js/support.js: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/support/js/support.js -------------------------------------------------------------------------------- /support/refc/Makefile: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/support/refc/Makefile -------------------------------------------------------------------------------- /support/refc/_datatypes.h: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/support/refc/_datatypes.h -------------------------------------------------------------------------------- /support/refc/buffer.c: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/support/refc/buffer.c -------------------------------------------------------------------------------- /support/refc/buffer.h: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/support/refc/buffer.h -------------------------------------------------------------------------------- /support/refc/cBackend.h: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/support/refc/cBackend.h -------------------------------------------------------------------------------- /support/refc/casts.c: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/support/refc/casts.c -------------------------------------------------------------------------------- /support/refc/casts.h: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/support/refc/casts.h -------------------------------------------------------------------------------- /support/refc/clock.c: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/support/refc/clock.c -------------------------------------------------------------------------------- /support/refc/clock.h: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/support/refc/clock.h -------------------------------------------------------------------------------- /support/refc/prim.c: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/support/refc/prim.c -------------------------------------------------------------------------------- /support/refc/prim.h: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/support/refc/prim.h -------------------------------------------------------------------------------- /support/refc/refc_util.c: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/support/refc/refc_util.c -------------------------------------------------------------------------------- /support/refc/refc_util.h: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/support/refc/refc_util.h -------------------------------------------------------------------------------- /support/refc/runtime.c: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/support/refc/runtime.c -------------------------------------------------------------------------------- /support/refc/runtime.h: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/support/refc/runtime.h -------------------------------------------------------------------------------- /support/refc/stringOps.c: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/support/refc/stringOps.c -------------------------------------------------------------------------------- /support/refc/stringOps.h: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/support/refc/stringOps.h -------------------------------------------------------------------------------- /support/refc/threads.c: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/support/refc/threads.c -------------------------------------------------------------------------------- /support/refc/threads.h: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/support/refc/threads.h -------------------------------------------------------------------------------- /tests/Main.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/Main.idr -------------------------------------------------------------------------------- /tests/Makefile: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/Makefile -------------------------------------------------------------------------------- /tests/README.md: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/README.md -------------------------------------------------------------------------------- /tests/allbackends/basic048/input: -------------------------------------------------------------------------------- 1 | function' 1 2 | :q 3 | -------------------------------------------------------------------------------- /tests/allbackends/basic048/input-ed: -------------------------------------------------------------------------------- 1 | :e 2 | -------------------------------------------------------------------------------- /tests/allbackends/evaluator005/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run Issue1200.idr 4 | -------------------------------------------------------------------------------- /tests/allbackends/issue2362/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run Issue2362.idr 4 | -------------------------------------------------------------------------------- /tests/allbackends/perf006/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run Issue775.idr 4 | -------------------------------------------------------------------------------- /tests/allschemes/channels001/expected: -------------------------------------------------------------------------------- 1 | Hello 2 | Goodbye 3 | -------------------------------------------------------------------------------- /tests/allschemes/channels001/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run Main.idr 4 | -------------------------------------------------------------------------------- /tests/allschemes/channels002/expected: -------------------------------------------------------------------------------- 1 | Success! 2 | -------------------------------------------------------------------------------- /tests/allschemes/channels002/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run Main.idr 4 | -------------------------------------------------------------------------------- /tests/allschemes/channels003/expected: -------------------------------------------------------------------------------- 1 | Success! 2 | -------------------------------------------------------------------------------- /tests/allschemes/channels003/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run Main.idr 4 | -------------------------------------------------------------------------------- /tests/allschemes/channels004/expected: -------------------------------------------------------------------------------- 1 | Success! 2 | -------------------------------------------------------------------------------- /tests/allschemes/channels004/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run Main.idr 4 | -------------------------------------------------------------------------------- /tests/allschemes/channels005/expected: -------------------------------------------------------------------------------- 1 | SUCCESS!!! 2 | -------------------------------------------------------------------------------- /tests/allschemes/channels005/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run Main.idr 4 | -------------------------------------------------------------------------------- /tests/allschemes/channels006/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run Main.idr 4 | -------------------------------------------------------------------------------- /tests/allschemes/ffi001/expected: -------------------------------------------------------------------------------- 1 | -------------------------------------------------------------------------------- /tests/allschemes/memo001/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run Memo.idr 4 | -------------------------------------------------------------------------------- /tests/allschemes/memo002/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run Memo.idr 4 | -------------------------------------------------------------------------------- /tests/allschemes/memo003/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run Memo.idr 4 | -------------------------------------------------------------------------------- /tests/allschemes/memo004/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run --find-ipkg Memo.idr 4 | -------------------------------------------------------------------------------- /tests/allschemes/memo004/test.ipkg: -------------------------------------------------------------------------------- 1 | package test 2 | 3 | main = Memo 4 | 5 | depends = contrib 6 | -------------------------------------------------------------------------------- /tests/allschemes/memo005/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run --find-ipkg Memo.idr 4 | -------------------------------------------------------------------------------- /tests/allschemes/memo005/test.ipkg: -------------------------------------------------------------------------------- 1 | package test 2 | 3 | main = Memo 4 | 5 | depends = contrib 6 | -------------------------------------------------------------------------------- /tests/allschemes/scheme001/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run CastStringDouble.idr 4 | -------------------------------------------------------------------------------- /tests/base/data_bits001/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run BitOps.idr 4 | -------------------------------------------------------------------------------- /tests/base/data_bits002/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run BitRotate.idr 4 | -------------------------------------------------------------------------------- /tests/base/data_fin/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/base/data_fin/run -------------------------------------------------------------------------------- /tests/base/data_integral/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run Integral.idr 4 | -------------------------------------------------------------------------------- /tests/base/data_list001/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run List.idr 4 | -------------------------------------------------------------------------------- /tests/base/data_list002/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run Prefix.idr 4 | -------------------------------------------------------------------------------- /tests/base/data_list003/expected: -------------------------------------------------------------------------------- 1 | "OK" 2 | -------------------------------------------------------------------------------- /tests/base/data_list003/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run Elem.idr 4 | -------------------------------------------------------------------------------- /tests/base/data_listone001/expected: -------------------------------------------------------------------------------- 1 | "OK" 2 | -------------------------------------------------------------------------------- /tests/base/data_listone001/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run Elem.idr 4 | -------------------------------------------------------------------------------- /tests/base/data_nat/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | check Properties.idr 4 | -------------------------------------------------------------------------------- /tests/base/data_ref_monadstate/a-test.ipkg: -------------------------------------------------------------------------------- 1 | package a-test 2 | -------------------------------------------------------------------------------- /tests/base/data_ref_monadstate/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run RefMonadState.idr 4 | -------------------------------------------------------------------------------- /tests/base/data_singleton/expected: -------------------------------------------------------------------------------- 1 | 1/1: Building RLE (RLE.idr) 2 | -------------------------------------------------------------------------------- /tests/base/data_singleton/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | check RLE.idr 4 | -------------------------------------------------------------------------------- /tests/base/data_snoclist001/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run SL.idr 4 | -------------------------------------------------------------------------------- /tests/base/data_snoclist002/expected: -------------------------------------------------------------------------------- 1 | "OK" 2 | -------------------------------------------------------------------------------- /tests/base/data_snoclist002/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run Elem.idr 4 | -------------------------------------------------------------------------------- /tests/base/data_string/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | check StringReduce.idr 4 | -------------------------------------------------------------------------------- /tests/base/data_string_lines001/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run Lines.idr 4 | -------------------------------------------------------------------------------- /tests/base/data_string_parse_proof/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | check StringParse.idr 4 | -------------------------------------------------------------------------------- /tests/base/data_string_unlines001/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run Unlines.idr 4 | -------------------------------------------------------------------------------- /tests/base/data_vect001/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run Vect.idr 4 | -------------------------------------------------------------------------------- /tests/base/data_vect002/expected: -------------------------------------------------------------------------------- 1 | "OK" 2 | -------------------------------------------------------------------------------- /tests/base/data_vect002/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run Elem.idr 4 | -------------------------------------------------------------------------------- /tests/base/deriving_foldable/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | check DeriveFoldable.idr 4 | -------------------------------------------------------------------------------- /tests/base/deriving_traversable/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | check DeriveTraversable.idr 4 | -------------------------------------------------------------------------------- /tests/base/system_directory/dir/a: -------------------------------------------------------------------------------- 1 | -------------------------------------------------------------------------------- /tests/base/system_directory/expected: -------------------------------------------------------------------------------- 1 | -------------------------------------------------------------------------------- /tests/base/system_env/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/base/system_env/run -------------------------------------------------------------------------------- /tests/base/system_errno/expected: -------------------------------------------------------------------------------- 1 | -------------------------------------------------------------------------------- /tests/base/system_fileError/read_only.txt: -------------------------------------------------------------------------------- 1 | This file should be read only. 2 | -------------------------------------------------------------------------------- /tests/base/system_file_copyFile/expected: -------------------------------------------------------------------------------- 1 | AQIDBA== 2 | -------------------------------------------------------------------------------- /tests/base/system_file_copyFile/source.bin: -------------------------------------------------------------------------------- 1 |  -------------------------------------------------------------------------------- /tests/base/system_file_fGetChars/empty.txt: -------------------------------------------------------------------------------- 1 | -------------------------------------------------------------------------------- /tests/base/system_file_fGetChars/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run ReadFile.idr 4 | -------------------------------------------------------------------------------- /tests/base/system_file_fGetChars/small.txt: -------------------------------------------------------------------------------- 1 | 12345 2 | -------------------------------------------------------------------------------- /tests/base/system_file_fRead/expected: -------------------------------------------------------------------------------- 1 | "Hello, world\nLorem ipsum\n" 2 | -------------------------------------------------------------------------------- /tests/base/system_file_fRead/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run ReadFile.idr 4 | -------------------------------------------------------------------------------- /tests/base/system_file_fRead/sampleFile.txt: -------------------------------------------------------------------------------- 1 | Hello, world 2 | Lorem ipsum 3 | -------------------------------------------------------------------------------- /tests/base/system_file_popen/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run Popen.idr 4 | -------------------------------------------------------------------------------- /tests/base/system_get_environment/expected: -------------------------------------------------------------------------------- 1 | False 2 | -------------------------------------------------------------------------------- /tests/base/system_info001/.gitignore: -------------------------------------------------------------------------------- 1 | /expected 2 | 3 | -------------------------------------------------------------------------------- /tests/base/system_info_os001/expected: -------------------------------------------------------------------------------- 1 | correct 2 | -------------------------------------------------------------------------------- /tests/base/system_run/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run Run.idr 4 | -------------------------------------------------------------------------------- /tests/base/system_signal001/expected: -------------------------------------------------------------------------------- 1 | before 2 | after 3 | done. 4 | -------------------------------------------------------------------------------- /tests/base/system_signal001/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run IgnoreSignal.idr 4 | -------------------------------------------------------------------------------- /tests/base/system_signal002/expected: -------------------------------------------------------------------------------- 1 | before 2 | after 3 | done. 4 | -------------------------------------------------------------------------------- /tests/base/system_signal002/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run HandleSignal.idr 4 | -------------------------------------------------------------------------------- /tests/base/system_signal003/expected: -------------------------------------------------------------------------------- 1 | -------------------------------------------------------------------------------- /tests/base/system_signal003/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run DefaultSignal.idr 2> /dev/null 4 | -------------------------------------------------------------------------------- /tests/base/system_signal004/expected: -------------------------------------------------------------------------------- 1 | before 2 | after 3 | done. 4 | -------------------------------------------------------------------------------- /tests/base/system_system/seventeen.sh: -------------------------------------------------------------------------------- 1 | #!/bin/sh -e 2 | 3 | echo "SEVENTEEN" 4 | exit 17 5 | -------------------------------------------------------------------------------- /tests/base/system_system/zero.sh: -------------------------------------------------------------------------------- 1 | #!/bin/sh -e 2 | 3 | echo "ZERO" 4 | exit 0 5 | -------------------------------------------------------------------------------- /tests/base/ttimp_show001/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | idris2 < input 4 | -------------------------------------------------------------------------------- /tests/base/void_error/expected: -------------------------------------------------------------------------------- 1 | No clauses in Prelude.Uninhabited.void 2 | -------------------------------------------------------------------------------- /tests/base/void_error/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run Main.idr 4 | -------------------------------------------------------------------------------- /tests/chez/barrier001/input: -------------------------------------------------------------------------------- 1 | -------------------------------------------------------------------------------- /tests/chez/barrier001/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run --cg chez Main.idr 4 | -------------------------------------------------------------------------------- /tests/chez/bitops/expected: -------------------------------------------------------------------------------- 1 | -------------------------------------------------------------------------------- /tests/chez/bitops/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run BitOps.idr 4 | -------------------------------------------------------------------------------- /tests/chez/buffer001/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run Main.idr 4 | rm tmp.bin 5 | -------------------------------------------------------------------------------- /tests/chez/casts/expected: -------------------------------------------------------------------------------- 1 | -------------------------------------------------------------------------------- /tests/chez/casts/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run Casts.idr 4 | -------------------------------------------------------------------------------- /tests/chez/channels007/expected: -------------------------------------------------------------------------------- 1 | Hello 2 | Goodbye 3 | Nothing 4 | -------------------------------------------------------------------------------- /tests/chez/channels007/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run Main.idr 4 | -------------------------------------------------------------------------------- /tests/chez/channels008/expected: -------------------------------------------------------------------------------- 1 | 55 2 | -------------------------------------------------------------------------------- /tests/chez/channels008/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run Main.idr 4 | -------------------------------------------------------------------------------- /tests/chez/channels009/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run Main.idr 4 | -------------------------------------------------------------------------------- /tests/chez/chez001/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run Total.idr 4 | -------------------------------------------------------------------------------- /tests/chez/chez002/input: -------------------------------------------------------------------------------- 1 | :exec printLn (pythag 200) 2 | :q 3 | -------------------------------------------------------------------------------- /tests/chez/chez002/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/chez/chez002/run -------------------------------------------------------------------------------- /tests/chez/chez003/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run IORef.idr 4 | -------------------------------------------------------------------------------- /tests/chez/chez004/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/chez/chez004/run -------------------------------------------------------------------------------- /tests/chez/chez005/input: -------------------------------------------------------------------------------- 1 | :exec printLn (Main.filter even [S Z,2,3,4,5,6]) 2 | :q 3 | -------------------------------------------------------------------------------- /tests/chez/chez005/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/chez/chez005/run -------------------------------------------------------------------------------- /tests/chez/chez006/input: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/chez/chez006/input -------------------------------------------------------------------------------- /tests/chez/chez006/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/chez/chez006/run -------------------------------------------------------------------------------- /tests/chez/chez007/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run TypeCase.idr 4 | -------------------------------------------------------------------------------- /tests/chez/chez008/expected: -------------------------------------------------------------------------------- 1 | 1 2 | 1 3 | 1 4 | -------------------------------------------------------------------------------- /tests/chez/chez008/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run Nat.idr 4 | -------------------------------------------------------------------------------- /tests/chez/chez009/expected: -------------------------------------------------------------------------------- 1 | 42 2 | ällo 3 | -------------------------------------------------------------------------------- /tests/chez/chez009/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run uni.idr 4 | -------------------------------------------------------------------------------- /tests/chez/chez010/CB.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/chez/chez010/CB.idr -------------------------------------------------------------------------------- /tests/chez/chez010/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/chez/chez010/run -------------------------------------------------------------------------------- /tests/chez/chez011/input: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/chez/chez011/input -------------------------------------------------------------------------------- /tests/chez/chez011/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/chez/chez011/run -------------------------------------------------------------------------------- /tests/chez/chez012/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run array.idr 4 | -------------------------------------------------------------------------------- /tests/chez/chez013/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/chez/chez013/run -------------------------------------------------------------------------------- /tests/chez/chez014/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run -p network Echo.idr 4 | -------------------------------------------------------------------------------- /tests/chez/chez015/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run Numbers.idr 4 | -------------------------------------------------------------------------------- /tests/chez/chez016/expected: -------------------------------------------------------------------------------- 1 | Running Chez program located in folder with spaces 2 | -------------------------------------------------------------------------------- /tests/chez/chez016/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/chez/chez016/run -------------------------------------------------------------------------------- /tests/chez/chez017/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/chez/chez017/run -------------------------------------------------------------------------------- /tests/chez/chez018/expected: -------------------------------------------------------------------------------- 1 | test test 2 | unfinished lineabc 3 | def 4 | File Not Found 5 | -------------------------------------------------------------------------------- /tests/chez/chez018/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/chez/chez018/run -------------------------------------------------------------------------------- /tests/chez/chez018/test.txt: -------------------------------------------------------------------------------- 1 | test test 2 | unfinished line -------------------------------------------------------------------------------- /tests/chez/chez019/input: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/chez/chez019/input -------------------------------------------------------------------------------- /tests/chez/chez019/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/chez/chez019/run -------------------------------------------------------------------------------- /tests/chez/chez020/expected: -------------------------------------------------------------------------------- 1 | opened 2 | closed 3 | Idris 2 4 | -------------------------------------------------------------------------------- /tests/chez/chez020/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/chez/chez020/run -------------------------------------------------------------------------------- /tests/chez/chez021/input: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/chez/chez021/input -------------------------------------------------------------------------------- /tests/chez/chez021/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/chez/chez021/run -------------------------------------------------------------------------------- /tests/chez/chez022/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/chez/chez022/run -------------------------------------------------------------------------------- /tests/chez/chez023/expected: -------------------------------------------------------------------------------- 1 | Hello 2 | 'I' 3 | dris! 4 | 5 | No exceptions occurred 6 | -------------------------------------------------------------------------------- /tests/chez/chez023/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/chez/chez023/run -------------------------------------------------------------------------------- /tests/chez/chez024/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run Envy.idr 4 | -------------------------------------------------------------------------------- /tests/chez/chez025/input: -------------------------------------------------------------------------------- 1 | :exec printLn (stsum [1..1000]) 2 | :q 3 | -------------------------------------------------------------------------------- /tests/chez/chez025/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/chez/chez025/run -------------------------------------------------------------------------------- /tests/chez/chez026/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/chez/chez026/run -------------------------------------------------------------------------------- /tests/chez/chez027/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/chez/chez027/run -------------------------------------------------------------------------------- /tests/chez/chez028/expected: -------------------------------------------------------------------------------- 1 | 5678 2 | -3 3 | 262145 4 | 10 5 | 7 6 | -------------------------------------------------------------------------------- /tests/chez/chez028/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run -p contrib ExpressionParser.idr 4 | -------------------------------------------------------------------------------- /tests/chez/chez029/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run BitCasts.idr 4 | -------------------------------------------------------------------------------- /tests/chez/chez030/expected: -------------------------------------------------------------------------------- 1 | 6 * 7 = 42 2 | -------------------------------------------------------------------------------- /tests/chez/chez030/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/chez/chez030/run -------------------------------------------------------------------------------- /tests/chez/chez031/input: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/chez/chez031/input -------------------------------------------------------------------------------- /tests/chez/chez031/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/chez/chez031/run -------------------------------------------------------------------------------- /tests/chez/chez032/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run BitOps.idr 4 | -------------------------------------------------------------------------------- /tests/chez/chez033/expected: -------------------------------------------------------------------------------- 1 | 10001 2 | -------------------------------------------------------------------------------- /tests/chez/chez033/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run Main.idr --inc chez 4 | -------------------------------------------------------------------------------- /tests/chez/chez034/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run ThreadData.idr 4 | -------------------------------------------------------------------------------- /tests/chez/chez035/input: -------------------------------------------------------------------------------- 1 | :q 2 | -------------------------------------------------------------------------------- /tests/chez/chez035/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/chez/chez035/run -------------------------------------------------------------------------------- /tests/chez/chez036/expected: -------------------------------------------------------------------------------- 1 | Ok 2 | Ok 3 | -------------------------------------------------------------------------------- /tests/chez/chez036/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/chez/chez036/run -------------------------------------------------------------------------------- /tests/chez/chez037/expected: -------------------------------------------------------------------------------- 1 | Error: INTERNAL ERROR: Chez exited with return code 1 2 | -------------------------------------------------------------------------------- /tests/chez/chez037/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/chez/chez037/run -------------------------------------------------------------------------------- /tests/chez/chez038/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run ThreadId.idr 4 | -------------------------------------------------------------------------------- /tests/chez/constfold/expected: -------------------------------------------------------------------------------- 1 | Constant expression correctly folded 2 | -------------------------------------------------------------------------------- /tests/chez/constfold/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/chez/constfold/run -------------------------------------------------------------------------------- /tests/chez/constfold2/expected: -------------------------------------------------------------------------------- 1 | Constant expression correctly folded 2 | -------------------------------------------------------------------------------- /tests/chez/constfold2/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/chez/constfold2/run -------------------------------------------------------------------------------- /tests/chez/constfold3/expected: -------------------------------------------------------------------------------- 1 | Constant expression correctly folded 2 | -------------------------------------------------------------------------------- /tests/chez/constfold3/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/chez/constfold3/run -------------------------------------------------------------------------------- /tests/chez/forkjoin001/expected: -------------------------------------------------------------------------------- 1 | Hello 2 | Goodbye 3 | -------------------------------------------------------------------------------- /tests/chez/forkjoin001/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run --cg chez Main.idr 4 | -------------------------------------------------------------------------------- /tests/chez/futures001/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/chez/futures001/run -------------------------------------------------------------------------------- /tests/chez/futures002/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/chez/futures002/run -------------------------------------------------------------------------------- /tests/chez/inlineiobind/expected: -------------------------------------------------------------------------------- 1 | io_bind correctly inlined 2 | -------------------------------------------------------------------------------- /tests/chez/integers/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/chez/integers/run -------------------------------------------------------------------------------- /tests/chez/nat2fin/expected: -------------------------------------------------------------------------------- 1 | natToFinLt optimized away 2 | -------------------------------------------------------------------------------- /tests/chez/nat2fin/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/chez/nat2fin/run -------------------------------------------------------------------------------- /tests/chez/newints/expected: -------------------------------------------------------------------------------- 1 | -------------------------------------------------------------------------------- /tests/chez/newints/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run IntOps.idr 4 | -------------------------------------------------------------------------------- /tests/chez/perf001/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/chez/perf001/run -------------------------------------------------------------------------------- /tests/chez/reg001/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run numbers.idr 4 | -------------------------------------------------------------------------------- /tests/chez/reg002/expected: -------------------------------------------------------------------------------- 1 | -------------------------------------------------------------------------------- /tests/chez/reg002/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run Main.idr 4 | -------------------------------------------------------------------------------- /tests/chez/semaphores001/expected: -------------------------------------------------------------------------------- 1 | Hello 2 | Goodbye 3 | -------------------------------------------------------------------------------- /tests/chez/semaphores001/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run --cg chez Main.idr 4 | -------------------------------------------------------------------------------- /tests/chez/semaphores002/expected: -------------------------------------------------------------------------------- 1 | Hello 2 | Goodbye 3 | -------------------------------------------------------------------------------- /tests/chez/semaphores002/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run --cg chez Main.idr 4 | -------------------------------------------------------------------------------- /tests/cli/exec001/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/cli/exec001/run -------------------------------------------------------------------------------- /tests/cli/exec002/expected: -------------------------------------------------------------------------------- 1 | Hello! 2 | 1 + 2 = 3 3 | Bye! 4 | -------------------------------------------------------------------------------- /tests/cli/exec002/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/cli/exec002/run -------------------------------------------------------------------------------- /tests/cli/exec003/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/cli/exec003/run -------------------------------------------------------------------------------- /tests/cli/exec004/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/cli/exec004/run -------------------------------------------------------------------------------- /tests/cli/optional001/expected: -------------------------------------------------------------------------------- 1 | -------------------------------------------------------------------------------- /tests/cli/optional001/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/cli/optional001/run -------------------------------------------------------------------------------- /tests/cli/optional001/test.ipkg: -------------------------------------------------------------------------------- 1 | package test 2 | -------------------------------------------------------------------------------- /tests/codegen/.gitignore: -------------------------------------------------------------------------------- 1 | *.cases 2 | -------------------------------------------------------------------------------- /tests/codegen/con001/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/codegen/con001/run -------------------------------------------------------------------------------- /tests/codegen/enum/expected: -------------------------------------------------------------------------------- 1 | Enum conversion optimized away 2 | -------------------------------------------------------------------------------- /tests/codegen/enum/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/codegen/enum/run -------------------------------------------------------------------------------- /tests/codegen/fix3375/expected: -------------------------------------------------------------------------------- 1 | -------------------------------------------------------------------------------- /tests/codegen/fix3375/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/codegen/fix3375/run -------------------------------------------------------------------------------- /tests/codegen/fix3515/expected: -------------------------------------------------------------------------------- 1 | 1 2 | 0 3 | -------------------------------------------------------------------------------- /tests/codegen/fix3515/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/codegen/fix3515/run -------------------------------------------------------------------------------- /tests/contrib/json_001/expected: -------------------------------------------------------------------------------- 1 | [] 2 | -------------------------------------------------------------------------------- /tests/contrib/json_001/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run -p contrib CharEncoding.idr 4 | -------------------------------------------------------------------------------- /tests/contrib/json_002/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run -p contrib ShowJSON.idr 4 | -------------------------------------------------------------------------------- /tests/contrib/json_003/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run -p contrib CastJSON.idr 4 | -------------------------------------------------------------------------------- /tests/contrib/json_004/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run -p contrib JSON.idr 4 | -------------------------------------------------------------------------------- /tests/contrib/lexer/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/contrib/lexer/run -------------------------------------------------------------------------------- /tests/contrib/list_alternating/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run -p contrib AlternatingList.idr 4 | -------------------------------------------------------------------------------- /tests/contrib/perf001/expected: -------------------------------------------------------------------------------- 1 | 4 2 | -------------------------------------------------------------------------------- /tests/contrib/perf001/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run -p contrib GCDPerf.idr 4 | -------------------------------------------------------------------------------- /tests/contrib/system_directory_tree_copyDir/templateDir/nestedDir/anotherFile.txt: -------------------------------------------------------------------------------- 1 | Hello, world 2 | -------------------------------------------------------------------------------- /tests/contrib/system_directory_tree_copyDir/templateDir/source.bin: -------------------------------------------------------------------------------- 1 |  -------------------------------------------------------------------------------- /tests/ideMode/ideMode001/dummy.ipkg: -------------------------------------------------------------------------------- 1 | package idemode001 2 | -------------------------------------------------------------------------------- /tests/ideMode/ideMode001/input2: -------------------------------------------------------------------------------- 1 | 00001b((:enable-syntax :False) 2) 2 | -------------------------------------------------------------------------------- /tests/ideMode/ideMode001/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | idris2 --ide-mode < input 4 | -------------------------------------------------------------------------------- /tests/ideMode/ideMode002/.gitignore: -------------------------------------------------------------------------------- 1 | /expected 2 | 3 | -------------------------------------------------------------------------------- /tests/ideMode/ideMode002/input: -------------------------------------------------------------------------------- 1 | 00000c(:version 1) 2 | -------------------------------------------------------------------------------- /tests/ideMode/ideMode003/dummy.ipkg: -------------------------------------------------------------------------------- 1 | package idemode003 2 | -------------------------------------------------------------------------------- /tests/ideMode/ideMode003/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | idris2 --ide-mode < input 4 | -------------------------------------------------------------------------------- /tests/ideMode/ideMode004/input: -------------------------------------------------------------------------------- 1 | 00001C((:interpret "\"Test\"") 32) 2 | -------------------------------------------------------------------------------- /tests/ideMode/ideMode004/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | idris2 --ide-mode < input 4 | -------------------------------------------------------------------------------- /tests/ideMode/ideMode006/dummy.ipkg: -------------------------------------------------------------------------------- 1 | package idemode005 2 | -------------------------------------------------------------------------------- /tests/ideMode/ideMode006/input: -------------------------------------------------------------------------------- 1 | 00001d((:load-file "Unsafe.idr") 1) -------------------------------------------------------------------------------- /tests/ideMode/ideMode006/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | idris2 --ide-mode < input 4 | -------------------------------------------------------------------------------- /tests/ideMode/ideMode007/dummy.ipkg: -------------------------------------------------------------------------------- 1 | package idemode005 2 | -------------------------------------------------------------------------------- /tests/ideMode/ideMode007/input: -------------------------------------------------------------------------------- 1 | 00001d((:load-file "Syntax.idr") 1) -------------------------------------------------------------------------------- /tests/ideMode/ideMode007/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | idris2 --ide-mode < input 4 | -------------------------------------------------------------------------------- /tests/ideMode/ideMode008/dummy.ipkg: -------------------------------------------------------------------------------- 1 | package idemode005 2 | -------------------------------------------------------------------------------- /tests/ideMode/ideMode008/input: -------------------------------------------------------------------------------- 1 | 000020((:load-file "Interface.idr") 1) -------------------------------------------------------------------------------- /tests/ideMode/ideMode008/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | idris2 --ide-mode < input 4 | -------------------------------------------------------------------------------- /tests/ideMode/ideMode009/expected: -------------------------------------------------------------------------------- 1 | 000018(:protocol-version 2 1) 2 | -------------------------------------------------------------------------------- /tests/ideMode/ideMode009/input: -------------------------------------------------------------------------------- 1 | 000021((:load-file "Ambiguity.idr") 1) -------------------------------------------------------------------------------- /tests/ideMode/ideMode009/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | idris2 --ide-mode < input 4 | -------------------------------------------------------------------------------- /tests/ideMode/ideMode010/dummy.ipkg: -------------------------------------------------------------------------------- 1 | package idemode005 2 | -------------------------------------------------------------------------------- /tests/ideMode/ideMode010/input: -------------------------------------------------------------------------------- 1 | 00001e((:load-file "Rainbow.idr") 1) -------------------------------------------------------------------------------- /tests/ideMode/ideMode010/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | idris2 --ide-mode < input 4 | -------------------------------------------------------------------------------- /tests/ideMode/ideMode011/dummy.ipkg: -------------------------------------------------------------------------------- 1 | package idemode005 2 | -------------------------------------------------------------------------------- /tests/ideMode/ideMode011/input: -------------------------------------------------------------------------------- 1 | 000025((:load-file "Implementation.idr") 1) -------------------------------------------------------------------------------- /tests/ideMode/ideMode011/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | idris2 --ide-mode < input 4 | -------------------------------------------------------------------------------- /tests/ideMode/ideMode012/dummy.ipkg: -------------------------------------------------------------------------------- 1 | package idemode005 2 | -------------------------------------------------------------------------------- /tests/ideMode/ideMode012/input: -------------------------------------------------------------------------------- 1 | 00001b((:load-file "Case.idr") 1) -------------------------------------------------------------------------------- /tests/ideMode/ideMode012/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | idris2 --ide-mode < input 4 | -------------------------------------------------------------------------------- /tests/ideMode/ideMode013/dummy.ipkg: -------------------------------------------------------------------------------- 1 | package idemode005 2 | -------------------------------------------------------------------------------- /tests/ideMode/ideMode013/input: -------------------------------------------------------------------------------- 1 | 000023((:load-file "RecordUpdate.idr") 1) -------------------------------------------------------------------------------- /tests/ideMode/ideMode013/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | idris2 --ide-mode < input 4 | -------------------------------------------------------------------------------- /tests/ideMode/ideMode014/dummy.ipkg: -------------------------------------------------------------------------------- 1 | package idemode005 2 | -------------------------------------------------------------------------------- /tests/ideMode/ideMode014/input: -------------------------------------------------------------------------------- 1 | 00001b((:load-file "With.idr") 1) -------------------------------------------------------------------------------- /tests/ideMode/ideMode014/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | idris2 --ide-mode < input 4 | -------------------------------------------------------------------------------- /tests/ideMode/ideMode015/dummy.ipkg: -------------------------------------------------------------------------------- 1 | package idemode005 2 | -------------------------------------------------------------------------------- /tests/ideMode/ideMode015/input: -------------------------------------------------------------------------------- 1 | 00001d((:load-file "Ranges.idr") 1) -------------------------------------------------------------------------------- /tests/ideMode/ideMode015/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | idris2 --ide-mode < input 4 | -------------------------------------------------------------------------------- /tests/ideMode/ideMode016/dummy.ipkg: -------------------------------------------------------------------------------- 1 | package idemode005 2 | -------------------------------------------------------------------------------- /tests/ideMode/ideMode016/input: -------------------------------------------------------------------------------- 1 | 000025((:load-file "StringLiterals.idr") 1) -------------------------------------------------------------------------------- /tests/ideMode/ideMode016/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | idris2 --ide-mode < input 4 | -------------------------------------------------------------------------------- /tests/ideMode/ideMode017/dummy.ipkg: -------------------------------------------------------------------------------- 1 | package idemode005 2 | -------------------------------------------------------------------------------- /tests/ideMode/ideMode017/input: -------------------------------------------------------------------------------- 1 | 00001e((:load-file "WithApp.idr") 1) -------------------------------------------------------------------------------- /tests/ideMode/ideMode017/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | idris2 --ide-mode < input 4 | -------------------------------------------------------------------------------- /tests/ideMode/ideMode018/dummy.ipkg: -------------------------------------------------------------------------------- 1 | package idemode005 2 | -------------------------------------------------------------------------------- /tests/ideMode/ideMode018/input: -------------------------------------------------------------------------------- 1 | 00001e((:load-file "Rewrite.idr") 1) -------------------------------------------------------------------------------- /tests/ideMode/ideMode018/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | idris2 --ide-mode < input 4 | -------------------------------------------------------------------------------- /tests/ideMode/ideMode019/dummy.ipkg: -------------------------------------------------------------------------------- 1 | package idemode005 2 | -------------------------------------------------------------------------------- /tests/ideMode/ideMode019/input: -------------------------------------------------------------------------------- 1 | 000028((:load-file "RecordProjections.idr") 1) -------------------------------------------------------------------------------- /tests/ideMode/ideMode019/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | idris2 --ide-mode < input 4 | -------------------------------------------------------------------------------- /tests/ideMode/ideMode020/dummy.ipkg: -------------------------------------------------------------------------------- 1 | package idemode005 2 | -------------------------------------------------------------------------------- /tests/ideMode/ideMode020/input: -------------------------------------------------------------------------------- 1 | 00001d((:load-file "Tuples.idr") 1) -------------------------------------------------------------------------------- /tests/ideMode/ideMode020/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | idris2 --ide-mode < input 4 | -------------------------------------------------------------------------------- /tests/ideMode/ideMode021/dummy.ipkg: -------------------------------------------------------------------------------- 1 | package idemode005 2 | -------------------------------------------------------------------------------- /tests/ideMode/ideMode021/input: -------------------------------------------------------------------------------- 1 | 000021((:load-file "LetBinders.idr") 1) -------------------------------------------------------------------------------- /tests/ideMode/ideMode021/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | idris2 --ide-mode < input 4 | -------------------------------------------------------------------------------- /tests/ideMode/ideMode022/dummy.ipkg: -------------------------------------------------------------------------------- 1 | package idemode005 2 | -------------------------------------------------------------------------------- /tests/ideMode/ideMode022/input: -------------------------------------------------------------------------------- 1 | 000022((:load-file "SnocRainbow.idr") 1) 2 | -------------------------------------------------------------------------------- /tests/ideMode/ideMode022/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | idris2 --ide-mode < input 4 | -------------------------------------------------------------------------------- /tests/ideMode/ideMode023/dummy.ipkg: -------------------------------------------------------------------------------- 1 | package idemode005 2 | -------------------------------------------------------------------------------- /tests/ideMode/ideMode023/input: -------------------------------------------------------------------------------- 1 | 00001b((:load-file "Fail.idr") 1) 2 | -------------------------------------------------------------------------------- /tests/ideMode/ideMode023/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | idris2 --ide-mode < input 4 | -------------------------------------------------------------------------------- /tests/ideMode/ideMode024/dummy.ipkg: -------------------------------------------------------------------------------- 1 | package idemode005 2 | -------------------------------------------------------------------------------- /tests/ideMode/ideMode024/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | idris2 --ide-mode < input 4 | -------------------------------------------------------------------------------- /tests/idris2/api/README: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/idris2/api/README -------------------------------------------------------------------------------- /tests/idris2/api/api001/expected: -------------------------------------------------------------------------------- 1 | I'd rather not. 2 | -------------------------------------------------------------------------------- /tests/idris2/basic/basic005/NoInfer.idr: -------------------------------------------------------------------------------- 1 | foo : ? -> Int 2 | foo x = 42 3 | -------------------------------------------------------------------------------- /tests/idris2/basic/basic009/input: -------------------------------------------------------------------------------- 1 | :t foo 2 | :q 3 | -------------------------------------------------------------------------------- /tests/idris2/basic/basic021/input: -------------------------------------------------------------------------------- 1 | :printdef foo 2 | :q 3 | -------------------------------------------------------------------------------- /tests/idris2/basic/basic024/input: -------------------------------------------------------------------------------- 1 | addToNums nums 2 | lengths vects 3 | :q 4 | -------------------------------------------------------------------------------- /tests/idris2/basic/basic026/expected: -------------------------------------------------------------------------------- 1 | 1/1: Building Erl (Erl.idr) 2 | -------------------------------------------------------------------------------- /tests/idris2/basic/basic038/input: -------------------------------------------------------------------------------- 1 | niceList 2 | :q -------------------------------------------------------------------------------- /tests/idris2/basic/basic047/input: -------------------------------------------------------------------------------- 1 | test 2 | :q 3 | -------------------------------------------------------------------------------- /tests/idris2/basic/basic050/input: -------------------------------------------------------------------------------- 1 | il 2 | lc 3 | ilc 4 | -------------------------------------------------------------------------------- /tests/idris2/basic/basic052/input: -------------------------------------------------------------------------------- 1 | h 9 2 | -------------------------------------------------------------------------------- /tests/idris2/basic/basic056/expected: -------------------------------------------------------------------------------- 1 | MkInUnit 0.25 _ 2 | MkNewtype 123.456 3 | -------------------------------------------------------------------------------- /tests/idris2/basic/basic064/input: -------------------------------------------------------------------------------- 1 | :m 2 | -------------------------------------------------------------------------------- /tests/idris2/basic/basic068/expected: -------------------------------------------------------------------------------- 1 | [B [A 5]] 2 | {B {A 6}} 3 | -------------------------------------------------------------------------------- /tests/idris2/basic/basic071/B.idr: -------------------------------------------------------------------------------- 1 | module B 2 | 3 | import A 4 | 5 | y : Nat 6 | y = x 7 | -------------------------------------------------------------------------------- /tests/idris2/basic/basic075/expected: -------------------------------------------------------------------------------- 1 | 2 2 | -------------------------------------------------------------------------------- /tests/idris2/basic/literals001/Test.idr: -------------------------------------------------------------------------------- 1 | {- 2 | c : Char 3 | c = '"' 4 | -} 5 | -------------------------------------------------------------------------------- /tests/idris2/builtin/builtin001/input: -------------------------------------------------------------------------------- 1 | :q 2 | -------------------------------------------------------------------------------- /tests/idris2/builtin/builtin002/input: -------------------------------------------------------------------------------- 1 | :q 2 | -------------------------------------------------------------------------------- /tests/idris2/builtin/builtin003/input: -------------------------------------------------------------------------------- 1 | :q 2 | -------------------------------------------------------------------------------- /tests/idris2/builtin/builtin004/input: -------------------------------------------------------------------------------- 1 | :q 2 | -------------------------------------------------------------------------------- /tests/idris2/builtin/builtin005/input: -------------------------------------------------------------------------------- 1 | :q 2 | -------------------------------------------------------------------------------- /tests/idris2/builtin/builtin006/input: -------------------------------------------------------------------------------- 1 | :q 2 | -------------------------------------------------------------------------------- /tests/idris2/builtin/builtin007/input: -------------------------------------------------------------------------------- 1 | :q 2 | -------------------------------------------------------------------------------- /tests/idris2/builtin/builtin008/input: -------------------------------------------------------------------------------- 1 | :q 2 | -------------------------------------------------------------------------------- /tests/idris2/builtin/builtin009/expected: -------------------------------------------------------------------------------- 1 | 3141592 2 | 12345 3 | True 4 | False 5 | -------------------------------------------------------------------------------- /tests/idris2/builtin/builtin010/input: -------------------------------------------------------------------------------- 1 | :q 2 | -------------------------------------------------------------------------------- /tests/idris2/builtin/builtin011/expected: -------------------------------------------------------------------------------- 1 | 3141592 2 | 12345 3 | 1100 4 | 17120 5 | -------------------------------------------------------------------------------- /tests/idris2/builtin/builtin012/expected: -------------------------------------------------------------------------------- 1 | 1 2 | -------------------------------------------------------------------------------- /tests/idris2/casetree/casetree003/input: -------------------------------------------------------------------------------- 1 | :di idL 2 | -------------------------------------------------------------------------------- /tests/idris2/casetree/heuristics001/input: -------------------------------------------------------------------------------- 1 | :di mergeLim 2 | -------------------------------------------------------------------------------- /tests/idris2/coverage/coverage004/input: -------------------------------------------------------------------------------- 1 | :missing okay 2 | :q 3 | -------------------------------------------------------------------------------- /tests/idris2/coverage/coverage006/input: -------------------------------------------------------------------------------- 1 | :total foo 2 | :q 3 | -------------------------------------------------------------------------------- /tests/idris2/coverage/coverage018/input: -------------------------------------------------------------------------------- 1 | :di test2 2 | :q -------------------------------------------------------------------------------- /tests/idris2/coverage/coverage023/X.idr: -------------------------------------------------------------------------------- 1 | data X = MkX 2 | -------------------------------------------------------------------------------- /tests/idris2/coverage/coverage023/Y.idr: -------------------------------------------------------------------------------- 1 | data Y = MkY 2 | -------------------------------------------------------------------------------- /tests/idris2/data/data001/Test.idr: -------------------------------------------------------------------------------- 1 | module Test 2 | 3 | export 4 | data Main : Type 5 | -------------------------------------------------------------------------------- /tests/idris2/data/data004/EmptySearch.idr: -------------------------------------------------------------------------------- 1 | data X : Type where 2 | [search] 3 | -------------------------------------------------------------------------------- /tests/idris2/data/record005/input: -------------------------------------------------------------------------------- 1 | :set showimplicits 2 | Bar 3 | :q 4 | -------------------------------------------------------------------------------- /tests/idris2/data/record006/input: -------------------------------------------------------------------------------- 1 | :set showimplicits 2 | three 3 | :q 4 | -------------------------------------------------------------------------------- /tests/idris2/data/record007/input: -------------------------------------------------------------------------------- 1 | :q 2 | -------------------------------------------------------------------------------- /tests/idris2/data/record015/expected: -------------------------------------------------------------------------------- 1 | [5, 6, 7, 3] 2 | [6, 9, 10, 5] 3 | -------------------------------------------------------------------------------- /tests/idris2/data/record018/expected: -------------------------------------------------------------------------------- 1 | 1/1: Building mut (mut.idr) 2 | -------------------------------------------------------------------------------- /tests/idris2/data/record022/EmptySearch.idr: -------------------------------------------------------------------------------- 1 | record R where 2 | [search] 3 | -------------------------------------------------------------------------------- /tests/idris2/error/error008/input: -------------------------------------------------------------------------------- 1 | :q 2 | -------------------------------------------------------------------------------- /tests/idris2/error/error009/input: -------------------------------------------------------------------------------- 1 | :q 2 | -------------------------------------------------------------------------------- /tests/idris2/error/error012/expected: -------------------------------------------------------------------------------- 1 | 2 | Error loading file "nothere.idr": File Not Found 3 | 4 | -------------------------------------------------------------------------------- /tests/idris2/error/error016/input: -------------------------------------------------------------------------------- 1 | :t nap 2 | :t lentgh 3 | :q -------------------------------------------------------------------------------- /tests/idris2/error/error020/Error.idr: -------------------------------------------------------------------------------- 1 | (a, b) = (1, 2) 2 | -------------------------------------------------------------------------------- /tests/idris2/error/perror007/StrError1.idr: -------------------------------------------------------------------------------- 1 | foo : String 2 | foo = "empty interp: \{}" 3 | -------------------------------------------------------------------------------- /tests/idris2/error/perror007/StrError3.idr: -------------------------------------------------------------------------------- 1 | foo : String 2 | foo = "incomplete: \{ a <+> }" 3 | -------------------------------------------------------------------------------- /tests/idris2/error/perror008/Issue1224b.idr: -------------------------------------------------------------------------------- 1 | import ggg 2 | 3 | t : Int 4 | t = yyy 5 | -------------------------------------------------------------------------------- /tests/idris2/error/perror008/Issue710b.idr: -------------------------------------------------------------------------------- 1 | module Issue710b 2 | 3 | data r : Type where 4 | -------------------------------------------------------------------------------- /tests/idris2/error/perror008/Issue710d.idr: -------------------------------------------------------------------------------- 1 | record T where 2 | constructor mkT 3 | -------------------------------------------------------------------------------- /tests/idris2/error/perror008/Issue710e.idr: -------------------------------------------------------------------------------- 1 | %default total 2 | 3 | namespace a 4 | -------------------------------------------------------------------------------- /tests/idris2/error/perror010/input: -------------------------------------------------------------------------------- 1 | :m 2 | :q -------------------------------------------------------------------------------- /tests/idris2/error/perror011/Issue1496-2.idr: -------------------------------------------------------------------------------- 1 | module X 2 | [ 3 | -------------------------------------------------------------------------------- /tests/idris2/error/perror013/x.ipkg: -------------------------------------------------------------------------------- 1 | package test 2 | -------------------------------------------------------------------------------- /tests/idris2/error/perror022/Indent.idr: -------------------------------------------------------------------------------- 1 | record Rec (a : Type) 2 | b : Int 3 | -------------------------------------------------------------------------------- /tests/idris2/error/perror023/ParseError.idr: -------------------------------------------------------------------------------- 1 | module ParseError 2 | 3 | String : Type 4 | -------------------------------------------------------------------------------- /tests/idris2/error/perror032/LambdaImpossible.idr: -------------------------------------------------------------------------------- 1 | foo : 2 = 3 -> Void 2 | foo = (\Refl impossible) 3 | -------------------------------------------------------------------------------- /tests/idris2/evaluator/evaluator002/input: -------------------------------------------------------------------------------- 1 | test 2 | :q -------------------------------------------------------------------------------- /tests/idris2/evaluator/interpreter001/input: -------------------------------------------------------------------------------- 1 | 3.5 - 2.0 2 | :q 3 | -------------------------------------------------------------------------------- /tests/idris2/evaluator/interpreter005/input: -------------------------------------------------------------------------------- 1 | test 2 | :q 3 | -------------------------------------------------------------------------------- /tests/idris2/interactive/interactive003/input2: -------------------------------------------------------------------------------- 1 | :cs 11 18 zs 2 | :q 3 | -------------------------------------------------------------------------------- /tests/idris2/interactive/interactive006/input: -------------------------------------------------------------------------------- 1 | :ml 8 empties 2 | :ml 10 transposeHelper 3 | :q 4 | -------------------------------------------------------------------------------- /tests/idris2/interactive/interactive007/input: -------------------------------------------------------------------------------- 1 | :gd 7 transposeHelper 2 | :q 3 | -------------------------------------------------------------------------------- /tests/idris2/interactive/interactive008/input: -------------------------------------------------------------------------------- 1 | :ps 8 baz 2 | :ps 15 foo 3 | :typeat 12 33 f 4 | :q 5 | -------------------------------------------------------------------------------- /tests/idris2/interactive/interactive010/input: -------------------------------------------------------------------------------- 1 | :gd 10 zipHere 2 | :q 3 | -------------------------------------------------------------------------------- /tests/idris2/interactive/interactive017/input: -------------------------------------------------------------------------------- 1 | :gd 15 uncompress 2 | :q 3 | -------------------------------------------------------------------------------- /tests/idris2/interactive/interactive033/input: -------------------------------------------------------------------------------- 1 | :cs 8 26 c 2 | :q 3 | -------------------------------------------------------------------------------- /tests/idris2/interactive/interactive034/input: -------------------------------------------------------------------------------- 1 | :gd 54 tailIsNotSound 2 | :q 3 | -------------------------------------------------------------------------------- /tests/idris2/interactive/interactive035/input: -------------------------------------------------------------------------------- 1 | :ps 7 vlength 2 | :q 3 | -------------------------------------------------------------------------------- /tests/idris2/interactive/interactive036/input: -------------------------------------------------------------------------------- 1 | :cs 3 3 bar 2 | :q 3 | -------------------------------------------------------------------------------- /tests/idris2/interactive/interactive037/input: -------------------------------------------------------------------------------- 1 | :m 2 | :q 3 | -------------------------------------------------------------------------------- /tests/idris2/interactive/interactive041/input: -------------------------------------------------------------------------------- 1 | :cs 4 10 i 2 | :q -------------------------------------------------------------------------------- /tests/idris2/interactive/interactive044/input: -------------------------------------------------------------------------------- 1 | :cs 5 7 c 2 | :r 3 | :q 4 | -------------------------------------------------------------------------------- /tests/idris2/interactive/interactive045/input: -------------------------------------------------------------------------------- 1 | :cs 5 4 x 2 | :r 3 | :q 4 | -------------------------------------------------------------------------------- /tests/idris2/interface/interface001/input1: -------------------------------------------------------------------------------- 1 | :t foo 2 | :q 3 | -------------------------------------------------------------------------------- /tests/idris2/interface/interface002/input: -------------------------------------------------------------------------------- 1 | :t foo 2 | :t bar 3 | :q 4 | -------------------------------------------------------------------------------- /tests/idris2/interface/interface003/input: -------------------------------------------------------------------------------- 1 | :t foo 2 | :q 3 | -------------------------------------------------------------------------------- /tests/idris2/interface/interface007/expected: -------------------------------------------------------------------------------- 1 | 1/1: Building A (A.idr) 2 | -------------------------------------------------------------------------------- /tests/idris2/interface/interface009/input: -------------------------------------------------------------------------------- 1 | :t bang 2 | :q 3 | 4 | -------------------------------------------------------------------------------- /tests/idris2/interface/interface010/expected: -------------------------------------------------------------------------------- 1 | 1/1: Building Dep (Dep.idr) 2 | -------------------------------------------------------------------------------- /tests/idris2/interface/interface023/input: -------------------------------------------------------------------------------- 1 | r1 2 | r2 3 | r3 4 | :q 5 | -------------------------------------------------------------------------------- /tests/idris2/interface/interface024/expected: -------------------------------------------------------------------------------- 1 | 1/1: Building EH (EH.idr) 2 | -------------------------------------------------------------------------------- /tests/idris2/interface/interface025/input: -------------------------------------------------------------------------------- 1 | :q 2 | -------------------------------------------------------------------------------- /tests/idris2/interface/interface026/input: -------------------------------------------------------------------------------- 1 | :q 2 | -------------------------------------------------------------------------------- /tests/idris2/linear/linear002/input: -------------------------------------------------------------------------------- 1 | :t foo 2 | :q 3 | -------------------------------------------------------------------------------- /tests/idris2/linear/linear006/input: -------------------------------------------------------------------------------- 1 | :set eval typecheck 2 | baz 3 | :q 4 | -------------------------------------------------------------------------------- /tests/idris2/linear/linear013/input: -------------------------------------------------------------------------------- 1 | :t what_is_f 2 | :q 3 | -------------------------------------------------------------------------------- /tests/idris2/linear/linear017/expected: -------------------------------------------------------------------------------- 1 | 1/1: Building As (As.idr) 2 | -------------------------------------------------------------------------------- /tests/idris2/literate/literate002/input2: -------------------------------------------------------------------------------- 1 | :cs 11 20 zs 2 | :q 3 | -------------------------------------------------------------------------------- /tests/idris2/literate/literate004/input: -------------------------------------------------------------------------------- 1 | :ml 8 empties 2 | :ml 10 transposeHelper 3 | :q 4 | -------------------------------------------------------------------------------- /tests/idris2/literate/literate005/input: -------------------------------------------------------------------------------- 1 | :gd 7 transposeHelper 2 | :q 3 | -------------------------------------------------------------------------------- /tests/idris2/literate/literate007/input: -------------------------------------------------------------------------------- 1 | :gd 10 zipHere 2 | :q 3 | -------------------------------------------------------------------------------- /tests/idris2/literate/literate007/input2: -------------------------------------------------------------------------------- 1 | :gd 12 zipHere 2 | :q 3 | -------------------------------------------------------------------------------- /tests/idris2/literate/literate011/input: -------------------------------------------------------------------------------- 1 | :gd 15 zipHere 2 | :q 3 | -------------------------------------------------------------------------------- /tests/idris2/literate/literate014/input: -------------------------------------------------------------------------------- 1 | :mw 4 dnat 2 | :q 3 | -------------------------------------------------------------------------------- /tests/idris2/literate/literate017/.gitignore: -------------------------------------------------------------------------------- 1 | project-output.ipkg 2 | -------------------------------------------------------------------------------- /tests/idris2/literate/literate017/input: -------------------------------------------------------------------------------- 1 | 2 | 3 | 4 | src/ 5 | 6 | -------------------------------------------------------------------------------- /tests/idris2/literate/literate017/src/A/A.org: -------------------------------------------------------------------------------- 1 | -------------------------------------------------------------------------------- /tests/idris2/literate/literate017/src/A/AB.lidr: -------------------------------------------------------------------------------- 1 | -------------------------------------------------------------------------------- /tests/idris2/literate/literate017/src/B/B.md: -------------------------------------------------------------------------------- 1 | -------------------------------------------------------------------------------- /tests/idris2/literate/literate017/src/B/BA.markdown: -------------------------------------------------------------------------------- 1 | -------------------------------------------------------------------------------- /tests/idris2/literate/literate017/src/Main.idr: -------------------------------------------------------------------------------- 1 | -------------------------------------------------------------------------------- /tests/idris2/literate/literate020/input: -------------------------------------------------------------------------------- 1 | :gd 15 zipHere 2 | :q 3 | -------------------------------------------------------------------------------- /tests/idris2/misc/golden001/000-hello/run: -------------------------------------------------------------------------------- 1 | echo "$1" 2 | 3 | $1 4 | -------------------------------------------------------------------------------- /tests/idris2/misc/import003/B.idr: -------------------------------------------------------------------------------- 1 | module B 2 | 3 | import A 4 | -------------------------------------------------------------------------------- /tests/idris2/misc/import003/C.idr: -------------------------------------------------------------------------------- 1 | module C 2 | 3 | import A 4 | 5 | A.defA = ?newHole 6 | -------------------------------------------------------------------------------- /tests/idris2/misc/import003/input: -------------------------------------------------------------------------------- 1 | :m 2 | :q 3 | 4 | -------------------------------------------------------------------------------- /tests/idris2/misc/import006/A/C.idr: -------------------------------------------------------------------------------- 1 | module A.C 2 | 3 | import A.B 4 | -------------------------------------------------------------------------------- /tests/idris2/misc/import006/cyclic.ipkg: -------------------------------------------------------------------------------- 1 | package cyclic 2 | 3 | modules = A.B, A.C 4 | -------------------------------------------------------------------------------- /tests/idris2/misc/namespace005/Lib2.idr: -------------------------------------------------------------------------------- 1 | module Lib2 2 | 3 | export infixl 5 %%% 4 | -------------------------------------------------------------------------------- /tests/idris2/misc/namespace005/LibPre2.idr: -------------------------------------------------------------------------------- 1 | module LibPre2 2 | 3 | export prefix 2 *! 4 | -------------------------------------------------------------------------------- /tests/idris2/misc/namespace005/NonConflict2.idr: -------------------------------------------------------------------------------- 1 | module NonConflict2 2 | 3 | export infixr 5 &&& 4 | -------------------------------------------------------------------------------- /tests/idris2/misc/params002/input: -------------------------------------------------------------------------------- 1 | :t whut 2 | :q 3 | -------------------------------------------------------------------------------- /tests/idris2/misc/params003/input: -------------------------------------------------------------------------------- 1 | :cs 3 7 n 2 | :q 3 | -------------------------------------------------------------------------------- /tests/idris2/misc/params004/input: -------------------------------------------------------------------------------- 1 | :cs 4 5 m 2 | :q 3 | -------------------------------------------------------------------------------- /tests/idris2/mkdoc/mkdoc001/Test1.idr: -------------------------------------------------------------------------------- 1 | ||| Single-line 2 | module Test1 3 | -------------------------------------------------------------------------------- /tests/idris2/mkdoc/mkdoc001/Test2.idr: -------------------------------------------------------------------------------- 1 | ||| Multi- 2 | ||| line 3 | module Test2 4 | -------------------------------------------------------------------------------- /tests/idris2/operators/operators002/Lin.idr: -------------------------------------------------------------------------------- 1 | module Lin 2 | 3 | export typebind infixr 0 =@ 4 | 5 | -------------------------------------------------------------------------------- /tests/idris2/operators/operators003/Error1.idr: -------------------------------------------------------------------------------- 1 | module Error1 2 | 3 | typebind infixl 0 =@ 4 | -------------------------------------------------------------------------------- /tests/idris2/operators/operators003/Error2.idr: -------------------------------------------------------------------------------- 1 | module Error2 2 | 3 | typebind infixr 3 =@ 4 | -------------------------------------------------------------------------------- /tests/idris2/operators/operators003/Error3.idr: -------------------------------------------------------------------------------- 1 | module Error3 2 | 3 | typebind infixl 3 =@ 4 | -------------------------------------------------------------------------------- /tests/idris2/operators/operators011/Test.idr: -------------------------------------------------------------------------------- 1 | 2 | %hide DoesNotExist.infixl.(+-+) 3 | -------------------------------------------------------------------------------- /tests/idris2/operators/operators012/expected: -------------------------------------------------------------------------------- 1 | 1/1: Building Y (Y.idr) 2 | -------------------------------------------------------------------------------- /tests/idris2/perf/perf001/expected: -------------------------------------------------------------------------------- 1 | 1/1: Building Big (Big.idr) 2 | -------------------------------------------------------------------------------- /tests/idris2/perf/perf002/expected: -------------------------------------------------------------------------------- 1 | 1/1: Building Big (Big.idr) 2 | -------------------------------------------------------------------------------- /tests/idris2/perf/perf005/Bad2.idr: -------------------------------------------------------------------------------- 1 | module Bad2 2 | 3 | badReturn : (whatever : Int) 4 | -------------------------------------------------------------------------------- /tests/idris2/perf/perf008/expected: -------------------------------------------------------------------------------- 1 | xs(500) = 500 2 | -------------------------------------------------------------------------------- /tests/idris2/pkg/pkg005/input: -------------------------------------------------------------------------------- 1 | :t hi 2 | hi 3 | :q 4 | -------------------------------------------------------------------------------- /tests/idris2/pkg/pkg006/depends/bar-1.0.1/bar.ipkg: -------------------------------------------------------------------------------- 1 | package bar 2 | version = 1.0.1 3 | -------------------------------------------------------------------------------- /tests/idris2/pkg/pkg006/depends/bar-baz/bar-baz.ipkg: -------------------------------------------------------------------------------- 1 | package bar-baz 2 | -- version = 1.0.1 3 | -------------------------------------------------------------------------------- /tests/idris2/pkg/pkg006/depends/foo-0.5/foo.ipkg: -------------------------------------------------------------------------------- 1 | package foo 2 | version = 0.5 3 | -------------------------------------------------------------------------------- /tests/idris2/pkg/pkg006/depends/foo-bar-1.3.1/foo-bar.ipkg: -------------------------------------------------------------------------------- 1 | package foo-bar 2 | version = 1.3.1 3 | -------------------------------------------------------------------------------- /tests/idris2/pkg/pkg006/depends/quux/quux.ipkg: -------------------------------------------------------------------------------- 1 | package quux 2 | -- version = 0.0.0 3 | -------------------------------------------------------------------------------- /tests/idris2/pkg/pkg006/test5.ipkg: -------------------------------------------------------------------------------- 1 | package test5 2 | version = "this one" 3 | -------------------------------------------------------------------------------- /tests/idris2/pkg/pkg007/input: -------------------------------------------------------------------------------- 1 | cool 2 | gallais 3 | -p contrib 4 | 5 | -------------------------------------------------------------------------------- /tests/idris2/pkg/pkg007/input2: -------------------------------------------------------------------------------- 1 | cool 2 | gallais 3 | -p contrib 4 | src 5 | -------------------------------------------------------------------------------- /tests/idris2/pkg/pkg008/Foo.idr: -------------------------------------------------------------------------------- 1 | module Foo 2 | -------------------------------------------------------------------------------- /tests/idris2/pkg/pkg013/depends/foo-0.1.0/foo.ipkg: -------------------------------------------------------------------------------- 1 | package foo 2 | version = 0.1.0 3 | -------------------------------------------------------------------------------- /tests/idris2/pkg/pkg013/test.ipkg: -------------------------------------------------------------------------------- 1 | package test 2 | depends = bar 3 | -------------------------------------------------------------------------------- /tests/idris2/pkg/pkg014/depends/baz-0.1.0/baz.ipkg: -------------------------------------------------------------------------------- 1 | package baz 2 | version = 0.1.0 3 | -------------------------------------------------------------------------------- /tests/idris2/pkg/pkg014/depends/baz-0.2.0/baz.ipkg: -------------------------------------------------------------------------------- 1 | package baz 2 | version = 0.2.0 3 | -------------------------------------------------------------------------------- /tests/idris2/pkg/pkg015/depends/baz-0.1.0/baz.ipkg: -------------------------------------------------------------------------------- 1 | package baz 2 | version = 0.1.0 3 | -------------------------------------------------------------------------------- /tests/idris2/pkg/pkg015/depends/baz-0.2.0/baz.ipkg: -------------------------------------------------------------------------------- 1 | package baz 2 | version = 0.2.0 3 | -------------------------------------------------------------------------------- /tests/idris2/pkg/pkg015/depends/prz-0.1.0/prz.ipkg: -------------------------------------------------------------------------------- 1 | package prz 2 | version = 0.1.0 3 | -------------------------------------------------------------------------------- /tests/idris2/pkg/pkg018/bad.ipkg: -------------------------------------------------------------------------------- 1 | package bad 2 | depend = contrib 3 | -------------------------------------------------------------------------------- /tests/idris2/pkg/pkg018/bad2.ipkg: -------------------------------------------------------------------------------- 1 | package bad 2 | sourcedir = src 3 | -------------------------------------------------------------------------------- /tests/idris2/pkg/pkg021/input: -------------------------------------------------------------------------------- 1 | :import Stuff 2 | :q 3 | -------------------------------------------------------------------------------- /tests/idris2/pkg/pkg021/src/Stuff.idr: -------------------------------------------------------------------------------- 1 | module Stuff 2 | 3 | -------------------------------------------------------------------------------- /tests/idris2/reflection/reflection004/input: -------------------------------------------------------------------------------- 1 | foo 4 5 2 | mkMult 3 3 | myplus 2 3 4 | :q 5 | -------------------------------------------------------------------------------- /tests/idris2/reflection/reflection005/input: -------------------------------------------------------------------------------- 1 | mkMult 100 2 | :q 3 | -------------------------------------------------------------------------------- /tests/idris2/reflection/reflection006/input: -------------------------------------------------------------------------------- 1 | mkMult 100 2 | :q 3 | -------------------------------------------------------------------------------- /tests/idris2/reflection/reflection011/input: -------------------------------------------------------------------------------- 1 | x 2 | :q 3 | -------------------------------------------------------------------------------- /tests/idris2/reflection/reflection012/input: -------------------------------------------------------------------------------- 1 | %runElab foo 2 | :q 3 | -------------------------------------------------------------------------------- /tests/idris2/reflection/reflection014/expected: -------------------------------------------------------------------------------- 1 | True 2 | False 3 | -------------------------------------------------------------------------------- /tests/idris2/reflection/reflection016/input: -------------------------------------------------------------------------------- 1 | :q 2 | -------------------------------------------------------------------------------- /tests/idris2/reflection/reflection019/input: -------------------------------------------------------------------------------- 1 | :t x 2 | x 3 | :q 4 | -------------------------------------------------------------------------------- /tests/idris2/reflection/reflection019/test.ipkg: -------------------------------------------------------------------------------- 1 | package a-test 2 | -------------------------------------------------------------------------------- /tests/idris2/reflection/reflection023/test.ipkg: -------------------------------------------------------------------------------- 1 | package a-test 2 | -------------------------------------------------------------------------------- /tests/idris2/reflection/reflection024/src/existentToRead: -------------------------------------------------------------------------------- 1 | existent to read 2 | second line 3 | -------------------------------------------------------------------------------- /tests/idris2/reflection/reflection025/test.ipkg: -------------------------------------------------------------------------------- 1 | package a-test 2 | -------------------------------------------------------------------------------- /tests/idris2/reflection/reflection026/test.ipkg: -------------------------------------------------------------------------------- 1 | package a-test 2 | -------------------------------------------------------------------------------- /tests/idris2/reflection/reflection027/test.ipkg: -------------------------------------------------------------------------------- 1 | package a-test 2 | -------------------------------------------------------------------------------- /tests/idris2/reflection/reflection028/test.ipkg: -------------------------------------------------------------------------------- 1 | package a-test 2 | -------------------------------------------------------------------------------- /tests/idris2/reflection/reflection034_2/expected: -------------------------------------------------------------------------------- 1 | -4 2 | -19 3 | -------------------------------------------------------------------------------- /tests/idris2/reg/reg001/expected: -------------------------------------------------------------------------------- 1 | 1/1: Building D (D.idr) 2 | -------------------------------------------------------------------------------- /tests/idris2/reg/reg006/expected: -------------------------------------------------------------------------------- 1 | 1/1: Building Cmd (Cmd.idr) 2 | -------------------------------------------------------------------------------- /tests/idris2/reg/reg008/input: -------------------------------------------------------------------------------- 1 | :missing runMachine 2 | :q 3 | -------------------------------------------------------------------------------- /tests/idris2/reg/reg011/expected: -------------------------------------------------------------------------------- 1 | 1/1: Building mut (mut.idr) 2 | -------------------------------------------------------------------------------- /tests/idris2/reg/reg012/expected: -------------------------------------------------------------------------------- 1 | 1/1: Building Foo (Foo.idr) 2 | -------------------------------------------------------------------------------- /tests/idris2/reg/reg020/input: -------------------------------------------------------------------------------- 1 | :printdef test1 2 | :q 3 | -------------------------------------------------------------------------------- /tests/idris2/reg/reg022/input: -------------------------------------------------------------------------------- 1 | :t foo 2 | :q 3 | -------------------------------------------------------------------------------- /tests/idris2/reg/reg024/input: -------------------------------------------------------------------------------- 1 | :cs 13 8 x 2 | :q 3 | -------------------------------------------------------------------------------- /tests/idris2/reg/reg025/input: -------------------------------------------------------------------------------- 1 | :ml 11 pbz_hole 2 | :q 3 | -------------------------------------------------------------------------------- /tests/idris2/reg/reg026/expected: -------------------------------------------------------------------------------- 1 | 1/1: Building Meh (Meh.idr) 2 | -------------------------------------------------------------------------------- /tests/idris2/reg/reg043/NotFake.idr: -------------------------------------------------------------------------------- 1 | module NotFake 2 | -------------------------------------------------------------------------------- /tests/idris2/reg/reg043/TestFake.idr: -------------------------------------------------------------------------------- 1 | import Fake 2 | -------------------------------------------------------------------------------- /tests/idris2/reg/reg046/input: -------------------------------------------------------------------------------- 1 | :q 2 | -------------------------------------------------------------------------------- /tests/idris2/reg/reg047/input: -------------------------------------------------------------------------------- 1 | propagateNSToBangs 2 | :q 3 | -------------------------------------------------------------------------------- /tests/idris2/reg/reg051/test.ipkg: -------------------------------------------------------------------------------- 1 | package a-test 2 | -------------------------------------------------------------------------------- /tests/idris2/reg/reg052/test.ipkg: -------------------------------------------------------------------------------- 1 | package a-test 2 | -------------------------------------------------------------------------------- /tests/idris2/reg/reg053/input: -------------------------------------------------------------------------------- 1 | :ti hole 2 | :q 3 | -------------------------------------------------------------------------------- /tests/idris2/repl/repl001/input: -------------------------------------------------------------------------------- 1 | :? 2 | :h 3 | :help 4 | -------------------------------------------------------------------------------- /tests/idris2/repl/repl007/input: -------------------------------------------------------------------------------- 1 | :di Bool 2 | :di True 3 | -------------------------------------------------------------------------------- /tests/idris2/schemeeval/schemeeval005/input: -------------------------------------------------------------------------------- 1 | :set eval scheme 2 | test 3 | :q 4 | -------------------------------------------------------------------------------- /tests/idris2/schemeeval/schemeeval006/input: -------------------------------------------------------------------------------- 1 | :set eval scheme 2 | unpack "foo" 3 | :q -------------------------------------------------------------------------------- /tests/idris2/total/total020/test.ipkg: -------------------------------------------------------------------------------- 1 | package a-test 2 | -------------------------------------------------------------------------------- /tests/idris2/total/total022/input: -------------------------------------------------------------------------------- 1 | :di f 2 | :q 3 | 4 | -------------------------------------------------------------------------------- /tests/idris2/total/total023/input: -------------------------------------------------------------------------------- 1 | :di addord 2 | :q 3 | -------------------------------------------------------------------------------- /tests/idris2/warning/warning004/Lib2.idr: -------------------------------------------------------------------------------- 1 | module Lib2 2 | 3 | export infixl 5 %%% 4 | -------------------------------------------------------------------------------- /tests/idris2/with/with004/input: -------------------------------------------------------------------------------- 1 | foo2 2 | :q -------------------------------------------------------------------------------- /tests/linear/system_concurrency_session/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run -p linear Main.idr 4 | -------------------------------------------------------------------------------- /tests/node/args/expected: -------------------------------------------------------------------------------- 1 | ["a", "b"] 2 | ["c"] 3 | -------------------------------------------------------------------------------- /tests/node/args/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/node/args/run -------------------------------------------------------------------------------- /tests/node/bitops/expected: -------------------------------------------------------------------------------- 1 | -------------------------------------------------------------------------------- /tests/node/bitops/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run --cg node BitOps.idr 4 | -------------------------------------------------------------------------------- /tests/node/casts/expected: -------------------------------------------------------------------------------- 1 | -------------------------------------------------------------------------------- /tests/node/casts/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run --cg node Casts.idr 4 | -------------------------------------------------------------------------------- /tests/node/double001/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/node/double001/run -------------------------------------------------------------------------------- /tests/node/double002/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/node/double002/run -------------------------------------------------------------------------------- /tests/node/double003/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/node/double003/run -------------------------------------------------------------------------------- /tests/node/doubles/expected: -------------------------------------------------------------------------------- 1 | -1 2 | -------------------------------------------------------------------------------- /tests/node/doubles/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/node/doubles/run -------------------------------------------------------------------------------- /tests/node/executable/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/node/executable/run -------------------------------------------------------------------------------- /tests/node/fastConcat/expected: -------------------------------------------------------------------------------- 1 | 34.. -------------------------------------------------------------------------------- /tests/node/fastConcat/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run --cg node FastConcat.idr 4 | -------------------------------------------------------------------------------- /tests/node/ffi001/expected: -------------------------------------------------------------------------------- 1 | hello, world 2 | -------------------------------------------------------------------------------- /tests/node/ffi001/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | run --cg node Foreign.idr 3 | -------------------------------------------------------------------------------- /tests/node/fix1839/OS.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/node/fix1839/OS.idr -------------------------------------------------------------------------------- /tests/node/fix1839/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/node/fix1839/run -------------------------------------------------------------------------------- /tests/node/idiom001/expected: -------------------------------------------------------------------------------- 1 | -------------------------------------------------------------------------------- /tests/node/idiom001/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run --cg node Main.idr 4 | -------------------------------------------------------------------------------- /tests/node/integer_array/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run --cg node array.idr 4 | -------------------------------------------------------------------------------- /tests/node/integers/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/node/integers/run -------------------------------------------------------------------------------- /tests/node/memo/Memo.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/node/memo/Memo.idr -------------------------------------------------------------------------------- /tests/node/memo/expected: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/node/memo/expected -------------------------------------------------------------------------------- /tests/node/memo/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run --cg node Memo.idr 4 | -------------------------------------------------------------------------------- /tests/node/newints/expected: -------------------------------------------------------------------------------- 1 | -------------------------------------------------------------------------------- /tests/node/newints/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run --cg node IntOps.idr 4 | -------------------------------------------------------------------------------- /tests/node/node001/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run --cg node Total.idr 4 | -------------------------------------------------------------------------------- /tests/node/node002/input: -------------------------------------------------------------------------------- 1 | :exec printLn (pythag 200) 2 | :q 3 | -------------------------------------------------------------------------------- /tests/node/node002/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/node/node002/run -------------------------------------------------------------------------------- /tests/node/node003/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run --cg node IORef.idr 4 | -------------------------------------------------------------------------------- /tests/node/node004/.gitignore: -------------------------------------------------------------------------------- 1 | test.buf 2 | -------------------------------------------------------------------------------- /tests/node/node004/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/node/node004/run -------------------------------------------------------------------------------- /tests/node/node005/input: -------------------------------------------------------------------------------- 1 | :exec printLn (Main.filter even [S Z,2,3,4,5,6]) 2 | :q 3 | -------------------------------------------------------------------------------- /tests/node/node005/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/node/node005/run -------------------------------------------------------------------------------- /tests/node/node006/input: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/node/node006/input -------------------------------------------------------------------------------- /tests/node/node006/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/node/node006/run -------------------------------------------------------------------------------- /tests/node/node007/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run --cg node TypeCase.idr 4 | -------------------------------------------------------------------------------- /tests/node/node008/expected: -------------------------------------------------------------------------------- 1 | 1 2 | 1 3 | 1 4 | -------------------------------------------------------------------------------- /tests/node/node008/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run --cg node Nat.idr 4 | -------------------------------------------------------------------------------- /tests/node/node009/expected: -------------------------------------------------------------------------------- 1 | 42 2 | ällo 3 | -------------------------------------------------------------------------------- /tests/node/node009/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run --cg node uni.idr 4 | -------------------------------------------------------------------------------- /tests/node/node011/input: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/node/node011/input -------------------------------------------------------------------------------- /tests/node/node011/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/node/node011/run -------------------------------------------------------------------------------- /tests/node/node012/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run --cg node array.idr 4 | -------------------------------------------------------------------------------- /tests/node/node015/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run --cg node Numbers.idr 4 | -------------------------------------------------------------------------------- /tests/node/node017/.gitignore: -------------------------------------------------------------------------------- 1 | testdir/ 2 | -------------------------------------------------------------------------------- /tests/node/node017/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/node/node017/run -------------------------------------------------------------------------------- /tests/node/node018/.gitignore: -------------------------------------------------------------------------------- 1 | testout.txt 2 | -------------------------------------------------------------------------------- /tests/node/node018/expected: -------------------------------------------------------------------------------- 1 | test test 2 | unfinished lineabc 3 | def 4 | File Not Found 5 | -------------------------------------------------------------------------------- /tests/node/node018/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/node/node018/run -------------------------------------------------------------------------------- /tests/node/node018/test.txt: -------------------------------------------------------------------------------- 1 | test test 2 | unfinished line -------------------------------------------------------------------------------- /tests/node/node019/input: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/node/node019/input -------------------------------------------------------------------------------- /tests/node/node019/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/node/node019/run -------------------------------------------------------------------------------- /tests/node/node020/expected: -------------------------------------------------------------------------------- 1 | opened 2 | closed 3 | Idris 2 4 | -------------------------------------------------------------------------------- /tests/node/node020/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/node/node020/run -------------------------------------------------------------------------------- /tests/node/node021/input: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/node/node021/input -------------------------------------------------------------------------------- /tests/node/node021/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/node/node021/run -------------------------------------------------------------------------------- /tests/node/node022/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run --cg node BitCasts.idr 4 | -------------------------------------------------------------------------------- /tests/node/node023/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run --cg node Casts.idr 4 | -------------------------------------------------------------------------------- /tests/node/node024/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run --cg node BitOps.idr 4 | -------------------------------------------------------------------------------- /tests/node/node025/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run --cg node Fix1037.idr 4 | -------------------------------------------------------------------------------- /tests/node/node026/expected: -------------------------------------------------------------------------------- 1 | Right ('1', 1) 2 | -------------------------------------------------------------------------------- /tests/node/node026/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run -p contrib --cg node Fix1795.idr 4 | -------------------------------------------------------------------------------- /tests/node/node027/expected: -------------------------------------------------------------------------------- 1 | -------------------------------------------------------------------------------- /tests/node/node027/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run --cg node PID.idr 4 | -------------------------------------------------------------------------------- /tests/node/node028/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/node/node028/run -------------------------------------------------------------------------------- /tests/node/perf001/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run --cg node Span.idr 4 | -------------------------------------------------------------------------------- /tests/node/reg001/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run --cg node numbers.idr 4 | -------------------------------------------------------------------------------- /tests/node/reg002/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run --cg node Issue1843.idr 4 | -------------------------------------------------------------------------------- /tests/node/stringcast/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run --cg node StringCast.idr 4 | -------------------------------------------------------------------------------- /tests/node/syntax001/expected: -------------------------------------------------------------------------------- 1 | 0 2 | 1 3 | -------------------------------------------------------------------------------- /tests/node/syntax001/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run --cg node caseBlock.idr 4 | -------------------------------------------------------------------------------- /tests/node/tailrec001/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run --cg node tailrec.idr 4 | -------------------------------------------------------------------------------- /tests/node/tailrec002/expected: -------------------------------------------------------------------------------- 1 | [] 2 | -------------------------------------------------------------------------------- /tests/node/tailrec002/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/node/tailrec002/run -------------------------------------------------------------------------------- /tests/node/tailrec_libs/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run --cg node tailrec.idr 4 | -------------------------------------------------------------------------------- /tests/prelude/bind001/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run bind.idr 4 | -------------------------------------------------------------------------------- /tests/prelude/char001/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | check chars.idr 4 | -------------------------------------------------------------------------------- /tests/prelude/double001/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run Types.idr 4 | -------------------------------------------------------------------------------- /tests/prelude/nat001/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | check nats.idr 4 | -------------------------------------------------------------------------------- /tests/prelude/reg001/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | check fixity.idr 4 | -------------------------------------------------------------------------------- /tests/prelude/unpack/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | check unpack.idr 4 | -------------------------------------------------------------------------------- /tests/racket/barrier001/input: -------------------------------------------------------------------------------- 1 | -------------------------------------------------------------------------------- /tests/racket/barrier001/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run --cg racket Main.idr 4 | -------------------------------------------------------------------------------- /tests/racket/conditions001/expected: -------------------------------------------------------------------------------- 1 | Hello 2 | Goodbye 3 | -------------------------------------------------------------------------------- /tests/racket/conditions001/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run --cg racket Main.idr 4 | -------------------------------------------------------------------------------- /tests/racket/conditions002/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run --cg racket Main.idr 4 | -------------------------------------------------------------------------------- /tests/racket/conditions003/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run --cg racket Main.idr 4 | -------------------------------------------------------------------------------- /tests/racket/conditions004/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run --cg racket Main.idr 4 | -------------------------------------------------------------------------------- /tests/racket/conditions005/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run --cg racket Main.idr 4 | -------------------------------------------------------------------------------- /tests/racket/conditions006/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run --cg racket Main.idr 4 | -------------------------------------------------------------------------------- /tests/racket/conditions007/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run --cg racket Main.idr 4 | -------------------------------------------------------------------------------- /tests/racket/ffi001/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/racket/ffi001/run -------------------------------------------------------------------------------- /tests/racket/forkjoin001/expected: -------------------------------------------------------------------------------- 1 | Hello 2 | Goodbye 3 | -------------------------------------------------------------------------------- /tests/racket/forkjoin001/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run --cg racket Main.idr 4 | -------------------------------------------------------------------------------- /tests/racket/mutex001/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run --cg racket Main.idr 4 | -------------------------------------------------------------------------------- /tests/racket/mutex002/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run --cg racket Main.idr 4 | -------------------------------------------------------------------------------- /tests/racket/mutex003/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run --cg racket Main.idr 4 | -------------------------------------------------------------------------------- /tests/racket/mutex004/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run --cg racket Main.idr 4 | -------------------------------------------------------------------------------- /tests/racket/mutex005/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run --cg racket Main.idr 4 | -------------------------------------------------------------------------------- /tests/racket/semaphores001/expected: -------------------------------------------------------------------------------- 1 | Hello 2 | Goodbye 3 | -------------------------------------------------------------------------------- /tests/racket/semaphores001/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run --cg racket Main.idr 4 | -------------------------------------------------------------------------------- /tests/racket/semaphores002/expected: -------------------------------------------------------------------------------- 1 | Hello 2 | Goodbye 3 | -------------------------------------------------------------------------------- /tests/racket/semaphores002/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | run --cg racket Main.idr 4 | -------------------------------------------------------------------------------- /tests/refc/args/expected: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/refc/args/expected -------------------------------------------------------------------------------- /tests/refc/args/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/refc/args/run -------------------------------------------------------------------------------- /tests/refc/buffer/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/refc/buffer/run -------------------------------------------------------------------------------- /tests/refc/clock/expected: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/refc/clock/expected -------------------------------------------------------------------------------- /tests/refc/clock/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/refc/clock/run -------------------------------------------------------------------------------- /tests/refc/doubles/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/refc/doubles/run -------------------------------------------------------------------------------- /tests/refc/integers/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/refc/integers/run -------------------------------------------------------------------------------- /tests/refc/issue1778/expected: -------------------------------------------------------------------------------- 1 | 34. -------------------------------------------------------------------------------- /tests/refc/issue1778/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/refc/issue1778/run -------------------------------------------------------------------------------- /tests/refc/issue2424/expected: -------------------------------------------------------------------------------- 1 | value is 42 2 | -------------------------------------------------------------------------------- /tests/refc/issue2424/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/refc/issue2424/run -------------------------------------------------------------------------------- /tests/refc/issue2452/expected: -------------------------------------------------------------------------------- 1 | good 2 | -------------------------------------------------------------------------------- /tests/refc/issue2452/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/refc/issue2452/run -------------------------------------------------------------------------------- /tests/refc/prims/Test.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/refc/prims/Test.idr -------------------------------------------------------------------------------- /tests/refc/prims/expected: -------------------------------------------------------------------------------- 1 | Nothing 2 | True 3 | Just 10 4 | "abcd" 5 | "ABCD" 6 | "refc" 7 | -------------------------------------------------------------------------------- /tests/refc/prims/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/refc/prims/run -------------------------------------------------------------------------------- /tests/refc/refc001/expected: -------------------------------------------------------------------------------- 1 | 2 | Hello World! 3 | -------------------------------------------------------------------------------- /tests/refc/refc001/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/refc/refc001/run -------------------------------------------------------------------------------- /tests/refc/refc002/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/refc/refc002/run -------------------------------------------------------------------------------- /tests/refc/refc003/expected: -------------------------------------------------------------------------------- 1 | 3 2 | -------------------------------------------------------------------------------- /tests/refc/refc003/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/refc/refc003/run -------------------------------------------------------------------------------- /tests/refc/reg001/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/refc/reg001/run -------------------------------------------------------------------------------- /tests/refc/reuse/Main.idr: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/refc/reuse/Main.idr -------------------------------------------------------------------------------- /tests/refc/reuse/expected: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/refc/reuse/expected -------------------------------------------------------------------------------- /tests/refc/reuse/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/refc/reuse/run -------------------------------------------------------------------------------- /tests/refc/strings/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/refc/strings/run -------------------------------------------------------------------------------- /tests/templates/simple-test/input: -------------------------------------------------------------------------------- 1 | 2 + 2 2 | :q 3 | -------------------------------------------------------------------------------- /tests/templates/ttimp/input: -------------------------------------------------------------------------------- 1 | test1 2 | test2 3 | :q 4 | -------------------------------------------------------------------------------- /tests/templates/ttimp/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/templates/ttimp/run -------------------------------------------------------------------------------- /tests/templates/with-ipkg/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | idris2 --build dummy.ipkg 4 | -------------------------------------------------------------------------------- /tests/tests.ipkg: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/tests.ipkg -------------------------------------------------------------------------------- /tests/testutils.sh: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/testutils.sh -------------------------------------------------------------------------------- /tests/ttimp/basic001/input: -------------------------------------------------------------------------------- 1 | test1 2 | test2 3 | :q 4 | -------------------------------------------------------------------------------- /tests/ttimp/basic001/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/ttimp/basic001/run -------------------------------------------------------------------------------- /tests/ttimp/basic002/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/ttimp/basic002/run -------------------------------------------------------------------------------- /tests/ttimp/basic003/input: -------------------------------------------------------------------------------- 1 | :t foo 2 | :q 3 | -------------------------------------------------------------------------------- /tests/ttimp/basic003/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/ttimp/basic003/run -------------------------------------------------------------------------------- /tests/ttimp/basic004/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/ttimp/basic004/run -------------------------------------------------------------------------------- /tests/ttimp/basic005/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/ttimp/basic005/run -------------------------------------------------------------------------------- /tests/ttimp/basic006/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/ttimp/basic006/run -------------------------------------------------------------------------------- /tests/ttimp/dot001/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/ttimp/dot001/run -------------------------------------------------------------------------------- /tests/ttimp/eta001/input: -------------------------------------------------------------------------------- 1 | eqTest 2 | :t etaGood1 3 | :q 4 | -------------------------------------------------------------------------------- /tests/ttimp/eta001/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/ttimp/eta001/run -------------------------------------------------------------------------------- /tests/ttimp/lazy001/input: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/ttimp/lazy001/input -------------------------------------------------------------------------------- /tests/ttimp/lazy001/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/ttimp/lazy001/run -------------------------------------------------------------------------------- /tests/ttimp/nest001/input: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/ttimp/nest001/input -------------------------------------------------------------------------------- /tests/ttimp/nest001/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/ttimp/nest001/run -------------------------------------------------------------------------------- /tests/ttimp/nest002/input: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/ttimp/nest002/input -------------------------------------------------------------------------------- /tests/ttimp/nest002/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/ttimp/nest002/run -------------------------------------------------------------------------------- /tests/ttimp/perf001/expected: -------------------------------------------------------------------------------- 1 | Processing as TTImp 2 | Written TTC 3 | Yaffle> Bye for now! 4 | -------------------------------------------------------------------------------- /tests/ttimp/perf001/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/ttimp/perf001/run -------------------------------------------------------------------------------- /tests/ttimp/perf002/input: -------------------------------------------------------------------------------- 1 | :t stuff 2 | :q 3 | -------------------------------------------------------------------------------- /tests/ttimp/perf002/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/ttimp/perf002/run -------------------------------------------------------------------------------- /tests/ttimp/perf003/input: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/ttimp/perf003/input -------------------------------------------------------------------------------- /tests/ttimp/perf003/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/ttimp/perf003/run -------------------------------------------------------------------------------- /tests/ttimp/qtt001/input: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/ttimp/qtt001/input -------------------------------------------------------------------------------- /tests/ttimp/qtt001/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/ttimp/qtt001/run -------------------------------------------------------------------------------- /tests/ttimp/qtt003/input: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/ttimp/qtt003/input -------------------------------------------------------------------------------- /tests/ttimp/qtt003/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/ttimp/qtt003/run -------------------------------------------------------------------------------- /tests/ttimp/record001/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/ttimp/record001/run -------------------------------------------------------------------------------- /tests/ttimp/record002/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/ttimp/record002/run -------------------------------------------------------------------------------- /tests/ttimp/record003/input: -------------------------------------------------------------------------------- 1 | :q 2 | 3 | -------------------------------------------------------------------------------- /tests/ttimp/record003/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/ttimp/record003/run -------------------------------------------------------------------------------- /tests/ttimp/record004/input: -------------------------------------------------------------------------------- 1 | :q 2 | -------------------------------------------------------------------------------- /tests/ttimp/record004/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/ttimp/record004/run -------------------------------------------------------------------------------- /tests/ttimp/total001/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/ttimp/total001/run -------------------------------------------------------------------------------- /tests/ttimp/total002/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/ttimp/total002/run -------------------------------------------------------------------------------- /tests/ttimp/total003/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/ttimp/total003/run -------------------------------------------------------------------------------- /tests/ttimp/total004/input: -------------------------------------------------------------------------------- 1 | :q 2 | -------------------------------------------------------------------------------- /tests/ttimp/total004/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/ttimp/total004/run -------------------------------------------------------------------------------- /tests/typedd-book/chapter01/input: -------------------------------------------------------------------------------- 1 | :t convert 2 | :q 3 | -------------------------------------------------------------------------------- /tests/typedd-book/chapter02/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | check All.idr 4 | -------------------------------------------------------------------------------- /tests/typedd-book/chapter03/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | check All.idr 4 | -------------------------------------------------------------------------------- /tests/typedd-book/chapter04/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | check All.idr 4 | -------------------------------------------------------------------------------- /tests/typedd-book/chapter05/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | check All.idr 4 | -------------------------------------------------------------------------------- /tests/typedd-book/chapter06/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | check All.idr 4 | -------------------------------------------------------------------------------- /tests/typedd-book/chapter07/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | check All.idr 4 | -------------------------------------------------------------------------------- /tests/typedd-book/chapter08/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | check All.idr 4 | -------------------------------------------------------------------------------- /tests/typedd-book/chapter09/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | check All.idr 4 | -------------------------------------------------------------------------------- /tests/typedd-book/chapter11/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | check All.idr 4 | -------------------------------------------------------------------------------- /tests/typedd-book/chapter12/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | check All.idr 4 | -------------------------------------------------------------------------------- /tests/typedd-book/chapter13/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | check All.idr 4 | -------------------------------------------------------------------------------- /tests/typedd-book/chapter14/run: -------------------------------------------------------------------------------- 1 | . ../../testutils.sh 2 | 3 | check All.idr 4 | -------------------------------------------------------------------------------- /tests/vmcode/basic001/run: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/tests/vmcode/basic001/run -------------------------------------------------------------------------------- /www/README.md: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/www/README.md -------------------------------------------------------------------------------- /www/katla.sh: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/www/katla.sh -------------------------------------------------------------------------------- /www/source/index.md: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/idris-lang/Idris2/HEAD/www/source/index.md --------------------------------------------------------------------------------