Skip to content

Commit

Permalink
better trace message for non quasi higher-order
Browse files Browse the repository at this point in the history
  • Loading branch information
PratherConid committed Jan 13, 2025
1 parent 57c655e commit d62b650
Showing 1 changed file with 6 additions and 1 deletion.
7 changes: 6 additions & 1 deletion Auto/Translation/Monomorphization.lean
Original file line number Diff line number Diff line change
Expand Up @@ -1104,7 +1104,12 @@ where
let liTypeRep? ← FVarRep.replacePolyWithFVar li.type
match liTypeRep? with
| .inl liTypeRep => return .some ⟨li.proof, liTypeRep, li.deriv⟩
| .inr m => if (← getIgnoreNonQuasiHigherOrder) then return .none else throwError m)
| .inr m =>
if (← getIgnoreNonQuasiHigherOrder) then
trace[auto.mono] "Don't know how to deal with fact {li.type}, ignoring it"
return .none
else
throwError m)
fvarRepMInductAction (ivals : Array (Array SimpleIndVal)) : FVarRep.FVarRepM (Array (Array SimpleIndVal)) :=
ivals.mapM (fun svals => svals.mapM (fun ⟨name, type, ctors, projs⟩ => do
let (type, _) ← FVarRep.processType type
Expand Down

0 comments on commit d62b650

Please sign in to comment.