aboutsummaryrefslogtreecommitdiff
path: root/src/Assembly/Pipeline.v
diff options
context:
space:
mode:
authorGravatar Robert Sloan <varomodt@gmail.com>2016-06-23 15:55:41 -0400
committerGravatar Robert Sloan <varomodt@gmail.com>2016-06-23 15:55:41 -0400
commitb9fcdc12c330b078574ba3feb2ab9e383fbc4e83 (patch)
tree7c5b98825e86a7c6cd59af0e785515de2bc966e9 /src/Assembly/Pipeline.v
parent8eba1b5866af0ec50c815d88f22198a88ac541dd (diff)
Pseudize Lemmas for Dual Operations
Diffstat (limited to 'src/Assembly/Pipeline.v')
-rw-r--r--src/Assembly/Pipeline.v16
1 files changed, 7 insertions, 9 deletions
diff --git a/src/Assembly/Pipeline.v b/src/Assembly/Pipeline.v
index 9299d9d52..9d6c4c9da 100644
--- a/src/Assembly/Pipeline.v
+++ b/src/Assembly/Pipeline.v
@@ -22,21 +22,19 @@ Module Pipeline.
End Pipeline.
Module PipelineExample.
- Import Pipeline ListNotations.
+ Import Pipeline ListNotations StateCommon EvalUtil ListState.
Local Notation "v [[ i ]]" := (nth i v (wzero _)) (at level 40).
Local Notation "$$ v" := (natToWord _ v) (at level 40).
Definition example: @pseudeq 32 W32 1 1 (fun v =>
- Let_In ($$ 1) (fun a =>
- Let_In (v[[0]]) (fun b => [
- a ^& b
- ]))).
-
+ plet a := $$ 1 in
+ plet b := v[[0]] in
+ plet c := multHigh a b in
+ plet d := a ^* b in
+ [b ^& d]).
pseudo_solve.
Defined.
- Definition exStr := Pipeline.toString (proj1_sig example).
-
- (* Eval vm_compute in exStr. *)
+ Eval vm_compute in (Pipeline.toString (proj1_sig example)).
End PipelineExample.