src/Pure/Isar/local_theory.ML
changeset 24949 5f00e3532418
parent 24933 5471b164813b
child 24984 952045a8dcf2
equal deleted inserted replaced
24948:c12c16a680a0 24949:5f00e3532418
    34   val type_syntax: declaration -> local_theory -> local_theory
    34   val type_syntax: declaration -> local_theory -> local_theory
    35   val term_syntax: declaration -> local_theory -> local_theory
    35   val term_syntax: declaration -> local_theory -> local_theory
    36   val declaration: declaration -> local_theory -> local_theory
    36   val declaration: declaration -> local_theory -> local_theory
    37   val note: string -> (bstring * Attrib.src list) * thm list ->
    37   val note: string -> (bstring * Attrib.src list) * thm list ->
    38     local_theory -> (bstring * thm list) * local_theory
    38     local_theory -> (bstring * thm list) * local_theory
    39   val notation: Syntax.mode -> (term * mixfix) list -> local_theory -> local_theory
    39   val notation: bool -> Syntax.mode -> (term * mixfix) list -> local_theory -> local_theory
    40   val target_morphism: local_theory -> morphism
    40   val target_morphism: local_theory -> morphism
    41   val target_naming: local_theory -> NameSpace.naming
    41   val target_naming: local_theory -> NameSpace.naming
    42   val target_name: local_theory -> bstring -> string
    42   val target_name: local_theory -> bstring -> string
    43   val init: string -> operations -> Proof.context -> local_theory
    43   val init: string -> operations -> Proof.context -> local_theory
    44   val restore: local_theory -> local_theory
    44   val restore: local_theory -> local_theory
   165 
   165 
   166 fun target_morphism lthy =
   166 fun target_morphism lthy =
   167   ProofContext.export_morphism lthy (target_of lthy) $>
   167   ProofContext.export_morphism lthy (target_of lthy) $>
   168   Morphism.thm_morphism Goal.norm_result;
   168   Morphism.thm_morphism Goal.norm_result;
   169 
   169 
   170 fun notation mode raw_args lthy =
   170 fun notation add mode raw_args lthy =
   171   let val args = map (apfst (Morphism.term (target_morphism lthy))) raw_args
   171   let val args = map (apfst (Morphism.term (target_morphism lthy))) raw_args
   172   in term_syntax (ProofContext.target_notation mode args) lthy end;
   172   in term_syntax (ProofContext.target_notation add mode args) lthy end;
   173 
   173 
   174 val target_name = NameSpace.full o target_naming;
   174 val target_name = NameSpace.full o target_naming;
   175 
   175 
   176 
   176 
   177 (* init -- exit *)
   177 (* init -- exit *)