Object

at.logic.gapt.proofs.lk

regularize

Related Doc: package lk

Permalink

object regularize extends LKVisitor[Set[Var]]

Proof regularization

Source
Utils.scala
Linear Supertypes
Ordering
  1. Alphabetic
  2. By Inheritance
Inherited
  1. regularize
  2. LKVisitor
  3. AnyRef
  4. Any
  1. Hide All
  2. Show All
Visibility
  1. Public
  2. All

Value Members

  1. final def !=(arg0: Any): Boolean

    Permalink
    Definition Classes
    AnyRef → Any
  2. final def ##(): Int

    Permalink
    Definition Classes
    AnyRef → Any
  3. final def ==(arg0: Any): Boolean

    Permalink
    Definition Classes
    AnyRef → Any
  4. def apply(proof: LKProof, blacklist: Seq[Var]): LKProof

    Permalink

    Renames at least the eigenvariables contains in blacklist so that proof becomes regular.

    Renames at least the eigenvariables contains in blacklist so that proof becomes regular.

    proof

    An LKProof.

    blacklist

    A sequence of variables that must be renamed if they occur as eigenvariables.

    returns

    A regular LKProof.

  5. def apply(proof: LKProof): LKProof

    Permalink

    Renames all eigenvariables in a proof so that it becomes regular.

    Renames all eigenvariables in a proof so that it becomes regular.

    proof

    An LKProof.

    returns

    A regular LKProof.

  6. final def apply(proof: LKProof, otherArg: Set[Var]): LKProof

    Permalink

    Applies the proof transformation to an LKProof.

    Applies the proof transformation to an LKProof.

    proof

    The input proof.

    returns

    The transformed proof.

    Definition Classes
    LKVisitor
  7. final def asInstanceOf[T0]: T0

    Permalink
    Definition Classes
    Any
  8. def clone(): AnyRef

    Permalink
    Attributes
    protected[java.lang]
    Definition Classes
    AnyRef
    Annotations
    @throws( ... )
  9. final def eq(arg0: AnyRef): Boolean

    Permalink
    Definition Classes
    AnyRef
  10. def equals(arg0: Any): Boolean

    Permalink
    Definition Classes
    AnyRef → Any
  11. def finalize(): Unit

    Permalink
    Attributes
    protected[java.lang]
    Definition Classes
    AnyRef
    Annotations
    @throws( classOf[java.lang.Throwable] )
  12. final def getClass(): Class[_]

    Permalink
    Definition Classes
    AnyRef → Any
  13. def hashCode(): Int

    Permalink
    Definition Classes
    AnyRef → Any
  14. final def isInstanceOf[T0]: Boolean

    Permalink
    Definition Classes
    Any
  15. final def ne(arg0: AnyRef): Boolean

    Permalink
    Definition Classes
    AnyRef
  16. final def notify(): Unit

    Permalink
    Definition Classes
    AnyRef
  17. final def notifyAll(): Unit

    Permalink
    Definition Classes
    AnyRef
  18. final def recurse(proof: LKProof, otherArg: Set[Var]): (LKProof, OccConnector[HOLFormula], Set[Var])

    Permalink
    Definition Classes
    LKVisitor
  19. final def synchronized[T0](arg0: ⇒ T0): T0

    Permalink
    Definition Classes
    AnyRef
  20. def toString(): String

    Permalink
    Definition Classes
    AnyRef → Any
  21. def visitAndLeft(proof: AndLeftRule, otherArg: Set[Var]): (LKProof, OccConnector[HOLFormula], Set[Var])

    Permalink
    Attributes
    protected
    Definition Classes
    LKVisitor
  22. def visitAndRight(proof: AndRightRule, otherArg: Set[Var]): (LKProof, OccConnector[HOLFormula], Set[Var])

    Permalink
    Attributes
    protected
    Definition Classes
    LKVisitor
  23. def visitBottomAxiom(otherArg: Set[Var]): (LKProof, OccConnector[HOLFormula], Set[Var])

    Permalink
    Attributes
    protected
    Definition Classes
    LKVisitor
  24. def visitContractionLeft(proof: ContractionLeftRule, otherArg: Set[Var]): (LKProof, OccConnector[HOLFormula], Set[Var])

    Permalink
    Attributes
    protected
    Definition Classes
    LKVisitor
  25. def visitContractionRight(proof: ContractionRightRule, otherArg: Set[Var]): (LKProof, OccConnector[HOLFormula], Set[Var])

    Permalink
    Attributes
    protected
    Definition Classes
    LKVisitor
  26. def visitCut(proof: CutRule, otherArg: Set[Var]): (LKProof, OccConnector[HOLFormula], Set[Var])

    Permalink
    Attributes
    protected
    Definition Classes
    LKVisitor
  27. def visitDefinitionLeft(proof: DefinitionLeftRule, otherArg: Set[Var]): (LKProof, OccConnector[HOLFormula], Set[Var])

    Permalink
    Attributes
    protected
    Definition Classes
    LKVisitor
  28. def visitDefinitionRight(proof: DefinitionRightRule, otherArg: Set[Var]): (LKProof, OccConnector[HOLFormula], Set[Var])

    Permalink
    Attributes
    protected
    Definition Classes
    LKVisitor
  29. def visitEqualityLeft(proof: EqualityLeftRule, otherArg: Set[Var]): (LKProof, OccConnector[HOLFormula], Set[Var])

    Permalink
    Attributes
    protected
    Definition Classes
    LKVisitor
  30. def visitEqualityRight(proof: EqualityRightRule, otherArg: Set[Var]): (LKProof, OccConnector[HOLFormula], Set[Var])

    Permalink
    Attributes
    protected
    Definition Classes
    LKVisitor
  31. def visitExistsLeft(proof: ExistsLeftRule, blacklist: Set[Var]): (ExistsLeftRule, OccConnector[HOLFormula], Set[Var])

    Permalink
    Attributes
    protected
    Definition Classes
    regularizeLKVisitor
  32. def visitExistsRight(proof: ExistsRightRule, otherArg: Set[Var]): (LKProof, OccConnector[HOLFormula], Set[Var])

    Permalink
    Attributes
    protected
    Definition Classes
    LKVisitor
  33. def visitForallLeft(proof: ForallLeftRule, otherArg: Set[Var]): (LKProof, OccConnector[HOLFormula], Set[Var])

    Permalink
    Attributes
    protected
    Definition Classes
    LKVisitor
  34. def visitForallRight(proof: ForallRightRule, blacklist: Set[Var]): (ForallRightRule, OccConnector[HOLFormula], Set[Var])

    Permalink
    Attributes
    protected
    Definition Classes
    regularizeLKVisitor
  35. def visitImpLeft(proof: ImpLeftRule, otherArg: Set[Var]): (LKProof, OccConnector[HOLFormula], Set[Var])

    Permalink
    Attributes
    protected
    Definition Classes
    LKVisitor
  36. def visitImpRight(proof: ImpRightRule, otherArg: Set[Var]): (LKProof, OccConnector[HOLFormula], Set[Var])

    Permalink
    Attributes
    protected
    Definition Classes
    LKVisitor
  37. def visitInduction(proof: InductionRule, blacklist: Set[Var]): (InductionRule, OccConnector[HOLFormula], Set[Var])

    Permalink
    Attributes
    protected
    Definition Classes
    regularizeLKVisitor
  38. def visitLogicalAxiom(proof: LogicalAxiom, otherArg: Set[Var]): (LKProof, OccConnector[HOLFormula], Set[Var])

    Permalink
    Attributes
    protected
    Definition Classes
    LKVisitor
  39. def visitNegLeft(proof: NegLeftRule, otherArg: Set[Var]): (LKProof, OccConnector[HOLFormula], Set[Var])

    Permalink
    Attributes
    protected
    Definition Classes
    LKVisitor
  40. def visitNegRight(proof: NegRightRule, otherArg: Set[Var]): (LKProof, OccConnector[HOLFormula], Set[Var])

    Permalink
    Attributes
    protected
    Definition Classes
    LKVisitor
  41. def visitOpenAssumption(proof: OpenAssumption, otherArg: Set[Var]): (LKProof, OccConnector[HOLFormula], Set[Var])

    Permalink
    Attributes
    protected
    Definition Classes
    LKVisitor
  42. def visitOrLeft(proof: OrLeftRule, otherArg: Set[Var]): (LKProof, OccConnector[HOLFormula], Set[Var])

    Permalink
    Attributes
    protected
    Definition Classes
    LKVisitor
  43. def visitOrRight(proof: OrRightRule, otherArg: Set[Var]): (LKProof, OccConnector[HOLFormula], Set[Var])

    Permalink
    Attributes
    protected
    Definition Classes
    LKVisitor
  44. def visitReflexivityAxiom(proof: ReflexivityAxiom, otherArg: Set[Var]): (LKProof, OccConnector[HOLFormula], Set[Var])

    Permalink
    Attributes
    protected
    Definition Classes
    LKVisitor
  45. def visitTheoryAxiom(proof: TheoryAxiom, otherArg: Set[Var]): (LKProof, OccConnector[HOLFormula], Set[Var])

    Permalink
    Attributes
    protected
    Definition Classes
    LKVisitor
  46. def visitTopAxiom(otherArg: Set[Var]): (LKProof, OccConnector[HOLFormula], Set[Var])

    Permalink
    Attributes
    protected
    Definition Classes
    LKVisitor
  47. def visitWeakeningLeft(proof: WeakeningLeftRule, otherArg: Set[Var]): (LKProof, OccConnector[HOLFormula], Set[Var])

    Permalink
    Attributes
    protected
    Definition Classes
    LKVisitor
  48. def visitWeakeningRight(proof: WeakeningRightRule, otherArg: Set[Var]): (LKProof, OccConnector[HOLFormula], Set[Var])

    Permalink
    Attributes
    protected
    Definition Classes
    LKVisitor
  49. final def wait(): Unit

    Permalink
    Definition Classes
    AnyRef
    Annotations
    @throws( ... )
  50. final def wait(arg0: Long, arg1: Int): Unit

    Permalink
    Definition Classes
    AnyRef
    Annotations
    @throws( ... )
  51. final def wait(arg0: Long): Unit

    Permalink
    Definition Classes
    AnyRef
    Annotations
    @throws( ... )
  52. final def withOccConnector(proof: LKProof, otherArg: Set[Var]): (LKProof, OccConnector[HOLFormula])

    Permalink

    Applies the proof transformation to an LKProof.

    Applies the proof transformation to an LKProof.

    proof

    The input proof.

    returns

    A pair consisting of the transformed proof and an OccConnector relating the two proofs.

    Definition Classes
    LKVisitor

Inherited from LKVisitor[Set[Var]]

Inherited from AnyRef

Inherited from Any

Ungrouped