src/Pure/Isar/outer_syntax.ML
changeset 20023 33124a9f5e31
parent 19482 9f11af8f7ef9
child 20323 ac413d7cc03d
--- a/src/Pure/Isar/outer_syntax.ML	Thu Jul 06 12:18:17 2006 +0200
+++ b/src/Pure/Isar/outer_syntax.ML	Thu Jul 06 15:21:33 2006 +0200
@@ -10,6 +10,7 @@
   structure Isar:
     sig
       val state: unit -> Toplevel.state
+      val context: unit -> Proof.context
       val exn: unit -> (exn * string) option
       val main: unit -> unit
       val loop: unit -> unit
@@ -323,6 +324,7 @@
 structure Isar =
 struct
   val state = Toplevel.get_state;
+  val context = Context.proof_of o Toplevel.context_of o state;
   val exn = Toplevel.exn;
   fun main () = gen_main false false;
   fun loop () = gen_loop false false;