aboutsummaryrefslogtreecommitdiff
path: root/src/Compilers/TestCase.v
diff options
context:
space:
mode:
authorGravatar Jason Gross <jgross@mit.edu>2017-04-14 21:51:50 -0400
committerGravatar Jason Gross <jgross@mit.edu>2017-04-14 21:51:50 -0400
commit1b732bd5dd2cedb821345f5772842c0994237722 (patch)
treeb8e3181441a0eefc46ca68189d30fdd6db22dd7e /src/Compilers/TestCase.v
parent0faedd6652a3d0c7c0f21b34761f494a310ea62b (diff)
Split off a-normal form from flattening
Now we can flatten let binders without putting operations in a-normal form
Diffstat (limited to 'src/Compilers/TestCase.v')
-rw-r--r--src/Compilers/TestCase.v4
1 files changed, 2 insertions, 2 deletions
diff --git a/src/Compilers/TestCase.v b/src/Compilers/TestCase.v
index 5240cf9c5..a7fd81328 100644
--- a/src/Compilers/TestCase.v
+++ b/src/Compilers/TestCase.v
@@ -99,7 +99,7 @@ Import Linearize Inline.
Goal True.
let x := Reify (fun xy => let '(x, y) := xy in (let a := 1 in let '(c, d) := (2, 3) in a + x - a + c + d) + y)%nat in
- pose (InlineConst is_const (Linearize x)) as e.
+ pose (InlineConst is_const (ANormal x)) as e.
vm_compute in e.
Abort.
@@ -190,7 +190,7 @@ Section cse.
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).
End cse.
-Definition example_expr_simplified := Eval vm_compute in InlineConst is_const (Linearize example_expr).
+Definition example_expr_simplified := Eval vm_compute in InlineConst is_const (ANormal example_expr).
Compute CSE example_expr_simplified.
Definition example_expr_compiled