aboutsummaryrefslogtreecommitdiff
path: root/src/Reflection/InputSyntax.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/InputSyntax.v
parent0cf72bdda642db646e25cba8af97f3c63d88764d (diff)
Split off some bits of Reflection.Syntax
Also split off some bits of Util.Tactics
Diffstat (limited to 'src/Reflection/InputSyntax.v')
-rw-r--r--src/Reflection/InputSyntax.v3
1 files changed, 2 insertions, 1 deletions
diff --git a/src/Reflection/InputSyntax.v b/src/Reflection/InputSyntax.v
index 3cd688cf3..42ac17069 100644
--- a/src/Reflection/InputSyntax.v
+++ b/src/Reflection/InputSyntax.v
@@ -1,6 +1,7 @@
(** * PHOAS Representation of Gallina which allows exact denotation *)
Require Import Coq.Strings.String.
Require Import Crypto.Reflection.Syntax.
+Require Import Crypto.Reflection.SmartMap.
Require Import Crypto.Reflection.Relations.
Require Import Crypto.Reflection.InterpProofs.
Require Import Crypto.Util.Tuple.
@@ -79,7 +80,7 @@ Section language.
Fixpoint compilef {t} (e : @exprf (interp_flat_type_gen var) t) : @Syntax.exprf base_type_code op var t
:= match e in exprf t return @Syntax.exprf _ _ _ t with
| Const _ x => @SmartConst _ x
- | Var _ x => Syntax.SmartVarf x
+ | Var _ x => SmartMap.SmartVarf x
| Op _ _ op args => Syntax.Op op (@compilef _ args)
| LetIn _ ex _ eC => Syntax.LetIn (@compilef _ ex) (fun x => @compilef _ (eC x))
| Pair _ ex _ ey => Syntax.Pair (@compilef _ ex) (@compilef _ ey)