@[reducible, inline]
abbrev
Lean.Compiler.LCNF.LetDecl.dependsOn
(decl : Lean.Compiler.LCNF.LetDecl)
(s : Lean.FVarIdSet)
:
Equations
- decl.dependsOn s = Lean.Compiler.LCNF.LetDecl.depOn✝ decl s
Instances For
@[reducible, inline]
abbrev
Lean.Compiler.LCNF.FunDecl.dependsOn
(decl : Lean.Compiler.LCNF.FunDecl)
(s : Lean.FVarIdSet)
:
Equations
- decl.dependsOn s = (Lean.Compiler.LCNF.typeDepOn✝ decl.type s || Lean.Compiler.LCNF.depOn✝ decl.value s)
Instances For
def
Lean.Compiler.LCNF.CodeDecl.dependsOn
(decl : Lean.Compiler.LCNF.CodeDecl)
(s : Lean.FVarIdSet)
:
Instances For
Return true
is c
depends on a free variable in s
.