aboutsummaryrefslogtreecommitdiffhomepage
path: root/checker/declarations.mli
diff options
context:
space:
mode:
authorGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2013-02-12 22:56:43 +0000
committerGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2013-02-12 22:56:43 +0000
commit33c0d04c1ae40fb3eded886f8d82eb941e588fc9 (patch)
tree2b3863afcfca8ccb73db473c889320f2ec24ac33 /checker/declarations.mli
parent351c92f5c61082e9e8f5e1c9364f1836416f17d3 (diff)
Checker: re-sync vo structures after Maxime's commit 16136
make validate still fails, but that's another issue (#2949) we're still working on... git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@16198 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'checker/declarations.mli')
-rw-r--r--checker/declarations.mli9
1 files changed, 8 insertions, 1 deletions
diff --git a/checker/declarations.mli b/checker/declarations.mli
index ad234a3f5..80c895bbe 100644
--- a/checker/declarations.mli
+++ b/checker/declarations.mli
@@ -5,6 +5,8 @@ open Term
type values
type reloc_table
type to_patch_substituted
+(* Native code *)
+type native_name
(*Retroknowledge *)
type action
type retroknowledge
@@ -57,7 +59,9 @@ type constant_body = {
const_body : constant_def;
const_type : constant_type;
const_body_code : to_patch_substituted;
- const_constraints : Univ.constraints }
+ const_constraints : Univ.constraints;
+ const_native_name : native_name ref;
+ const_inline_code : bool }
val body_of_constant : constant_body -> constr_substituted option
val constant_has_body : constant_body -> bool
@@ -167,6 +171,9 @@ type mutual_inductive_body = {
(* Universes constraints enforced by the inductive declaration *)
mind_constraints : Univ.constraints;
+ (* Data for native compilation *)
+ mind_native_name : native_name ref;
+
}
(* Modules *)