aboutsummaryrefslogtreecommitdiffhomepage
path: root/kernel/retroknowledge.mli
diff options
context:
space:
mode:
authorGravatar glondu <glondu@85f007b7-540e-0410-9357-904b9bb8a0f7>2009-09-17 15:58:14 +0000
committerGravatar glondu <glondu@85f007b7-540e-0410-9357-904b9bb8a0f7>2009-09-17 15:58:14 +0000
commit61ccbc81a2f3b4662ed4a2bad9d07d2003dda3a2 (patch)
tree961cc88c714aa91a0276ea9fbf8bc53b2b9d5c28 /kernel/retroknowledge.mli
parent6d3fbdf36c6a47b49c2a4b16f498972c93c07574 (diff)
Delete trailing whitespaces in all *.{v,ml*} files
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@12337 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'kernel/retroknowledge.mli')
-rw-r--r--kernel/retroknowledge.mli38
1 files changed, 19 insertions, 19 deletions
diff --git a/kernel/retroknowledge.mli b/kernel/retroknowledge.mli
index 2baf38285..0f1cdc8e2 100644
--- a/kernel/retroknowledge.mli
+++ b/kernel/retroknowledge.mli
@@ -24,8 +24,8 @@ type nat_field =
| NatType
| NatPlus
| NatTimes
-
-type n_field =
+
+type n_field =
| NPositive
| NType
| NTwice
@@ -35,7 +35,7 @@ type n_field =
| NPlus
| NTimes
-type int31_field =
+type int31_field =
| Int31Bits
| Int31Type
| Int31Twice
@@ -81,14 +81,14 @@ val initial_retroknowledge : retroknowledge
returns the compilation of id in cont if it has a specific treatment
or raises Not_found if id should be compiled as usual *)
val get_vm_compiling_info : retroknowledge -> entry -> Cbytecodes.comp_env ->
- constr array ->
+ constr array ->
int -> Cbytecodes.bytecodes-> Cbytecodes.bytecodes
(*Given an identifier id (usually Construct _)
and its argument array, returns a function that tries an ad-hoc optimisated
compilation (in the case of the 31-bit integers it means compiling them
directly into an integer)
raises Not_found if id should be compiled as usual, and expectingly
- CBytecodes.NotClosed if the term is not a closed constructor pattern
+ CBytecodes.NotClosed if the term is not a closed constructor pattern
(a constant for the compiler) *)
val get_vm_constant_static_info : retroknowledge -> entry ->
constr array ->
@@ -99,19 +99,19 @@ val get_vm_constant_static_info : retroknowledge -> entry ->
of id+args+cont when id has a specific treatment (in the case of
31-bit integers, that would be the dynamic compilation into integers)
or raises Not_found if id should be compiled as usual *)
-val get_vm_constant_dynamic_info : retroknowledge -> entry ->
- Cbytecodes.comp_env ->
- Cbytecodes.block array ->
+val get_vm_constant_dynamic_info : retroknowledge -> entry ->
+ Cbytecodes.comp_env ->
+ Cbytecodes.block array ->
int -> Cbytecodes.bytecodes -> Cbytecodes.bytecodes
-(* Given a type identifier, this function is used before compiling a match
- over this type. In the case of 31-bit integers for instance, it is used
+(* Given a type identifier, this function is used before compiling a match
+ over this type. In the case of 31-bit integers for instance, it is used
to add the instruction sequence which would perform a dynamic decompilation
in case the argument of the match is not in coq representation *)
val get_vm_before_match_info : retroknowledge -> entry -> Cbytecodes.bytecodes
-> Cbytecodes.bytecodes
-(* Given a type identifier, this function is used by pretyping/vnorm.ml to
- recover the elements of that type from their compiled form if it's non
+(* Given a type identifier, this function is used by pretyping/vnorm.ml to
+ recover the elements of that type from their compiled form if it's non
standard (it is used (and can be used) only when the compiled form
is not a block *)
val get_vm_decompile_constant_info : retroknowledge -> entry -> int -> Term.constr
@@ -127,26 +127,26 @@ val find : retroknowledge -> field -> entry
(* the following function manipulate the reactive information of values
they are only used by the functions of Pre_env, and Environ to implement
the functions register and unregister of Environ *)
-val add_vm_compiling_info : retroknowledge-> entry ->
+val add_vm_compiling_info : retroknowledge-> entry ->
(bool -> Cbytecodes.comp_env -> constr array -> int ->
Cbytecodes.bytecodes -> Cbytecodes.bytecodes) ->
retroknowledge
-val add_vm_constant_static_info : retroknowledge-> entry ->
+val add_vm_constant_static_info : retroknowledge-> entry ->
(bool->constr array->
Cbytecodes.structured_constant) ->
retroknowledge
-val add_vm_constant_dynamic_info : retroknowledge-> entry ->
- (bool -> Cbytecodes.comp_env ->
- Cbytecodes.block array -> int ->
+val add_vm_constant_dynamic_info : retroknowledge-> entry ->
+ (bool -> Cbytecodes.comp_env ->
+ Cbytecodes.block array -> int ->
Cbytecodes.bytecodes -> Cbytecodes.bytecodes) ->
retroknowledge
val add_vm_before_match_info : retroknowledge -> entry ->
(bool->Cbytecodes.bytecodes->Cbytecodes.bytecodes) ->
retroknowledge
-val add_vm_decompile_constant_info : retroknowledge -> entry ->
+val add_vm_decompile_constant_info : retroknowledge -> entry ->
(int -> constr) -> retroknowledge
-
+
val clear_info : retroknowledge-> entry -> retroknowledge