src/Pure/sign.ML
changeset 42224 578a51fae383
parent 42204 b3277168c1e7
child 42247 12fe41a92cd5
equal deleted inserted replaced
42223:098c86e53153 42224:578a51fae383
    89   val add_const_constraint: string * typ option -> theory -> theory
    89   val add_const_constraint: string * typ option -> theory -> theory
    90   val primitive_class: binding * class list -> theory -> theory
    90   val primitive_class: binding * class list -> theory -> theory
    91   val primitive_classrel: class * class -> theory -> theory
    91   val primitive_classrel: class * class -> theory -> theory
    92   val primitive_arity: arity -> theory -> theory
    92   val primitive_arity: arity -> theory -> theory
    93   val add_trfuns:
    93   val add_trfuns:
    94     (string * (ast list -> ast)) list *
    94     (string * (Ast.ast list -> Ast.ast)) list *
    95     (string * (term list -> term)) list *
    95     (string * (term list -> term)) list *
    96     (string * (term list -> term)) list *
    96     (string * (term list -> term)) list *
    97     (string * (ast list -> ast)) list -> theory -> theory
    97     (string * (Ast.ast list -> Ast.ast)) list -> theory -> theory
    98   val add_trfunsT:
    98   val add_trfunsT:
    99     (string * (bool -> typ -> term list -> term)) list -> theory -> theory
    99     (string * (bool -> typ -> term list -> term)) list -> theory -> theory
   100   val add_advanced_trfuns:
   100   val add_advanced_trfuns:
   101     (string * (Proof.context -> ast list -> ast)) list *
   101     (string * (Proof.context -> Ast.ast list -> Ast.ast)) list *
   102     (string * (Proof.context -> term list -> term)) list *
   102     (string * (Proof.context -> term list -> term)) list *
   103     (string * (Proof.context -> term list -> term)) list *
   103     (string * (Proof.context -> term list -> term)) list *
   104     (string * (Proof.context -> ast list -> ast)) list -> theory -> theory
   104     (string * (Proof.context -> Ast.ast list -> Ast.ast)) list -> theory -> theory
   105   val add_advanced_trfunsT:
   105   val add_advanced_trfunsT:
   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: ast Syntax.trrule list -> theory -> theory
   111   val add_trrules: Ast.ast Syntax.trrule list -> theory -> theory
   112   val del_trrules: ast Syntax.trrule list -> theory -> theory
   112   val del_trrules: Ast.ast Syntax.trrule list -> theory -> theory
   113   val new_group: theory -> theory
   113   val new_group: theory -> theory
   114   val reset_group: theory -> theory
   114   val reset_group: theory -> theory
   115   val add_path: string -> theory -> theory
   115   val add_path: string -> theory -> theory
   116   val root_path: theory -> theory
   116   val root_path: theory -> theory
   117   val parent_path: theory -> theory
   117   val parent_path: theory -> theory