aboutsummaryrefslogtreecommitdiffhomepage
path: root/kernel/cemitcodes.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/cemitcodes.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/cemitcodes.mli')
-rw-r--r--kernel/cemitcodes.mli16
1 files changed, 8 insertions, 8 deletions
diff --git a/kernel/cemitcodes.mli b/kernel/cemitcodes.mli
index ca6da65e1..965228fa1 100644
--- a/kernel/cemitcodes.mli
+++ b/kernel/cemitcodes.mli
@@ -2,17 +2,17 @@ open Names
open Cbytecodes
type reloc_info =
- | Reloc_annot of annot_switch
+ | Reloc_annot of annot_switch
| Reloc_const of structured_constant
| Reloc_getglobal of constant
-type patch = reloc_info * int
+type patch = reloc_info * int
(* A virer *)
val subst_patch : Mod_subst.substitution -> patch -> patch
-
-type emitcodes
-val length : emitcodes -> int
+type emitcodes
+
+val length : emitcodes -> int
val patch_int : emitcodes -> (*pos*)int -> int -> unit
@@ -26,9 +26,9 @@ type body_code =
| BCconstant
-type to_patch_substituted
+type to_patch_substituted
-val from_val : body_code -> to_patch_substituted
+val from_val : body_code -> to_patch_substituted
val force : to_patch_substituted -> body_code
@@ -37,4 +37,4 @@ val is_boxed : to_patch_substituted -> bool
val subst_to_patch_subst : Mod_subst.substitution -> to_patch_substituted -> to_patch_substituted
val to_memory : bytecodes * bytecodes * fv -> to_patch
- (* init code, fun code, fv *)
+ (* init code, fun code, fv *)