aboutsummaryrefslogtreecommitdiff
path: root/src/Reflection/InterpProofs.v
diff options
context:
space:
mode:
authorGravatar Jason Gross <jgross@mit.edu>2017-01-26 18:19:54 -0500
committerGravatar Jason Gross <jgross@mit.edu>2017-01-26 18:20:08 -0500
commit39c70ae2abd720ec76e01c85d2aa0e56aeae3414 (patch)
treeb8ca8c8c4e935a078813d1f753f29db7e95f91d4 /src/Reflection/InterpProofs.v
parent0cf72bdda642db646e25cba8af97f3c63d88764d (diff)
Split off some bits of Reflection.Syntax
Also split off some bits of Util.Tactics
Diffstat (limited to 'src/Reflection/InterpProofs.v')
-rw-r--r--src/Reflection/InterpProofs.v6
1 files changed, 4 insertions, 2 deletions
diff --git a/src/Reflection/InterpProofs.v b/src/Reflection/InterpProofs.v
index abd54ec3b..b0aa20ccf 100644
--- a/src/Reflection/InterpProofs.v
+++ b/src/Reflection/InterpProofs.v
@@ -1,4 +1,6 @@
Require Import Crypto.Reflection.Syntax.
+Require Import Crypto.Reflection.Wf.
+Require Import Crypto.Reflection.SmartMap.
Require Import Crypto.Reflection.WfProofs.
Require Import Crypto.Util.LetIn.
Require Import Crypto.Util.Tactics Crypto.Util.Sigma Crypto.Util.Prod.
@@ -37,7 +39,7 @@ Section language.
(Hin : List.In
(existT (fun t : base_type_code => (exprf base_type_code op (Tbase t) * interp_base_type t)%type)
t (x, x'))
- (flatten_binding_list (t := t') base_type_code (SmartVarVarf v) v))
+ (flatten_binding_list (t := t') (SmartVarVarf v) v))
: interpf interp_op x = x'.
Proof.
clear -Hin.
@@ -52,7 +54,7 @@ Section language.
(Hin : List.In
(existT (fun t : base_type_code => (exprf base_type_code op (Tbase t) * interp_base_type t)%type)
t (x, x'))
- (flatten_binding_list (t := t') base_type_code (SmartVarVarf v') v))
+ (flatten_binding_list (t := t') (SmartVarVarf v') v))
: interpf interp_op x = x'.
Proof.
subst; eapply interpf_SmartVarVarf; eassumption.