src/Pure/context_position.ML
changeset 25953 03937086b1fe
parent 25952 2152b47a87ed
child 25954 682e84b60e5c
--- a/src/Pure/context_position.ML	Thu Jan 24 12:02:44 2008 +0100
+++ /dev/null	Thu Jan 01 00:00:00 1970 +0000
@@ -1,35 +0,0 @@
-(*  Title:      Pure/context_position.ML
-    ID:         $Id$
-    Author:     Makarius
-
-Context positions.
-*)
-
-signature CONTEXT_POSITION =
-sig
-  val put: Position.T -> Context.generic -> Context.generic
-  val put_ctxt: Position.T -> Proof.context -> Proof.context
-  val get: Proof.context -> Position.T
-  val str_of: Proof.context -> string
-  val properties_of: Proof.context -> Markup.property list
-end;
-
-structure ContextPosition: CONTEXT_POSITION =
-struct
-
-structure Data = GenericDataFun
-(
-  type T = Position.T;
-  val empty = Position.none;
-  fun extend _ = empty;
-  fun merge _ _ = empty;
-);
-
-val put = Data.put;
-val put_ctxt = Context.proof_map o put;
-
-val get = Data.get o Context.Proof;
-val str_of = Position.str_of o get;
-val properties_of = Position.properties_of o get;
-
-end;