(***********************************************************************) (* v * The Coq Proof Assistant / The Coq Development Team *) (* bool * strength -> Coqast.t -> Coqast.t option -> global_reference val definition_body_red : Tacred.red_expr option -> identifier -> bool * strength -> Coqast.t -> Coqast.t option -> global_reference val syntax_definition : identifier -> Coqast.t -> unit (*i val abstraction_definition : identifier -> int array -> Coqast.t -> unit i*) val hypothesis_def_var : bool -> identifier -> strength -> Coqast.t -> global_reference val parameter_def_var : identifier -> Coqast.t -> constant_path val build_mutual : (identifier * Coqast.t) list -> (identifier * Coqast.t * (identifier * Coqast.t) list) list -> bool -> unit val declare_mutual_with_eliminations : Declarations.mutual_inductive_entry -> section_path val build_recursive : (identifier * ((identifier * Coqast.t) list) * Coqast.t * Coqast.t) list -> unit val build_corecursive : (identifier * Coqast.t * Coqast.t) list -> unit val build_scheme : (identifier * bool * identifier * Coqast.t) list -> unit val start_proof_com : identifier option -> strength -> Coqast.t -> unit (*s [save_named b] saves the current completed proof under the name it was started; boolean [b] tells if the theorem is declared opaque; it fails if the proof is not completed *) val save_named : bool -> unit (* [save_anonymous b name] behaves as [save_named] but declares the theorem under the name [name] and respects the strength of the declaration *) val save_anonymous : bool -> identifier -> unit (* [save_anonymous_with_strength s b name] behaves as [save_anonymous] but declares the theorem under the name [name] and gives it the strength [strength] *) val save_anonymous_with_strength : strength -> bool -> identifier -> unit (* [get_current_context ()] returns the evar context and env of the current open proof if any, otherwise returns the empty evar context and the current global env *) val get_current_context : unit -> Proof_type.enamed_declarations * Environ.env