We read every piece of feedback, and take your input very seriously.
To see all available qualifiers, see our documentation.
There was an error while loading. Please reload this page.
1 parent 1328e6e commit aafb96fCopy full SHA for aafb96f
Mathlib/Lean/Expr/Basic.lean
@@ -103,7 +103,7 @@ def isInternal' (declName : Name) : Bool :=
103
open Meta
104
105
-- from Lean.Server.Completion
106
-def isBlackListed (declName : Name) : CoreM Bool := do
+def isBlackListed {m} [Monad m] [MonadEnv m] (declName : Name) : m Bool := do
107
if declName == ``sorryAx then return true
108
if declName matches .str _ "inj" then return true
109
if declName matches .str _ "noConfusionType" then return true
0 commit comments