SumOfOnesExampleProof

gapt.examples.sequence.SumOfOnesExampleProof

Functions to construct cut-free FOL LK proofs of the sequents

Refl, Trans, CongSuc, ABase, ASuc :- sum( n ) = s^n^(0)

where n is an Integer parameter >= 0.

Attributes

Source
SumOfOnesExampleProof.scala
Graph
Supertypes
class Object
trait Matchable
class Any
Self type

Members list

Value members

Concrete methods

def apply(n: Int): LKProof

Attributes

Source
SumOfOnesExampleProof.scala

Inherited methods

def name: String

Attributes

Inherited from:
ProofSequence
Source
ProofSequence.scala