blob: c2e8ac386c86ed8e6ad387b7f342e00b1eec49ff (
plain)
1
2
3
4
5
6
7
8
9
10
11
12
13
14
15
16
17
18
19
20
21
22
23
24
25
26
27
28
29
30
31
32
33
34
35
36
37
38
39
40
41
42
43
44
45
46
47
48
49
50
51
52
53
54
55
56
57
58
59
60
61
|
(* $Id$ *)
(*i*)
open Names
open Univ
open Term
open Sign
open Declarations
open Inductive
open Environ
open Safe_typing
(*i*)
(* This module defines the global environment of Coq.
The functions below are exactly the same as the ones in [Typing],
operating on that global environment. *)
val safe_env : unit -> safe_environment
val env : unit -> env
val universes : unit -> universes
val context : unit -> context
val var_context : unit -> var_context
val push_var_decl : identifier * constr -> unit
val push_var_def : identifier * constr -> unit
(*
val push_var : identifier * constr option * constr -> unit
val push_rel_decl : name * constr -> unit
val push_rel_def : name * constr -> unit
*)
val add_constant : section_path -> constant_entry -> unit
val add_parameter : section_path -> constr -> unit
val add_mind : section_path -> mutual_inductive_entry -> unit
val add_constraints : constraints -> unit
val pop_vars : identifier list -> unit
val lookup_var : identifier -> constr option * typed_type
(*val lookup_rel : int -> name * typed_type*)
val lookup_constant : section_path -> constant_body
val lookup_mind : section_path -> mutual_inductive_body
val lookup_mind_specif : inductive -> inductive_instance
val export : string -> compiled_env
val import : compiled_env -> unit
(*s Some functions of [Environ] instanciated on the global environment. *)
val id_of_global : sorts oper -> identifier
(*s Re-exported functions of [Inductive], composed with
[lookup_mind_specif]. *)
val mind_is_recursive : inductive -> bool
val mind_nconstr : inductive -> int
val mind_nparams : inductive -> int
val mind_arity : inductive -> constr
val mind_lc : inductive -> constr array
|