object pushEqualityInferencesToLeaves2 extends LKVisitor[Unit]
- Alphabetic
- By Inheritance
- pushEqualityInferencesToLeaves2
- LKVisitor
- AnyRef
- Any
- Hide All
- Show All
- Public
- Protected
Value Members
- final def !=(arg0: Any): Boolean
- Definition Classes
- AnyRef → Any
- final def ##: Int
- Definition Classes
- AnyRef → Any
- final def ==(arg0: Any): Boolean
- Definition Classes
- AnyRef → Any
- def apply(p: LKProof): LKProof
- final def apply(proof: LKProof, otherArg: Unit): LKProof
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
- final def asInstanceOf[T0]: T0
- Definition Classes
- Any
- def clone(): AnyRef
- Attributes
- protected[lang]
- Definition Classes
- AnyRef
- Annotations
- @throws(classOf[java.lang.CloneNotSupportedException]) @native() @IntrinsicCandidate()
- def contractAfter[A](visitingFunction: (LKProof, A) => (LKProof, SequentConnector)): (LKProof, A) => (LKProof, SequentConnector)
Transforms a visiting function by inserting contractions after it.
Transforms a visiting function by inserting contractions after it. Only formula occurrences that were not in the old proof -- i.e., that have been added by the visitor -- are contracted.
- visitingFunction
The visiting function after which contractions should be inserted. In most cases, just using
recurse
here should be fine.- returns
A new visiting function that behaves the same as the old one, but contracts all duplicate new formulas at the end.
- Definition Classes
- LKVisitor
- final def eq(arg0: AnyRef): Boolean
- Definition Classes
- AnyRef
- def equals(arg0: AnyRef): Boolean
- Definition Classes
- AnyRef → Any
- final def getClass(): Class[_ <: AnyRef]
- Definition Classes
- AnyRef → Any
- Annotations
- @native() @IntrinsicCandidate()
- def hashCode(): Int
- Definition Classes
- AnyRef → Any
- Annotations
- @native() @IntrinsicCandidate()
- final def isInstanceOf[T0]: Boolean
- Definition Classes
- Any
- final def ne(arg0: AnyRef): Boolean
- Definition Classes
- AnyRef
- final def notify(): Unit
- Definition Classes
- AnyRef
- Annotations
- @native() @IntrinsicCandidate()
- final def notifyAll(): Unit
- Definition Classes
- AnyRef
- Annotations
- @native() @IntrinsicCandidate()
- def one2one(proof: LKProof, arg: Unit)(func: (Seq[(LKProof, SequentConnector)]) => LKProof): (LKProof, SequentConnector)
- Definition Classes
- LKVisitor
- def push(proof: EqualityRule): LKProof
- def push(p: LKProof, eq: Formula, aux: SequentIndex, ctx: Abs): LKProof
Pushes a single equality inferences as far to the leaves as possible, that is, until it reaches an initial sequent or another equality inference.
- def recurse(proof: LKProof, otherArg: Unit): (LKProof, SequentConnector)
- Attributes
- protected
- Definition Classes
- LKVisitor
- final def synchronized[T0](arg0: => T0): T0
- Definition Classes
- AnyRef
- def toString(): String
- Definition Classes
- AnyRef → Any
- def transportToSubProof(arg: Unit, proof: LKProof, subProofIdx: Int): Unit
- Definition Classes
- LKVisitor
- def visitAndLeft(proof: AndLeftRule, otherArg: Unit): (LKProof, SequentConnector)
- Attributes
- protected
- Definition Classes
- LKVisitor
- def visitAndRight(proof: AndRightRule, otherArg: Unit): (LKProof, SequentConnector)
- Attributes
- protected
- Definition Classes
- LKVisitor
- def visitBottomAxiom(otherArg: Unit): (LKProof, SequentConnector)
- Attributes
- protected
- Definition Classes
- LKVisitor
- def visitContractionLeft(proof: ContractionLeftRule, otherArg: Unit): (LKProof, SequentConnector)
- Attributes
- protected
- Definition Classes
- LKVisitor
- def visitContractionRight(proof: ContractionRightRule, otherArg: Unit): (LKProof, SequentConnector)
- Attributes
- protected
- Definition Classes
- LKVisitor
- def visitCut(proof: CutRule, otherArg: Unit): (LKProof, SequentConnector)
- Attributes
- protected
- Definition Classes
- LKVisitor
- def visitDefinitionLeft(proof: ConversionLeftRule, otherArg: Unit): (LKProof, SequentConnector)
- Attributes
- protected
- Definition Classes
- LKVisitor
- def visitDefinitionRight(proof: ConversionRightRule, otherArg: Unit): (LKProof, SequentConnector)
- Attributes
- protected
- Definition Classes
- LKVisitor
- def visitEquality(proof: EqualityRule): (LKProof, SequentConnector)
- def visitEqualityLeft(proof: EqualityLeftRule, otherArg: Unit): (LKProof, SequentConnector)
- Definition Classes
- pushEqualityInferencesToLeaves2 → LKVisitor
- def visitEqualityRight(proof: EqualityRightRule, otherArg: Unit): (LKProof, SequentConnector)
- Definition Classes
- pushEqualityInferencesToLeaves2 → LKVisitor
- def visitExistsLeft(proof: ExistsLeftRule, otherArg: Unit): (LKProof, SequentConnector)
- Attributes
- protected
- Definition Classes
- LKVisitor
- def visitExistsRight(proof: ExistsRightRule, otherArg: Unit): (LKProof, SequentConnector)
- Attributes
- protected
- Definition Classes
- LKVisitor
- def visitExistsSkLeft(proof: ExistsSkLeftRule, otherArg: Unit): (LKProof, SequentConnector)
- Attributes
- protected
- Definition Classes
- LKVisitor
- def visitForallLeft(proof: ForallLeftRule, otherArg: Unit): (LKProof, SequentConnector)
- Attributes
- protected
- Definition Classes
- LKVisitor
- def visitForallRight(proof: ForallRightRule, otherArg: Unit): (LKProof, SequentConnector)
- Attributes
- protected
- Definition Classes
- LKVisitor
- def visitForallSkRight(proof: ForallSkRightRule, otherArg: Unit): (LKProof, SequentConnector)
- Attributes
- protected
- Definition Classes
- LKVisitor
- def visitImpLeft(proof: ImpLeftRule, otherArg: Unit): (LKProof, SequentConnector)
- Attributes
- protected
- Definition Classes
- LKVisitor
- def visitImpRight(proof: ImpRightRule, otherArg: Unit): (LKProof, SequentConnector)
- Attributes
- protected
- Definition Classes
- LKVisitor
- def visitInduction(proof: InductionRule, otherArg: Unit): (LKProof, SequentConnector)
- Attributes
- protected
- Definition Classes
- LKVisitor
- def visitLogicalAxiom(proof: LogicalAxiom, otherArg: Unit): (LKProof, SequentConnector)
- Attributes
- protected
- Definition Classes
- LKVisitor
- def visitNegLeft(proof: NegLeftRule, otherArg: Unit): (LKProof, SequentConnector)
- Attributes
- protected
- Definition Classes
- LKVisitor
- def visitNegRight(proof: NegRightRule, otherArg: Unit): (LKProof, SequentConnector)
- Attributes
- protected
- Definition Classes
- LKVisitor
- def visitOpenAssumption(proof: OpenAssumption, otherArg: Unit): (LKProof, SequentConnector)
- Attributes
- protected
- Definition Classes
- LKVisitor
- def visitOrLeft(proof: OrLeftRule, otherArg: Unit): (LKProof, SequentConnector)
- Attributes
- protected
- Definition Classes
- LKVisitor
- def visitOrRight(proof: OrRightRule, otherArg: Unit): (LKProof, SequentConnector)
- Attributes
- protected
- Definition Classes
- LKVisitor
- def visitProofLink(proof: ProofLink, otherArg: Unit): (LKProof, SequentConnector)
- Attributes
- protected
- Definition Classes
- LKVisitor
- def visitReflexivityAxiom(proof: ReflexivityAxiom, otherArg: Unit): (LKProof, SequentConnector)
- Attributes
- protected
- Definition Classes
- LKVisitor
- def visitTopAxiom(otherArg: Unit): (LKProof, SequentConnector)
- Attributes
- protected
- Definition Classes
- LKVisitor
- def visitWeakeningLeft(proof: WeakeningLeftRule, otherArg: Unit): (LKProof, SequentConnector)
- Attributes
- protected
- Definition Classes
- LKVisitor
- def visitWeakeningRight(proof: WeakeningRightRule, otherArg: Unit): (LKProof, SequentConnector)
- Attributes
- protected
- Definition Classes
- LKVisitor
- final def wait(arg0: Long, arg1: Int): Unit
- Definition Classes
- AnyRef
- Annotations
- @throws(classOf[java.lang.InterruptedException])
- final def wait(arg0: Long): Unit
- Definition Classes
- AnyRef
- Annotations
- @throws(classOf[java.lang.InterruptedException]) @native()
- final def wait(): Unit
- Definition Classes
- AnyRef
- Annotations
- @throws(classOf[java.lang.InterruptedException])
- def withIdentitySequentConnector(proof: LKProof): (LKProof, SequentConnector)
- Definition Classes
- LKVisitor
- final def withSequentConnector(proof: LKProof, otherArg: Unit): (LKProof, SequentConnector)
Applies the proof transformation to an LKProof.
Applies the proof transformation to an LKProof.
- proof
The input proof.
- returns
Transformed proof, and the sequent connector with the new proof as lower sequent and the old proof as upper sequent.
- Definition Classes
- LKVisitor
This is the API documentation for GAPT.
The main package is gapt.