src/Pure/PIDE/markup.scala
changeset 72116 7773ec172572
parent 72112 3546dd4ade74
child 72119 d115d50a19c0
--- a/src/Pure/PIDE/markup.scala	Fri Aug 07 21:21:44 2020 +0200
+++ b/src/Pure/PIDE/markup.scala	Fri Aug 07 22:19:32 2020 +0200
@@ -576,11 +576,11 @@
       }
   }
 
-  object ML_Pid extends Function("ML_pid")
+  object ML_Statistics extends Function("ML_statistics")
   {
     def unapply(props: Properties.T): Option[Long] =
       props match {
-        case List(PROPERTY, (ID, Value.Long(pid))) => Some(pid)
+        case List(PROPERTY, ("pid", Value.Long(pid))) => Some(pid)
         case _ => None
       }
   }
@@ -593,7 +593,6 @@
   {
     val Threads = new Properties.Int("threads")
   }
-  object ML_Statistics extends Properties_Function("ML_statistics")
   object Task_Statistics extends Properties_Function("task_statistics")
 
   object Loading_Theory extends Name_Function("loading_theory")