src/Pure/variable.ML
changeset 36603 d5d6111761a6
parent 33957 e9afca2118d4
child 36610 bafd82950e24
equal deleted inserted replaced
36602:0cbcdfd9e527 36603:d5d6111761a6
    26   val declare_constraints: term -> Proof.context -> Proof.context
    26   val declare_constraints: term -> Proof.context -> Proof.context
    27   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
    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 global_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 bind_term: indexname * term option -> Proof.context -> Proof.context
    33   val bind_term: indexname * term option -> Proof.context -> Proof.context
    34   val expand_binds: Proof.context -> term -> term
    34   val expand_binds: Proof.context -> term -> term
    35   val lookup_const: Proof.context -> string -> string option
    35   val lookup_const: Proof.context -> string -> string option
    36   val is_const: Proof.context -> string -> bool
    36   val is_const: Proof.context -> string -> bool
   233 val declare_typ = declare_term o Logic.mk_type;
   233 val declare_typ = declare_term o Logic.mk_type;
   234 
   234 
   235 val declare_prf = Proofterm.fold_proof_terms declare_internal (declare_internal o Logic.mk_type);
   235 val declare_prf = Proofterm.fold_proof_terms declare_internal (declare_internal o Logic.mk_type);
   236 
   236 
   237 val declare_thm = Thm.fold_terms declare_internal;
   237 val declare_thm = Thm.fold_terms declare_internal;
   238 fun thm_context th = declare_thm th (ProofContext.init (Thm.theory_of_thm th));
   238 fun global_thm_context th = declare_thm th (ProofContext.init (Thm.theory_of_thm th));
   239 
   239 
   240 
   240 
   241 (* renaming term/type frees *)
   241 (* renaming term/type frees *)
   242 
   242 
   243 fun variant_frees ctxt ts frees =
   243 fun variant_frees ctxt ts frees =