src/Pure/variable.ML
changeset 27280 2a38802d3649
parent 27119 c36c88fcdd22
child 28625 d51a14105e53
equal deleted inserted replaced
27279:39ff18c0f07f 27280:2a38802d3649
    20   val newly_fixed: Proof.context -> Proof.context -> string -> bool
    20   val newly_fixed: Proof.context -> Proof.context -> string -> bool
    21   val add_fixed: Proof.context -> term -> (string * typ) list -> (string * typ) list
    21   val add_fixed: Proof.context -> term -> (string * typ) list -> (string * typ) list
    22   val default_type: Proof.context -> string -> typ option
    22   val default_type: Proof.context -> string -> typ option
    23   val def_type: Proof.context -> bool -> indexname -> typ option
    23   val def_type: Proof.context -> bool -> indexname -> typ option
    24   val def_sort: Proof.context -> indexname -> sort option
    24   val def_sort: Proof.context -> indexname -> sort option
       
    25   val declare_names: term -> Proof.context -> Proof.context
    25   val declare_constraints: term -> Proof.context -> Proof.context
    26   val declare_constraints: term -> Proof.context -> Proof.context
    26   val declare_names: term -> Proof.context -> Proof.context
       
    27   val declare_internal: term -> Proof.context -> Proof.context
       
    28   val declare_term: term -> Proof.context -> Proof.context
    27   val declare_term: term -> Proof.context -> Proof.context
       
    28   val declare_typ: typ -> Proof.context -> Proof.context
    29   val declare_prf: Proofterm.proof -> Proof.context -> Proof.context
    29   val declare_prf: Proofterm.proof -> Proof.context -> Proof.context
    30   val declare_thm: thm -> Proof.context -> Proof.context
    30   val declare_thm: thm -> Proof.context -> Proof.context
    31   val thm_context: thm -> Proof.context
    31   val thm_context: thm -> Proof.context
    32   val variant_frees: Proof.context -> term list -> (string * 'a) list -> (string * 'a) list
    32   val variant_frees: Proof.context -> term list -> (string * 'a) list -> (string * 'a) list
    33   val add_binds: (indexname * term option) list -> Proof.context -> Proof.context
    33   val add_binds: (indexname * term option) list -> Proof.context -> Proof.context
   220 
   220 
   221 fun declare_term t =
   221 fun declare_term t =
   222   declare_internal t #>
   222   declare_internal t #>
   223   declare_constraints t;
   223   declare_constraints t;
   224 
   224 
       
   225 val declare_typ = declare_term o Logic.mk_type;
       
   226 
   225 val declare_prf = Proofterm.fold_proof_terms declare_internal (declare_internal o Logic.mk_type);
   227 val declare_prf = Proofterm.fold_proof_terms declare_internal (declare_internal o Logic.mk_type);
   226 
   228 
   227 val declare_thm = Thm.fold_terms declare_internal;
   229 val declare_thm = Thm.fold_terms declare_internal;
   228 fun thm_context th = declare_thm th (ProofContext.init (Thm.theory_of_thm th));
   230 fun thm_context th = declare_thm th (ProofContext.init (Thm.theory_of_thm th));
   229 
   231