Skip to content

Commit

Permalink
ignoreUsableFacts option bug fix
Browse files Browse the repository at this point in the history
  • Loading branch information
JOSHCLUNE committed Oct 15, 2024
1 parent a0afb1e commit e68416d
Showing 1 changed file with 2 additions and 1 deletion.
3 changes: 2 additions & 1 deletion Duper/Tactic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -67,7 +67,8 @@ def elabFact (stx : Term) : TacticM (Array (Expr × Expr × Array Name)) := do
match stx with
| `($id:ident) =>
let some expr ← Term.resolveId? id
| throwError "Unknown identifier {id}"
| if ← getIgnoreUsableFactsM then return #[]
else throwError "Unknown identifier {id}"
match expr with
| .const exprConstName _ =>
match (← getEnv).find? exprConstName with
Expand Down

0 comments on commit e68416d

Please sign in to comment.