src/Pure/Isar/toplevel.ML
changeset 38351 ea1ee55aa41f
parent 38350 480b2de9927c
parent 38337 f6c1e169f51b
child 38384 07c33be08476
equal deleted inserted replaced
38350:480b2de9927c 38351:ea1ee55aa41f
    18   val context_of: state -> Proof.context
    18   val context_of: state -> Proof.context
    19   val generic_theory_of: state -> generic_theory
    19   val generic_theory_of: state -> generic_theory
    20   val theory_of: state -> theory
    20   val theory_of: state -> theory
    21   val proof_of: state -> Proof.state
    21   val proof_of: state -> Proof.state
    22   val proof_position_of: state -> int
    22   val proof_position_of: state -> int
    23   val enter_proof_body: state -> Proof.state
       
    24   val end_theory: Position.T -> state -> theory
    23   val end_theory: Position.T -> state -> theory
    25   val print_state_context: state -> unit
    24   val print_state_context: state -> unit
    26   val print_state: bool -> state -> unit
    25   val print_state: bool -> state -> unit
    27   val pretty_abstract: state -> Pretty.T
    26   val pretty_abstract: state -> Pretty.T
    28   val quiet: bool Unsynchronized.ref
    27   val quiet: bool Unsynchronized.ref
   184 fun proof_position_of state =
   183 fun proof_position_of state =
   185   (case node_of state of
   184   (case node_of state of
   186     Proof (prf, _) => Proof_Node.position prf
   185     Proof (prf, _) => Proof_Node.position prf
   187   | _ => raise UNDEF);
   186   | _ => raise UNDEF);
   188 
   187 
   189 val enter_proof_body = node_case (Proof.init o Context.proof_of) Proof.enter_forward;
       
   190 
       
   191 fun end_theory _ (State (NONE, SOME (Theory (Context.Theory thy, _)))) = Theory.end_theory thy
   188 fun end_theory _ (State (NONE, SOME (Theory (Context.Theory thy, _)))) = Theory.end_theory thy
   192   | end_theory pos _ = error ("Unfinished theory at end of input" ^ Position.str_of pos);
   189   | end_theory pos _ = error ("Unfinished theory at end of input" ^ Position.str_of pos);
   193 
   190 
   194 
   191 
   195 (* print state *)
   192 (* print state *)