aboutsummaryrefslogtreecommitdiff
path: root/src/Assembly/QhasmUtil.v
diff options
context:
space:
mode:
authorGravatar Robert Sloan <varomodt@google.com>2016-10-17 14:39:18 -0700
committerGravatar Robert Sloan <varomodt@google.com>2016-10-17 14:39:18 -0700
commitf8680ec8e73f8acb39cb55f6e616a0e5d10347f8 (patch)
treed13ad67b22fcce1dd72946d3aef2532e785ef9ac /src/Assembly/QhasmUtil.v
parent075347c125e6bdb77c1e0f4ed229d5019b213584 (diff)
Converting to bounded machinery
Diffstat (limited to 'src/Assembly/QhasmUtil.v')
-rw-r--r--src/Assembly/QhasmUtil.v5
1 files changed, 4 insertions, 1 deletions
diff --git a/src/Assembly/QhasmUtil.v b/src/Assembly/QhasmUtil.v
index f6a342fc0..79591d40d 100644
--- a/src/Assembly/QhasmUtil.v
+++ b/src/Assembly/QhasmUtil.v
@@ -74,7 +74,10 @@ Section Util.
x ^+ y ^+ (natToWord _ (if c then 1 else 0)).
Definition omap {A B} (x: option A) (f: A -> option B) :=
- match x with | Some y => f y | _ => None end.
+ match x with
+ | Some y => f y
+ | _ => None
+ end.
Notation "A <- X ; B" := (omap X (fun A => B)) (at level 70, right associativity).
End Util.