SquareDiagonalExampleProof

gapt.examples.sequence.SquareDiagonalExampleProof

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

P(0,0), ∀x,y. P(x,y) → P(s(x),y), ∀x,y. P(x,y) → P(x,s(y)) :- P(s^n^(0),s^n^(0))

where n is an Integer parameter >= 0.

The proofs constructed here go along the diagonal of P, i.e. one x-step, then one y-step, etc.

Attributes

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

Members list

Value members

Concrete methods

def apply(n: Int): LKProof

Value parameters

n

An integer >= 0.

Attributes

Returns

A proof of P(0,0), ∀x,y. P(x,y) → P(s(x),y), ∀x,y. P(x,y) → P(x,s(y)) :- P(s^n^(0),s^n^(0))

Source
SquareDiagonalExampleProof.scala

Inherited methods

def name: String

Attributes

Inherited from:
ProofSequence
Source
ProofSequence.scala