aboutsummaryrefslogtreecommitdiffhomepage
path: root/kernel/typeops.mli
blob: a271dc9ecbec0a046837bce40fadd8527e722676 (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
62
63
64
65
66
67
68
69
70
71
72
73
74
75
76
77
78
79
80
81
82
83
84
85
86
87
88
89
(* $Id$ *)

(*i*)
open Names
open Univ
open Term
open Evd
open Environ
(*i*)


(* Basic operations of the typing machine. *)

val make_judge : constr -> typed_type -> unsafe_judgment

val j_val_only : unsafe_judgment -> constr

(* If [j] is the judgement $c:t:s$, then [typed_type_of_judgment env j]
   constructs the typed type $t:s$, while [assumption_of_judgement env j]
   cosntructs the type type $c:t$, checking that $t$ is a sort. *)

val typed_type_of_judgment : 
  env -> 'a evar_map -> unsafe_judgment -> typed_type
val assumption_of_judgment : 
  env -> 'a evar_map -> unsafe_judgment -> typed_type

val relative : env -> int -> unsafe_judgment

val type_of_constant : env -> 'a evar_map -> constr -> typed_type

val type_of_inductive : env -> 'a evar_map -> constr -> typed_type

val type_of_constructor : env -> 'a evar_map -> constr -> constr

val type_of_existential : env -> 'a evar_map -> constr -> constr

val type_of_case : env -> 'a evar_map 
  -> unsafe_judgment -> unsafe_judgment 
    -> unsafe_judgment array -> unsafe_judgment

val type_case_branches :
  env -> 'a evar_map -> constr -> constr -> constr -> constr 
    -> constr * constr array * constr 

val judge_of_prop_contents : contents -> unsafe_judgment

val judge_of_type : universe -> unsafe_judgment * constraints

val abs_rel : 
  env -> 'a evar_map -> name -> typed_type -> unsafe_judgment 
    -> unsafe_judgment * constraints

val gen_rel :
  env -> 'a evar_map -> name -> typed_type -> unsafe_judgment 
    -> unsafe_judgment * constraints

val cast_rel : 
  env -> 'a evar_map -> unsafe_judgment -> unsafe_judgment 
    -> unsafe_judgment

val apply_rel_list : 
  env -> 'a evar_map -> bool -> unsafe_judgment list -> unsafe_judgment
    -> unsafe_judgment * constraints

val check_fix : env -> 'a evar_map -> constr -> unit
val check_cofix : env -> 'a evar_map -> constr -> unit
val control_only_guard : env -> 'a evar_map -> constr -> unit

val type_fixpoint : env -> 'a evar_map -> name list -> typed_type array 
    -> unsafe_judgment array -> constraints

val type_one_branch_dep : env -> 'a evar_map -> 
  int * constr list * constr -> constr -> constr -> constr 

val type_one_branch_nodep : env -> 'a evar_map -> 
  int * constr list * constr -> constr -> constr 

val make_arity_dep : 
  env -> 'a evar_map -> constr -> constr -> constr -> constr 

val make_arity_nodep : 
  env -> 'a evar_map -> constr -> constr -> constr 

val find_case_dep_nparams :
  env -> 'a evar_map -> constr * constr ->
    constr * constr list ->
      constr -> bool * (int * constr list * constr list) 

val type_inst_construct : env -> 'a evar_map -> int -> constr -> constr