aboutsummaryrefslogtreecommitdiff
path: root/src/Assembly/QhasmCommon.v
diff options
context:
space:
mode:
authorGravatar Robert Sloan <varomodt@gmail.com>2016-05-18 22:22:47 -0400
committerGravatar Robert Sloan <varomodt@gmail.com>2016-06-22 13:43:30 -0400
commitb4895166bfc9cc73e18805e88bef4cf6f280364d (patch)
tree694ae707cbc3c60b17c3ad8203f1870f3078e596 /src/Assembly/QhasmCommon.v
parenta263361224a46fb8416c1b66a3af6f2d6cc7cff7 (diff)
Tuple-ization tactics work
Most of Medial, less the conversions Most of Medial, less the conversions Most of Medial, less the conversions Most of Medial, less the conversions More of Medial MedialConversions done
Diffstat (limited to 'src/Assembly/QhasmCommon.v')
-rw-r--r--src/Assembly/QhasmCommon.v1
1 files changed, 0 insertions, 1 deletions
diff --git a/src/Assembly/QhasmCommon.v b/src/Assembly/QhasmCommon.v
index f213dc9a4..5e2077c5a 100644
--- a/src/Assembly/QhasmCommon.v
+++ b/src/Assembly/QhasmCommon.v
@@ -4,7 +4,6 @@ Require Export Bedrock.Word.
(* A formalization of x86 qhasm *)
Definition Label := nat.
Definition Index (limit: nat) := {x: nat | (x < limit)%nat}.
-Definition Invert := bool.
(* Sugar and Tactics *)