src/Pure/Isar/proof_context.ML
changeset 30420 ebbec8d8d7a9
parent 30364 577edc39b501
child 30424 692279df7cc2
equal deleted inserted replaced
30419:c944e299eaf9 30420:ebbec8d8d7a9
    95   val get_fact: Proof.context -> Facts.ref -> thm list
    95   val get_fact: Proof.context -> Facts.ref -> thm list
    96   val get_fact_single: Proof.context -> Facts.ref -> thm
    96   val get_fact_single: Proof.context -> Facts.ref -> thm
    97   val get_thms: Proof.context -> xstring -> thm list
    97   val get_thms: Proof.context -> xstring -> thm list
    98   val get_thm: Proof.context -> xstring -> thm
    98   val get_thm: Proof.context -> xstring -> thm
    99   val add_path: string -> Proof.context -> Proof.context
    99   val add_path: string -> Proof.context -> Proof.context
   100   val no_base_names: Proof.context -> Proof.context
   100   val sticky_prefix: string -> Proof.context -> Proof.context
   101   val qualified_names: Proof.context -> Proof.context
   101   val qualified_names: Proof.context -> Proof.context
   102   val sticky_prefix: string -> Proof.context -> Proof.context
       
   103   val restore_naming: Proof.context -> Proof.context -> Proof.context
   102   val restore_naming: Proof.context -> Proof.context -> Proof.context
   104   val reset_naming: Proof.context -> Proof.context
   103   val reset_naming: Proof.context -> Proof.context
   105   val note_thmss: string -> (Thm.binding * (Facts.ref * attribute list) list) list ->
   104   val note_thmss: string -> (Thm.binding * (Facts.ref * attribute list) list) list ->
   106     Proof.context -> (string * thm list) list * Proof.context
   105     Proof.context -> (string * thm list) list * Proof.context
   107   val note_thmss_i: string -> (Thm.binding * (thm list * attribute list) list) list ->
   106   val note_thmss_i: string -> (Thm.binding * (thm list * attribute list) list) list ->
   943 
   942 
   944 
   943 
   945 (* name space operations *)
   944 (* name space operations *)
   946 
   945 
   947 val add_path        = map_naming o NameSpace.add_path;
   946 val add_path        = map_naming o NameSpace.add_path;
   948 val no_base_names   = map_naming NameSpace.no_base_names;
   947 val sticky_prefix   = map_naming o NameSpace.sticky_prefix;
   949 val qualified_names = map_naming NameSpace.qualified_names;
   948 val qualified_names = map_naming NameSpace.qualified_names;
   950 val sticky_prefix   = map_naming o NameSpace.sticky_prefix;
       
   951 val restore_naming  = map_naming o K o naming_of;
   949 val restore_naming  = map_naming o K o naming_of;
   952 val reset_naming    = map_naming (K local_naming);
   950 val reset_naming    = map_naming (K local_naming);
   953 
   951 
   954 
   952 
   955 (* facts *)
   953 (* facts *)