src/Pure/Isar/proof_context.ML
changeset 22352 f15118a79c0e
parent 21824 153fad1e7318
child 22358 4d8a9e3a29f8
equal deleted inserted replaced
22351:587845efb4cf 22352:f15118a79c0e
   102   val get_thm_closure: Proof.context -> thmref -> thm
   102   val get_thm_closure: Proof.context -> thmref -> thm
   103   val get_thms: Proof.context -> thmref -> thm list
   103   val get_thms: Proof.context -> thmref -> thm list
   104   val get_thms_closure: Proof.context -> thmref -> thm list
   104   val get_thms_closure: Proof.context -> thmref -> thm list
   105   val valid_thms: Proof.context -> string * thm list -> bool
   105   val valid_thms: Proof.context -> string * thm list -> bool
   106   val lthms_containing: Proof.context -> FactIndex.spec -> (string * thm list) list
   106   val lthms_containing: Proof.context -> FactIndex.spec -> (string * thm list) list
       
   107   val add_path: string -> Proof.context -> Proof.context
   107   val no_base_names: Proof.context -> Proof.context
   108   val no_base_names: Proof.context -> Proof.context
   108   val qualified_names: Proof.context -> Proof.context
   109   val qualified_names: Proof.context -> Proof.context
   109   val sticky_prefix: string -> Proof.context -> Proof.context
   110   val sticky_prefix: string -> Proof.context -> Proof.context
   110   val restore_naming: Proof.context -> Proof.context -> Proof.context
   111   val restore_naming: Proof.context -> Proof.context -> Proof.context
   111   val reset_naming: Proof.context -> Proof.context
   112   val reset_naming: Proof.context -> Proof.context
   761     else (NameSpace.hidden (if name = "" then "unnamed" else name), ths));
   762     else (NameSpace.hidden (if name = "" then "unnamed" else name), ths));
   762 
   763 
   763 
   764 
   764 (* name space operations *)
   765 (* name space operations *)
   765 
   766 
       
   767 val add_path        = map_naming o NameSpace.add_path;
   766 val no_base_names   = map_naming NameSpace.no_base_names;
   768 val no_base_names   = map_naming NameSpace.no_base_names;
   767 val qualified_names = map_naming NameSpace.qualified_names;
   769 val qualified_names = map_naming NameSpace.qualified_names;
   768 val sticky_prefix   = map_naming o NameSpace.sticky_prefix;
   770 val sticky_prefix   = map_naming o NameSpace.sticky_prefix;
   769 val restore_naming  = map_naming o K o naming_of;
   771 val restore_naming  = map_naming o K o naming_of;
   770 val reset_naming    = map_naming (K local_naming);
   772 val reset_naming    = map_naming (K local_naming);