aboutsummaryrefslogtreecommitdiff
path: root/src/Compilers/TestCase.v
diff options
context:
space:
mode:
authorGravatar Jason Gross <jgross@mit.edu>2017-04-15 02:01:56 -0400
committerGravatar Jason Gross <jasongross9@gmail.com>2017-05-14 00:52:04 -0400
commit096a24265d4df0bbb5321c6fa794577bee5cae25 (patch)
tree4b7cbeefaf12fc5ce836e80864a6221c7b44dcf9 /src/Compilers/TestCase.v
parent63e036b685457b7ecfb44e6caf966c4a7e8462d1 (diff)
CSE without inlining arithmetic expressions
This takes care of most of #158. The remaining bits are reworking the Wf and interpretation lemmas to actually work. (The former needs a only bit of rethinking and rephrasing to handle the fact that sometimes we change the stored symbolic expression from a complicated one to a fresh variable, while the latter needs major surgery, which Adam tells me is easy, and this is a note that when I come back to it, I should look at the email thread with Adam about CSE from last summer.)
Diffstat (limited to 'src/Compilers/TestCase.v')
-rw-r--r--src/Compilers/TestCase.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/src/Compilers/TestCase.v b/src/Compilers/TestCase.v
index a7fd81328..36774e4e3 100644
--- a/src/Compilers/TestCase.v
+++ b/src/Compilers/TestCase.v
@@ -187,7 +187,7 @@ Section cse.
| Mul => SMul
| Sub => SSub
end.
- Definition CSE {t} e := @CSE base_type op_code base_type_beq op_code_beq internal_base_type_dec_bl op symbolicify_op (fun _ x => x) t e (fun _ => nil).
+ Definition CSE {t} e := @CSE base_type op_code base_type_beq op_code_beq internal_base_type_dec_bl op symbolicify_op (fun _ x => x) true t e (fun _ => nil).
End cse.
Definition example_expr_simplified := Eval vm_compute in InlineConst is_const (ANormal example_expr).