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.v1
1 files changed, 1 insertions, 0 deletions
diff --git a/src/Assembly/QhasmCommon.v b/src/Assembly/QhasmCommon.v
index fe6746382..8a9d0d51f 100644
--- a/src/Assembly/QhasmCommon.v
+++ b/src/Assembly/QhasmCommon.v
@@ -71,6 +71,7 @@ Inductive Operation :=
| IOpConst: forall {n}, IntOp -> Reg n -> Const n -> Operation
| IOpReg: forall {n}, IntOp -> Reg n -> Reg n -> Operation
| IOpMem: forall {n m}, IntOp -> Reg n -> Mem n m -> Index m -> Operation
+ | IOpStack: forall {n}, IntOp -> Reg n -> Stack n -> Operation
| DOp: forall {n}, DualOp -> Reg n -> Reg n -> option (Reg n) -> Operation
| ROp: forall {n}, RotOp -> Reg n -> Index n -> Operation
| COp: forall {n}, CarryOp -> Reg n -> Reg n -> Operation.