aboutsummaryrefslogtreecommitdiffhomepage
path: root/kernel/term.ml
diff options
context:
space:
mode:
Diffstat (limited to 'kernel/term.ml')
-rw-r--r--kernel/term.ml6
1 files changed, 3 insertions, 3 deletions
diff --git a/kernel/term.ml b/kernel/term.ml
index 9a25de1bc..16649b181 100644
--- a/kernel/term.ml
+++ b/kernel/term.ml
@@ -108,6 +108,8 @@ type ('constr, 'types) kind_of_term =
-rectypes of the Caml compiler to be set *)
type constr = (constr,constr) kind_of_term
+type strategy = types option
+
type existential = existential_key * constr array
type rec_declaration = name array * constr array * constr array
type fixpoint = (int array * int) * rec_declaration
@@ -429,7 +431,7 @@ let rec under_casts f c = match kind_of_term c with
(******************************************************************)
(* flattens application lists throwing casts in-between *)
-let rec collapse_appl c = match kind_of_term c with
+let collapse_appl c = match kind_of_term c with
| App (f,cl) ->
let rec collapse_rec f cl2 =
match kind_of_term (strip_outer_cast f) with
@@ -647,8 +649,6 @@ let rec constr_ord m n=
type types = constr
-type strategy = types option
-
type named_declaration = identifier * constr option * types
type rel_declaration = name * constr option * types