Skip to content

Commit

Permalink
better error message for monomorphization failure
Browse files Browse the repository at this point in the history
  • Loading branch information
PratherConid committed Dec 18, 2024
1 parent 027d8de commit d3963a3
Showing 1 changed file with 3 additions and 1 deletion.
4 changes: 3 additions & 1 deletion Auto/Translation/Monomorphization.lean
Original file line number Diff line number Diff line change
Expand Up @@ -813,7 +813,9 @@ namespace FVarRep
let m₃ := m!"· Type argument with bound variables, e.g. `@Fin.add (n + 2) a b` where `n` is a bound variable"
let m₄ := m!"· λ binders whose type contain bound variables, e.g. `fun (x : a) => x` where `a` is a bound variable"
let m₅ := m!"· Other (TODO)"
m₁ ++ "\n" ++ m₂ ++ "\n" ++ m₃ ++ "\n" ++ m₄ ++ "\n" ++ m₅
let m₆ := m!"`set_option auto.mono.ignoreNonQuasiHigherOrder true` will instruct Lean-auto to ignore " ++
m!"all the `LemmaInst`s which contain expressions that cannot be handeled by the current procedure"
m₁ ++ "\n" ++ m₂ ++ "\n" ++ m₃ ++ "\n" ++ m₄ ++ "\n" ++ m₅ ++ "\n" ++ m₆

def unknownExpr2FVar (e : Expr) : FVarRepM (Expr ⊕ MessageData) := do
let bfvarSet ← getBfvarSet
Expand Down

0 comments on commit d3963a3

Please sign in to comment.