aboutsummaryrefslogtreecommitdiffhomepage
path: root/kernel
diff options
context:
space:
mode:
authorGravatar regisgia <regisgia@85f007b7-540e-0410-9357-904b9bb8a0f7>2012-09-14 10:04:47 +0000
committerGravatar regisgia <regisgia@85f007b7-540e-0410-9357-904b9bb8a0f7>2012-09-14 10:04:47 +0000
commit20a663fc7c2636833d7c789ca70efebe545df747 (patch)
tree2467027e1c8170997a50ce30d1d8d0f99879db8f /kernel
parent18ebb3f525a965358d96eab7df493450009517b5 (diff)
kernel/Term:
Backtrack on a type definition that was moved by error by the previous patch. git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@15798 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'kernel')
-rw-r--r--kernel/term.ml6
1 files changed, 3 insertions, 3 deletions
diff --git a/kernel/term.ml b/kernel/term.ml
index 16649b181..07152d4b6 100644
--- a/kernel/term.ml
+++ b/kernel/term.ml
@@ -108,8 +108,6 @@ 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
@@ -649,10 +647,12 @@ 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
-let map_named_declaration f (id, v, ty) = (id, Option.map f v, f ty)
+let map_named_declaration f (id, (v : strategy), ty) = (id, Option.map f v, f ty)
let map_rel_declaration = map_named_declaration
let fold_named_declaration f (_, v, ty) a = f ty (Option.fold_right f v a)