aboutsummaryrefslogtreecommitdiff
path: root/src/Assembly/Compile.v
diff options
context:
space:
mode:
Diffstat (limited to 'src/Assembly/Compile.v')
-rw-r--r--src/Assembly/Compile.v7
1 files changed, 5 insertions, 2 deletions
diff --git a/src/Assembly/Compile.v b/src/Assembly/Compile.v
index 9db4f7188..f0ee42e7c 100644
--- a/src/Assembly/Compile.v
+++ b/src/Assembly/Compile.v
@@ -15,9 +15,9 @@ Module CompileHL.
Section Compilation.
Context {T: Type}.
- Fixpoint compile {t} (e:@HL.expr T (@LL.arg T T) t) : @LL.expr T T t :=
+ Fixpoint compile {T t} (e:@HL.expr T (@LL.arg T T) t) : @LL.expr T T t :=
match e with
- | HL.Const n => LL.Return (LL.Const n)
+ | HL.Const _ n => LL.Return (LL.Const n)
| HL.Var _ arg => LL.Return arg
@@ -41,6 +41,9 @@ Module CompileHL.
let (a1, a2) := LL.match_arg_Prod arg in
compile (eC a1 a2))
end.
+
+ Definition Compile {T t} (e:@HL.Expr T t) : @LL.expr T T t :=
+ compile (e (@LL.arg T T)).
End Compilation.
Section Correctness.