Agda
Safe HaskellNone
LanguageHaskell2010

Agda.Interaction.Options.Errors

Description

Provide names for the errors Agda throws.Options/Er

Synopsis

Documentation

data CannotQuoteTerm Source #

Extra information for error CannotQuoteTerm.

Instances

Instances details
NFData CannotQuoteTerm Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

Methods

rnf :: CannotQuoteTerm -> () #

Bounded CannotQuoteTerm Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

Enum CannotQuoteTerm Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

Generic CannotQuoteTerm Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

Associated Types

type Rep CannotQuoteTerm 
Instance details

Defined in Agda.Interaction.Options.Errors

type Rep CannotQuoteTerm = D1 ('MetaData "CannotQuoteTerm" "Agda.Interaction.Options.Errors" "Agda-2.8.0-inplace" 'False) (C1 ('MetaCons "CannotQuoteTermHidden" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "CannotQuoteTermNothing" 'PrefixI 'False) (U1 :: Type -> Type))
Show CannotQuoteTerm Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

type Rep CannotQuoteTerm Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

type Rep CannotQuoteTerm = D1 ('MetaData "CannotQuoteTerm" "Agda.Interaction.Options.Errors" "Agda-2.8.0-inplace" 'False) (C1 ('MetaCons "CannotQuoteTermHidden" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "CannotQuoteTermNothing" 'PrefixI 'False) (U1 :: Type -> Type))

data DataRecOrFun_ Source #

What kind of declaration?

See also DataRecOrFun.

Constructors

DataName_

Name of a data type.

RecName_

Name of a record type.

FunName_

Name of a function.

Instances

Instances details
Bounded DataRecOrFun_ Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

Enum DataRecOrFun_ Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

Generic DataRecOrFun_ Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

Associated Types

type Rep DataRecOrFun_ 
Instance details

Defined in Agda.Interaction.Options.Errors

type Rep DataRecOrFun_ = D1 ('MetaData "DataRecOrFun_" "Agda.Interaction.Options.Errors" "Agda-2.8.0-inplace" 'False) (C1 ('MetaCons "DataName_" 'PrefixI 'False) (U1 :: Type -> Type) :+: (C1 ('MetaCons "RecName_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "FunName_" 'PrefixI 'False) (U1 :: Type -> Type)))
Show DataRecOrFun_ Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

type Rep DataRecOrFun_ Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

type Rep DataRecOrFun_ = D1 ('MetaData "DataRecOrFun_" "Agda.Interaction.Options.Errors" "Agda-2.8.0-inplace" 'False) (C1 ('MetaCons "DataName_" 'PrefixI 'False) (U1 :: Type -> Type) :+: (C1 ('MetaCons "RecName_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "FunName_" 'PrefixI 'False) (U1 :: Type -> Type)))

data ErasedDatatypeReason Source #

The reason for an ErasedDatatype error.

Constructors

SeveralConstructors

There are several constructors.

NoErasedMatches

The flag --erased-matches is not used.

NoK

The K rule is not activated.

Instances

Instances details
NFData ErasedDatatypeReason Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

Methods

rnf :: ErasedDatatypeReason -> () #

Bounded ErasedDatatypeReason Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

Enum ErasedDatatypeReason Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

Generic ErasedDatatypeReason Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

Associated Types

type Rep ErasedDatatypeReason 
Instance details

Defined in Agda.Interaction.Options.Errors

type Rep ErasedDatatypeReason = D1 ('MetaData "ErasedDatatypeReason" "Agda.Interaction.Options.Errors" "Agda-2.8.0-inplace" 'False) (C1 ('MetaCons "SeveralConstructors" 'PrefixI 'False) (U1 :: Type -> Type) :+: (C1 ('MetaCons "NoErasedMatches" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "NoK" 'PrefixI 'False) (U1 :: Type -> Type)))
Show ErasedDatatypeReason Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

type Rep ErasedDatatypeReason Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

type Rep ErasedDatatypeReason = D1 ('MetaData "ErasedDatatypeReason" "Agda.Interaction.Options.Errors" "Agda-2.8.0-inplace" 'False) (C1 ('MetaCons "SeveralConstructors" 'PrefixI 'False) (U1 :: Type -> Type) :+: (C1 ('MetaCons "NoErasedMatches" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "NoK" 'PrefixI 'False) (U1 :: Type -> Type)))

data NotAllowedInDotPatterns Source #

Things not allowed in dot patterns.

Instances

Instances details
NFData NotAllowedInDotPatterns Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

Methods

rnf :: NotAllowedInDotPatterns -> () #

Bounded NotAllowedInDotPatterns Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

Enum NotAllowedInDotPatterns Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

Generic NotAllowedInDotPatterns Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

Associated Types

type Rep NotAllowedInDotPatterns 
Instance details

Defined in Agda.Interaction.Options.Errors

type Rep NotAllowedInDotPatterns = D1 ('MetaData "NotAllowedInDotPatterns" "Agda.Interaction.Options.Errors" "Agda-2.8.0-inplace" 'False) (C1 ('MetaCons "LetExpressions" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "PatternLambdas" 'PrefixI 'False) (U1 :: Type -> Type))
Show NotAllowedInDotPatterns Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

type Rep NotAllowedInDotPatterns Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

type Rep NotAllowedInDotPatterns = D1 ('MetaData "NotAllowedInDotPatterns" "Agda.Interaction.Options.Errors" "Agda-2.8.0-inplace" 'False) (C1 ('MetaCons "LetExpressions" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "PatternLambdas" 'PrefixI 'False) (U1 :: Type -> Type))

data NotAValidLetBinding Source #

Reasons for error NotAValidLetBinding.

Instances

Instances details
NFData NotAValidLetBinding Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

Methods

rnf :: NotAValidLetBinding -> () #

Bounded NotAValidLetBinding Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

Enum NotAValidLetBinding Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

Generic NotAValidLetBinding Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

Associated Types

type Rep NotAValidLetBinding 
Instance details

Defined in Agda.Interaction.Options.Errors

type Rep NotAValidLetBinding = D1 ('MetaData "NotAValidLetBinding" "Agda.Interaction.Options.Errors" "Agda-2.8.0-inplace" 'False) (C1 ('MetaCons "MissingRHS" 'PrefixI 'False) (U1 :: Type -> Type) :+: (C1 ('MetaCons "NotAValidLetPattern" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "WhereClausesNotAllowed" 'PrefixI 'False) (U1 :: Type -> Type)))
Show NotAValidLetBinding Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

type Rep NotAValidLetBinding Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

type Rep NotAValidLetBinding = D1 ('MetaData "NotAValidLetBinding" "Agda.Interaction.Options.Errors" "Agda-2.8.0-inplace" 'False) (C1 ('MetaCons "MissingRHS" 'PrefixI 'False) (U1 :: Type -> Type) :+: (C1 ('MetaCons "NotAValidLetPattern" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "WhereClausesNotAllowed" 'PrefixI 'False) (U1 :: Type -> Type)))

data NotAValidLetExpression Source #

Reasons for error NotAValidLetExpression.

Constructors

MissingBody 

Instances

Instances details
NFData NotAValidLetExpression Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

Methods

rnf :: NotAValidLetExpression -> () #

Bounded NotAValidLetExpression Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

Enum NotAValidLetExpression Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

Generic NotAValidLetExpression Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

Associated Types

type Rep NotAValidLetExpression 
Instance details

Defined in Agda.Interaction.Options.Errors

type Rep NotAValidLetExpression = D1 ('MetaData "NotAValidLetExpression" "Agda.Interaction.Options.Errors" "Agda-2.8.0-inplace" 'False) (C1 ('MetaCons "MissingBody" 'PrefixI 'False) (U1 :: Type -> Type))
Show NotAValidLetExpression Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

type Rep NotAValidLetExpression Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

type Rep NotAValidLetExpression = D1 ('MetaData "NotAValidLetExpression" "Agda.Interaction.Options.Errors" "Agda-2.8.0-inplace" 'False) (C1 ('MetaCons "MissingBody" 'PrefixI 'False) (U1 :: Type -> Type))

data ErrorName Source #

Symbolic name of an Agda error.

Constructors

ExecError_ ExecError_ 
GHCBackendError_ GHCBackendError_ 
ImpossibleConstructor_ NegativeUnification_ 
InteractionError_ InteractionError_ 
JSBackendError_ JSBackendError_ 
NicifierError_ DeclarationException_ 
SplitError_ SplitError_ 
UnquoteError_ UnquoteError_ 
CompilationError_ 
CustomBackendError_ 
GenericError_ 
GenericDocError_ 
InternalError_ 
LibraryError_ 
NonFatalErrors_ 
NotImplemented_ 
NotSupported_ 
OptionError_ 
SyntaxError_ 
AbsentRHSRequiresAbsurdPattern_ 
AbstractConstructorNotInScope_ 
AmbiguousConstructor_ 
AmbiguousField_ 
AmbiguousModule_ 
AmbiguousName_ 
AmbiguousOverloadedProjection_ 
AmbiguousParseForApplication_ 
AmbiguousParseForLHS_ 
AmbiguousProjection_ 
AmbiguousTopLevelModuleName_ 
AsPatternInPatternSynonym_ 
AttributeKindNotEnabled_ 
BackendDoesNotSupportOnlyScopeChecking_ 
BadArgumentsToPatternSynonym_ 
BothWithAndRHS_ 
BuiltinInParameterisedModule_ 
BuiltinMustBeConstructor_ 
BuiltinMustBeData_ 
BuiltinMustBeDef_ 
BuiltinMustBeFunction_ 
BuiltinMustBePostulate_ 
CannotApply_ 
CannotEliminateWithPattern_ 
CannotEliminateWithProjection_ 
CannotGenerateHCompClause_ 
CannotGenerateTransportClause_ 
CannotQuote_ CannotQuote_ 
CannotQuoteTerm_ CannotQuoteTerm 
CannotResolveAmbiguousPatternSynonym_ 
CannotRewriteByNonEquation_ 
CannotSolveSizeConstraints_ 
CantResolveOverloadedConstructorsTargetingSameDatatype_ 
ClashingDefinition_ 
ClashingModule_ 
ComatchingDisabledForRecord_ 
ConstructorDoesNotTargetGivenType_ 
ConstructorPatternInWrongDatatype_ 
ContradictorySizeConstraint_ 
CopatternHeadNotProjection_ 
CubicalCompilationNotSupported_ 
CubicalNotErasure_ 
CubicalPrimitiveNotFullyApplied_ 
CyclicModuleDependency_ 
DatatypeIndexPolarity_ 
DeBruijnIndexOutOfScope_ 
DeclarationsAfterTopLevelModule_ 
DefinitionInDifferentModule_ 
DefinitionIsErased_ 
DefinitionIsIrrelevant_ 
DoNotationError_ 
DoesNotMentionTicks_ 
DotPatternInPatternSynonym_ 
DuplicateBuiltinBinding_ 
DuplicateConstructors_ 
DuplicateFields_ 
DuplicateImports_ 
DuplicateOverlapPragma_ 
DuplicatePrimitiveBinding_ 
EmptyTypeOfSizes_ 
ExpectedBindingForParameter_ 
ExpectedIntervalLiteral_ 
FieldOutsideRecord_ 
FaceConstraintDisjunction_ 
FaceConstraintUnsatisfiable_ 
FileNotFound_ 
ForcedConstructorNotInstantiated_ 
FunctionTypeInSizeUniv_ 
GeneralizeCyclicDependency_ 
GeneralizeNotSupportedHere_ 
GeneralizedVarInLetOpenedModule_ 
ModuleNameHashCollision_ 
HidingMismatch_ 
IdiomBracketError_ 
InvalidBuiltin_ 
InvalidDottedExpression_ 
IllTypedPatternAfterWithAbstraction_ 
IllegalDeclarationBeforeTopLevelModule_ 
IllegalDeclarationInDataDefinition_ 
IllegalHidingInPostfixProjection_ 
IllegalInstanceVariableInPatternSynonym_ 
IllegalLetInTelescope_ 
IllegalPatternInTelescope_ 
IllformedProjectionPatternAbstract_ 
IllformedProjectionPatternConcrete_ 
IncorrectTypeForRewriteRelation_ 
InstanceNoCandidate_ 
InstanceSearchDepthExhausted_ 
InvalidFileName_ 
InvalidModalTelescopeUse_ 
InvalidPattern_ 
InvalidProjectionParameter_ 
InvalidPun_ ConstructorOrPatternSynonym 
InvalidTypeSort_ 
LambdaIsErased_ 
LibTooFarDown_ 
LiteralTooBig_ 
MacroResultTypeMismatch_ 
MetaCannotDependOn_ 
MetaErasedSolution_ 
MetaIrrelevantSolution_ 
MismatchedProjectionsError_ 
MissingTypeSignature_ DataRecOrFun_ 
ModuleArityMismatch_ 
ModuleDefinedInOtherFile_ 
ModuleNameDoesntMatchFileName_ 
ModuleNameUnexpected_ 
MultipleFixityDecls_ 
MultiplePolarityPragmas_ 
ExplicitPolarityVsPragma_ 
ConstructorNameOfNonRecord_ 
NamedWhereModuleInRefinedContext_ 
NeedOptionAllowExec_ 
NeedOptionCopatterns_ 
NeedOptionCubical_ 
NeedOptionPatternMatching_ 
NeedOptionProp_ 
NeedOptionRewriting_ 
NeedOptionSizedTypes_ 
NeedOptionTwoLevel_ 
NeedOptionUniversePolymorphism_ 
NegativeLiteralInPattern_ 
NoBindingForBuiltin_ 
NoBindingForPrimitive_ 
NoKnownRecordWithSuchFields_ 
NoParameterOfName_ 
NoParseForApplication_ 
NoParseForLHS_ 
NoSuchBuiltinName_ 
NoSuchModule_ 
NoSuchPrimitiveFunction_ 
NotAValidLetBinding_ (Maybe NotAValidLetBinding) 
NotAValidLetExpression_ NotAValidLetExpression 
NotAllowedInDotPatterns_ NotAllowedInDotPatterns 
NotAnExpression_ 
NotInScope_ 
NotLeqSort_ 
NotValidBeforeField_ 
OpenEverythingInRecordWhere_ 
OverlappingProjects_ 
PathAbstractionFailed_ 
PatternInPathLambda_ 
PatternInSystem_ 
PatternSynonymArgumentShadows_ ConstructorOrPatternSynonym 
PostulatedSizeInModule_ 
PrivateRecordField_ 
ProjectionIsIrrelevant_ 
QualifiedLocalModule_ 
QuantityMismatch_ 
RecordIsErased_ 
RecursiveRecordNeedsInductivity_ 
ReferencesFutureVariables_ 
RelevanceMismatch_ 
RepeatedNamesInImportDirective_ 
RepeatedVariablesInPattern_ 
ShadowedModule_ 
ShouldBeASort_ 
ShouldBeEmpty_ 
ShouldBePath_ 
ShouldBePi_ 
ShouldBeRecordPattern_ 
ShouldBeRecordType_ 
ShouldEndInApplicationOfTheDatatype_ 
SolvedButOpenHoles_ 
SortCannotDependOnItsIndex_ 
SortDoesNotAdmitDataDefinitions_ 
SortOfSplitVarError_ 
SplitInProp_ 
SplitOnAbstract_ 
SplitOnCoinductive_ 
SplitOnIrrelevant_ 
SplitOnNonEtaRecord_ 
SplitOnNonVariable_ 
SplitOnPartial_ 
SplitOnUnchecked_ 
SplitOnUnusableCohesion_ 
SplitOnUnusablePolarity_ 
TacticAttributeNotAllowed_ 
TooFewArgumentsToPatternSynonym_ 
TooFewPatternsInWithClause_ 
TooManyFields_ 
TooManyPatternsInWithClause_ 
TriedToCopyConstrainedPrim_ 
InvalidInstanceHeadType_ 
UnboundVariablesInPatternSynonym_ 
UnequalCohesion_ 
UnequalFiniteness_ 
UnequalHiding_ 
UnequalLevel_ 
UnequalQuantity_ 
UnequalRelevance_ 
UnequalPolarity_ 
UnequalSorts_ 
UnequalTerms_ 
UnexpectedModalityAnnotationInParameter_ 
UnexpectedParameter_ 
UnexpectedTypeSignatureForParameter_ 
UnexpectedWithPatterns_ 
UnknownBackend_ 
UnusableAtModality_ 
UnusedVariableInPatternSynonym_ 
VariableIsErased_ 
VariableIsIrrelevant_ 
VariableIsOfUnusableCohesion_ 
VariableIsOfUnusablePolarity_ 
WithClausePatternMismatch_ 
WithOnFreeVariable_ 
WrongAnnotationInLambda_ 
WrongArgInfoForPrimitive_ 
WrongCohesionInLambda_ 
WrongPolarityInLambda_ 
WrongHidingInApplication_ 
WrongHidingInLHS_ 
WrongHidingInLambda_ 
WrongHidingInProjection_ 
WrongIrrelevanceInLambda_ 
WrongNamedArgument_ 
WrongNumberOfConstructorArguments_ 
WrongQuantityInLambda_ 
WrongSharpArity_ 

Instances

Instances details
Bounded ErrorName Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

Enum ErrorName Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

Generic ErrorName Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

Associated Types

type Rep ErrorName 
Instance details

Defined in Agda.Interaction.Options.Errors

type Rep ErrorName = D1 ('MetaData "ErrorName" "Agda.Interaction.Options.Errors" "Agda-2.8.0-inplace" 'False) (((((((C1 ('MetaCons "ExecError_" 'PrefixI 'False) (S1 ('MetaSel ('Nothing :: Maybe Symbol) 'NoSourceUnpackedness 'NoSourceStrictness 'DecidedLazy) (Rec0 ExecError_)) :+: (C1 ('MetaCons "GHCBackendError_" 'PrefixI 'False) (S1 ('MetaSel ('Nothing :: Maybe Symbol) 'NoSourceUnpackedness 'NoSourceStrictness 'DecidedLazy) (Rec0 GHCBackendError_)) :+: C1 ('MetaCons "ImpossibleConstructor_" 'PrefixI 'False) (S1 ('MetaSel ('Nothing :: Maybe Symbol) 'NoSourceUnpackedness 'NoSourceStrictness 'DecidedLazy) (Rec0 NegativeUnification_)))) :+: ((C1 ('MetaCons "InteractionError_" 'PrefixI 'False) (S1 ('MetaSel ('Nothing :: Maybe Symbol) 'NoSourceUnpackedness 'NoSourceStrictness 'DecidedLazy) (Rec0 InteractionError_)) :+: C1 ('MetaCons "JSBackendError_" 'PrefixI 'False) (S1 ('MetaSel ('Nothing :: Maybe Symbol) 'NoSourceUnpackedness 'NoSourceStrictness 'DecidedLazy) (Rec0 JSBackendError_))) :+: (C1 ('MetaCons "NicifierError_" 'PrefixI 'False) (S1 ('MetaSel ('Nothing :: Maybe Symbol) 'NoSourceUnpackedness 'NoSourceStrictness 'DecidedLazy) (Rec0 DeclarationException_)) :+: C1 ('MetaCons "SplitError_" 'PrefixI 'False) (S1 ('MetaSel ('Nothing :: Maybe Symbol) 'NoSourceUnpackedness 'NoSourceStrictness 'DecidedLazy) (Rec0 SplitError_))))) :+: ((C1 ('MetaCons "UnquoteError_" 'PrefixI 'False) (S1 ('MetaSel ('Nothing :: Maybe Symbol) 'NoSourceUnpackedness 'NoSourceStrictness 'DecidedLazy) (Rec0 UnquoteError_)) :+: (C1 ('MetaCons "CompilationError_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "CustomBackendError_" 'PrefixI 'False) (U1 :: Type -> Type))) :+: ((C1 ('MetaCons "GenericError_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "GenericDocError_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "InternalError_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "LibraryError_" 'PrefixI 'False) (U1 :: Type -> Type))))) :+: (((C1 ('MetaCons "NonFatalErrors_" 'PrefixI 'False) (U1 :: Type -> Type) :+: (C1 ('MetaCons "NotImplemented_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "NotSupported_" 'PrefixI 'False) (U1 :: Type -> Type))) :+: ((C1 ('MetaCons "OptionError_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "SyntaxError_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "AbsentRHSRequiresAbsurdPattern_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "AbstractConstructorNotInScope_" 'PrefixI 'False) (U1 :: Type -> Type)))) :+: (((C1 ('MetaCons "AmbiguousConstructor_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "AmbiguousField_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "AmbiguousModule_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "AmbiguousName_" 'PrefixI 'False) (U1 :: Type -> Type))) :+: ((C1 ('MetaCons "AmbiguousOverloadedProjection_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "AmbiguousParseForApplication_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "AmbiguousParseForLHS_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "AmbiguousProjection_" 'PrefixI 'False) (U1 :: Type -> Type)))))) :+: ((((C1 ('MetaCons "AmbiguousTopLevelModuleName_" 'PrefixI 'False) (U1 :: Type -> Type) :+: (C1 ('MetaCons "AsPatternInPatternSynonym_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "AttributeKindNotEnabled_" 'PrefixI 'False) (U1 :: Type -> Type))) :+: ((C1 ('MetaCons "BackendDoesNotSupportOnlyScopeChecking_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "BadArgumentsToPatternSynonym_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "BothWithAndRHS_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "BuiltinInParameterisedModule_" 'PrefixI 'False) (U1 :: Type -> Type)))) :+: (((C1 ('MetaCons "BuiltinMustBeConstructor_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "BuiltinMustBeData_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "BuiltinMustBeDef_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "BuiltinMustBeFunction_" 'PrefixI 'False) (U1 :: Type -> Type))) :+: ((C1 ('MetaCons "BuiltinMustBePostulate_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "CannotApply_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "CannotEliminateWithPattern_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "CannotEliminateWithProjection_" 'PrefixI 'False) (U1 :: Type -> Type))))) :+: (((C1 ('MetaCons "CannotGenerateHCompClause_" 'PrefixI 'False) (U1 :: Type -> Type) :+: (C1 ('MetaCons "CannotGenerateTransportClause_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "CannotQuote_" 'PrefixI 'False) (S1 ('MetaSel ('Nothing :: Maybe Symbol) 'NoSourceUnpackedness 'NoSourceStrictness 'DecidedLazy) (Rec0 CannotQuote_)))) :+: ((C1 ('MetaCons "CannotQuoteTerm_" 'PrefixI 'False) (S1 ('MetaSel ('Nothing :: Maybe Symbol) 'NoSourceUnpackedness 'NoSourceStrictness 'DecidedLazy) (Rec0 CannotQuoteTerm)) :+: C1 ('MetaCons "CannotResolveAmbiguousPatternSynonym_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "CannotRewriteByNonEquation_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "CannotSolveSizeConstraints_" 'PrefixI 'False) (U1 :: Type -> Type)))) :+: (((C1 ('MetaCons "CantResolveOverloadedConstructorsTargetingSameDatatype_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "ClashingDefinition_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "ClashingModule_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "ComatchingDisabledForRecord_" 'PrefixI 'False) (U1 :: Type -> Type))) :+: ((C1 ('MetaCons "ConstructorDoesNotTargetGivenType_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "ConstructorPatternInWrongDatatype_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "ContradictorySizeConstraint_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "CopatternHeadNotProjection_" 'PrefixI 'False) (U1 :: Type -> Type))))))) :+: (((((C1 ('MetaCons "CubicalCompilationNotSupported_" 'PrefixI 'False) (U1 :: Type -> Type) :+: (C1 ('MetaCons "CubicalNotErasure_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "CubicalPrimitiveNotFullyApplied_" 'PrefixI 'False) (U1 :: Type -> Type))) :+: ((C1 ('MetaCons "CyclicModuleDependency_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "DatatypeIndexPolarity_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "DeBruijnIndexOutOfScope_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "DeclarationsAfterTopLevelModule_" 'PrefixI 'False) (U1 :: Type -> Type)))) :+: (((C1 ('MetaCons "DefinitionInDifferentModule_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "DefinitionIsErased_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "DefinitionIsIrrelevant_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "DoNotationError_" 'PrefixI 'False) (U1 :: Type -> Type))) :+: ((C1 ('MetaCons "DoesNotMentionTicks_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "DotPatternInPatternSynonym_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "DuplicateBuiltinBinding_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "DuplicateConstructors_" 'PrefixI 'False) (U1 :: Type -> Type))))) :+: (((C1 ('MetaCons "DuplicateFields_" 'PrefixI 'False) (U1 :: Type -> Type) :+: (C1 ('MetaCons "DuplicateImports_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "DuplicateOverlapPragma_" 'PrefixI 'False) (U1 :: Type -> Type))) :+: ((C1 ('MetaCons "DuplicatePrimitiveBinding_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "EmptyTypeOfSizes_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "ExpectedBindingForParameter_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "ExpectedIntervalLiteral_" 'PrefixI 'False) (U1 :: Type -> Type)))) :+: (((C1 ('MetaCons "FieldOutsideRecord_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "FaceConstraintDisjunction_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "FaceConstraintUnsatisfiable_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "FileNotFound_" 'PrefixI 'False) (U1 :: Type -> Type))) :+: ((C1 ('MetaCons "ForcedConstructorNotInstantiated_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "FunctionTypeInSizeUniv_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "GeneralizeCyclicDependency_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "GeneralizeNotSupportedHere_" 'PrefixI 'False) (U1 :: Type -> Type)))))) :+: ((((C1 ('MetaCons "GeneralizedVarInLetOpenedModule_" 'PrefixI 'False) (U1 :: Type -> Type) :+: (C1 ('MetaCons "ModuleNameHashCollision_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "HidingMismatch_" 'PrefixI 'False) (U1 :: Type -> Type))) :+: ((C1 ('MetaCons "IdiomBracketError_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "InvalidBuiltin_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "InvalidDottedExpression_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "IllTypedPatternAfterWithAbstraction_" 'PrefixI 'False) (U1 :: Type -> Type)))) :+: (((C1 ('MetaCons "IllegalDeclarationBeforeTopLevelModule_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "IllegalDeclarationInDataDefinition_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "IllegalHidingInPostfixProjection_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "IllegalInstanceVariableInPatternSynonym_" 'PrefixI 'False) (U1 :: Type -> Type))) :+: ((C1 ('MetaCons "IllegalLetInTelescope_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "IllegalPatternInTelescope_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "IllformedProjectionPatternAbstract_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "IllformedProjectionPatternConcrete_" 'PrefixI 'False) (U1 :: Type -> Type))))) :+: (((C1 ('MetaCons "IncorrectTypeForRewriteRelation_" 'PrefixI 'False) (U1 :: Type -> Type) :+: (C1 ('MetaCons "InstanceNoCandidate_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "InstanceSearchDepthExhausted_" 'PrefixI 'False) (U1 :: Type -> Type))) :+: ((C1 ('MetaCons "InvalidFileName_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "InvalidModalTelescopeUse_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "InvalidPattern_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "InvalidProjectionParameter_" 'PrefixI 'False) (U1 :: Type -> Type)))) :+: (((C1 ('MetaCons "InvalidPun_" 'PrefixI 'False) (S1 ('MetaSel ('Nothing :: Maybe Symbol) 'NoSourceUnpackedness 'NoSourceStrictness 'DecidedLazy) (Rec0 ConstructorOrPatternSynonym)) :+: C1 ('MetaCons "InvalidTypeSort_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "LambdaIsErased_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "LibTooFarDown_" 'PrefixI 'False) (U1 :: Type -> Type))) :+: ((C1 ('MetaCons "LiteralTooBig_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "MacroResultTypeMismatch_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "MetaCannotDependOn_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "MetaErasedSolution_" 'PrefixI 'False) (U1 :: Type -> Type)))))))) :+: ((((((C1 ('MetaCons "MetaIrrelevantSolution_" 'PrefixI 'False) (U1 :: Type -> Type) :+: (C1 ('MetaCons "MismatchedProjectionsError_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "MissingTypeSignature_" 'PrefixI 'False) (S1 ('MetaSel ('Nothing :: Maybe Symbol) 'NoSourceUnpackedness 'NoSourceStrictness 'DecidedLazy) (Rec0 DataRecOrFun_)))) :+: ((C1 ('MetaCons "ModuleArityMismatch_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "ModuleDefinedInOtherFile_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "ModuleNameDoesntMatchFileName_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "ModuleNameUnexpected_" 'PrefixI 'False) (U1 :: Type -> Type)))) :+: (((C1 ('MetaCons "MultipleFixityDecls_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "MultiplePolarityPragmas_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "ExplicitPolarityVsPragma_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "ConstructorNameOfNonRecord_" 'PrefixI 'False) (U1 :: Type -> Type))) :+: ((C1 ('MetaCons "NamedWhereModuleInRefinedContext_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "NeedOptionAllowExec_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "NeedOptionCopatterns_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "NeedOptionCubical_" 'PrefixI 'False) (U1 :: Type -> Type))))) :+: (((C1 ('MetaCons "NeedOptionPatternMatching_" 'PrefixI 'False) (U1 :: Type -> Type) :+: (C1 ('MetaCons "NeedOptionProp_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "NeedOptionRewriting_" 'PrefixI 'False) (U1 :: Type -> Type))) :+: ((C1 ('MetaCons "NeedOptionSizedTypes_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "NeedOptionTwoLevel_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "NeedOptionUniversePolymorphism_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "NegativeLiteralInPattern_" 'PrefixI 'False) (U1 :: Type -> Type)))) :+: (((C1 ('MetaCons "NoBindingForBuiltin_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "NoBindingForPrimitive_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "NoKnownRecordWithSuchFields_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "NoParameterOfName_" 'PrefixI 'False) (U1 :: Type -> Type))) :+: ((C1 ('MetaCons "NoParseForApplication_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "NoParseForLHS_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "NoSuchBuiltinName_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "NoSuchModule_" 'PrefixI 'False) (U1 :: Type -> Type)))))) :+: ((((C1 ('MetaCons "NoSuchPrimitiveFunction_" 'PrefixI 'False) (U1 :: Type -> Type) :+: (C1 ('MetaCons "NotAValidLetBinding_" 'PrefixI 'False) (S1 ('MetaSel ('Nothing :: Maybe Symbol) 'NoSourceUnpackedness 'NoSourceStrictness 'DecidedLazy) (Rec0 (Maybe NotAValidLetBinding))) :+: C1 ('MetaCons "NotAValidLetExpression_" 'PrefixI 'False) (S1 ('MetaSel ('Nothing :: Maybe Symbol) 'NoSourceUnpackedness 'NoSourceStrictness 'DecidedLazy) (Rec0 NotAValidLetExpression)))) :+: ((C1 ('MetaCons "NotAllowedInDotPatterns_" 'PrefixI 'False) (S1 ('MetaSel ('Nothing :: Maybe Symbol) 'NoSourceUnpackedness 'NoSourceStrictness 'DecidedLazy) (Rec0 NotAllowedInDotPatterns)) :+: C1 ('MetaCons "NotAnExpression_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "NotInScope_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "NotLeqSort_" 'PrefixI 'False) (U1 :: Type -> Type)))) :+: (((C1 ('MetaCons "NotValidBeforeField_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "OpenEverythingInRecordWhere_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "OverlappingProjects_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "PathAbstractionFailed_" 'PrefixI 'False) (U1 :: Type -> Type))) :+: ((C1 ('MetaCons "PatternInPathLambda_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "PatternInSystem_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "PatternSynonymArgumentShadows_" 'PrefixI 'False) (S1 ('MetaSel ('Nothing :: Maybe Symbol) 'NoSourceUnpackedness 'NoSourceStrictness 'DecidedLazy) (Rec0 ConstructorOrPatternSynonym)) :+: C1 ('MetaCons "PostulatedSizeInModule_" 'PrefixI 'False) (U1 :: Type -> Type))))) :+: (((C1 ('MetaCons "PrivateRecordField_" 'PrefixI 'False) (U1 :: Type -> Type) :+: (C1 ('MetaCons "ProjectionIsIrrelevant_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "QualifiedLocalModule_" 'PrefixI 'False) (U1 :: Type -> Type))) :+: ((C1 ('MetaCons "QuantityMismatch_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "RecordIsErased_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "RecursiveRecordNeedsInductivity_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "ReferencesFutureVariables_" 'PrefixI 'False) (U1 :: Type -> Type)))) :+: (((C1 ('MetaCons "RelevanceMismatch_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "RepeatedNamesInImportDirective_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "RepeatedVariablesInPattern_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "ShadowedModule_" 'PrefixI 'False) (U1 :: Type -> Type))) :+: ((C1 ('MetaCons "ShouldBeASort_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "ShouldBeEmpty_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "ShouldBePath_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "ShouldBePi_" 'PrefixI 'False) (U1 :: Type -> Type))))))) :+: (((((C1 ('MetaCons "ShouldBeRecordPattern_" 'PrefixI 'False) (U1 :: Type -> Type) :+: (C1 ('MetaCons "ShouldBeRecordType_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "ShouldEndInApplicationOfTheDatatype_" 'PrefixI 'False) (U1 :: Type -> Type))) :+: ((C1 ('MetaCons "SolvedButOpenHoles_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "SortCannotDependOnItsIndex_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "SortDoesNotAdmitDataDefinitions_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "SortOfSplitVarError_" 'PrefixI 'False) (U1 :: Type -> Type)))) :+: (((C1 ('MetaCons "SplitInProp_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "SplitOnAbstract_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "SplitOnCoinductive_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "SplitOnIrrelevant_" 'PrefixI 'False) (U1 :: Type -> Type))) :+: ((C1 ('MetaCons "SplitOnNonEtaRecord_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "SplitOnNonVariable_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "SplitOnPartial_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "SplitOnUnchecked_" 'PrefixI 'False) (U1 :: Type -> Type))))) :+: (((C1 ('MetaCons "SplitOnUnusableCohesion_" 'PrefixI 'False) (U1 :: Type -> Type) :+: (C1 ('MetaCons "SplitOnUnusablePolarity_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "TacticAttributeNotAllowed_" 'PrefixI 'False) (U1 :: Type -> Type))) :+: ((C1 ('MetaCons "TooFewArgumentsToPatternSynonym_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "TooFewPatternsInWithClause_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "TooManyFields_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "TooManyPatternsInWithClause_" 'PrefixI 'False) (U1 :: Type -> Type)))) :+: (((C1 ('MetaCons "TriedToCopyConstrainedPrim_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "InvalidInstanceHeadType_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "UnboundVariablesInPatternSynonym_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "UnequalCohesion_" 'PrefixI 'False) (U1 :: Type -> Type))) :+: ((C1 ('MetaCons "UnequalFiniteness_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "UnequalHiding_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "UnequalLevel_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "UnequalQuantity_" 'PrefixI 'False) (U1 :: Type -> Type)))))) :+: ((((C1 ('MetaCons "UnequalRelevance_" 'PrefixI 'False) (U1 :: Type -> Type) :+: (C1 ('MetaCons "UnequalPolarity_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "UnequalSorts_" 'PrefixI 'False) (U1 :: Type -> Type))) :+: ((C1 ('MetaCons "UnequalTerms_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "UnexpectedModalityAnnotationInParameter_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "UnexpectedParameter_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "UnexpectedTypeSignatureForParameter_" 'PrefixI 'False) (U1 :: Type -> Type)))) :+: (((C1 ('MetaCons "UnexpectedWithPatterns_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "UnknownBackend_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "UnusableAtModality_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "UnusedVariableInPatternSynonym_" 'PrefixI 'False) (U1 :: Type -> Type))) :+: ((C1 ('MetaCons "VariableIsErased_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "VariableIsIrrelevant_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "VariableIsOfUnusableCohesion_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "VariableIsOfUnusablePolarity_" 'PrefixI 'False) (U1 :: Type -> Type))))) :+: (((C1 ('MetaCons "WithClausePatternMismatch_" 'PrefixI 'False) (U1 :: Type -> Type) :+: (C1 ('MetaCons "WithOnFreeVariable_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "WrongAnnotationInLambda_" 'PrefixI 'False) (U1 :: Type -> Type))) :+: ((C1 ('MetaCons "WrongArgInfoForPrimitive_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "WrongCohesionInLambda_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "WrongPolarityInLambda_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "WrongHidingInApplication_" 'PrefixI 'False) (U1 :: Type -> Type)))) :+: (((C1 ('MetaCons "WrongHidingInLHS_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "WrongHidingInLambda_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "WrongHidingInProjection_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "WrongIrrelevanceInLambda_" 'PrefixI 'False) (U1 :: Type -> Type))) :+: ((C1 ('MetaCons "WrongNamedArgument_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "WrongNumberOfConstructorArguments_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "WrongQuantityInLambda_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "WrongSharpArity_" 'PrefixI 'False) (U1 :: Type -> Type)))))))))
Show ErrorName Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

type Rep ErrorName Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

type Rep ErrorName = D1 ('MetaData "ErrorName" "Agda.Interaction.Options.Errors" "Agda-2.8.0-inplace" 'False) (((((((C1 ('MetaCons "ExecError_" 'PrefixI 'False) (S1 ('MetaSel ('Nothing :: Maybe Symbol) 'NoSourceUnpackedness 'NoSourceStrictness 'DecidedLazy) (Rec0 ExecError_)) :+: (C1 ('MetaCons "GHCBackendError_" 'PrefixI 'False) (S1 ('MetaSel ('Nothing :: Maybe Symbol) 'NoSourceUnpackedness 'NoSourceStrictness 'DecidedLazy) (Rec0 GHCBackendError_)) :+: C1 ('MetaCons "ImpossibleConstructor_" 'PrefixI 'False) (S1 ('MetaSel ('Nothing :: Maybe Symbol) 'NoSourceUnpackedness 'NoSourceStrictness 'DecidedLazy) (Rec0 NegativeUnification_)))) :+: ((C1 ('MetaCons "InteractionError_" 'PrefixI 'False) (S1 ('MetaSel ('Nothing :: Maybe Symbol) 'NoSourceUnpackedness 'NoSourceStrictness 'DecidedLazy) (Rec0 InteractionError_)) :+: C1 ('MetaCons "JSBackendError_" 'PrefixI 'False) (S1 ('MetaSel ('Nothing :: Maybe Symbol) 'NoSourceUnpackedness 'NoSourceStrictness 'DecidedLazy) (Rec0 JSBackendError_))) :+: (C1 ('MetaCons "NicifierError_" 'PrefixI 'False) (S1 ('MetaSel ('Nothing :: Maybe Symbol) 'NoSourceUnpackedness 'NoSourceStrictness 'DecidedLazy) (Rec0 DeclarationException_)) :+: C1 ('MetaCons "SplitError_" 'PrefixI 'False) (S1 ('MetaSel ('Nothing :: Maybe Symbol) 'NoSourceUnpackedness 'NoSourceStrictness 'DecidedLazy) (Rec0 SplitError_))))) :+: ((C1 ('MetaCons "UnquoteError_" 'PrefixI 'False) (S1 ('MetaSel ('Nothing :: Maybe Symbol) 'NoSourceUnpackedness 'NoSourceStrictness 'DecidedLazy) (Rec0 UnquoteError_)) :+: (C1 ('MetaCons "CompilationError_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "CustomBackendError_" 'PrefixI 'False) (U1 :: Type -> Type))) :+: ((C1 ('MetaCons "GenericError_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "GenericDocError_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "InternalError_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "LibraryError_" 'PrefixI 'False) (U1 :: Type -> Type))))) :+: (((C1 ('MetaCons "NonFatalErrors_" 'PrefixI 'False) (U1 :: Type -> Type) :+: (C1 ('MetaCons "NotImplemented_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "NotSupported_" 'PrefixI 'False) (U1 :: Type -> Type))) :+: ((C1 ('MetaCons "OptionError_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "SyntaxError_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "AbsentRHSRequiresAbsurdPattern_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "AbstractConstructorNotInScope_" 'PrefixI 'False) (U1 :: Type -> Type)))) :+: (((C1 ('MetaCons "AmbiguousConstructor_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "AmbiguousField_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "AmbiguousModule_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "AmbiguousName_" 'PrefixI 'False) (U1 :: Type -> Type))) :+: ((C1 ('MetaCons "AmbiguousOverloadedProjection_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "AmbiguousParseForApplication_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "AmbiguousParseForLHS_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "AmbiguousProjection_" 'PrefixI 'False) (U1 :: Type -> Type)))))) :+: ((((C1 ('MetaCons "AmbiguousTopLevelModuleName_" 'PrefixI 'False) (U1 :: Type -> Type) :+: (C1 ('MetaCons "AsPatternInPatternSynonym_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "AttributeKindNotEnabled_" 'PrefixI 'False) (U1 :: Type -> Type))) :+: ((C1 ('MetaCons "BackendDoesNotSupportOnlyScopeChecking_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "BadArgumentsToPatternSynonym_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "BothWithAndRHS_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "BuiltinInParameterisedModule_" 'PrefixI 'False) (U1 :: Type -> Type)))) :+: (((C1 ('MetaCons "BuiltinMustBeConstructor_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "BuiltinMustBeData_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "BuiltinMustBeDef_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "BuiltinMustBeFunction_" 'PrefixI 'False) (U1 :: Type -> Type))) :+: ((C1 ('MetaCons "BuiltinMustBePostulate_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "CannotApply_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "CannotEliminateWithPattern_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "CannotEliminateWithProjection_" 'PrefixI 'False) (U1 :: Type -> Type))))) :+: (((C1 ('MetaCons "CannotGenerateHCompClause_" 'PrefixI 'False) (U1 :: Type -> Type) :+: (C1 ('MetaCons "CannotGenerateTransportClause_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "CannotQuote_" 'PrefixI 'False) (S1 ('MetaSel ('Nothing :: Maybe Symbol) 'NoSourceUnpackedness 'NoSourceStrictness 'DecidedLazy) (Rec0 CannotQuote_)))) :+: ((C1 ('MetaCons "CannotQuoteTerm_" 'PrefixI 'False) (S1 ('MetaSel ('Nothing :: Maybe Symbol) 'NoSourceUnpackedness 'NoSourceStrictness 'DecidedLazy) (Rec0 CannotQuoteTerm)) :+: C1 ('MetaCons "CannotResolveAmbiguousPatternSynonym_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "CannotRewriteByNonEquation_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "CannotSolveSizeConstraints_" 'PrefixI 'False) (U1 :: Type -> Type)))) :+: (((C1 ('MetaCons "CantResolveOverloadedConstructorsTargetingSameDatatype_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "ClashingDefinition_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "ClashingModule_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "ComatchingDisabledForRecord_" 'PrefixI 'False) (U1 :: Type -> Type))) :+: ((C1 ('MetaCons "ConstructorDoesNotTargetGivenType_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "ConstructorPatternInWrongDatatype_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "ContradictorySizeConstraint_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "CopatternHeadNotProjection_" 'PrefixI 'False) (U1 :: Type -> Type))))))) :+: (((((C1 ('MetaCons "CubicalCompilationNotSupported_" 'PrefixI 'False) (U1 :: Type -> Type) :+: (C1 ('MetaCons "CubicalNotErasure_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "CubicalPrimitiveNotFullyApplied_" 'PrefixI 'False) (U1 :: Type -> Type))) :+: ((C1 ('MetaCons "CyclicModuleDependency_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "DatatypeIndexPolarity_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "DeBruijnIndexOutOfScope_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "DeclarationsAfterTopLevelModule_" 'PrefixI 'False) (U1 :: Type -> Type)))) :+: (((C1 ('MetaCons "DefinitionInDifferentModule_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "DefinitionIsErased_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "DefinitionIsIrrelevant_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "DoNotationError_" 'PrefixI 'False) (U1 :: Type -> Type))) :+: ((C1 ('MetaCons "DoesNotMentionTicks_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "DotPatternInPatternSynonym_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "DuplicateBuiltinBinding_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "DuplicateConstructors_" 'PrefixI 'False) (U1 :: Type -> Type))))) :+: (((C1 ('MetaCons "DuplicateFields_" 'PrefixI 'False) (U1 :: Type -> Type) :+: (C1 ('MetaCons "DuplicateImports_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "DuplicateOverlapPragma_" 'PrefixI 'False) (U1 :: Type -> Type))) :+: ((C1 ('MetaCons "DuplicatePrimitiveBinding_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "EmptyTypeOfSizes_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "ExpectedBindingForParameter_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "ExpectedIntervalLiteral_" 'PrefixI 'False) (U1 :: Type -> Type)))) :+: (((C1 ('MetaCons "FieldOutsideRecord_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "FaceConstraintDisjunction_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "FaceConstraintUnsatisfiable_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "FileNotFound_" 'PrefixI 'False) (U1 :: Type -> Type))) :+: ((C1 ('MetaCons "ForcedConstructorNotInstantiated_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "FunctionTypeInSizeUniv_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "GeneralizeCyclicDependency_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "GeneralizeNotSupportedHere_" 'PrefixI 'False) (U1 :: Type -> Type)))))) :+: ((((C1 ('MetaCons "GeneralizedVarInLetOpenedModule_" 'PrefixI 'False) (U1 :: Type -> Type) :+: (C1 ('MetaCons "ModuleNameHashCollision_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "HidingMismatch_" 'PrefixI 'False) (U1 :: Type -> Type))) :+: ((C1 ('MetaCons "IdiomBracketError_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "InvalidBuiltin_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "InvalidDottedExpression_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "IllTypedPatternAfterWithAbstraction_" 'PrefixI 'False) (U1 :: Type -> Type)))) :+: (((C1 ('MetaCons "IllegalDeclarationBeforeTopLevelModule_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "IllegalDeclarationInDataDefinition_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "IllegalHidingInPostfixProjection_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "IllegalInstanceVariableInPatternSynonym_" 'PrefixI 'False) (U1 :: Type -> Type))) :+: ((C1 ('MetaCons "IllegalLetInTelescope_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "IllegalPatternInTelescope_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "IllformedProjectionPatternAbstract_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "IllformedProjectionPatternConcrete_" 'PrefixI 'False) (U1 :: Type -> Type))))) :+: (((C1 ('MetaCons "IncorrectTypeForRewriteRelation_" 'PrefixI 'False) (U1 :: Type -> Type) :+: (C1 ('MetaCons "InstanceNoCandidate_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "InstanceSearchDepthExhausted_" 'PrefixI 'False) (U1 :: Type -> Type))) :+: ((C1 ('MetaCons "InvalidFileName_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "InvalidModalTelescopeUse_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "InvalidPattern_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "InvalidProjectionParameter_" 'PrefixI 'False) (U1 :: Type -> Type)))) :+: (((C1 ('MetaCons "InvalidPun_" 'PrefixI 'False) (S1 ('MetaSel ('Nothing :: Maybe Symbol) 'NoSourceUnpackedness 'NoSourceStrictness 'DecidedLazy) (Rec0 ConstructorOrPatternSynonym)) :+: C1 ('MetaCons "InvalidTypeSort_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "LambdaIsErased_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "LibTooFarDown_" 'PrefixI 'False) (U1 :: Type -> Type))) :+: ((C1 ('MetaCons "LiteralTooBig_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "MacroResultTypeMismatch_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "MetaCannotDependOn_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "MetaErasedSolution_" 'PrefixI 'False) (U1 :: Type -> Type)))))))) :+: ((((((C1 ('MetaCons "MetaIrrelevantSolution_" 'PrefixI 'False) (U1 :: Type -> Type) :+: (C1 ('MetaCons "MismatchedProjectionsError_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "MissingTypeSignature_" 'PrefixI 'False) (S1 ('MetaSel ('Nothing :: Maybe Symbol) 'NoSourceUnpackedness 'NoSourceStrictness 'DecidedLazy) (Rec0 DataRecOrFun_)))) :+: ((C1 ('MetaCons "ModuleArityMismatch_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "ModuleDefinedInOtherFile_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "ModuleNameDoesntMatchFileName_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "ModuleNameUnexpected_" 'PrefixI 'False) (U1 :: Type -> Type)))) :+: (((C1 ('MetaCons "MultipleFixityDecls_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "MultiplePolarityPragmas_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "ExplicitPolarityVsPragma_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "ConstructorNameOfNonRecord_" 'PrefixI 'False) (U1 :: Type -> Type))) :+: ((C1 ('MetaCons "NamedWhereModuleInRefinedContext_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "NeedOptionAllowExec_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "NeedOptionCopatterns_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "NeedOptionCubical_" 'PrefixI 'False) (U1 :: Type -> Type))))) :+: (((C1 ('MetaCons "NeedOptionPatternMatching_" 'PrefixI 'False) (U1 :: Type -> Type) :+: (C1 ('MetaCons "NeedOptionProp_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "NeedOptionRewriting_" 'PrefixI 'False) (U1 :: Type -> Type))) :+: ((C1 ('MetaCons "NeedOptionSizedTypes_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "NeedOptionTwoLevel_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "NeedOptionUniversePolymorphism_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "NegativeLiteralInPattern_" 'PrefixI 'False) (U1 :: Type -> Type)))) :+: (((C1 ('MetaCons "NoBindingForBuiltin_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "NoBindingForPrimitive_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "NoKnownRecordWithSuchFields_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "NoParameterOfName_" 'PrefixI 'False) (U1 :: Type -> Type))) :+: ((C1 ('MetaCons "NoParseForApplication_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "NoParseForLHS_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "NoSuchBuiltinName_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "NoSuchModule_" 'PrefixI 'False) (U1 :: Type -> Type)))))) :+: ((((C1 ('MetaCons "NoSuchPrimitiveFunction_" 'PrefixI 'False) (U1 :: Type -> Type) :+: (C1 ('MetaCons "NotAValidLetBinding_" 'PrefixI 'False) (S1 ('MetaSel ('Nothing :: Maybe Symbol) 'NoSourceUnpackedness 'NoSourceStrictness 'DecidedLazy) (Rec0 (Maybe NotAValidLetBinding))) :+: C1 ('MetaCons "NotAValidLetExpression_" 'PrefixI 'False) (S1 ('MetaSel ('Nothing :: Maybe Symbol) 'NoSourceUnpackedness 'NoSourceStrictness 'DecidedLazy) (Rec0 NotAValidLetExpression)))) :+: ((C1 ('MetaCons "NotAllowedInDotPatterns_" 'PrefixI 'False) (S1 ('MetaSel ('Nothing :: Maybe Symbol) 'NoSourceUnpackedness 'NoSourceStrictness 'DecidedLazy) (Rec0 NotAllowedInDotPatterns)) :+: C1 ('MetaCons "NotAnExpression_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "NotInScope_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "NotLeqSort_" 'PrefixI 'False) (U1 :: Type -> Type)))) :+: (((C1 ('MetaCons "NotValidBeforeField_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "OpenEverythingInRecordWhere_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "OverlappingProjects_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "PathAbstractionFailed_" 'PrefixI 'False) (U1 :: Type -> Type))) :+: ((C1 ('MetaCons "PatternInPathLambda_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "PatternInSystem_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "PatternSynonymArgumentShadows_" 'PrefixI 'False) (S1 ('MetaSel ('Nothing :: Maybe Symbol) 'NoSourceUnpackedness 'NoSourceStrictness 'DecidedLazy) (Rec0 ConstructorOrPatternSynonym)) :+: C1 ('MetaCons "PostulatedSizeInModule_" 'PrefixI 'False) (U1 :: Type -> Type))))) :+: (((C1 ('MetaCons "PrivateRecordField_" 'PrefixI 'False) (U1 :: Type -> Type) :+: (C1 ('MetaCons "ProjectionIsIrrelevant_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "QualifiedLocalModule_" 'PrefixI 'False) (U1 :: Type -> Type))) :+: ((C1 ('MetaCons "QuantityMismatch_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "RecordIsErased_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "RecursiveRecordNeedsInductivity_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "ReferencesFutureVariables_" 'PrefixI 'False) (U1 :: Type -> Type)))) :+: (((C1 ('MetaCons "RelevanceMismatch_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "RepeatedNamesInImportDirective_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "RepeatedVariablesInPattern_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "ShadowedModule_" 'PrefixI 'False) (U1 :: Type -> Type))) :+: ((C1 ('MetaCons "ShouldBeASort_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "ShouldBeEmpty_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "ShouldBePath_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "ShouldBePi_" 'PrefixI 'False) (U1 :: Type -> Type))))))) :+: (((((C1 ('MetaCons "ShouldBeRecordPattern_" 'PrefixI 'False) (U1 :: Type -> Type) :+: (C1 ('MetaCons "ShouldBeRecordType_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "ShouldEndInApplicationOfTheDatatype_" 'PrefixI 'False) (U1 :: Type -> Type))) :+: ((C1 ('MetaCons "SolvedButOpenHoles_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "SortCannotDependOnItsIndex_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "SortDoesNotAdmitDataDefinitions_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "SortOfSplitVarError_" 'PrefixI 'False) (U1 :: Type -> Type)))) :+: (((C1 ('MetaCons "SplitInProp_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "SplitOnAbstract_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "SplitOnCoinductive_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "SplitOnIrrelevant_" 'PrefixI 'False) (U1 :: Type -> Type))) :+: ((C1 ('MetaCons "SplitOnNonEtaRecord_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "SplitOnNonVariable_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "SplitOnPartial_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "SplitOnUnchecked_" 'PrefixI 'False) (U1 :: Type -> Type))))) :+: (((C1 ('MetaCons "SplitOnUnusableCohesion_" 'PrefixI 'False) (U1 :: Type -> Type) :+: (C1 ('MetaCons "SplitOnUnusablePolarity_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "TacticAttributeNotAllowed_" 'PrefixI 'False) (U1 :: Type -> Type))) :+: ((C1 ('MetaCons "TooFewArgumentsToPatternSynonym_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "TooFewPatternsInWithClause_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "TooManyFields_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "TooManyPatternsInWithClause_" 'PrefixI 'False) (U1 :: Type -> Type)))) :+: (((C1 ('MetaCons "TriedToCopyConstrainedPrim_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "InvalidInstanceHeadType_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "UnboundVariablesInPatternSynonym_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "UnequalCohesion_" 'PrefixI 'False) (U1 :: Type -> Type))) :+: ((C1 ('MetaCons "UnequalFiniteness_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "UnequalHiding_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "UnequalLevel_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "UnequalQuantity_" 'PrefixI 'False) (U1 :: Type -> Type)))))) :+: ((((C1 ('MetaCons "UnequalRelevance_" 'PrefixI 'False) (U1 :: Type -> Type) :+: (C1 ('MetaCons "UnequalPolarity_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "UnequalSorts_" 'PrefixI 'False) (U1 :: Type -> Type))) :+: ((C1 ('MetaCons "UnequalTerms_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "UnexpectedModalityAnnotationInParameter_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "UnexpectedParameter_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "UnexpectedTypeSignatureForParameter_" 'PrefixI 'False) (U1 :: Type -> Type)))) :+: (((C1 ('MetaCons "UnexpectedWithPatterns_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "UnknownBackend_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "UnusableAtModality_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "UnusedVariableInPatternSynonym_" 'PrefixI 'False) (U1 :: Type -> Type))) :+: ((C1 ('MetaCons "VariableIsErased_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "VariableIsIrrelevant_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "VariableIsOfUnusableCohesion_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "VariableIsOfUnusablePolarity_" 'PrefixI 'False) (U1 :: Type -> Type))))) :+: (((C1 ('MetaCons "WithClausePatternMismatch_" 'PrefixI 'False) (U1 :: Type -> Type) :+: (C1 ('MetaCons "WithOnFreeVariable_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "WrongAnnotationInLambda_" 'PrefixI 'False) (U1 :: Type -> Type))) :+: ((C1 ('MetaCons "WrongArgInfoForPrimitive_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "WrongCohesionInLambda_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "WrongPolarityInLambda_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "WrongHidingInApplication_" 'PrefixI 'False) (U1 :: Type -> Type)))) :+: (((C1 ('MetaCons "WrongHidingInLHS_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "WrongHidingInLambda_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "WrongHidingInProjection_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "WrongIrrelevanceInLambda_" 'PrefixI 'False) (U1 :: Type -> Type))) :+: ((C1 ('MetaCons "WrongNamedArgument_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "WrongNumberOfConstructorArguments_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "WrongQuantityInLambda_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "WrongSharpArity_" 'PrefixI 'False) (U1 :: Type -> Type)))))))))

data DeclarationException_ Source #

Nicifier errors.

Instances

Instances details
Bounded DeclarationException_ Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

Enum DeclarationException_ Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

Generic DeclarationException_ Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

Associated Types

type Rep DeclarationException_ 
Instance details

Defined in Agda.Interaction.Options.Errors

type Rep DeclarationException_ = D1 ('MetaData "DeclarationException_" "Agda.Interaction.Options.Errors" "Agda-2.8.0-inplace" 'False) (((C1 ('MetaCons "AmbiguousConstructorN_" 'PrefixI 'False) (U1 :: Type -> Type) :+: (C1 ('MetaCons "AmbiguousFunClauses_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "BadMacroDef_" 'PrefixI 'False) (U1 :: Type -> Type))) :+: ((C1 ('MetaCons "DisallowedInterleavedMutual_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "DuplicateAnonDeclaration_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "DuplicateDefinition_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "InvalidMeasureMutual_" 'PrefixI 'False) (U1 :: Type -> Type)))) :+: ((C1 ('MetaCons "MissingWithClauses_" 'PrefixI 'False) (U1 :: Type -> Type) :+: (C1 ('MetaCons "MultipleEllipses_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "OpaqueInMutual_" 'PrefixI 'False) (U1 :: Type -> Type))) :+: ((C1 ('MetaCons "UnfoldingOutsideOpaque_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "UnquoteDefRequiresSignature_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "WrongContentBlock_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "WrongDefinition_" 'PrefixI 'False) (U1 :: Type -> Type)))))
Show DeclarationException_ Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

type Rep DeclarationException_ Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

type Rep DeclarationException_ = D1 ('MetaData "DeclarationException_" "Agda.Interaction.Options.Errors" "Agda-2.8.0-inplace" 'False) (((C1 ('MetaCons "AmbiguousConstructorN_" 'PrefixI 'False) (U1 :: Type -> Type) :+: (C1 ('MetaCons "AmbiguousFunClauses_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "BadMacroDef_" 'PrefixI 'False) (U1 :: Type -> Type))) :+: ((C1 ('MetaCons "DisallowedInterleavedMutual_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "DuplicateAnonDeclaration_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "DuplicateDefinition_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "InvalidMeasureMutual_" 'PrefixI 'False) (U1 :: Type -> Type)))) :+: ((C1 ('MetaCons "MissingWithClauses_" 'PrefixI 'False) (U1 :: Type -> Type) :+: (C1 ('MetaCons "MultipleEllipses_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "OpaqueInMutual_" 'PrefixI 'False) (U1 :: Type -> Type))) :+: ((C1 ('MetaCons "UnfoldingOutsideOpaque_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "UnquoteDefRequiresSignature_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "WrongContentBlock_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "WrongDefinition_" 'PrefixI 'False) (U1 :: Type -> Type)))))

data GHCBackendError_ Source #

Instances

Instances details
Bounded GHCBackendError_ Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

Enum GHCBackendError_ Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

Generic GHCBackendError_ Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

Associated Types

type Rep GHCBackendError_ 
Instance details

Defined in Agda.Interaction.Options.Errors

type Rep GHCBackendError_ = D1 ('MetaData "GHCBackendError_" "Agda.Interaction.Options.Errors" "Agda-2.8.0-inplace" 'False) (C1 ('MetaCons "ConstructorCountMismatch_" 'PrefixI 'False) (U1 :: Type -> Type) :+: (C1 ('MetaCons "NotAHaskellType_" 'PrefixI 'False) (S1 ('MetaSel ('Nothing :: Maybe Symbol) 'NoSourceUnpackedness 'NoSourceStrictness 'DecidedLazy) (Rec0 NotAHaskellType_)) :+: C1 ('MetaCons "WrongTypeOfMain_" 'PrefixI 'False) (U1 :: Type -> Type)))
Show GHCBackendError_ Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

type Rep GHCBackendError_ Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

type Rep GHCBackendError_ = D1 ('MetaData "GHCBackendError_" "Agda.Interaction.Options.Errors" "Agda-2.8.0-inplace" 'False) (C1 ('MetaCons "ConstructorCountMismatch_" 'PrefixI 'False) (U1 :: Type -> Type) :+: (C1 ('MetaCons "NotAHaskellType_" 'PrefixI 'False) (S1 ('MetaSel ('Nothing :: Maybe Symbol) 'NoSourceUnpackedness 'NoSourceStrictness 'DecidedLazy) (Rec0 NotAHaskellType_)) :+: C1 ('MetaCons "WrongTypeOfMain_" 'PrefixI 'False) (U1 :: Type -> Type)))

