Skip to content

Commit

Permalink
Merge pull request #4190 from jfdm/fix-haddock-copyright
Browse files Browse the repository at this point in the history
Remove the empty haddock property 'copyright'.
  • Loading branch information
jfdm authored Nov 10, 2017
2 parents a4258cd + 3ccb494 commit f92ecd2
Show file tree
Hide file tree
Showing 102 changed files with 102 additions and 102 deletions.
2 changes: 1 addition & 1 deletion src/IRTS/Bytecode.hs
Original file line number Diff line number Diff line change
Expand Up @@ -2,7 +2,7 @@
Module : IRTS.Bytecode
Description : Bytecode for a stack based VM (e.g. for generating C code with an accurate hand written GC)
Copyright :
License : BSD3
Maintainer : The Idris Community.
Expand Down
2 changes: 1 addition & 1 deletion src/IRTS/CodegenC.hs
Original file line number Diff line number Diff line change
@@ -1,7 +1,7 @@
{-|
Module : IRTS.CodegenC
Description : The default code generator for Idris, generating C code.
Copyright :
License : BSD3
Maintainer : The Idris Community.
-}
Expand Down
2 changes: 1 addition & 1 deletion src/IRTS/CodegenCommon.hs
Original file line number Diff line number Diff line change
Expand Up @@ -2,7 +2,7 @@
{-|
Module : IRTS.CodegenCommon
Description : Common data structures required for all code generators.
Copyright :
License : BSD3
Maintainer : The Idris Community.
-}
Expand Down
2 changes: 1 addition & 1 deletion src/IRTS/CodegenJavaScript.hs
Original file line number Diff line number Diff line change
@@ -1,7 +1,7 @@
{-|
Module : IRTS.CodegenJavaScript
Description : The JavaScript code generator.
Copyright :
License : BSD3
Maintainer : The Idris Community.
-}
Expand Down
2 changes: 1 addition & 1 deletion src/IRTS/Compiler.hs
Original file line number Diff line number Diff line change
@@ -1,7 +1,7 @@
{-|
Module : IRTS.Compiler
Description : Coordinates the compilation process.
Copyright :
License : BSD3
Maintainer : The Idris Community.
-}
Expand Down
2 changes: 1 addition & 1 deletion src/IRTS/Defunctionalise.hs
Original file line number Diff line number Diff line change
@@ -1,7 +1,7 @@
{-|
Module : IRTS.Defunctionalise
Description : Defunctionalise Idris' IR.
Copyright :
License : BSD3
Maintainer : The Idris Community.
Expand Down
2 changes: 1 addition & 1 deletion src/IRTS/DumpBC.hs
Original file line number Diff line number Diff line change
@@ -1,7 +1,7 @@
{-|
Module : IRTS.DumpBC
Description : Serialise Idris to its IBC format.
Copyright :
License : BSD3
Maintainer : The Idris Community.
-}
Expand Down
2 changes: 1 addition & 1 deletion src/IRTS/Exports.hs
Original file line number Diff line number Diff line change
@@ -1,7 +1,7 @@
{-|
Module : IRTS.Exports
Description : Deal with external things.
Copyright :
License : BSD3
Maintainer : The Idris Community.
-}
Expand Down
2 changes: 1 addition & 1 deletion src/IRTS/Inliner.hs
Original file line number Diff line number Diff line change
@@ -1,7 +1,7 @@
{-|
Module : IRTS.Inliner
Description : Inline expressions.
Copyright :
License : BSD3
Maintainer : The Idris Community.
-}
Expand Down
2 changes: 1 addition & 1 deletion src/IRTS/JavaScript/AST.hs
Original file line number Diff line number Diff line change
@@ -1,7 +1,7 @@
{-|
Module : IRTS.JavaScript.AST
Description : The JavaScript AST.
Copyright :
License : BSD3
Maintainer : The Idris Community.
-}
Expand Down
2 changes: 1 addition & 1 deletion src/IRTS/JavaScript/Codegen.hs
Original file line number Diff line number Diff line change
@@ -1,7 +1,7 @@
{-|
Module : IRTS.JavaScript.Codegen
Description : The JavaScript common code generator.
Copyright :
License : BSD3
Maintainer : The Idris Community.
-}
Expand Down
2 changes: 1 addition & 1 deletion src/IRTS/JavaScript/LangTransforms.hs
Original file line number Diff line number Diff line change
@@ -1,7 +1,7 @@
{-|
Module : IRTS.JavaScript.LangTransforms
Description : The JavaScript LDecl Transformations.
Copyright :
License : BSD3
Maintainer : The Idris Community.
-}
Expand Down
2 changes: 1 addition & 1 deletion src/IRTS/JavaScript/Name.hs
Original file line number Diff line number Diff line change
@@ -1,7 +1,7 @@
{-|
Module : IRTS.JavaScript.Name
Description : The JavaScript name mangler.
Copyright :
License : BSD3
Maintainer : The Idris Community.
-}
Expand Down
2 changes: 1 addition & 1 deletion src/IRTS/JavaScript/PrimOp.hs
Original file line number Diff line number Diff line change
@@ -1,7 +1,7 @@
{-|
Module : IRTS.JavaScript.PrimOp
Description : The JavaScript primitive operations.
Copyright :
License : BSD3
Maintainer : The Idris Community.
-}
Expand Down
2 changes: 1 addition & 1 deletion src/IRTS/JavaScript/Specialize.hs
Original file line number Diff line number Diff line change
@@ -1,7 +1,7 @@
{-|
Module : IRTS.JavaScript.Specialize
Description : The JavaScript specializer.
Copyright :
License : BSD3
Maintainer : The Idris Community.
-}
Expand Down
2 changes: 1 addition & 1 deletion src/IRTS/Lang.hs
Original file line number Diff line number Diff line change
@@ -1,7 +1,7 @@
{-|
Module : IRTS.Lang
Description : Internal representation of Idris' constructs.
Copyright :
License : BSD3
Maintainer : The Idris Community.
-}
Expand Down
2 changes: 1 addition & 1 deletion src/IRTS/LangOpts.hs
Original file line number Diff line number Diff line change
@@ -1,7 +1,7 @@
{-|
Module : IRTS.LangOpts
Description : Transformations to apply to Idris' IR.
Copyright :
License : BSD3
Maintainer : The Idris Community.
-}
Expand Down
2 changes: 1 addition & 1 deletion src/IRTS/Portable.hs
Original file line number Diff line number Diff line change
@@ -1,7 +1,7 @@
{-|
Module : IRTS.Portable
Description : Serialise Idris' IR to JSON.
Copyright :
License : BSD3
Maintainer : The Idris Community.
-}
Expand Down
2 changes: 1 addition & 1 deletion src/IRTS/Simplified.hs
Original file line number Diff line number Diff line change
@@ -1,7 +1,7 @@
{-|
Module : IRTS.Simplified
Description : Simplified expressions, where functions/constructors can only be applied to variables.
Copyright :
License : BSD3
Maintainer : The Idris Community.
-}
Expand Down
2 changes: 1 addition & 1 deletion src/IRTS/System.hs
Original file line number Diff line number Diff line change
@@ -1,7 +1,7 @@
{-|
Module : IRTS.System
Description : Utilities for interacting with the System.
Copyright :
License : BSD3
Maintainer : The Idris Community.
-}
Expand Down
2 changes: 1 addition & 1 deletion src/Idris/ASTUtils.hs
Original file line number Diff line number Diff line change
Expand Up @@ -2,7 +2,7 @@
{-|
Module : Idris.ASTUtils
Description : This implements just a few basic lens-like concepts to ease state updates. Similar to fclabels in approach, just without the extra dependency.
Copyright :
License : BSD3
Maintainer : The Idris Community.
Expand Down
2 changes: 1 addition & 1 deletion src/Idris/AbsSyntax.hs
Original file line number Diff line number Diff line change
@@ -1,7 +1,7 @@
{-|
Module : Idris.AbsSyntax
Description : Provides Idris' core data definitions and utility code.
Copyright :
License : BSD3
Maintainer : The Idris Community.
-}
Expand Down
2 changes: 1 addition & 1 deletion src/Idris/AbsSyntaxTree.hs
Original file line number Diff line number Diff line change
@@ -1,7 +1,7 @@
{-|
Module : Idris.AbsSyntaxTree
Description : Core data definitions used in Idris.
Copyright :
License : BSD3
Maintainer : The Idris Community.
-}
Expand Down
2 changes: 1 addition & 1 deletion src/Idris/Apropos.hs
Original file line number Diff line number Diff line change
@@ -1,7 +1,7 @@
{-|
Module : Idris.Apropos
Description : Search loaded Idris code and named modules for things.
Copyright :
License : BSD3
Maintainer : The Idris Community.
-}
Expand Down
2 changes: 1 addition & 1 deletion src/Idris/CaseSplit.hs
Original file line number Diff line number Diff line change
@@ -1,7 +1,7 @@
{-|
Module : Idris.CaseSplit
Description : Module to provide case split functionality.
Copyright :
License : BSD3
Maintainer : The Idris Community.
Expand Down
2 changes: 1 addition & 1 deletion src/Idris/Chaser.hs
Original file line number Diff line number Diff line change
@@ -1,7 +1,7 @@
{-|
Module : Idris.Chaser
Description : Module chaser to determine cycles and import modules.
Copyright :
License : BSD3
Maintainer : The Idris Community.
-}
Expand Down
2 changes: 1 addition & 1 deletion src/Idris/Colours.hs
Original file line number Diff line number Diff line change
Expand Up @@ -2,7 +2,7 @@
{-|
Module : Idris.Colours
Description : Support for colours within Idris.
Copyright :
License : BSD3
Maintainer : The Idris Community.
-}
Expand Down
2 changes: 1 addition & 1 deletion src/Idris/Completion.hs
Original file line number Diff line number Diff line change
@@ -1,7 +1,7 @@
{-|
Module : Idris.Completion
Description : Support for command-line completion at the REPL and in the prover.
Copyright :
License : BSD3
Maintainer : The Idris Community.
-}
Expand Down
2 changes: 1 addition & 1 deletion src/Idris/Core/Binary.hs
Original file line number Diff line number Diff line change
@@ -1,7 +1,7 @@
{-|
Module : Idris.Core.Binary
Description : Binary instances for the core datatypes
Copyright :
License : BSD3
Maintainer : The Idris Community.
-}
Expand Down
2 changes: 1 addition & 1 deletion src/Idris/Core/CaseTree.hs
Original file line number Diff line number Diff line change
@@ -1,7 +1,7 @@
{-|
Module : Idris.Core.CaseTree
Description : Module to define and interact with case trees.
Copyright :
License : BSD3
Maintainer : The Idris Community.
Expand Down
2 changes: 1 addition & 1 deletion src/Idris/Core/Constraints.hs
Original file line number Diff line number Diff line change
Expand Up @@ -2,7 +2,7 @@
{-|
Module : Idris.Core.Constraints
Description : Check universe constraints.
Copyright :
License : BSD3
Maintainer : The Idris Community.
-}
Expand Down
2 changes: 1 addition & 1 deletion src/Idris/Core/DeepSeq.hs
Original file line number Diff line number Diff line change
@@ -1,7 +1,7 @@
{-|
Module : Idris.Core.DeepSeq
Description : NFData instances for TT.
Copyright :
License : BSD3
Maintainer : The Idris Community.
-}
Expand Down
2 changes: 1 addition & 1 deletion src/Idris/Core/Elaborate.hs
Original file line number Diff line number Diff line change
@@ -1,7 +1,7 @@
{-|
Module : Idris.Core.Elaborate
Description : A high level language of tactic composition, for building elaborators from a high level language into the core theory.
Copyright :
License : BSD3
Maintainer : The Idris Community.
Expand Down
2 changes: 1 addition & 1 deletion src/Idris/Core/Evaluate.hs
Original file line number Diff line number Diff line change
@@ -1,7 +1,7 @@
{-|
Module : Idris.Core.Evaluate
Description : Evaluate Idris expressions.
Copyright :
License : BSD3
Maintainer : The Idris Community.
-}
Expand Down
2 changes: 1 addition & 1 deletion src/Idris/Core/Execute.hs
Original file line number Diff line number Diff line change
@@ -1,7 +1,7 @@
{-|
Module : Idris.Core.Execute
Description : Execute Idris code and deal with FFI.
Copyright :
License : BSD3
Maintainer : The Idris Community.
-}
Expand Down
2 changes: 1 addition & 1 deletion src/Idris/Core/ProofState.hs
Original file line number Diff line number Diff line change
@@ -1,7 +1,7 @@
{-|
Module : Idris.Core.ProofState
Description : Proof state implementation.
Copyright :
License : BSD3
Maintainer : The Idris Community.
Expand Down
2 changes: 1 addition & 1 deletion src/Idris/Core/ProofTerm.hs
Original file line number Diff line number Diff line change
@@ -1,7 +1,7 @@
{-|
Module : Idris.Core.ProofTerm
Description : Proof term. implementation and utilities.
Copyright :
License : BSD3
Maintainer : The Idris Community.
-}
Expand Down
2 changes: 1 addition & 1 deletion src/Idris/Core/TT.hs
Original file line number Diff line number Diff line change
@@ -1,7 +1,7 @@
{-|
Module : Idris.Core.TT
Description : The core language of Idris, TT.
Copyright :
License : BSD3
Maintainer : The Idris Community.
Expand Down
2 changes: 1 addition & 1 deletion src/Idris/Core/Typecheck.hs
Original file line number Diff line number Diff line change
@@ -1,7 +1,7 @@
{-|
Module : Idris.Core.Typecheck
Description : Idris' type checker.
Copyright :
License : BSD3
Maintainer : The Idris Community.
-}
Expand Down
2 changes: 1 addition & 1 deletion src/Idris/Core/Unify.hs
Original file line number Diff line number Diff line change
@@ -1,7 +1,7 @@
{-|
Module : Idris.Core.Unify
Description : Idris' unification code.
Copyright :
License : BSD3
Maintainer : The Idris Community.
Expand Down
2 changes: 1 addition & 1 deletion src/Idris/Core/WHNF.hs
Original file line number Diff line number Diff line change
@@ -1,7 +1,7 @@
{-|
Module : Idris.Core.WHNF
Description : Reduction to Weak Head Normal Form
Copyright :
License : BSD3
Maintainer : The Idris Community.
-}
Expand Down
2 changes: 1 addition & 1 deletion src/Idris/Coverage.hs
Original file line number Diff line number Diff line change
@@ -1,7 +1,7 @@
{-|
Module : Idris.Coverage
Description : Clause generation for coverage checking
Copyright :
License : BSD3
Maintainer : The Idris Community.
-}
Expand Down
2 changes: 1 addition & 1 deletion src/Idris/DSL.hs
Original file line number Diff line number Diff line change
@@ -1,7 +1,7 @@
{-|
Module : Idris.DSL
Description : Code to deal with DSL blocks.
Copyright :
License : BSD3
Maintainer : The Idris Community.
-}
Expand Down
2 changes: 1 addition & 1 deletion src/Idris/DataOpts.hs
Original file line number Diff line number Diff line change
@@ -1,7 +1,7 @@
{-|
Module : Idris.DataOpts
Description : Optimisations for Idris code i.e. Forcing, detagging and collapsing.
Copyright :
License : BSD3
Maintainer : The Idris Community.
-}
Expand Down
Loading

0 comments on commit f92ecd2

Please sign in to comment.