src/Pure/theory.ML
changeset 67384 e32b0eb63666
parent 67380 8bef51521f21
child 68164 738071699826
equal deleted inserted replaced
67383:aacea75450b4 67384:e32b0eb63666
     9   val parents_of: theory -> theory list
     9   val parents_of: theory -> theory list
    10   val ancestors_of: theory -> theory list
    10   val ancestors_of: theory -> theory list
    11   val nodes_of: theory -> theory list
    11   val nodes_of: theory -> theory list
    12   val setup: (theory -> theory) -> unit
    12   val setup: (theory -> theory) -> unit
    13   val local_setup: (Proof.context -> Proof.context) -> unit
    13   val local_setup: (Proof.context -> Proof.context) -> unit
       
    14   val install_pure: theory -> unit
    14   val get_pure: unit -> theory
    15   val get_pure: unit -> theory
    15   val install_pure: theory -> unit
       
    16   val get_markup: theory -> Markup.T
    16   val get_markup: theory -> Markup.T
    17   val check: Proof.context -> string * Position.T -> theory
    17   val check: Proof.context -> string * Position.T -> theory
    18   val axiom_table: theory -> term Name_Space.table
    18   val axiom_table: theory -> term Name_Space.table
    19   val axiom_space: theory -> Name_Space.T
    19   val axiom_space: theory -> Name_Space.T
    20   val axioms_of: theory -> (string * term) list
    20   val axioms_of: theory -> (string * term) list
    45 fun nodes_of thy = thy :: ancestors_of thy;
    45 fun nodes_of thy = thy :: ancestors_of thy;
    46 
    46 
    47 fun setup f = Context.>> (Context.map_theory f);
    47 fun setup f = Context.>> (Context.map_theory f);
    48 fun local_setup f = Context.>> (Context.map_proof f);
    48 fun local_setup f = Context.>> (Context.map_proof f);
    49 
    49 
       
    50 
       
    51 (* implicit theory Pure *)
       
    52 
    50 val pure: theory Single_Assignment.var = Single_Assignment.var "pure";
    53 val pure: theory Single_Assignment.var = Single_Assignment.var "pure";
    51 fun get_pure () = the (Single_Assignment.peek pure);
    54 
    52 fun install_pure thy = Single_Assignment.assign pure thy;
    55 fun install_pure thy = Single_Assignment.assign pure thy;
       
    56 
       
    57 fun get_pure () =
       
    58   (case Single_Assignment.peek pure of
       
    59     SOME thy => thy
       
    60   | NONE => raise Fail "Theory Pure not present");
    53 
    61 
    54 
    62 
    55 
    63 
    56 (** datatype thy **)
    64 (** datatype thy **)
    57 
    65