src/Pure/PIDE/document_status.scala
changeset 69818 60d0ee8f2ddb
parent 69817 5f160df596c1
child 69844 b21ddfa7042b
equal deleted inserted replaced
69817:5f160df596c1 69818:60d0ee8f2ddb
   132       }
   132       }
   133       val initialized = state.node_initialized(version, name)
   133       val initialized = state.node_initialized(version, name)
   134       val consolidated = state.node_consolidated(version, name)
   134       val consolidated = state.node_consolidated(version, name)
   135 
   135 
   136       Node_Status(
   136       Node_Status(
       
   137         is_suppressed = version.nodes.is_suppressed(name),
   137         unprocessed = unprocessed,
   138         unprocessed = unprocessed,
   138         running = running,
   139         running = running,
   139         warned = warned,
   140         warned = warned,
   140         failed = failed,
   141         failed = failed,
   141         finished = finished,
   142         finished = finished,
   146         consolidated = consolidated)
   147         consolidated = consolidated)
   147     }
   148     }
   148   }
   149   }
   149 
   150 
   150   sealed case class Node_Status(
   151   sealed case class Node_Status(
       
   152     is_suppressed: Boolean,
   151     unprocessed: Int,
   153     unprocessed: Int,
   152     running: Int,
   154     running: Int,
   153     warned: Int,
   155     warned: Int,
   154     failed: Int,
   156     failed: Int,
   155     finished: Int,
   157     finished: Int,
   228   {
   230   {
   229     def is_empty: Boolean = rep.isEmpty
   231     def is_empty: Boolean = rep.isEmpty
   230     def apply(name: Document.Node.Name): Node_Status = rep(name)
   232     def apply(name: Document.Node.Name): Node_Status = rep(name)
   231     def get(name: Document.Node.Name): Option[Node_Status] = rep.get(name)
   233     def get(name: Document.Node.Name): Option[Node_Status] = rep.get(name)
   232 
   234 
   233     def present(snapshot: Document.Snapshot): List[(Document.Node.Name, Node_Status)] =
   235     def present: List[(Document.Node.Name, Node_Status)] =
   234       (for {
   236       (for {
   235         name <- nodes.topological_order.iterator
   237         name <- nodes.topological_order.iterator
   236         node_status <- get(name)
   238         node_status <- get(name)
   237         if !snapshot.version.nodes.is_suppressed(name)
       
   238       } yield (name, node_status)).toList
   239       } yield (name, node_status)).toList
   239 
   240 
   240     def quasi_consolidated(name: Document.Node.Name): Boolean =
   241     def quasi_consolidated(name: Document.Node.Name): Boolean =
   241       rep.get(name) match {
   242       rep.get(name) match {
   242         case Some(st) => st.quasi_consolidated
   243         case Some(st) => st.quasi_consolidated