src/Pure/context_position.ML
author wenzelm
Fri, 03 Aug 2007 22:33:09 +0200
changeset 24150 ed724867099a
parent 23354 a189707c1d76
child 24773 ec3a04e6f1a9
permissions -rw-r--r--
sort indexes according to symbolic update_time (multithreading-safe);

(*  Title:      Pure/context_position.ML
    ID:         $Id$
    Author:     Makarius

Context positions.
*)

signature CONTEXT_POSITION =
sig
  val put: Position.T -> Proof.context -> Proof.context
  val get: Proof.context -> Position.T
  val str_of: Proof.context -> string
end;

structure ContextPosition: CONTEXT_POSITION =
struct

structure Data = ProofDataFun
(
  type T = Position.T;
  fun init _ = Position.none;
);

val put = Data.put;
val get = Data.get;
val str_of = Position.str_of o get;

end;