o

gapt.examples.sequence

FactorialFunctionEqualityExampleProof

object FactorialFunctionEqualityExampleProof extends ProofSequence

Proof of f(n) = g(n, 1), where f is the head recursive and g the tail recursive formulation of the factorial function

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

Value Members

  1. final def !=(arg0: Any): Boolean
    Definition Classes
    AnyRef → Any
  2. final def ##(): Int
    Definition Classes
    AnyRef → Any
  3. final def ==(arg0: Any): Boolean
    Definition Classes
    AnyRef → Any
  4. def apply(n: Int): LKProof
  5. final def asInstanceOf[T0]: T0
    Definition Classes
    Any
  6. val assoc_mul_axiom: AllQuantifiedConditionalAxiomHelper
  7. def clone(): AnyRef
    Attributes
    protected[java.lang]
    Definition Classes
    AnyRef
    Annotations
    @throws(classOf[java.lang.CloneNotSupportedException]) @native()
  8. val compat_mul_axiom: AllQuantifiedConditionalAxiomHelper
  9. final def eq(arg0: AnyRef): Boolean
    Definition Classes
    AnyRef
  10. def equals(arg0: AnyRef): Boolean
    Definition Classes
    AnyRef → Any
  11. val f: String
  12. def f1(sym: String, arg: FOLTerm): FOLTerm
  13. def f2(arg1: FOLTerm, sym: String, arg2: FOLTerm): FOLTerm
  14. def f2(sym: String, arg1: FOLTerm, arg2: FOLTerm): FOLTerm
  15. val f_ax_1: FOLAtom
  16. val f_ax_2: FOLFormula
  17. def finalize(): Unit
    Attributes
    protected[java.lang]
    Definition Classes
    AnyRef
    Annotations
    @throws(classOf[java.lang.Throwable])
  18. val g: String
  19. val g_ax_1: AllQuantifiedConditionalAxiomHelper
  20. val g_ax_2: FOLFormula
  21. val g_compat_2: AllQuantifiedConditionalAxiomHelper
  22. final def getClass(): Class[_ <: AnyRef]
    Definition Classes
    AnyRef → Any
    Annotations
    @native()
  23. def hashCode(): Int
    Definition Classes
    AnyRef → Any
    Annotations
    @native()
  24. def induction_steps(n: Int): LKProof
  25. final def isInstanceOf[T0]: Boolean
    Definition Classes
    Any
  26. val m: String
  27. val mul_neutral_axiom: AllQuantifiedConditionalAxiomHelper
  28. val mul_neutral_axiom_2: AllQuantifiedConditionalAxiomHelper
  29. def name: String
    Definition Classes
    ProofSequence
  30. final def ne(arg0: AnyRef): Boolean
    Definition Classes
    AnyRef
  31. final def notify(): Unit
    Definition Classes
    AnyRef
    Annotations
    @native()
  32. final def notifyAll(): Unit
    Definition Classes
    AnyRef
    Annotations
    @native()
  33. val p: String
  34. val refl_axiom: AllQuantifiedConditionalAxiomHelper
  35. val s: String
  36. val symm_axiom: FOLFormula
  37. final def synchronized[T0](arg0: => T0): T0
    Definition Classes
    AnyRef
  38. def toString(): String
    Definition Classes
    AnyRef → Any
  39. val trans_axiom: AllQuantifiedConditionalAxiomHelper
  40. final def wait(): Unit
    Definition Classes
    AnyRef
    Annotations
    @throws(classOf[java.lang.InterruptedException])
  41. final def wait(arg0: Long, arg1: Int): Unit
    Definition Classes
    AnyRef
    Annotations
    @throws(classOf[java.lang.InterruptedException])
  42. final def wait(arg0: Long): Unit
    Definition Classes
    AnyRef
    Annotations
    @throws(classOf[java.lang.InterruptedException]) @native()
  43. val x: FOLVar
  44. val y: FOLVar
  45. val z: FOLVar

Inherited from ProofSequence

Inherited from AnyRef

Inherited from Any

Ungrouped