aboutsummaryrefslogtreecommitdiffhomepage
path: root/library/global.mli
blob: d21509e3211f6aae9b8ca7749d34bf5a961082b2 (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

(* $Id$ *)

(*i*)
open Names
open Univ
open Term
open Sign
open Evd
open Constant
open Inductive
open Environ
(*i*)

(* This module defines the global environment of Coq. 
   The functions below are the exactly the same as the ones in [Typing],
   operating on that global environment. *)

val evar_map : unit -> unit evar_map
val universes : unit -> universes
val metamap : unit -> (int * constr) list
val context : unit -> context

val push_var : identifier * constr -> unit
val push_rel : 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 lookup_var : identifier -> name * 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 : constr -> mind_specif
val lookup_meta : int -> constr

val export : string -> compiled_env
val import : compiled_env -> unit