src/Pure/sign.ML
changeset 42204 b3277168c1e7
parent 40959 49765c1104d4
child 42224 578a51fae383
equal deleted inserted replaced
42203:9c9c97a5040d 42204:b3277168c1e7
   106     (string * (Proof.context -> bool -> typ -> term list -> term)) list -> theory -> theory
   106     (string * (Proof.context -> bool -> typ -> term list -> term)) list -> theory -> theory
   107   val add_tokentrfuns:
   107   val add_tokentrfuns:
   108     (string * string * (Proof.context -> string -> Pretty.T)) list -> theory -> theory
   108     (string * string * (Proof.context -> string -> Pretty.T)) list -> theory -> theory
   109   val add_mode_tokentrfuns: string -> (string * (Proof.context -> string -> Pretty.T)) list
   109   val add_mode_tokentrfuns: string -> (string * (Proof.context -> string -> Pretty.T)) list
   110     -> theory -> theory
   110     -> theory -> theory
   111   val add_trrules: (xstring * string) Syntax.trrule list -> theory -> theory
   111   val add_trrules: ast Syntax.trrule list -> theory -> theory
   112   val del_trrules: (xstring * string) Syntax.trrule list -> theory -> theory
   112   val del_trrules: ast Syntax.trrule list -> theory -> theory
   113   val add_trrules_i: ast Syntax.trrule list -> theory -> theory
       
   114   val del_trrules_i: ast Syntax.trrule list -> theory -> theory
       
   115   val new_group: theory -> theory
   113   val new_group: theory -> theory
   116   val reset_group: theory -> theory
   114   val reset_group: theory -> theory
   117   val add_path: string -> theory -> theory
   115   val add_path: string -> theory -> theory
   118   val root_path: theory -> theory
   116   val root_path: theory -> theory
   119   val parent_path: theory -> theory
   117   val parent_path: theory -> theory
   495 fun add_mode_tokentrfuns m = add_tokentrfuns o map (fn (s, f) => (m, s, f));
   493 fun add_mode_tokentrfuns m = add_tokentrfuns o map (fn (s, f) => (m, s, f));
   496 
   494 
   497 
   495 
   498 (* translation rules *)
   496 (* translation rules *)
   499 
   497 
   500 fun gen_trrules f args thy = thy |> map_syn (fn syn =>
   498 val add_trrules = map_syn o Syntax.update_trrules;
   501   let val rules = map (Syntax.map_trrule (apfst (intern_type thy))) args
   499 val del_trrules = map_syn o Syntax.remove_trrules;
   502   in f (ProofContext.init_global thy) syn rules syn end);
       
   503 
       
   504 val add_trrules = gen_trrules Syntax.update_trrules;
       
   505 val del_trrules = gen_trrules Syntax.remove_trrules;
       
   506 val add_trrules_i = map_syn o Syntax.update_trrules_i;
       
   507 val del_trrules_i = map_syn o Syntax.remove_trrules_i;
       
   508 
   500 
   509 
   501 
   510 (* naming *)
   502 (* naming *)
   511 
   503 
   512 val new_group = map_naming Name_Space.new_group;
   504 val new_group = map_naming Name_Space.new_group;