aboutsummaryrefslogtreecommitdiff
path: root/src/Assembly/DSL.v
diff options
context:
space:
mode:
authorGravatar Jason Gross <jgross@mit.edu>2016-02-05 15:24:42 -0500
committerGravatar Robert Sloan <varomodt@gmail.com>2016-06-22 13:39:02 -0400
commitc33166b756b0b6bd8141130bcdf8053ffff790e5 (patch)
tree3e93aa97f5b2c308c11d9abf94abd86bc8f1cf9b /src/Assembly/DSL.v
parentceb005a2bfde307ccfe6a3a52efd5f07f5483f84 (diff)
Update build process to use COQPATH & _CoqProject
Removed all of the files not built by default; they can be resurrected from git history. _CoqProject is the standard way to list the files in a project and to give information to coq_makefile. COQPATH is the standard way to make use of not-yet-installed libraries that are not part of your project (i.e., you don't want to remove them when you `make clean`, etc.).
Diffstat (limited to 'src/Assembly/DSL.v')
-rw-r--r--src/Assembly/DSL.v28
1 files changed, 0 insertions, 28 deletions
diff --git a/src/Assembly/DSL.v b/src/Assembly/DSL.v
deleted file mode 100644
index 2cb07a5d4..000000000
--- a/src/Assembly/DSL.v
+++ /dev/null
@@ -1,28 +0,0 @@
-
-Require Export ConstrainedComputation.
-
-Notation "const A" := CConst A.
-Notation "var A" := CVar A.
-Notation "A : B" := CJoin A B.
-Notation "left A" := CLeft A.
-Notation "right A" := CRight A.
-
-Notation "~ A" := UnaryExpr CNot A.
-Notation "- A" := UnaryExpr COpp A.
-Notation "A + B" := BinaryExpr CPlus A B.
-Notation "A - B" := BinaryExpr CMinus A B.
-Notation "A * B" := BinaryExpr CMult A B.
-Notation "A / B" := BinaryExpr CDiv A B.
-Notation "A & B" := BinaryExpr CAnd A B.
-Notation "A | B" := BinaryExpr COr A B.
-Notation "A ^ B" := BinaryExpr CXor A B.
-Notation "A >> B" := BinaryExpr CRShift A B.
-Notation "A << B" := BinaryExpr CLShift A B.
-
-Definition toExpr {type} (term: CTerm type) = TermExpr term.
-Coersion toExpr: {type} CTerm type >-> CExpr type.
-
-Notation "ret A" := CRet A
-Notation "A . B" := CCompose A B
-Notation "A ? B : C" := CIte A B C
-Notation "set A to B in C" := CLet A B C