data JSBackendError_ Source #

Constructors

BadCompilePragma_ 

Instances

Instances details
Bounded JSBackendError_ Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

Enum JSBackendError_ Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

Generic JSBackendError_ Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

Associated Types

type Rep JSBackendError_ 
Instance details

Defined in Agda.Interaction.Options.Errors

type Rep JSBackendError_ = D1 ('MetaData "JSBackendError_" "Agda.Interaction.Options.Errors" "Agda-2.8.0-inplace" 'False) (C1 ('MetaCons "BadCompilePragma_" 'PrefixI 'False) (U1 :: Type -> Type))
Show JSBackendError_ Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

type Rep JSBackendError_ Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

type Rep JSBackendError_ = D1 ('MetaData "JSBackendError_" "Agda.Interaction.Options.Errors" "Agda-2.8.0-inplace" 'False) (C1 ('MetaCons "BadCompilePragma_" 'PrefixI 'False) (U1 :: Type -> Type))

data InteractionError_ Source #

Instances

Instances details
Bounded InteractionError_ Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

Enum InteractionError_ Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

Generic InteractionError_ Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

Associated Types

type Rep InteractionError_ 
Instance details

Defined in Agda.Interaction.Options.Errors

type Rep InteractionError_ = D1 ('MetaData "InteractionError_" "Agda.Interaction.Options.Errors" "Agda-2.8.0-inplace" 'False) (((C1 ('MetaCons "CannotGive_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "CannotRefine_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "CaseSplitError_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "ExpectedIdentifier_" 'PrefixI 'False) (U1 :: Type -> Type))) :+: ((C1 ('MetaCons "ExpectedApplication_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "NoActionForInteractionPoint_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "NoSuchInteractionPoint_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "UnexpectedWhere_" 'PrefixI 'False) (U1 :: Type -> Type))))
Show InteractionError_ Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

type Rep InteractionError_ Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

type Rep InteractionError_ = D1 ('MetaData "InteractionError_" "Agda.Interaction.Options.Errors" "Agda-2.8.0-inplace" 'False) (((C1 ('MetaCons "CannotGive_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "CannotRefine_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "CaseSplitError_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "ExpectedIdentifier_" 'PrefixI 'False) (U1 :: Type -> Type))) :+: ((C1 ('MetaCons "ExpectedApplication_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "NoActionForInteractionPoint_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "NoSuchInteractionPoint_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "UnexpectedWhere_" 'PrefixI 'False) (U1 :: Type -> Type))))

data NegativeUnification_ Source #

Instances

Instances details
Bounded NegativeUnification_ Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

Enum NegativeUnification_ Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

Generic NegativeUnification_ Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

Associated Types

type Rep NegativeUnification_ 
Instance details

Defined in Agda.Interaction.Options.Errors

type Rep NegativeUnification_ = D1 ('MetaData "NegativeUnification_" "Agda.Interaction.Options.Errors" "Agda-2.8.0-inplace" 'False) (C1 ('MetaCons "UnifyConflict_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "UnifyCycle_" 'PrefixI 'False) (U1 :: Type -> Type))
Show NegativeUnification_ Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

type Rep NegativeUnification_ Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

type Rep NegativeUnification_ = D1 ('MetaData "NegativeUnification_" "Agda.Interaction.Options.Errors" "Agda-2.8.0-inplace" 'False) (C1 ('MetaCons "UnifyConflict_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "UnifyCycle_" 'PrefixI 'False) (U1 :: Type -> Type))

data NotAHaskellType_ Source #

Instances

Instances details
Bounded NotAHaskellType_ Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

Enum NotAHaskellType_ Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

Generic NotAHaskellType_ Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

Associated Types

type Rep NotAHaskellType_ 
Instance details

Defined in Agda.Interaction.Options.Errors

type Rep NotAHaskellType_ = D1 ('MetaData "NotAHaskellType_" "Agda.Interaction.Options.Errors" "Agda-2.8.0-inplace" 'False) ((C1 ('MetaCons "BadDontCare_" 'PrefixI 'False) (U1 :: Type -> Type) :+: (C1 ('MetaCons "BadLambda_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "BadMeta_" 'PrefixI 'False) (U1 :: Type -> Type))) :+: (C1 ('MetaCons "NoPragmaFor_" 'PrefixI 'False) (U1 :: Type -> Type) :+: (C1 ('MetaCons "NotCompiled_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "WrongPragmaFor_" 'PrefixI 'False) (U1 :: Type -> Type))))
Show NotAHaskellType_ Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

type Rep NotAHaskellType_ Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

type Rep NotAHaskellType_ = D1 ('MetaData "NotAHaskellType_" "Agda.Interaction.Options.Errors" "Agda-2.8.0-inplace" 'False) ((C1 ('MetaCons "BadDontCare_" 'PrefixI 'False) (U1 :: Type -> Type) :+: (C1 ('MetaCons "BadLambda_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "BadMeta_" 'PrefixI 'False) (U1 :: Type -> Type))) :+: (C1 ('MetaCons "NoPragmaFor_" 'PrefixI 'False) (U1 :: Type -> Type) :+: (C1 ('MetaCons "NotCompiled_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "WrongPragmaFor_" 'PrefixI 'False) (U1 :: Type -> Type))))

data SplitError_ Source #

Instances

Instances details
Bounded SplitError_ Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

Enum SplitError_ Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

Generic SplitError_ Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

Associated Types

type Rep SplitError_ 
Instance details

Defined in Agda.Interaction.Options.Errors

type Rep SplitError_ = D1 ('MetaData "SplitError_" "Agda.Interaction.Options.Errors" "Agda-2.8.0-inplace" 'False) (((C1 ('MetaCons "ErasedDatatype_" 'PrefixI 'False) (S1 ('MetaSel ('Nothing :: Maybe Symbol) 'NoSourceUnpackedness 'NoSourceStrictness 'DecidedLazy) (Rec0 ErasedDatatypeReason)) :+: C1 ('MetaCons "GenericSplitError_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "BlockedType_" 'PrefixI 'False) (U1 :: Type -> Type) :+: (C1 ('MetaCons "CannotCreateMissingClause_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "CoinductiveDatatype_" 'PrefixI 'False) (U1 :: Type -> Type)))) :+: ((C1 ('MetaCons "CosplitCatchall_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "CosplitNoRecordType_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "CosplitNoTarget_" 'PrefixI 'False) (U1 :: Type -> Type) :+: (C1 ('MetaCons "NotADatatype_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "UnificationStuck_" 'PrefixI 'False) (U1 :: Type -> Type)))))
Show SplitError_ Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

type Rep SplitError_ Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

type Rep SplitError_ = D1 ('MetaData "SplitError_" "Agda.Interaction.Options.Errors" "Agda-2.8.0-inplace" 'False) (((C1 ('MetaCons "ErasedDatatype_" 'PrefixI 'False) (S1 ('MetaSel ('Nothing :: Maybe Symbol) 'NoSourceUnpackedness 'NoSourceStrictness 'DecidedLazy) (Rec0 ErasedDatatypeReason)) :+: C1 ('MetaCons "GenericSplitError_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "BlockedType_" 'PrefixI 'False) (U1 :: Type -> Type) :+: (C1 ('MetaCons "CannotCreateMissingClause_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "CoinductiveDatatype_" 'PrefixI 'False) (U1 :: Type -> Type)))) :+: ((C1 ('MetaCons "CosplitCatchall_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "CosplitNoRecordType_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "CosplitNoTarget_" 'PrefixI 'False) (U1 :: Type -> Type) :+: (C1 ('MetaCons "NotADatatype_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "UnificationStuck_" 'PrefixI 'False) (U1 :: Type -> Type)))))

data CannotQuote_ Source #

Instances

Instances details
Bounded CannotQuote_ Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

Enum CannotQuote_ Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

Generic CannotQuote_ Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

Associated Types

type Rep CannotQuote_ 
Instance details

Defined in Agda.Interaction.Options.Errors

type Rep CannotQuote_ = D1 ('MetaData "CannotQuote_" "Agda.Interaction.Options.Errors" "Agda-2.8.0-inplace" 'False) ((C1 ('MetaCons "CannotQuoteAmbiguous_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "CannotQuoteExpression_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "CannotQuoteHidden_" 'PrefixI 'False) (U1 :: Type -> Type) :+: (C1 ('MetaCons "CannotQuoteNothing_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "CannotQuotePattern_" 'PrefixI 'False) (U1 :: Type -> Type))))
Show CannotQuote_ Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

type Rep CannotQuote_ Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

type Rep CannotQuote_ = D1 ('MetaData "CannotQuote_" "Agda.Interaction.Options.Errors" "Agda-2.8.0-inplace" 'False) ((C1 ('MetaCons "CannotQuoteAmbiguous_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "CannotQuoteExpression_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "CannotQuoteHidden_" 'PrefixI 'False) (U1 :: Type -> Type) :+: (C1 ('MetaCons "CannotQuoteNothing_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "CannotQuotePattern_" 'PrefixI 'False) (U1 :: Type -> Type))))

data ExecError_ Source #

Instances

Instances details
Bounded ExecError_ Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

Enum ExecError_ Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

Generic ExecError_ Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

Associated Types

type Rep ExecError_ 
Instance details

Defined in Agda.Interaction.Options.Errors

type Rep ExecError_ = D1 ('MetaData "ExecError_" "Agda.Interaction.Options.Errors" "Agda-2.8.0-inplace" 'False) (C1 ('MetaCons "ExeNotTrusted_" 'PrefixI 'False) (U1 :: Type -> Type) :+: (C1 ('MetaCons "ExeNotFound_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "ExeNotExecutable_" 'PrefixI 'False) (U1 :: Type -> Type)))
Show ExecError_ Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

type Rep ExecError_ Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

type Rep ExecError_ = D1 ('MetaData "ExecError_" "Agda.Interaction.Options.Errors" "Agda-2.8.0-inplace" 'False) (C1 ('MetaCons "ExeNotTrusted_" 'PrefixI 'False) (U1 :: Type -> Type) :+: (C1 ('MetaCons "ExeNotFound_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "ExeNotExecutable_" 'PrefixI 'False) (U1 :: Type -> Type)))

data UnquoteError_ Source #

Instances

Instances details
Bounded UnquoteError_ Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

Enum UnquoteError_ Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

Generic UnquoteError_ Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

Associated Types

type Rep UnquoteError_ 
Instance details

Defined in Agda.Interaction.Options.Errors

type Rep UnquoteError_ = D1 ('MetaData "UnquoteError_" "Agda.Interaction.Options.Errors" "Agda-2.8.0-inplace" 'False) (((C1 ('MetaCons "BlockedOnMeta_" 'PrefixI 'False) (U1 :: Type -> Type) :+: (C1 ('MetaCons "CannotDeclareHiddenFunction_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "CommitAfterDef_" 'PrefixI 'False) (U1 :: Type -> Type))) :+: ((C1 ('MetaCons "ConInsteadOfDef_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "DefineDataNotData_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "DefInsteadOfCon_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "MissingDeclaration_" 'PrefixI 'False) (U1 :: Type -> Type)))) :+: ((C1 ('MetaCons "MissingDefinition_" 'PrefixI 'False) (U1 :: Type -> Type) :+: (C1 ('MetaCons "NakedUnquote_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "NonCanonical_" 'PrefixI 'False) (U1 :: Type -> Type))) :+: ((C1 ('MetaCons "PatLamWithoutClauses_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "StaleMeta_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "TooManyParameters_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "UnboundName_" 'PrefixI 'False) (U1 :: Type -> Type)))))
Show UnquoteError_ Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

type Rep UnquoteError_ Source # 
Instance details

Defined in Agda.Interaction.Options.Errors

type Rep UnquoteError_ = D1 ('MetaData "UnquoteError_" "Agda.Interaction.Options.Errors" "Agda-2.8.0-inplace" 'False) (((C1 ('MetaCons "BlockedOnMeta_" 'PrefixI 'False) (U1 :: Type -> Type) :+: (C1 ('MetaCons "CannotDeclareHiddenFunction_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "CommitAfterDef_" 'PrefixI 'False) (U1 :: Type -> Type))) :+: ((C1 ('MetaCons "ConInsteadOfDef_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "DefineDataNotData_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "DefInsteadOfCon_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "MissingDeclaration_" 'PrefixI 'False) (U1 :: Type -> Type)))) :+: ((C1 ('MetaCons "MissingDefinition_" 'PrefixI 'False) (U1 :: Type -> Type) :+: (C1 ('MetaCons "NakedUnquote_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "NonCanonical_" 'PrefixI 'False) (U1 :: Type -> Type))) :+: ((C1 ('MetaCons "PatLamWithoutClauses_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "StaleMeta_" 'PrefixI 'False) (U1 :: Type -> Type)) :+: (C1 ('MetaCons "TooManyParameters_" 'PrefixI 'False) (U1 :: Type -> Type) :+: C1 ('MetaCons "UnboundName_" 'PrefixI 'False) (U1 :: Type -> Type)))))

Printing error names

helpErrors :: String Source #

Print list of errors.

Print error messages

Orphan instances

(Bounded a, Enum a) => Bounded (Maybe a) Source # 
Instance details

Methods

minBound :: Maybe a #

maxBound :: Maybe a #

(Bounded a, Enum a) => Enum (Maybe a) Source # 
Instance details

Methods

succ :: Maybe a -> Maybe a #

pred :: Maybe a -> Maybe a #

toEnum :: Int -> Maybe a #

fromEnum :: Maybe a -> Int #

enumFrom :: Maybe a -> [Maybe a] #

enumFromThen :: Maybe a -> Maybe a -> [Maybe a] #

enumFromTo :: Maybe a -> Maybe a -> [Maybe a] #

enumFromThenTo :: Maybe a -> Maybe a -> Maybe a -> [Maybe a] #