src/Pure/Concurrent/counter.scala
author wenzelm
Wed, 22 Jan 2025 22:22:19 +0100
changeset 81954 6f2bcdfa9a19
parent 78243 0e221a8128e4
permissions -rw-r--r--
misc tuning: more concise operations on prems (without change of exceptions); discontinue odd clone Drule.cprems_of (see also 991a3feaf270);

/*  Title:      Pure/Concurrent/counter.scala
    Author:     Makarius

Synchronized counter for unique identifiers < 0.

NB: ML ticks forwards, JVM ticks backwards.
*/

package isabelle


object Counter {
  type ID = Long
  def make(): Counter = new Counter
}

final class Counter private {
  private var count: Counter.ID = 0

  def apply(): Counter.ID = synchronized {
    require(count > Long.MinValue, "counter overflow")
    count -= 1
    count
  }

  override def toString: String = count.toString
}