| Safe Haskell | None |
|---|---|
| Language | Haskell98 |
TPDB.CPF.Proof.Type
Description
internal representation of CPF termination proofs, see http://cl-informatik.uibk.ac.at/software/cpf/
Synopsis
- data ACTerminationProof = ACTerminationProofFIXME ()
- data ArgumentFilterEntry = ArgumentFilterEntry {}
- data PrecedenceEntry = PrecedenceEntry {}
- data PathOrder = PathOrder [PrecedenceEntry] [ArgumentFilterEntry]
- class ToExotic a where
- data Exotic
- data Coefficient
- = Vector [Coefficient]
- | Matrix [Coefficient]
- | (Eq a, XmlContent a) => Coefficient_Coefficient a
- data Label
- data Symbol
- data ArithFunction
- data Polynomial
- data Value
- data Interpret = Interpret {}
- data Domain
- data Interpretation_Type = Matrix_Interpretation {}
- data Interpretation = Interpretation {}
- data RedPair
- data OrderingConstraintProof = OCPRedPair RedPair
- data DepGraphComponent = DepGraphComponent {
- dgcRealScc :: Bool
- dgcDps :: DPS
- dgcDpProof :: DpProof
- data DpProof
- = PIsEmpty
- | RedPairProc { }
- | DepGraphProc [DepGraphComponent]
- | SemLabProc { }
- | UnlabProc { }
- data Model = FiniteModel Int [Interpret]
- data Transition_Lhs
- data Transition = Transition {}
- data State = State Int
- data TreeAutomaton = TreeAutomaton {
- ta_finalStates :: [State]
- ta_transitions :: [Transition]
- data Criterion = Compatibility
- data ClosedTreeAutomaton = ClosedTreeAutomaton {}
- data Bounds_Type
- data TrsTerminationProof
- = RIsEmpty
- | RuleRemoval { }
- | DpTrans { }
- | Semlab { }
- | Unlab { }
- | StringReversal { }
- | Bounds { }
- data TrsNonterminationProof = TrsNonterminationProofFIXME ()
- data ComplexityClass = ComplexityClassPolynomial {}
- data ComplexityMeasure
- data ComplexityProof = ComplexityProofFIXME ()
- data DPS = (XmlContent s, Typeable s, Eq s) => DPS [Rule (Term Identifier s)]
- data Proof
- data CertificationProblemInput
- = TrsInput { }
- | ComplexityInput { }
- | ACRewriteSystem {
- trsinput_trs :: TRS Identifier Identifier
- asymbols :: [Identifier]
- csymbols :: [Identifier]
- data Tool = Tool {}
- data Origin = ProofOrigin {}
- data CertificationProblem = CertificationProblem {}
- ignoredOrigin :: Origin
- data Identifier
- type TES = TRS Identifier Identifier
Documentation
data ACTerminationProof Source #
Constructors
| ACTerminationProofFIXME () |
Instances
| Eq ACTerminationProof Source # | |
Defined in TPDB.CPF.Proof.Type Methods (==) :: ACTerminationProof -> ACTerminationProof -> Bool # (/=) :: ACTerminationProof -> ACTerminationProof -> Bool # | |
data ArgumentFilterEntry Source #
Constructors
| ArgumentFilterEntry | |
Instances
| Eq ArgumentFilterEntry Source # | |
Defined in TPDB.CPF.Proof.Type Methods (==) :: ArgumentFilterEntry -> ArgumentFilterEntry -> Bool # (/=) :: ArgumentFilterEntry -> ArgumentFilterEntry -> Bool # | |
| XmlContent ArgumentFilterEntry Source # | |
Defined in TPDB.CPF.Proof.Write Methods toContents :: ArgumentFilterEntry -> [Node] Source # parseContents :: Cursor -> [ArgumentFilterEntry] Source # | |
data PrecedenceEntry Source #
Constructors
| PrecedenceEntry | |
Instances
| Eq PrecedenceEntry Source # | |
Defined in TPDB.CPF.Proof.Type Methods (==) :: PrecedenceEntry -> PrecedenceEntry -> Bool # (/=) :: PrecedenceEntry -> PrecedenceEntry -> Bool # | |
| XmlContent PrecedenceEntry Source # | |
Defined in TPDB.CPF.Proof.Write Methods toContents :: PrecedenceEntry -> [Node] Source # parseContents :: Cursor -> [PrecedenceEntry] Source # | |
Constructors
| PathOrder [PrecedenceEntry] [ArgumentFilterEntry] |
Instances
| Eq PathOrder Source # | |
| XmlContent PathOrder Source # | |
Defined in TPDB.CPF.Proof.Write | |
Constructors
| Minus_Infinite | |
| E_Integer Integer | |
| E_Rational Rational | |
| Plus_Infinite |
data Coefficient Source #
Constructors
| Vector [Coefficient] | |
| Matrix [Coefficient] | |
| (Eq a, XmlContent a) => Coefficient_Coefficient a |
Instances
| Eq Coefficient Source # | |
Defined in TPDB.CPF.Proof.Type | |
| XmlContent Coefficient Source # | |
Defined in TPDB.CPF.Proof.Write Methods toContents :: Coefficient -> [Node] Source # parseContents :: Cursor -> [Coefficient] Source # | |
Instances
| Eq Symbol Source # | |
| XmlContent Symbol Source # | |
Defined in TPDB.CPF.Proof.Write | |
| XmlContent (TRS Identifier Symbol) Source # | |
Defined in TPDB.CPF.Proof.Write Methods toContents :: TRS Identifier Symbol -> [Node] Source # parseContents :: Cursor -> [TRS Identifier Symbol] Source # | |
data ArithFunction Source #
Constructors
| AFNatural Integer | |
| AFVariable Integer | |
| AFSum [ArithFunction] | |
| AFProduct [ArithFunction] | |
| AFMin [ArithFunction] | |
| AFMax [ArithFunction] | |
| AFIfEqual ArithFunction ArithFunction ArithFunction ArithFunction |
Instances
| Eq ArithFunction Source # | |
Defined in TPDB.CPF.Proof.Type Methods (==) :: ArithFunction -> ArithFunction -> Bool # (/=) :: ArithFunction -> ArithFunction -> Bool # | |
| XmlContent ArithFunction Source # | |
Defined in TPDB.CPF.Proof.Write Methods toContents :: ArithFunction -> [Node] Source # parseContents :: Cursor -> [ArithFunction] Source # | |
data Polynomial Source #
Constructors
| Sum [Polynomial] | |
| Product [Polynomial] | |
| Polynomial_Coefficient Coefficient | |
| Polynomial_Variable Text |
Instances
| Eq Polynomial Source # | |
Defined in TPDB.CPF.Proof.Type | |
| XmlContent Polynomial Source # | |
Defined in TPDB.CPF.Proof.Write | |
Constructors
| Polynomial Polynomial | |
| ArithFunction ArithFunction |
Instances
| Eq Interpret Source # | |
| XmlContent Interpret Source # | |
Defined in TPDB.CPF.Proof.Write | |
data Interpretation_Type Source #
Constructors
| Matrix_Interpretation | |
Instances
| Eq Interpretation_Type Source # | |
Defined in TPDB.CPF.Proof.Type Methods (==) :: Interpretation_Type -> Interpretation_Type -> Bool # (/=) :: Interpretation_Type -> Interpretation_Type -> Bool # | |
| XmlContent Interpretation_Type Source # | |
Defined in TPDB.CPF.Proof.Write Methods toContents :: Interpretation_Type -> [Node] Source # parseContents :: Cursor -> [Interpretation_Type] Source # | |
data Interpretation Source #
Constructors
| Interpretation | |
Fields | |
Instances
| Eq Interpretation Source # | |
Defined in TPDB.CPF.Proof.Type Methods (==) :: Interpretation -> Interpretation -> Bool # (/=) :: Interpretation -> Interpretation -> Bool # | |
| XmlContent Interpretation Source # | |
Defined in TPDB.CPF.Proof.Write Methods toContents :: Interpretation -> [Node] Source # parseContents :: Cursor -> [Interpretation] Source # | |
Constructors
| RPInterpretation Interpretation | |
| RPPathOrder PathOrder |
data OrderingConstraintProof Source #
Constructors
| OCPRedPair RedPair |
Instances
| Eq OrderingConstraintProof Source # | |
Defined in TPDB.CPF.Proof.Type Methods (==) :: OrderingConstraintProof -> OrderingConstraintProof -> Bool # (/=) :: OrderingConstraintProof -> OrderingConstraintProof -> Bool # | |
| XmlContent OrderingConstraintProof Source # | |
Defined in TPDB.CPF.Proof.Write Methods toContents :: OrderingConstraintProof -> [Node] Source # parseContents :: Cursor -> [OrderingConstraintProof] Source # | |
data DepGraphComponent Source #
Constructors
| DepGraphComponent | |
Fields
| |
Instances
| Eq DepGraphComponent Source # | |
Defined in TPDB.CPF.Proof.Type Methods (==) :: DepGraphComponent -> DepGraphComponent -> Bool # (/=) :: DepGraphComponent -> DepGraphComponent -> Bool # | |
| XmlContent DepGraphComponent Source # | |
Defined in TPDB.CPF.Proof.Write Methods toContents :: DepGraphComponent -> [Node] Source # parseContents :: Cursor -> [DepGraphComponent] Source # | |
Constructors
| PIsEmpty | |
| RedPairProc | |
Fields | |
| DepGraphProc [DepGraphComponent] | |
| SemLabProc | |
| UnlabProc | |
Constructors
| FiniteModel Int [Interpret] |
data Transition_Lhs Source #
Constructors
| Transition_Symbol | |
| Transition_Epsilon State | |
Instances
| Eq Transition_Lhs Source # | |
Defined in TPDB.CPF.Proof.Type Methods (==) :: Transition_Lhs -> Transition_Lhs -> Bool # (/=) :: Transition_Lhs -> Transition_Lhs -> Bool # | |
| XmlContent Transition_Lhs Source # | |
Defined in TPDB.CPF.Proof.Write Methods toContents :: Transition_Lhs -> [Node] Source # parseContents :: Cursor -> [Transition_Lhs] Source # | |
data Transition Source #
Constructors
| Transition | |
Fields | |
Instances
| Eq Transition Source # | |
Defined in TPDB.CPF.Proof.Type | |
| XmlContent Transition Source # | |
Defined in TPDB.CPF.Proof.Write | |
data TreeAutomaton Source #
Constructors
| TreeAutomaton | |
Fields
| |
Instances
| Eq TreeAutomaton Source # | |
Defined in TPDB.CPF.Proof.Type Methods (==) :: TreeAutomaton -> TreeAutomaton -> Bool # (/=) :: TreeAutomaton -> TreeAutomaton -> Bool # | |
| XmlContent TreeAutomaton Source # | |
Defined in TPDB.CPF.Proof.Write Methods toContents :: TreeAutomaton -> [Node] Source # parseContents :: Cursor -> [TreeAutomaton] Source # | |
Constructors
| Compatibility |
Instances
| Eq Criterion Source # | |
| XmlContent Criterion Source # | |
Defined in TPDB.CPF.Proof.Write | |
data ClosedTreeAutomaton Source #
Constructors
| ClosedTreeAutomaton | |
Fields | |
Instances
| Eq ClosedTreeAutomaton Source # | |
Defined in TPDB.CPF.Proof.Type Methods (==) :: ClosedTreeAutomaton -> ClosedTreeAutomaton -> Bool # (/=) :: ClosedTreeAutomaton -> ClosedTreeAutomaton -> Bool # | |
| XmlContent ClosedTreeAutomaton Source # | |
Defined in TPDB.CPF.Proof.Write Methods toContents :: ClosedTreeAutomaton -> [Node] Source # parseContents :: Cursor -> [ClosedTreeAutomaton] Source # | |
data Bounds_Type Source #
Instances
| Eq Bounds_Type Source # | |
Defined in TPDB.CPF.Proof.Type | |
| XmlContent Bounds_Type Source # | |
Defined in TPDB.CPF.Proof.Write Methods toContents :: Bounds_Type -> [Node] Source # parseContents :: Cursor -> [Bounds_Type] Source # | |
data TrsTerminationProof Source #
Constructors
| RIsEmpty | |
| RuleRemoval | |
| DpTrans | |
Fields
| |
| Semlab | |
Fields | |
| Unlab | |
Fields | |
| StringReversal | |
Fields | |
| Bounds | |
Fields | |
Instances
| Eq TrsTerminationProof Source # | |
Defined in TPDB.CPF.Proof.Type Methods (==) :: TrsTerminationProof -> TrsTerminationProof -> Bool # (/=) :: TrsTerminationProof -> TrsTerminationProof -> Bool # | |
| XmlContent TrsTerminationProof Source # | |
Defined in TPDB.CPF.Proof.Write Methods toContents :: TrsTerminationProof -> [Node] Source # parseContents :: Cursor -> [TrsTerminationProof] Source # | |
data TrsNonterminationProof Source #
Constructors
| TrsNonterminationProofFIXME () |
Instances
| Eq TrsNonterminationProof Source # | |
Defined in TPDB.CPF.Proof.Type Methods (==) :: TrsNonterminationProof -> TrsNonterminationProof -> Bool # (/=) :: TrsNonterminationProof -> TrsNonterminationProof -> Bool # | |
data ComplexityClass Source #
Constructors
| ComplexityClassPolynomial | it seems the degree must always be given in CPF, although the category spec also allows POLY http://cl-informatik.uibk.ac.at/users/georg/cbr/competition/rules.php |
Instances
| Eq ComplexityClass Source # | |
Defined in TPDB.CPF.Proof.Type Methods (==) :: ComplexityClass -> ComplexityClass -> Bool # (/=) :: ComplexityClass -> ComplexityClass -> Bool # | |
| Show ComplexityClass Source # | |
Defined in TPDB.CPF.Proof.Type Methods showsPrec :: Int -> ComplexityClass -> ShowS # show :: ComplexityClass -> String # showList :: [ComplexityClass] -> ShowS # | |
data ComplexityMeasure Source #
Constructors
| DerivationalComplexity | |
| RuntimeComplexity |
Instances
| Eq ComplexityMeasure Source # | |
Defined in TPDB.CPF.Proof.Type Methods (==) :: ComplexityMeasure -> ComplexityMeasure -> Bool # (/=) :: ComplexityMeasure -> ComplexityMeasure -> Bool # | |
| Show ComplexityMeasure Source # | |
Defined in TPDB.CPF.Proof.Type Methods showsPrec :: Int -> ComplexityMeasure -> ShowS # show :: ComplexityMeasure -> String # showList :: [ComplexityMeasure] -> ShowS # | |
data ComplexityProof Source #
Constructors
| ComplexityProofFIXME () |
Instances
| Eq ComplexityProof Source # | |
Defined in TPDB.CPF.Proof.Type Methods (==) :: ComplexityProof -> ComplexityProof -> Bool # (/=) :: ComplexityProof -> ComplexityProof -> Bool # | |
Constructors
| (XmlContent s, Typeable s, Eq s) => DPS [Rule (Term Identifier s)] |
data CertificationProblemInput Source #
Constructors
| TrsInput | this is actually not true, since instead of copying from XTC, CPF format repeats the definition of TRS, and it's a different one (relative rules are extra) |
Fields | |
| ComplexityInput | |
| ACRewriteSystem | |
Fields
| |
Instances
| Eq CertificationProblemInput Source # | |
Defined in TPDB.CPF.Proof.Type Methods (==) :: CertificationProblemInput -> CertificationProblemInput -> Bool # (/=) :: CertificationProblemInput -> CertificationProblemInput -> Bool # | |
| Pretty CertificationProblemInput Source # | |
Defined in TPDB.CPF.Proof.Type Methods pretty :: CertificationProblemInput -> Doc ann # prettyList :: [CertificationProblemInput] -> Doc ann # | |
| XmlContent CertificationProblemInput Source # | |
Defined in TPDB.CPF.Proof.Write Methods toContents :: CertificationProblemInput -> [Node] Source # parseContents :: Cursor -> [CertificationProblemInput] Source # | |
Constructors
| ProofOrigin | |
data CertificationProblem Source #
Constructors
| CertificationProblem | |
Fields
| |
Instances
| Eq CertificationProblem Source # | |
Defined in TPDB.CPF.Proof.Type Methods (==) :: CertificationProblem -> CertificationProblem -> Bool # (/=) :: CertificationProblem -> CertificationProblem -> Bool # | |
| XmlContent CertificationProblem Source # | |
Defined in TPDB.CPF.Proof.Write Methods toContents :: CertificationProblem -> [Node] Source # parseContents :: Cursor -> [CertificationProblem] Source # | |
data Identifier Source #
Instances
type TES = TRS Identifier Identifier Source #
legacy stuff (used in matchbox)