src/Pure/PIDE/session.scala
changeset 71655 dad29591645a
parent 71652 721f143a679b
child 71667 4d2de35214c5
equal deleted inserted replaced
71654:0aef1812ae3a 71655:dad29591645a
   484             msg.properties match {
   484             msg.properties match {
   485               case Markup.Protocol_Handler(name) if prover.defined =>
   485               case Markup.Protocol_Handler(name) if prover.defined =>
   486                 init_protocol_handler(name)
   486                 init_protocol_handler(name)
   487 
   487 
   488               case Protocol.Command_Timing(state_id, timing) if prover.defined =>
   488               case Protocol.Command_Timing(state_id, timing) if prover.defined =>
   489                 command_timings.post(Session.Command_Timing(msg.properties))
   489                 command_timings.post(Session.Command_Timing(msg.properties.tail))
   490                 val message = XML.elem(Markup.STATUS, List(XML.Elem(Markup.Timing(timing), Nil)))
   490                 val message = XML.elem(Markup.STATUS, List(XML.Elem(Markup.Timing(timing), Nil)))
   491                 change_command(_.accumulate(state_id, xml_cache.elem(message), xml_cache))
   491                 change_command(_.accumulate(state_id, xml_cache.elem(message), xml_cache))
   492 
   492 
   493               case Protocol.Theory_Timing(_, _) =>
   493               case Protocol.Theory_Timing(_, _) =>
   494                 theory_timings.post(Session.Theory_Timing(msg.properties))
   494                 theory_timings.post(Session.Theory_Timing(msg.properties.tail))
   495 
   495 
   496               case Protocol.Export(args)
   496               case Protocol.Export(args)
   497               if args.id.isDefined && Value.Long.unapply(args.id.get).isDefined =>
   497               if args.id.isDefined && Value.Long.unapply(args.id.get).isDefined =>
   498                 val id = Value.Long.unapply(args.id.get).get
   498                 val id = Value.Long.unapply(args.id.get).get
   499                 val export = Export.make_entry("", args, msg.bytes, cache = xz_cache)
   499                 val export = Export.make_entry("", args, msg.bytes, cache = xz_cache)