src/Pure/General/logger.scala
author wenzelm
Sun, 21 May 2017 23:41:46 +0200
changeset 65895 744878d72021
parent 64606 a871fa7c24fc
child 65921 5b42937d3b2d
permissions -rw-r--r--
more general workaround for failed sessions (again, see also 2edb89630a80, ed7b5cd3a7f2);

/*  Title:      Pure/General/logger.scala
    Author:     Makarius

Minimal logging support.
*/

package isabelle


object Logger
{
  def make(log_file: Option[Path]): Logger =
    log_file match { case Some(file) => new File_Logger(file) case None => No_Logger }
}

trait Logger
{
  def apply(msg: => String): Unit
}

object No_Logger extends Logger
{
  def apply(msg: => String) { }
}

class File_Logger(path: Path) extends Logger
{
  def apply(msg: => String) { synchronized { File.append(path, msg + "\n") } }

  override def toString: String = path.toString
}