aboutsummaryrefslogtreecommitdiff
path: root/src/Compilers/Z/InlineConstAndOpInterp.v
diff options
context:
space:
mode:
Diffstat (limited to 'src/Compilers/Z/InlineConstAndOpInterp.v')
-rw-r--r--src/Compilers/Z/InlineConstAndOpInterp.v11
1 files changed, 0 insertions, 11 deletions
diff --git a/src/Compilers/Z/InlineConstAndOpInterp.v b/src/Compilers/Z/InlineConstAndOpInterp.v
deleted file mode 100644
index 417085929..000000000
--- a/src/Compilers/Z/InlineConstAndOpInterp.v
+++ /dev/null
@@ -1,11 +0,0 @@
-Require Import Crypto.Compilers.Syntax.
-Require Import Crypto.Compilers.Wf.
-Require Import Crypto.Compilers.InlineConstAndOpInterp.
-Require Import Crypto.Compilers.Z.Syntax.
-Require Import Crypto.Compilers.Z.InlineConstAndOp.
-
-Definition InterpInlineConstAndOp {t} (e : Expr t) (Hwf : Wf e)
- : forall x, Interp (InlineConstAndOp e) x = Interp e x
- := @InterpInlineConstAndOp _ _ _ _ _ t e Hwf Syntax.Util.make_const_correct.
-
-Hint Rewrite @InterpInlineConstAndOp using solve_wf_side_condition : reflective_interp.