aboutsummaryrefslogtreecommitdiffhomepage
path: root/interp/topconstr.mli
diff options
context:
space:
mode:
authorGravatar bertot <bertot@85f007b7-540e-0410-9357-904b9bb8a0f7>2004-02-26 13:35:24 +0000
committerGravatar bertot <bertot@85f007b7-540e-0410-9357-904b9bb8a0f7>2004-02-26 13:35:24 +0000
commit67fe536720c5ef5bb509249b9a30cbc6f2cebd92 (patch)
tree54964d8e58b41b401d097f044d50b03ee68da118 /interp/topconstr.mli
parente6370d38bd56ccd070cb33d257147ace238efc8b (diff)
Keep structure information for Fixpoint declaration and Fix terms
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@5386 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'interp/topconstr.mli')
-rw-r--r--interp/topconstr.mli2
1 files changed, 1 insertions, 1 deletions
diff --git a/interp/topconstr.mli b/interp/topconstr.mli
index c6be36028..d35418b51 100644
--- a/interp/topconstr.mli
+++ b/interp/topconstr.mli
@@ -107,7 +107,7 @@ type constr_expr =
| CDelimiters of loc * string * constr_expr
| CDynamic of loc * Dyn.t
-and fixpoint_expr = identifier * int * constr_expr * constr_expr
+and fixpoint_expr = identifier * int * int option * constr_expr * constr_expr
and cofixpoint_expr = identifier * constr_expr * constr_expr