├── .gitignore ├── INSTALL.txt ├── LICENSE ├── README.md ├── READMEconsolePrograms.txt ├── docs ├── Agda.Builtin.Bool.html ├── Agda.Builtin.Char.html ├── Agda.Builtin.Coinduction.html ├── Agda.Builtin.Equality.html ├── Agda.Builtin.List.html ├── Agda.Builtin.Nat.html ├── Agda.Builtin.Size.html ├── Agda.Builtin.String.html ├── Agda.Builtin.TrustMe.html ├── Agda.Builtin.Unit.html ├── Agda.Primitive.html ├── Agda.css ├── Algebra.FunctionProperties.Core.html ├── Algebra.FunctionProperties.html ├── Algebra.Morphism.html ├── Algebra.Operations.html ├── Algebra.Properties.AbelianGroup.html ├── Algebra.Properties.BooleanAlgebra.Expression.html ├── Algebra.Properties.BooleanAlgebra.html ├── Algebra.Properties.DistributiveLattice.html ├── Algebra.Properties.Group.html ├── Algebra.Properties.Lattice.html ├── Algebra.Properties.Ring.html ├── Algebra.RingSolver.AlmostCommutativeRing.html ├── Algebra.RingSolver.Lemmas.html ├── Algebra.RingSolver.Simple.html ├── Algebra.RingSolver.html ├── Algebra.Structures.html ├── Algebra.html ├── Category.Applicative.Indexed.html ├── Category.Applicative.html ├── Category.Functor.Identity.html ├── Category.Functor.html ├── Category.Monad.Identity.html ├── Category.Monad.Indexed.html ├── Category.Monad.html ├── Coinduction.html ├── Data.Bool.Base.html ├── Data.Bool.Properties.html ├── Data.Bool.html ├── Data.BoundedVec.Inefficient.html ├── Data.Char.Base.html ├── Data.Char.Core.html ├── Data.Char.html ├── Data.Colist.html ├── Data.Conat.html ├── Data.Empty.html ├── Data.Fin.Dec.html ├── Data.Fin.Properties.html ├── Data.Fin.Subset.Properties.html ├── Data.Fin.Subset.html ├── Data.Fin.html ├── Data.List.Any.html ├── Data.List.Base.html ├── Data.List.NonEmpty.html ├── Data.List.html ├── Data.Maybe.Base.html ├── Data.Maybe.html ├── Data.Nat.Base.html ├── Data.Nat.Properties.Simple.html ├── Data.Nat.Properties.html ├── Data.Nat.html ├── Data.Plus.html ├── Data.Product.html ├── Data.String.Base.html ├── Data.String.html ├── Data.Sum.html ├── Data.Unit.Base.html ├── Data.Unit.NonEta.html ├── Data.Unit.html ├── Data.Vec.Equality.html ├── Data.Vec.N-ary.html ├── Data.Vec.Properties.html ├── Data.Vec.html ├── Function.Bijection.html ├── Function.Equality.html ├── Function.Equivalence.html ├── Function.Injection.html ├── Function.Inverse.html ├── Function.LeftInverse.html ├── Function.Related.html ├── Function.Surjection.html ├── Function.html ├── Level.html ├── NativeIO.html ├── Relation.Binary.Consequences.Core.html ├── Relation.Binary.Consequences.html ├── Relation.Binary.Core.html ├── Relation.Binary.EqReasoning.html ├── Relation.Binary.HeterogeneousEquality.Core.html ├── Relation.Binary.HeterogeneousEquality.html ├── Relation.Binary.Indexed.Core.html ├── Relation.Binary.Indexed.html ├── Relation.Binary.InducedPreorders.html ├── Relation.Binary.Lattice.html ├── Relation.Binary.List.Pointwise.html ├── Relation.Binary.List.StrictLex.html ├── Relation.Binary.On.html ├── Relation.Binary.PartialOrderReasoning.html ├── Relation.Binary.PreorderReasoning.html ├── Relation.Binary.PropositionalEquality.Core.html ├── Relation.Binary.PropositionalEquality.TrustMe.html ├── Relation.Binary.PropositionalEquality.html ├── Relation.Binary.Reflection.html ├── Relation.Binary.Vec.Pointwise.html ├── Relation.Binary.html ├── Relation.Nullary.Decidable.html ├── Relation.Nullary.Negation.html ├── Relation.Nullary.html ├── Relation.Unary.html ├── Size.html ├── SizedIO.Base.html ├── SizedIO.Console.html ├── SizedIO.Object.html ├── StateSizedIO.Base.html ├── StateSizedIO.IOObject.html ├── StateSizedIO.Object.html ├── StateSizedIO.RObject.html ├── StateSizedIO.cellStateDependent.html ├── StateSizedIO.writingOOsUsingIO.html ├── StateSizedIO.writingOOsUsingIOVers4ReaderMethods.html ├── Unit.html ├── examples.heap.ALL.html ├── examples.heap.correctnessLinkedList.html ├── examples.heap.correctnessLinkedListStep2.html ├── heap.library.html ├── heap.libraryBool.html ├── heap.libraryFin.html ├── heap.libraryMaybe.html ├── heap.libraryNat.html ├── src.heap.heapAsObject.html ├── src.heap.heapAsObjectBase.html ├── src.heap.heapAsObjectExample.html ├── src.heap.heapAsObjectGeneric.html ├── src.heap.heapAsObjectNativeHeap.html └── src.heap.worldModule.html ├── exampleCode ├── helloWorld.agda └── myExample.agda-lib ├── examples ├── DrawingProgram │ ├── IOExampleGraphicsDrawingProgram.agda │ ├── IOExampleGraphicsDrawingProgramWhenJust.agda │ ├── IOExampleGraphicsMovingText.agda │ └── Main.agda-lib ├── Sized │ ├── ConsoleExample.agda │ ├── CounterCell.agda │ ├── Parrot.agda │ ├── SelfRef.agda │ ├── SimpleCell.agda │ └── StatefulCell.agda ├── SizedPoly │ ├── Console.agda │ └── SimpleCell.agda ├── StateSized │ ├── GUI │ │ ├── BitMaps.agda │ │ ├── ShipBitMap.agda │ │ ├── SpaceShipAdvanced.agda │ │ ├── SpaceShipCell.agda │ │ ├── SpaceShipExtendedExample.agda │ │ ├── SpaceShipSimpleVar.agda │ │ └── ship.ico │ ├── StackStateDependent.agda │ └── cellStateDependent.agda ├── UnSized │ ├── Console.agda │ ├── Parrot.agda │ ├── SelfRef.agda │ └── SimpleCell.agda ├── consoleExamples │ ├── helloWorld.agda │ ├── passwordCheckSimple.agda │ └── simpleLoop.agda ├── examplesPaperJFP │ ├── BasicIO.agda │ ├── CatNonTerm.agda │ ├── CatTerm.agda │ ├── Coalgebra.agda │ ├── Colists.agda │ ├── Collatz.agda │ ├── Console.agda │ ├── ConsoleInterface.agda │ ├── CounterCell.agda │ ├── Equality.agda │ ├── ExampleDrawingProgram.agda │ ├── IOExampleConsole.agda │ ├── IOGraphicsLib.agda │ ├── NativeIOSafe.agda │ ├── Object.agda │ ├── Sized.agda │ ├── SpaceShipAdvanced.agda │ ├── SpaceShipCell.agda │ ├── SpaceShipSimpleVar.agda │ ├── StackBisim.agda │ ├── StateDependentIO.agda │ ├── StatefulObject.agda │ ├── VariableList.agda │ ├── VariableListForDispatchOnly.agda │ ├── WxGraphicsLib.agda │ ├── agdaCodeBrady.agda │ ├── exampleFinFun.agda │ ├── finn.agda │ ├── loadAllOOAgdaFilesAsInLibrary.agda │ ├── loadAllOOAgdaPart1.agda │ ├── loadAllOOAgdaPart2.agda │ ├── safeFibStackMachineObjectOriented.agda │ └── triangleRightOperator.agda ├── java │ ├── Cell.java │ ├── CounterCell.java │ ├── Makefile │ ├── Parrot.java │ ├── SelfRefExample.java │ ├── SimpleCell.java │ ├── Stack │ │ ├── README │ │ ├── Stack.java │ │ └── StackLinkedList.java │ └── StatsCell.java └── ooAgdaExamples.agda-lib ├── presentationsAndExampleCode └── agdaImplementorsMeetingGlasgow22April2016AntonSetzer │ ├── NativeIOSafe.agda │ ├── StateSized │ └── GUI │ │ └── ship.ico │ ├── drawingProgram.agda │ ├── interactiveProgramsAgda.agda │ ├── interactiveProgramsAgda.old.agda │ ├── interactiveProgramsAgdaUnsized.agda │ ├── interfaceExtensionAndDelegation.agda │ ├── main.agda │ ├── objectOrientedGui.agda │ ├── objectsInAgda.agda │ ├── objectsInAgdaUnsized.agda │ ├── ship.ico │ ├── spaceShipAdvanced.agda │ ├── spaceShipCell.agda │ ├── spaceShipSimpleVar.agda │ ├── stateDependentIO.agda │ ├── stateDependentObjects.agda │ └── talkGlasgow.agda-lib └── src ├── ConsoleLib.agda ├── NativeIO.agda ├── NativeInt.agda ├── NativePolyIO.agda ├── SizedIO ├── Base.agda ├── Console.agda ├── ConsoleObject.agda ├── IOGraphicsLib.agda ├── IOObject.agda ├── Object.agda ├── coIOIO.agda └── coIOIOObject.agda ├── SizedPolyIO ├── Base.agda ├── Console.agda ├── ConsoleObject.agda ├── IOObject.agda └── Object.agda ├── StateSizedIO ├── Base.agda ├── Base.agda.README.txt ├── GUI │ ├── BaseStateDependent.agda │ ├── VariableList.agda │ ├── WxBindingsFFI.agda │ └── WxGraphicsLib.agda ├── IOObject.agda └── Object.agda ├── UnSizedIO ├── Base.agda ├── Console.agda ├── ConsoleObject.agda ├── IOObject.agda └── Object.agda ├── Unit.agda ├── lib ├── libraryDec.agda └── libraryString.agda └── ooAgda.agda-lib /.gitignore: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/.gitignore -------------------------------------------------------------------------------- /INSTALL.txt: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/INSTALL.txt -------------------------------------------------------------------------------- /LICENSE: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/LICENSE -------------------------------------------------------------------------------- /README.md: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/README.md -------------------------------------------------------------------------------- /READMEconsolePrograms.txt: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/READMEconsolePrograms.txt -------------------------------------------------------------------------------- /docs/Agda.Builtin.Bool.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Agda.Builtin.Bool.html -------------------------------------------------------------------------------- /docs/Agda.Builtin.Char.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Agda.Builtin.Char.html -------------------------------------------------------------------------------- /docs/Agda.Builtin.Coinduction.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Agda.Builtin.Coinduction.html -------------------------------------------------------------------------------- /docs/Agda.Builtin.Equality.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Agda.Builtin.Equality.html -------------------------------------------------------------------------------- /docs/Agda.Builtin.List.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Agda.Builtin.List.html -------------------------------------------------------------------------------- /docs/Agda.Builtin.Nat.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Agda.Builtin.Nat.html -------------------------------------------------------------------------------- /docs/Agda.Builtin.Size.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Agda.Builtin.Size.html -------------------------------------------------------------------------------- /docs/Agda.Builtin.String.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Agda.Builtin.String.html -------------------------------------------------------------------------------- /docs/Agda.Builtin.TrustMe.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Agda.Builtin.TrustMe.html -------------------------------------------------------------------------------- /docs/Agda.Builtin.Unit.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Agda.Builtin.Unit.html -------------------------------------------------------------------------------- /docs/Agda.Primitive.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Agda.Primitive.html -------------------------------------------------------------------------------- /docs/Agda.css: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Agda.css -------------------------------------------------------------------------------- /docs/Algebra.FunctionProperties.Core.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Algebra.FunctionProperties.Core.html -------------------------------------------------------------------------------- /docs/Algebra.FunctionProperties.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Algebra.FunctionProperties.html -------------------------------------------------------------------------------- /docs/Algebra.Morphism.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Algebra.Morphism.html -------------------------------------------------------------------------------- /docs/Algebra.Operations.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Algebra.Operations.html -------------------------------------------------------------------------------- /docs/Algebra.Properties.AbelianGroup.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Algebra.Properties.AbelianGroup.html -------------------------------------------------------------------------------- /docs/Algebra.Properties.BooleanAlgebra.Expression.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Algebra.Properties.BooleanAlgebra.Expression.html -------------------------------------------------------------------------------- /docs/Algebra.Properties.BooleanAlgebra.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Algebra.Properties.BooleanAlgebra.html -------------------------------------------------------------------------------- /docs/Algebra.Properties.DistributiveLattice.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Algebra.Properties.DistributiveLattice.html -------------------------------------------------------------------------------- /docs/Algebra.Properties.Group.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Algebra.Properties.Group.html -------------------------------------------------------------------------------- /docs/Algebra.Properties.Lattice.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Algebra.Properties.Lattice.html -------------------------------------------------------------------------------- /docs/Algebra.Properties.Ring.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Algebra.Properties.Ring.html -------------------------------------------------------------------------------- /docs/Algebra.RingSolver.AlmostCommutativeRing.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Algebra.RingSolver.AlmostCommutativeRing.html -------------------------------------------------------------------------------- /docs/Algebra.RingSolver.Lemmas.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Algebra.RingSolver.Lemmas.html -------------------------------------------------------------------------------- /docs/Algebra.RingSolver.Simple.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Algebra.RingSolver.Simple.html -------------------------------------------------------------------------------- /docs/Algebra.RingSolver.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Algebra.RingSolver.html -------------------------------------------------------------------------------- /docs/Algebra.Structures.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Algebra.Structures.html -------------------------------------------------------------------------------- /docs/Algebra.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Algebra.html -------------------------------------------------------------------------------- /docs/Category.Applicative.Indexed.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Category.Applicative.Indexed.html -------------------------------------------------------------------------------- /docs/Category.Applicative.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Category.Applicative.html -------------------------------------------------------------------------------- /docs/Category.Functor.Identity.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Category.Functor.Identity.html -------------------------------------------------------------------------------- /docs/Category.Functor.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Category.Functor.html -------------------------------------------------------------------------------- /docs/Category.Monad.Identity.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Category.Monad.Identity.html -------------------------------------------------------------------------------- /docs/Category.Monad.Indexed.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Category.Monad.Indexed.html -------------------------------------------------------------------------------- /docs/Category.Monad.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Category.Monad.html -------------------------------------------------------------------------------- /docs/Coinduction.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Coinduction.html -------------------------------------------------------------------------------- /docs/Data.Bool.Base.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Data.Bool.Base.html -------------------------------------------------------------------------------- /docs/Data.Bool.Properties.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Data.Bool.Properties.html -------------------------------------------------------------------------------- /docs/Data.Bool.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Data.Bool.html -------------------------------------------------------------------------------- /docs/Data.BoundedVec.Inefficient.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Data.BoundedVec.Inefficient.html -------------------------------------------------------------------------------- /docs/Data.Char.Base.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Data.Char.Base.html -------------------------------------------------------------------------------- /docs/Data.Char.Core.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Data.Char.Core.html -------------------------------------------------------------------------------- /docs/Data.Char.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Data.Char.html -------------------------------------------------------------------------------- /docs/Data.Colist.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Data.Colist.html -------------------------------------------------------------------------------- /docs/Data.Conat.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Data.Conat.html -------------------------------------------------------------------------------- /docs/Data.Empty.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Data.Empty.html -------------------------------------------------------------------------------- /docs/Data.Fin.Dec.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Data.Fin.Dec.html -------------------------------------------------------------------------------- /docs/Data.Fin.Properties.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Data.Fin.Properties.html -------------------------------------------------------------------------------- /docs/Data.Fin.Subset.Properties.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Data.Fin.Subset.Properties.html -------------------------------------------------------------------------------- /docs/Data.Fin.Subset.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Data.Fin.Subset.html -------------------------------------------------------------------------------- /docs/Data.Fin.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Data.Fin.html -------------------------------------------------------------------------------- /docs/Data.List.Any.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Data.List.Any.html -------------------------------------------------------------------------------- /docs/Data.List.Base.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Data.List.Base.html -------------------------------------------------------------------------------- /docs/Data.List.NonEmpty.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Data.List.NonEmpty.html -------------------------------------------------------------------------------- /docs/Data.List.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Data.List.html -------------------------------------------------------------------------------- /docs/Data.Maybe.Base.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Data.Maybe.Base.html -------------------------------------------------------------------------------- /docs/Data.Maybe.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Data.Maybe.html -------------------------------------------------------------------------------- /docs/Data.Nat.Base.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Data.Nat.Base.html -------------------------------------------------------------------------------- /docs/Data.Nat.Properties.Simple.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Data.Nat.Properties.Simple.html -------------------------------------------------------------------------------- /docs/Data.Nat.Properties.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Data.Nat.Properties.html -------------------------------------------------------------------------------- /docs/Data.Nat.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Data.Nat.html -------------------------------------------------------------------------------- /docs/Data.Plus.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Data.Plus.html -------------------------------------------------------------------------------- /docs/Data.Product.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Data.Product.html -------------------------------------------------------------------------------- /docs/Data.String.Base.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Data.String.Base.html -------------------------------------------------------------------------------- /docs/Data.String.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Data.String.html -------------------------------------------------------------------------------- /docs/Data.Sum.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Data.Sum.html -------------------------------------------------------------------------------- /docs/Data.Unit.Base.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Data.Unit.Base.html -------------------------------------------------------------------------------- /docs/Data.Unit.NonEta.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Data.Unit.NonEta.html -------------------------------------------------------------------------------- /docs/Data.Unit.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Data.Unit.html -------------------------------------------------------------------------------- /docs/Data.Vec.Equality.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Data.Vec.Equality.html -------------------------------------------------------------------------------- /docs/Data.Vec.N-ary.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Data.Vec.N-ary.html -------------------------------------------------------------------------------- /docs/Data.Vec.Properties.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Data.Vec.Properties.html -------------------------------------------------------------------------------- /docs/Data.Vec.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Data.Vec.html -------------------------------------------------------------------------------- /docs/Function.Bijection.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Function.Bijection.html -------------------------------------------------------------------------------- /docs/Function.Equality.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Function.Equality.html -------------------------------------------------------------------------------- /docs/Function.Equivalence.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Function.Equivalence.html -------------------------------------------------------------------------------- /docs/Function.Injection.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Function.Injection.html -------------------------------------------------------------------------------- /docs/Function.Inverse.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Function.Inverse.html -------------------------------------------------------------------------------- /docs/Function.LeftInverse.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Function.LeftInverse.html -------------------------------------------------------------------------------- /docs/Function.Related.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Function.Related.html -------------------------------------------------------------------------------- /docs/Function.Surjection.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Function.Surjection.html -------------------------------------------------------------------------------- /docs/Function.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Function.html -------------------------------------------------------------------------------- /docs/Level.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Level.html -------------------------------------------------------------------------------- /docs/NativeIO.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/NativeIO.html -------------------------------------------------------------------------------- /docs/Relation.Binary.Consequences.Core.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Relation.Binary.Consequences.Core.html -------------------------------------------------------------------------------- /docs/Relation.Binary.Consequences.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Relation.Binary.Consequences.html -------------------------------------------------------------------------------- /docs/Relation.Binary.Core.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Relation.Binary.Core.html -------------------------------------------------------------------------------- /docs/Relation.Binary.EqReasoning.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Relation.Binary.EqReasoning.html -------------------------------------------------------------------------------- /docs/Relation.Binary.HeterogeneousEquality.Core.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Relation.Binary.HeterogeneousEquality.Core.html -------------------------------------------------------------------------------- /docs/Relation.Binary.HeterogeneousEquality.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Relation.Binary.HeterogeneousEquality.html -------------------------------------------------------------------------------- /docs/Relation.Binary.Indexed.Core.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Relation.Binary.Indexed.Core.html -------------------------------------------------------------------------------- /docs/Relation.Binary.Indexed.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Relation.Binary.Indexed.html -------------------------------------------------------------------------------- /docs/Relation.Binary.InducedPreorders.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Relation.Binary.InducedPreorders.html -------------------------------------------------------------------------------- /docs/Relation.Binary.Lattice.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Relation.Binary.Lattice.html -------------------------------------------------------------------------------- /docs/Relation.Binary.List.Pointwise.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Relation.Binary.List.Pointwise.html -------------------------------------------------------------------------------- /docs/Relation.Binary.List.StrictLex.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Relation.Binary.List.StrictLex.html -------------------------------------------------------------------------------- /docs/Relation.Binary.On.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Relation.Binary.On.html -------------------------------------------------------------------------------- /docs/Relation.Binary.PartialOrderReasoning.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Relation.Binary.PartialOrderReasoning.html -------------------------------------------------------------------------------- /docs/Relation.Binary.PreorderReasoning.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Relation.Binary.PreorderReasoning.html -------------------------------------------------------------------------------- /docs/Relation.Binary.PropositionalEquality.Core.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Relation.Binary.PropositionalEquality.Core.html -------------------------------------------------------------------------------- /docs/Relation.Binary.PropositionalEquality.TrustMe.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Relation.Binary.PropositionalEquality.TrustMe.html -------------------------------------------------------------------------------- /docs/Relation.Binary.PropositionalEquality.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Relation.Binary.PropositionalEquality.html -------------------------------------------------------------------------------- /docs/Relation.Binary.Reflection.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Relation.Binary.Reflection.html -------------------------------------------------------------------------------- /docs/Relation.Binary.Vec.Pointwise.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Relation.Binary.Vec.Pointwise.html -------------------------------------------------------------------------------- /docs/Relation.Binary.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Relation.Binary.html -------------------------------------------------------------------------------- /docs/Relation.Nullary.Decidable.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Relation.Nullary.Decidable.html -------------------------------------------------------------------------------- /docs/Relation.Nullary.Negation.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Relation.Nullary.Negation.html -------------------------------------------------------------------------------- /docs/Relation.Nullary.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Relation.Nullary.html -------------------------------------------------------------------------------- /docs/Relation.Unary.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Relation.Unary.html -------------------------------------------------------------------------------- /docs/Size.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Size.html -------------------------------------------------------------------------------- /docs/SizedIO.Base.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/SizedIO.Base.html -------------------------------------------------------------------------------- /docs/SizedIO.Console.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/SizedIO.Console.html -------------------------------------------------------------------------------- /docs/SizedIO.Object.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/SizedIO.Object.html -------------------------------------------------------------------------------- /docs/StateSizedIO.Base.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/StateSizedIO.Base.html -------------------------------------------------------------------------------- /docs/StateSizedIO.IOObject.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/StateSizedIO.IOObject.html -------------------------------------------------------------------------------- /docs/StateSizedIO.Object.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/StateSizedIO.Object.html -------------------------------------------------------------------------------- /docs/StateSizedIO.RObject.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/StateSizedIO.RObject.html -------------------------------------------------------------------------------- /docs/StateSizedIO.cellStateDependent.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/StateSizedIO.cellStateDependent.html -------------------------------------------------------------------------------- /docs/StateSizedIO.writingOOsUsingIO.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/StateSizedIO.writingOOsUsingIO.html -------------------------------------------------------------------------------- /docs/StateSizedIO.writingOOsUsingIOVers4ReaderMethods.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/StateSizedIO.writingOOsUsingIOVers4ReaderMethods.html -------------------------------------------------------------------------------- /docs/Unit.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/Unit.html -------------------------------------------------------------------------------- /docs/examples.heap.ALL.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/examples.heap.ALL.html -------------------------------------------------------------------------------- /docs/examples.heap.correctnessLinkedList.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/examples.heap.correctnessLinkedList.html -------------------------------------------------------------------------------- /docs/examples.heap.correctnessLinkedListStep2.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/examples.heap.correctnessLinkedListStep2.html -------------------------------------------------------------------------------- /docs/heap.library.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/heap.library.html -------------------------------------------------------------------------------- /docs/heap.libraryBool.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/heap.libraryBool.html -------------------------------------------------------------------------------- /docs/heap.libraryFin.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/heap.libraryFin.html -------------------------------------------------------------------------------- /docs/heap.libraryMaybe.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/heap.libraryMaybe.html -------------------------------------------------------------------------------- /docs/heap.libraryNat.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/heap.libraryNat.html -------------------------------------------------------------------------------- /docs/src.heap.heapAsObject.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/src.heap.heapAsObject.html -------------------------------------------------------------------------------- /docs/src.heap.heapAsObjectBase.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/src.heap.heapAsObjectBase.html -------------------------------------------------------------------------------- /docs/src.heap.heapAsObjectExample.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/src.heap.heapAsObjectExample.html -------------------------------------------------------------------------------- /docs/src.heap.heapAsObjectGeneric.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/src.heap.heapAsObjectGeneric.html -------------------------------------------------------------------------------- /docs/src.heap.heapAsObjectNativeHeap.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/src.heap.heapAsObjectNativeHeap.html -------------------------------------------------------------------------------- /docs/src.heap.worldModule.html: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/docs/src.heap.worldModule.html -------------------------------------------------------------------------------- /exampleCode/helloWorld.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/exampleCode/helloWorld.agda -------------------------------------------------------------------------------- /exampleCode/myExample.agda-lib: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/exampleCode/myExample.agda-lib -------------------------------------------------------------------------------- /examples/DrawingProgram/IOExampleGraphicsDrawingProgram.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/examples/DrawingProgram/IOExampleGraphicsDrawingProgram.agda -------------------------------------------------------------------------------- /examples/DrawingProgram/IOExampleGraphicsDrawingProgramWhenJust.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/examples/DrawingProgram/IOExampleGraphicsDrawingProgramWhenJust.agda -------------------------------------------------------------------------------- /examples/DrawingProgram/IOExampleGraphicsMovingText.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/examples/DrawingProgram/IOExampleGraphicsMovingText.agda -------------------------------------------------------------------------------- /examples/DrawingProgram/Main.agda-lib: -------------------------------------------------------------------------------- 1 | name: Main 2 | depend: std-lib ionew 3 | include: . 4 | -------------------------------------------------------------------------------- /examples/Sized/ConsoleExample.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/examples/Sized/ConsoleExample.agda -------------------------------------------------------------------------------- /examples/Sized/CounterCell.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/examples/Sized/CounterCell.agda -------------------------------------------------------------------------------- /examples/Sized/Parrot.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/examples/Sized/Parrot.agda -------------------------------------------------------------------------------- /examples/Sized/SelfRef.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/examples/Sized/SelfRef.agda -------------------------------------------------------------------------------- /examples/Sized/SimpleCell.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/examples/Sized/SimpleCell.agda -------------------------------------------------------------------------------- /examples/Sized/StatefulCell.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/examples/Sized/StatefulCell.agda -------------------------------------------------------------------------------- /examples/SizedPoly/Console.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/examples/SizedPoly/Console.agda -------------------------------------------------------------------------------- /examples/SizedPoly/SimpleCell.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/examples/SizedPoly/SimpleCell.agda -------------------------------------------------------------------------------- /examples/StateSized/GUI/BitMaps.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/examples/StateSized/GUI/BitMaps.agda -------------------------------------------------------------------------------- /examples/StateSized/GUI/ShipBitMap.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/examples/StateSized/GUI/ShipBitMap.agda -------------------------------------------------------------------------------- /examples/StateSized/GUI/SpaceShipAdvanced.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/examples/StateSized/GUI/SpaceShipAdvanced.agda -------------------------------------------------------------------------------- /examples/StateSized/GUI/SpaceShipCell.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/examples/StateSized/GUI/SpaceShipCell.agda -------------------------------------------------------------------------------- /examples/StateSized/GUI/SpaceShipExtendedExample.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/examples/StateSized/GUI/SpaceShipExtendedExample.agda -------------------------------------------------------------------------------- /examples/StateSized/GUI/SpaceShipSimpleVar.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/examples/StateSized/GUI/SpaceShipSimpleVar.agda -------------------------------------------------------------------------------- /examples/StateSized/GUI/ship.ico: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/examples/StateSized/GUI/ship.ico -------------------------------------------------------------------------------- /examples/StateSized/StackStateDependent.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/examples/StateSized/StackStateDependent.agda -------------------------------------------------------------------------------- /examples/StateSized/cellStateDependent.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/examples/StateSized/cellStateDependent.agda -------------------------------------------------------------------------------- /examples/UnSized/Console.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/examples/UnSized/Console.agda -------------------------------------------------------------------------------- /examples/UnSized/Parrot.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/examples/UnSized/Parrot.agda -------------------------------------------------------------------------------- /examples/UnSized/SelfRef.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/examples/UnSized/SelfRef.agda -------------------------------------------------------------------------------- /examples/UnSized/SimpleCell.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/examples/UnSized/SimpleCell.agda -------------------------------------------------------------------------------- /examples/consoleExamples/helloWorld.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/examples/consoleExamples/helloWorld.agda -------------------------------------------------------------------------------- /examples/consoleExamples/passwordCheckSimple.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/examples/consoleExamples/passwordCheckSimple.agda -------------------------------------------------------------------------------- /examples/consoleExamples/simpleLoop.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/examples/consoleExamples/simpleLoop.agda -------------------------------------------------------------------------------- /examples/examplesPaperJFP/BasicIO.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/examples/examplesPaperJFP/BasicIO.agda -------------------------------------------------------------------------------- /examples/examplesPaperJFP/CatNonTerm.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/examples/examplesPaperJFP/CatNonTerm.agda -------------------------------------------------------------------------------- /examples/examplesPaperJFP/CatTerm.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/examples/examplesPaperJFP/CatTerm.agda -------------------------------------------------------------------------------- /examples/examplesPaperJFP/Coalgebra.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/examples/examplesPaperJFP/Coalgebra.agda -------------------------------------------------------------------------------- /examples/examplesPaperJFP/Colists.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/examples/examplesPaperJFP/Colists.agda -------------------------------------------------------------------------------- /examples/examplesPaperJFP/Collatz.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/examples/examplesPaperJFP/Collatz.agda -------------------------------------------------------------------------------- /examples/examplesPaperJFP/Console.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/examples/examplesPaperJFP/Console.agda -------------------------------------------------------------------------------- /examples/examplesPaperJFP/ConsoleInterface.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/examples/examplesPaperJFP/ConsoleInterface.agda -------------------------------------------------------------------------------- /examples/examplesPaperJFP/CounterCell.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/examples/examplesPaperJFP/CounterCell.agda -------------------------------------------------------------------------------- /examples/examplesPaperJFP/Equality.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/examples/examplesPaperJFP/Equality.agda -------------------------------------------------------------------------------- /examples/examplesPaperJFP/ExampleDrawingProgram.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/examples/examplesPaperJFP/ExampleDrawingProgram.agda -------------------------------------------------------------------------------- /examples/examplesPaperJFP/IOExampleConsole.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/examples/examplesPaperJFP/IOExampleConsole.agda -------------------------------------------------------------------------------- /examples/examplesPaperJFP/IOGraphicsLib.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/examples/examplesPaperJFP/IOGraphicsLib.agda -------------------------------------------------------------------------------- /examples/examplesPaperJFP/NativeIOSafe.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/examples/examplesPaperJFP/NativeIOSafe.agda -------------------------------------------------------------------------------- /examples/examplesPaperJFP/Object.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/examples/examplesPaperJFP/Object.agda -------------------------------------------------------------------------------- /examples/examplesPaperJFP/Sized.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/examples/examplesPaperJFP/Sized.agda -------------------------------------------------------------------------------- /examples/examplesPaperJFP/SpaceShipAdvanced.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/examples/examplesPaperJFP/SpaceShipAdvanced.agda -------------------------------------------------------------------------------- /examples/examplesPaperJFP/SpaceShipCell.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/examples/examplesPaperJFP/SpaceShipCell.agda -------------------------------------------------------------------------------- /examples/examplesPaperJFP/SpaceShipSimpleVar.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/examples/examplesPaperJFP/SpaceShipSimpleVar.agda -------------------------------------------------------------------------------- /examples/examplesPaperJFP/StackBisim.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/examples/examplesPaperJFP/StackBisim.agda -------------------------------------------------------------------------------- /examples/examplesPaperJFP/StateDependentIO.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/examples/examplesPaperJFP/StateDependentIO.agda -------------------------------------------------------------------------------- /examples/examplesPaperJFP/StatefulObject.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/examples/examplesPaperJFP/StatefulObject.agda -------------------------------------------------------------------------------- /examples/examplesPaperJFP/VariableList.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/examples/examplesPaperJFP/VariableList.agda -------------------------------------------------------------------------------- /examples/examplesPaperJFP/VariableListForDispatchOnly.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/examples/examplesPaperJFP/VariableListForDispatchOnly.agda -------------------------------------------------------------------------------- /examples/examplesPaperJFP/WxGraphicsLib.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/examples/examplesPaperJFP/WxGraphicsLib.agda -------------------------------------------------------------------------------- /examples/examplesPaperJFP/agdaCodeBrady.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/examples/examplesPaperJFP/agdaCodeBrady.agda -------------------------------------------------------------------------------- /examples/examplesPaperJFP/exampleFinFun.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/examples/examplesPaperJFP/exampleFinFun.agda -------------------------------------------------------------------------------- /examples/examplesPaperJFP/finn.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/examples/examplesPaperJFP/finn.agda -------------------------------------------------------------------------------- /examples/examplesPaperJFP/loadAllOOAgdaFilesAsInLibrary.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/examples/examplesPaperJFP/loadAllOOAgdaFilesAsInLibrary.agda -------------------------------------------------------------------------------- /examples/examplesPaperJFP/loadAllOOAgdaPart1.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/examples/examplesPaperJFP/loadAllOOAgdaPart1.agda -------------------------------------------------------------------------------- /examples/examplesPaperJFP/loadAllOOAgdaPart2.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/examples/examplesPaperJFP/loadAllOOAgdaPart2.agda -------------------------------------------------------------------------------- /examples/examplesPaperJFP/safeFibStackMachineObjectOriented.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/examples/examplesPaperJFP/safeFibStackMachineObjectOriented.agda -------------------------------------------------------------------------------- /examples/examplesPaperJFP/triangleRightOperator.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/examples/examplesPaperJFP/triangleRightOperator.agda -------------------------------------------------------------------------------- /examples/java/Cell.java: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/examples/java/Cell.java -------------------------------------------------------------------------------- /examples/java/CounterCell.java: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/examples/java/CounterCell.java -------------------------------------------------------------------------------- /examples/java/Makefile: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/examples/java/Makefile -------------------------------------------------------------------------------- /examples/java/Parrot.java: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/examples/java/Parrot.java -------------------------------------------------------------------------------- /examples/java/SelfRefExample.java: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/examples/java/SelfRefExample.java -------------------------------------------------------------------------------- /examples/java/SimpleCell.java: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/examples/java/SimpleCell.java -------------------------------------------------------------------------------- /examples/java/Stack/README: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/examples/java/Stack/README -------------------------------------------------------------------------------- /examples/java/Stack/Stack.java: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/examples/java/Stack/Stack.java -------------------------------------------------------------------------------- /examples/java/Stack/StackLinkedList.java: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/examples/java/Stack/StackLinkedList.java -------------------------------------------------------------------------------- /examples/java/StatsCell.java: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/examples/java/StatsCell.java -------------------------------------------------------------------------------- /examples/ooAgdaExamples.agda-lib: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/examples/ooAgdaExamples.agda-lib -------------------------------------------------------------------------------- /presentationsAndExampleCode/agdaImplementorsMeetingGlasgow22April2016AntonSetzer/NativeIOSafe.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/presentationsAndExampleCode/agdaImplementorsMeetingGlasgow22April2016AntonSetzer/NativeIOSafe.agda -------------------------------------------------------------------------------- /presentationsAndExampleCode/agdaImplementorsMeetingGlasgow22April2016AntonSetzer/StateSized/GUI/ship.ico: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/presentationsAndExampleCode/agdaImplementorsMeetingGlasgow22April2016AntonSetzer/StateSized/GUI/ship.ico -------------------------------------------------------------------------------- /presentationsAndExampleCode/agdaImplementorsMeetingGlasgow22April2016AntonSetzer/drawingProgram.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/presentationsAndExampleCode/agdaImplementorsMeetingGlasgow22April2016AntonSetzer/drawingProgram.agda -------------------------------------------------------------------------------- /presentationsAndExampleCode/agdaImplementorsMeetingGlasgow22April2016AntonSetzer/interactiveProgramsAgda.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/presentationsAndExampleCode/agdaImplementorsMeetingGlasgow22April2016AntonSetzer/interactiveProgramsAgda.agda -------------------------------------------------------------------------------- /presentationsAndExampleCode/agdaImplementorsMeetingGlasgow22April2016AntonSetzer/interactiveProgramsAgda.old.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/presentationsAndExampleCode/agdaImplementorsMeetingGlasgow22April2016AntonSetzer/interactiveProgramsAgda.old.agda -------------------------------------------------------------------------------- /presentationsAndExampleCode/agdaImplementorsMeetingGlasgow22April2016AntonSetzer/interactiveProgramsAgdaUnsized.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/presentationsAndExampleCode/agdaImplementorsMeetingGlasgow22April2016AntonSetzer/interactiveProgramsAgdaUnsized.agda -------------------------------------------------------------------------------- /presentationsAndExampleCode/agdaImplementorsMeetingGlasgow22April2016AntonSetzer/interfaceExtensionAndDelegation.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/presentationsAndExampleCode/agdaImplementorsMeetingGlasgow22April2016AntonSetzer/interfaceExtensionAndDelegation.agda -------------------------------------------------------------------------------- /presentationsAndExampleCode/agdaImplementorsMeetingGlasgow22April2016AntonSetzer/main.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/presentationsAndExampleCode/agdaImplementorsMeetingGlasgow22April2016AntonSetzer/main.agda -------------------------------------------------------------------------------- /presentationsAndExampleCode/agdaImplementorsMeetingGlasgow22April2016AntonSetzer/objectOrientedGui.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/presentationsAndExampleCode/agdaImplementorsMeetingGlasgow22April2016AntonSetzer/objectOrientedGui.agda -------------------------------------------------------------------------------- /presentationsAndExampleCode/agdaImplementorsMeetingGlasgow22April2016AntonSetzer/objectsInAgda.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/presentationsAndExampleCode/agdaImplementorsMeetingGlasgow22April2016AntonSetzer/objectsInAgda.agda -------------------------------------------------------------------------------- /presentationsAndExampleCode/agdaImplementorsMeetingGlasgow22April2016AntonSetzer/objectsInAgdaUnsized.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/presentationsAndExampleCode/agdaImplementorsMeetingGlasgow22April2016AntonSetzer/objectsInAgdaUnsized.agda -------------------------------------------------------------------------------- /presentationsAndExampleCode/agdaImplementorsMeetingGlasgow22April2016AntonSetzer/ship.ico: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/presentationsAndExampleCode/agdaImplementorsMeetingGlasgow22April2016AntonSetzer/ship.ico -------------------------------------------------------------------------------- /presentationsAndExampleCode/agdaImplementorsMeetingGlasgow22April2016AntonSetzer/spaceShipAdvanced.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/presentationsAndExampleCode/agdaImplementorsMeetingGlasgow22April2016AntonSetzer/spaceShipAdvanced.agda -------------------------------------------------------------------------------- /presentationsAndExampleCode/agdaImplementorsMeetingGlasgow22April2016AntonSetzer/spaceShipCell.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/presentationsAndExampleCode/agdaImplementorsMeetingGlasgow22April2016AntonSetzer/spaceShipCell.agda -------------------------------------------------------------------------------- /presentationsAndExampleCode/agdaImplementorsMeetingGlasgow22April2016AntonSetzer/spaceShipSimpleVar.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/presentationsAndExampleCode/agdaImplementorsMeetingGlasgow22April2016AntonSetzer/spaceShipSimpleVar.agda -------------------------------------------------------------------------------- /presentationsAndExampleCode/agdaImplementorsMeetingGlasgow22April2016AntonSetzer/stateDependentIO.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/presentationsAndExampleCode/agdaImplementorsMeetingGlasgow22April2016AntonSetzer/stateDependentIO.agda -------------------------------------------------------------------------------- /presentationsAndExampleCode/agdaImplementorsMeetingGlasgow22April2016AntonSetzer/stateDependentObjects.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/presentationsAndExampleCode/agdaImplementorsMeetingGlasgow22April2016AntonSetzer/stateDependentObjects.agda -------------------------------------------------------------------------------- /presentationsAndExampleCode/agdaImplementorsMeetingGlasgow22April2016AntonSetzer/talkGlasgow.agda-lib: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/presentationsAndExampleCode/agdaImplementorsMeetingGlasgow22April2016AntonSetzer/talkGlasgow.agda-lib -------------------------------------------------------------------------------- /src/ConsoleLib.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/src/ConsoleLib.agda -------------------------------------------------------------------------------- /src/NativeIO.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/src/NativeIO.agda -------------------------------------------------------------------------------- /src/NativeInt.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/src/NativeInt.agda -------------------------------------------------------------------------------- /src/NativePolyIO.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/src/NativePolyIO.agda -------------------------------------------------------------------------------- /src/SizedIO/Base.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/src/SizedIO/Base.agda -------------------------------------------------------------------------------- /src/SizedIO/Console.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/src/SizedIO/Console.agda -------------------------------------------------------------------------------- /src/SizedIO/ConsoleObject.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/src/SizedIO/ConsoleObject.agda -------------------------------------------------------------------------------- /src/SizedIO/IOGraphicsLib.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/src/SizedIO/IOGraphicsLib.agda -------------------------------------------------------------------------------- /src/SizedIO/IOObject.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/src/SizedIO/IOObject.agda -------------------------------------------------------------------------------- /src/SizedIO/Object.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/src/SizedIO/Object.agda -------------------------------------------------------------------------------- /src/SizedIO/coIOIO.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/src/SizedIO/coIOIO.agda -------------------------------------------------------------------------------- /src/SizedIO/coIOIOObject.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/src/SizedIO/coIOIOObject.agda -------------------------------------------------------------------------------- /src/SizedPolyIO/Base.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/src/SizedPolyIO/Base.agda -------------------------------------------------------------------------------- /src/SizedPolyIO/Console.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/src/SizedPolyIO/Console.agda -------------------------------------------------------------------------------- /src/SizedPolyIO/ConsoleObject.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/src/SizedPolyIO/ConsoleObject.agda -------------------------------------------------------------------------------- /src/SizedPolyIO/IOObject.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/src/SizedPolyIO/IOObject.agda -------------------------------------------------------------------------------- /src/SizedPolyIO/Object.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/src/SizedPolyIO/Object.agda -------------------------------------------------------------------------------- /src/StateSizedIO/Base.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/src/StateSizedIO/Base.agda -------------------------------------------------------------------------------- /src/StateSizedIO/Base.agda.README.txt: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/src/StateSizedIO/Base.agda.README.txt -------------------------------------------------------------------------------- /src/StateSizedIO/GUI/BaseStateDependent.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/src/StateSizedIO/GUI/BaseStateDependent.agda -------------------------------------------------------------------------------- /src/StateSizedIO/GUI/VariableList.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/src/StateSizedIO/GUI/VariableList.agda -------------------------------------------------------------------------------- /src/StateSizedIO/GUI/WxBindingsFFI.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/src/StateSizedIO/GUI/WxBindingsFFI.agda -------------------------------------------------------------------------------- /src/StateSizedIO/GUI/WxGraphicsLib.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/src/StateSizedIO/GUI/WxGraphicsLib.agda -------------------------------------------------------------------------------- /src/StateSizedIO/IOObject.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/src/StateSizedIO/IOObject.agda -------------------------------------------------------------------------------- /src/StateSizedIO/Object.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/src/StateSizedIO/Object.agda -------------------------------------------------------------------------------- /src/UnSizedIO/Base.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/src/UnSizedIO/Base.agda -------------------------------------------------------------------------------- /src/UnSizedIO/Console.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/src/UnSizedIO/Console.agda -------------------------------------------------------------------------------- /src/UnSizedIO/ConsoleObject.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/src/UnSizedIO/ConsoleObject.agda -------------------------------------------------------------------------------- /src/UnSizedIO/IOObject.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/src/UnSizedIO/IOObject.agda -------------------------------------------------------------------------------- /src/UnSizedIO/Object.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/src/UnSizedIO/Object.agda -------------------------------------------------------------------------------- /src/Unit.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/src/Unit.agda -------------------------------------------------------------------------------- /src/lib/libraryDec.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/src/lib/libraryDec.agda -------------------------------------------------------------------------------- /src/lib/libraryString.agda: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/src/lib/libraryString.agda -------------------------------------------------------------------------------- /src/ooAgda.agda-lib: -------------------------------------------------------------------------------- https://raw.githubusercontent.com/agda/ooAgda/HEAD/src/ooAgda.agda-lib --------------------------------------------------------------------------------