aboutsummaryrefslogtreecommitdiff
path: root/src/Reflection/InlineWf.v
diff options
context:
space:
mode:
Diffstat (limited to 'src/Reflection/InlineWf.v')
-rw-r--r--src/Reflection/InlineWf.v5
1 files changed, 3 insertions, 2 deletions
diff --git a/src/Reflection/InlineWf.v b/src/Reflection/InlineWf.v
index 5e402bf97..d721f9ce7 100644
--- a/src/Reflection/InlineWf.v
+++ b/src/Reflection/InlineWf.v
@@ -1,5 +1,6 @@
(** * Inline: Remove some [Let] expressions *)
Require Import Crypto.Reflection.Syntax.
+Require Import Crypto.Reflection.Wf.
Require Import Crypto.Reflection.WfProofs.
Require Import Crypto.Reflection.Inline.
Require Import Crypto.Util.Tactics.SpecializeBy Crypto.Util.Tactics.DestructHead Crypto.Util.Sigma Crypto.Util.Prod.
@@ -21,11 +22,11 @@ Section language.
Section with_var.
Context {var1 var2 : base_type_code -> Type}.
- Local Hint Constructors Syntax.wff.
+ Local Hint Constructors Wf.wff.
Local Hint Resolve List.in_app_or List.in_or_app.
Local Hint Constructors or.
- Local Hint Constructors Syntax.wff.
+ Local Hint Constructors Wf.wff.
Local Hint Extern 1 => progress unfold List.In in *.
Local Hint Resolve wff_in_impl_Proper.
Local Hint Resolve wff_SmartVarf.