aboutsummaryrefslogtreecommitdiff
path: root/src/Assembly/AlmostQhasm.v
diff options
context:
space:
mode:
authorGravatar Robert Sloan <varomodt@gmail.com>2016-04-04 19:38:00 -0400
committerGravatar Robert Sloan <varomodt@gmail.com>2016-06-22 13:43:15 -0400
commit366b62f01f7931b91bb6b7671d2e481ab0585075 (patch)
tree493d50e94bb0d94dde970a1431b66a11173b13df /src/Assembly/AlmostQhasm.v
parent55c24be6c27a807cfdd8c4ac392bbd288819622d (diff)
Fix Qhasm and AlmostQhasm with new State machinery
Diffstat (limited to 'src/Assembly/AlmostQhasm.v')
-rw-r--r--src/Assembly/AlmostQhasm.v5
1 files changed, 3 insertions, 2 deletions
diff --git a/src/Assembly/AlmostQhasm.v b/src/Assembly/AlmostQhasm.v
index 31128fbfb..0ec47fc37 100644
--- a/src/Assembly/AlmostQhasm.v
+++ b/src/Assembly/AlmostQhasm.v
@@ -4,6 +4,7 @@ Require Import List.
Module AlmostQhasm <: Language.
Import ListNotations.
+ Import State.
(* A constant upper-bound on the number of operations we run *)
Definition maxOps: nat := 1000.
@@ -44,8 +45,8 @@ Module AlmostQhasm <: Language.
| (Some st') => eval b st'
| _ => None
end
- | AAssign a => Some (evalAssignment a state)
- | AOp a => Some (evalOperation a state)
+ | AAssign a => evalAssignment a state
+ | AOp a => evalOperation a state
| ACond c a b =>
if (evalCond c state)
then eval a state