object Mizar

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

Type Members

  1. class Quantifier extends AnyRef

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. val HiddenTh: MPath
  5. val MizarInformal: MPath
  6. val MizarPatternsTh: MPath
  7. val MizarTh: MPath
  8. def adjective(cluster: Term, typ: Term): Term
  9. def and(tms: List[Term]): Term
  10. def andCon: GlobalName
  11. val any: Term
  12. def apply(f: Term, args: Term*): Term
  13. final def asInstanceOf[T0]: T0
    Definition Classes
    Any
  14. def attr(t: Term): Term
  15. def be(t1: Term, t2: Term): Term
  16. def by: Term
  17. def choice(tp: Term): Term
  18. def clone(): AnyRef
    Attributes
    protected[lang]
    Definition Classes
    AnyRef
    Annotations
    @throws( ... ) @native()
  19. def cluster(a1: Term, a2: Term): Term
  20. def compact(t: Term): Term
  21. def constant(name: String): Term
  22. def constantName(name: String): GlobalName
  23. final def eq(arg0: AnyRef): Boolean
    Definition Classes
    AnyRef
  24. def eqCon: GlobalName
  25. def equals(arg0: Any): Boolean
    Definition Classes
    AnyRef → Any
  26. def falseCon: Term
  27. def finalize(): Unit
    Attributes
    protected[lang]
    Definition Classes
    AnyRef
    Annotations
    @throws( classOf[java.lang.Throwable] )
  28. def fraenkel(v: String, t: Term, p: Term, f: Term): Term
  29. def from: Term
  30. final def getClass(): Class[_]
    Definition Classes
    AnyRef → Any
    Annotations
    @native()
  31. def hashCode(): Int
    Definition Classes
    AnyRef → Any
    Annotations
    @native()
  32. def is(t1: Term, t2: Term): Term
  33. final def isInstanceOf[T0]: Boolean
    Definition Classes
    Any
  34. val mathHubBase: String
  35. val mmlBase: URI
  36. final def ne(arg0: AnyRef): Boolean
    Definition Classes
    AnyRef
  37. final def notify(): Unit
    Definition Classes
    AnyRef
    Annotations
    @native()
  38. final def notifyAll(): Unit
    Definition Classes
    AnyRef
    Annotations
    @native()
  39. def num(i: Int): OMLIT
  40. val numRT: RepresentedRealizedType[BigInt]
  41. def or(tms: List[Term]): Term
  42. def orCon: GlobalName
  43. def prop: Term
  44. def seqConn(connective: String, length: Term, seq: Term): Term
  45. def set: Term
  46. final def synchronized[T0](arg0: ⇒ T0): T0
    Definition Classes
    AnyRef
  47. def toString(): String
    Definition Classes
    AnyRef → Any
  48. def tp: Term
  49. def trueCon: Term
  50. final def wait(): Unit
    Definition Classes
    AnyRef
    Annotations
    @throws( ... )
  51. final def wait(arg0: Long, arg1: Int): Unit
    Definition Classes
    AnyRef
    Annotations
    @throws( ... )
  52. final def wait(arg0: Long): Unit
    Definition Classes
    AnyRef
    Annotations
    @throws( ... ) @native()
  53. object eq extends BinaryLFConstantScala
  54. object exists extends Quantifier
  55. object forall extends Quantifier
  56. object iff extends BinaryLFConstantScala
  57. object implies extends BinaryLFConstantScala
  58. object not extends UnaryLFConstantScala
  59. object proof extends UnaryLFConstantScala

Inherited from AnyRef

Inherited from Any

Ungrouped