| author | wenzelm | 
| Fri, 17 Aug 2012 18:04:49 +0200 | |
| changeset 48846 | fd3cba82c446 | 
| parent 46712 | 8650d9a95736 | 
| child 56685 | 535d59d4ed12 | 
| permissions | -rw-r--r-- | 
/* Title: Pure/Concurrent/volatile.scala Module: PIDE Author: Makarius Volatile variables. */ package isabelle object Volatile { def apply[A](init: A): Volatile[A] = new Volatile(init) } final class Volatile[A] private(init: A) { @volatile private var state: A = init def apply(): A = state def >> (f: A => A) { state = f(state) } def >>>[B] (f: A => (B, A)): B = { val (result, new_state) = f(state) state = new_state result } }