moved to Pure/context.ML;
authorwenzelm
Wed, 03 Feb 1999 17:21:12 +0100
changeset 6202 7306d37f7929
parent 6201 27a94d4a8c15
child 6203 328b4377755c
moved to Pure/context.ML;
src/Pure/Thy/context.ML
--- a/src/Pure/Thy/context.ML	Wed Feb 03 17:20:55 1999 +0100
+++ /dev/null	Thu Jan 01 00:00:00 1970 +0000
@@ -1,101 +0,0 @@
-(*  Title:      Pure/Thy/context.ML
-    ID:         $Id$
-    Author:     Markus Wenzel, TU Muenchen
-
-Global contexts: session and theory.
-*)
-
-signature BASIC_CONTEXT =
-sig
-  val context: theory -> unit
-  val the_context: unit -> theory
-  val thm: xstring -> thm
-  val thms: xstring -> thm list
-  val Goal: string -> thm list
-  val Goalw: thm list -> string -> thm list
-  val Open_locale: xstring -> unit
-  val Close_locale: xstring -> unit
-  val Print_scope: unit -> unit
-  val Export: thm -> thm
-end;
-
-signature CONTEXT =
-sig
-  include BASIC_CONTEXT
-  val get_session: unit -> string list
-  val add_session: string -> unit
-  val reset_session: unit -> unit
-  val welcome: unit -> string
-  val get_context: unit -> theory option
-  val set_context: theory option -> unit
-  val reset_context: unit -> unit
-  val >> : (theory -> theory) -> unit
-end;
-
-structure Context: CONTEXT =
-struct
-
-
-(** session **)
-
-val current_session = ref ([]: string list);
-
-fun get_session () = ! current_session;
-fun add_session s = current_session := ! current_session @ [s];
-fun reset_session () = current_session := [];
-
-fun welcome () =
-  "Welcome to Isabelle/" ^
-    (case get_session () of [] => "Pure" | ss => space_implode "/" ss) ^
-    " (" ^ version ^ ")";
-
-
-
-(** theory context **)
-
-local
-  val current_theory = ref (None: theory option);
-in
-  fun get_context () = ! current_theory;
-  fun set_context opt_thy = current_theory := opt_thy;
-end;
-
-fun the_context () =
-  (case get_context () of
-    Some thy => thy
-  | _ => error "Unknown theory context");
-
-fun context thy = set_context (Some thy);
-fun reset_context () = set_context None;
-
-
-(* map context *)
-
-nonfix >>;
-fun >> f = set_context (Some (f (the_context ())));
-
-
-(* retrieve thms *)
-
-fun thm name = Locale.get_thm (the_context ()) name;
-fun thms name = Locale.get_thms (the_context ()) name;
-
-
-(* shortcut goal commands *)
-
-fun Goal s = Goals.atomic_goal (the_context ()) s;
-fun Goalw thms s = Goals.atomic_goalw (the_context ()) thms s;
-
-
-(* scope manipulation *)
-
-fun Open_locale xname = (Locale.open_locale xname (the_context ()); ());
-fun Close_locale xname = (Locale.close_locale xname (the_context ()); ());
-fun Print_scope () = (Locale.print_scope (the_context()); ());
-fun Export th = export_thy (the_context ()) th;
-
-end;
-
-
-structure BasicContext: BASIC_CONTEXT = Context;
-open BasicContext;