Packages

case object WDiGraph extends Product with Serializable

Factory for weighted directed graphs.

Linear Supertypes
Ordering
  1. Alphabetic
  2. By Inheritance
Inherited
  1. WDiGraph
  2. Serializable
  3. Product
  4. Equals
  5. AnyRef
  6. Any
  1. Hide All
  2. Show All
Visibility
  1. Public
  2. Protected

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[T, X](vertices: Set[T], edges: Set[WDiEdge[Node[T]]])(implicit arg0: ClassTag[X]): WDiGraph[T]

    Creates a weighted directed graph from a set of base values and a set of edges.

    Creates a weighted directed graph from a set of base values and a set of edges.

    Will map base values to the Node wrapper and then construct the directed graph.

    T

    The type of the directed graph vertices.

    X

    A scala.reflect.ClassTag to prevent type erasure of the edges.

    vertices

    The set of base values representing the vertices.

    edges

    The set of edges.

    returns

    A directed graph.

  5. def apply[T, X](edges: Set[WDiEdge[Node[T]]])(implicit arg0: ClassTag[X]): WDiGraph[T]

    Creates a weighted directed graph from a set of edges.

    Creates a weighted directed graph from a set of edges.

    Will automatically add the vertices from the edges, without explicitly passing them to the constructor.

    T

    The type of the directed graph vertices.

    X

    A scala.reflect.ClassTag to prevent type erasure of the edges.

    edges

    The set of edges.

    returns

    A directed graph of type T.

  6. def apply[T](vertices: Set[Node[T]]): WDiGraph[T]

    Creates a weighted directed graph without edges from a set of vertices.

    Creates a weighted directed graph without edges from a set of vertices.

    T

    The type of the directed graph vertices.

    vertices

    A set of vertices.

    returns

    A directed graph of type T with only the vertices.

  7. final def asInstanceOf[T0]: T0
    Definition Classes
    Any
  8. def clone(): AnyRef
    Attributes
    protected[lang]
    Definition Classes
    AnyRef
    Annotations
    @throws(classOf[java.lang.CloneNotSupportedException]) @native() @IntrinsicCandidate()
  9. def empty[T]: WDiGraph[T]

    Creates an empty weighted directed graph of type T.

    Creates an empty weighted directed graph of type T.

    T

    The type of the directed graph vertices.

    returns

    An empty directed graph of type T.

  10. final def eq(arg0: AnyRef): Boolean
    Definition Classes
    AnyRef
  11. def equals(arg0: AnyRef): Boolean
    Definition Classes
    AnyRef → Any
  12. final def getClass(): Class[_ <: AnyRef]
    Definition Classes
    AnyRef → Any
    Annotations
    @native() @IntrinsicCandidate()
  13. final def isInstanceOf[T0]: Boolean
    Definition Classes
    Any
  14. final def ne(arg0: AnyRef): Boolean
    Definition Classes
    AnyRef
  15. final def notify(): Unit
    Definition Classes
    AnyRef
    Annotations
    @native() @IntrinsicCandidate()
  16. final def notifyAll(): Unit
    Definition Classes
    AnyRef
    Annotations
    @native() @IntrinsicCandidate()
  17. def productElementName(n: Int): String
    Definition Classes
    Product
  18. def productElementNames: Iterator[String]
    Definition Classes
    Product
  19. def productIterator: Iterator[Any]
    Definition Classes
    Product
  20. def random(n: Int, p: Double): WDiGraph[String]

    Helper factory to generate a random weighted directed graph of type java.lang.String for n vertices.

    Helper factory to generate a random weighted directed graph of type java.lang.String for n vertices.

    Uses the Erdős–Rényi–Gilbert model. Weights are random sampled between 0 and 1.

    n

    The number of vertices.

    p

    The probability of an edge existing.

    returns

    A random graph.

  21. def random[T](objects: Set[T], p: Double): WDiGraph[T]

    Generate a random weighted directed graph.

    Generate a random weighted directed graph.

    Graphs are generated according to the Erdős–Rényi–Gilbert model, which states that between each pair of objects there is a p probability of an edge existing. Weights are random sampled between 0 and 1.

    T

    The type of the graph and objects.

    objects

    The set of objects representing the vertices.

    p

    The probability of an edge existing.

    returns

    A random graph.

  22. final def synchronized[T0](arg0: => T0): T0
    Definition Classes
    AnyRef
  23. def uniform(n: Int, numberEdges: Int): WDiGraph[String]

    Helper factory to generate a random weighted directed graph of type java.lang.String for n vertices.

    Helper factory to generate a random weighted directed graph of type java.lang.String for n vertices.

    Uses the uniform model and weights are random sampled between 0 and 1.

    n

    The number of vertices.

    numberEdges

    The number of edges.

    returns

    A random graph.

  24. def uniform[T](objects: Set[T], numberEdges: Int): WDiGraph[T]

    Generate a random weighted directed graph.

    Generate a random weighted directed graph.

    Graphs are generated according to the uniform model, which states that given a number of fixed edges will uniformly distribute those edges between all pairs of objects. Weights are random sampled between 0 and 1. The probability of an edge existing in the final graph is the same as in the Erdős–Rényi–Gilbert model.

    T

    The type of the graph and objects.

    objects

    The set of objects representing the vertices.

    numberEdges

    The number of edges.

    returns

    A random graph.

  25. final def wait(arg0: Long, arg1: Int): Unit
    Definition Classes
    AnyRef
    Annotations
    @throws(classOf[java.lang.InterruptedException])
  26. final def wait(arg0: Long): Unit
    Definition Classes
    AnyRef
    Annotations
    @throws(classOf[java.lang.InterruptedException])
  27. final def wait(): Unit
    Definition Classes
    AnyRef
    Annotations
    @throws(classOf[java.lang.InterruptedException])

Deprecated Value Members

  1. def finalize(): Unit
    Attributes
    protected[lang]
    Definition Classes
    AnyRef
    Annotations
    @throws(classOf[java.lang.Throwable]) @Deprecated
    Deprecated

Inherited from Serializable

Inherited from Product

Inherited from Equals

Inherited from AnyRef

Inherited from Any

Ungrouped