aboutsummaryrefslogtreecommitdiffhomepage
path: root/kernel/byterun
diff options
context:
space:
mode:
authorGravatar Guillaume Melquiond <guillaume.melquiond@inria.fr>2015-10-14 10:39:55 +0200
committerGravatar Guillaume Melquiond <guillaume.melquiond@inria.fr>2015-10-14 10:39:55 +0200
commitf617aeef08441e83b13f839ce767b840fddbcf7d (patch)
tree9a0c914031262f5491745d9773d7c2a0e5bdaa41 /kernel/byterun
parented95f122f3c68becc09c653471dc2982b346d343 (diff)
Fix some typos.
Diffstat (limited to 'kernel/byterun')
-rw-r--r--kernel/byterun/coq_interp.c2
1 files changed, 1 insertions, 1 deletions
diff --git a/kernel/byterun/coq_interp.c b/kernel/byterun/coq_interp.c
index 399fa843f..1653c3b01 100644
--- a/kernel/byterun/coq_interp.c
+++ b/kernel/byterun/coq_interp.c
@@ -1271,7 +1271,7 @@ value coq_interprete
Instruct (COMPAREINT31) {
/* returns Eq if equal, Lt if accu is less than *sp, Gt otherwise */
- /* assumes Inudctive _ : _ := Eq | Lt | Gt */
+ /* assumes Inductive _ : _ := Eq | Lt | Gt */
print_instr("COMPAREINT31");
if ((uint32_t)accu == (uint32_t)*sp) {
accu = 1; /* 2*0+1 */