aboutsummaryrefslogtreecommitdiffhomepage
path: root/interp/coqlib.mli
diff options
context:
space:
mode:
authorGravatar msozeau <msozeau@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-06-30 19:43:44 +0000
committerGravatar msozeau <msozeau@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-06-30 19:43:44 +0000
commit4f70016289f15526b162582fc267374e2b60448e (patch)
tree47abfac4e62dfe1dc5dcfad34050634480518709 /interp/coqlib.mli
parent13e53564fdc4beb14bd04612214a648630549417 (diff)
Move [delayed] to util and use [force_delayed] everywhere to force
thunks. Move from [lazy] to [delayed] in subtac. git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@13227 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'interp/coqlib.mli')
-rw-r--r--interp/coqlib.mli6
1 files changed, 3 insertions, 3 deletions
diff --git a/interp/coqlib.mli b/interp/coqlib.mli
index 73427d902..c4693479b 100644
--- a/interp/coqlib.mli
+++ b/interp/coqlib.mli
@@ -11,6 +11,7 @@ open Libnames
open Nametab
open Term
open Pattern
+open Util
(** This module collects the global references, constructions and
patterns of the standard library used in ocaml files *)
@@ -84,9 +85,8 @@ val glob_jmeq : global_reference
at compile time. Therefore, we can only provide methods to build
them at runtime. This is the purpose of the [constr delayed] and
[constr_pattern delayed] types. Objects of this time needs to be
- applied to [()] to get the actual constr or pattern at runtime *)
-
-type 'a delayed = unit -> 'a
+ forced with [delayed_force] to get the actual constr or pattern
+ at runtime. *)
type coq_bool_data = {
andb : constr;