aboutsummaryrefslogtreecommitdiff
path: root/src/Compilers/Named/Wf.v
diff options
context:
space:
mode:
Diffstat (limited to 'src/Compilers/Named/Wf.v')
-rw-r--r--src/Compilers/Named/Wf.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/src/Compilers/Named/Wf.v b/src/Compilers/Named/Wf.v
index 736d0bd81..79f620edb 100644
--- a/src/Compilers/Named/Wf.v
+++ b/src/Compilers/Named/Wf.v
@@ -18,7 +18,7 @@ Module Export Named.
Fixpoint wff_gen (ctx : Context) {t} (e : @exprf base_type_code op Name t) : option pointed_Prop
:= match e with
| TT => Some trivial
- | Var t n => match lookupb ctx n t return bool with
+ | Var t n => match lookupb t ctx n return bool with
| Some _ => true
| None => false
end