aboutsummaryrefslogtreecommitdiff
path: root/src/Compilers/ZExtended/Syntax.v
diff options
context:
space:
mode:
authorGravatar Jason Gross <jgross@mit.edu>2017-10-31 23:26:25 -0400
committerGravatar Jason Gross <jgross@mit.edu>2017-10-31 23:26:25 -0400
commit824e4fff531916aeb0870dfd8d8d51b5c68ebfa4 (patch)
tree4d01fe6b712f7175f03923ccd2acadacdd12f0a6 /src/Compilers/ZExtended/Syntax.v
parentcda816c48795e49b049e0cce87cf04426a420a2d (diff)
Switch to AddWithGetCarry in ZExtended
Diffstat (limited to 'src/Compilers/ZExtended/Syntax.v')
-rw-r--r--src/Compilers/ZExtended/Syntax.v8
1 files changed, 4 insertions, 4 deletions
diff --git a/src/Compilers/ZExtended/Syntax.v b/src/Compilers/ZExtended/Syntax.v
index 0a40abb8b..38141c7c2 100644
--- a/src/Compilers/ZExtended/Syntax.v
+++ b/src/Compilers/ZExtended/Syntax.v
@@ -24,9 +24,9 @@ Definition interp_base_type (v : base_type) : Set :=
end.
Inductive op : flat_type base_type -> flat_type base_type -> Set :=
-| AddGetCarry : op (tuple tZ 3) (tuple tZ 2)
+| AddWithGetCarry : op (tuple tZ 4) (tuple tZ 2)
| MulSplitAtBitwidth : op (tuple tZ 3) (tuple tZ 2)
-| AddGetCarryZ (bitwidth : Z) : op (tuple tZ 2) (tuple tZ 2)
+| AddWithGetCarryZ (bitwidth : Z) : op (tuple tZ 3) (tuple tZ 2)
| MulSplitAtBitwidthZ (bitwidth : Z) : op (tuple tZ 2) (tuple tZ 2)
| Zselect : op (tuple tZ 3) (tuple tZ 1)
| Zmul : op (tuple tZ 2) (tuple tZ 1)
@@ -54,9 +54,9 @@ Definition Const {t} : interp_base_type t -> op Unit (Tbase t)
Definition interp_op {s d} (opv : op s d) : interp_flat_type interp_base_type s -> interp_flat_type interp_base_type d
:= match opv with
- | AddGetCarry => curry3 Z.add_get_carry
+ | AddWithGetCarry => curry4 Z.add_with_get_carry
| MulSplitAtBitwidth => curry3 Z.mul_split_at_bitwidth
- | AddGetCarryZ bitwidth => curry2 (Z.add_get_carry bitwidth)
+ | AddWithGetCarryZ bitwidth => curry3 (Z.add_with_get_carry bitwidth)
| MulSplitAtBitwidthZ bitwidth => curry2 (Z.mul_split_at_bitwidth bitwidth)
| Zselect => curry3 Z.zselect
| Zmul => curry2 Z.mul