aboutsummaryrefslogtreecommitdiffhomepage
path: root/checker/declarations.mli
diff options
context:
space:
mode:
authorGravatar Enrico Tassi <Enrico.Tassi@inria.fr>2014-02-21 18:24:59 +0100
committerGravatar Enrico Tassi <Enrico.Tassi@inria.fr>2014-02-26 14:53:08 +0100
commit0499f51cedb38eba6b8ecd01ce94ddfb1b6ae9c8 (patch)
treeeb43b12647b93e52784c9118d77c7a64199989a5 /checker/declarations.mli
parentf7338257584ba69e7e815c7ef9ac0d24f0dec36c (diff)
checker and votour ported to new vo format (after -vi2vo)
Diffstat (limited to 'checker/declarations.mli')
-rw-r--r--checker/declarations.mli2
1 files changed, 2 insertions, 0 deletions
diff --git a/checker/declarations.mli b/checker/declarations.mli
index a5785b52a..3c6db6ab7 100644
--- a/checker/declarations.mli
+++ b/checker/declarations.mli
@@ -2,9 +2,11 @@ open Names
open Cic
val force_constr : constr_substituted -> constr
+val force_lazy_constr_univs : Cic.constant_def -> Univ.constraints
val from_val : constr -> constr_substituted
val indirect_opaque_access : (DirPath.t -> int -> constr) ref
+val indirect_opaque_univ_access : (DirPath.t -> int -> Univ.constraints) ref
(** Constant_body *)