aboutsummaryrefslogtreecommitdiff
path: root/src/Assembly/Compile.v
diff options
context:
space:
mode:
authorGravatar Jason Gross <jgross@mit.edu>2016-10-22 16:06:49 -0400
committerGravatar Jason Gross <jgross@mit.edu>2016-10-22 16:06:49 -0400
commit7a0ca3b4172584368a3d83053db77f287f3d5ddd (patch)
tree511af6c9667f11f3d52f949bec852bb2234032aa /src/Assembly/Compile.v
parent75e070f25b8f17643f8cfee38f6fa0ef38de6171 (diff)
Fix 8.4 build
Diffstat (limited to 'src/Assembly/Compile.v')
-rw-r--r--src/Assembly/Compile.v5
1 files changed, 3 insertions, 2 deletions
diff --git a/src/Assembly/Compile.v b/src/Assembly/Compile.v
index 9948be50a..e072342a5 100644
--- a/src/Assembly/Compile.v
+++ b/src/Assembly/Compile.v
@@ -283,11 +283,12 @@ Module CompileLL.
(fun rt var op x y out => Some out)
(fun t' a => Some (vars a)).
- Fixpoint fillInputs {t inputs} (prog: NAry inputs Z (WExpr t)) {struct inputs}: WExpr t :=
+ Fixpoint fillInputs t inputs (prog: NAry inputs Z (WExpr t)) {struct inputs}: WExpr t :=
match inputs as inputs' return NAry inputs' Z (WExpr t) -> NAry O Z (WExpr t) with
| O => fun p => p
- | S inputs'' => fun p => fillInputs (p (Z.of_nat inputs))
+ | S inputs'' => fun p => @fillInputs _ _ (p (Z.of_nat inputs))
end prog.
+ Global Arguments fillInputs {t inputs} _.
Definition compile {t inputs} (p: NAry inputs Z (WExpr t)): option (Program * list nat) :=
let p' := fillInputs p in