aboutsummaryrefslogtreecommitdiff
path: root/src/Assembly/QhasmCommon.v
diff options
context:
space:
mode:
Diffstat (limited to 'src/Assembly/QhasmCommon.v')
-rw-r--r--src/Assembly/QhasmCommon.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/src/Assembly/QhasmCommon.v b/src/Assembly/QhasmCommon.v
index 8a9d0d51f..21f846cb5 100644
--- a/src/Assembly/QhasmCommon.v
+++ b/src/Assembly/QhasmCommon.v
@@ -93,7 +93,7 @@ Inductive Conditional :=
Inductive Mapping (n: nat) :=
| regM: forall (r: Reg n), Mapping n
| stackM: forall (s: Stack n), Mapping n
- | memM: forall {m} (x: Mem n m), Mapping n
+ | memM: forall {m} (x: Mem n m) (i: Index m), Mapping n
| constM: forall (x: Const n), Mapping n.
(* Parameter Accessors *)