Skip to content

Commit

Permalink
fix
Browse files Browse the repository at this point in the history
  • Loading branch information
kim-em committed Nov 19, 2024
1 parent d2b159a commit 479f69a
Showing 1 changed file with 4 additions and 1 deletion.
5 changes: 4 additions & 1 deletion Plausible/Testable.lean
Original file line number Diff line number Diff line change
Expand Up @@ -365,7 +365,10 @@ partial def minimizeAux [SampleableExt α] {β : α → Prop} [∀ x, Testable (
if res.isFailure then
if cfg.traceShrink then
slimTrace s!"{var} shrunk to {repr candidate} from {repr x}"
let currentStep := OptionT.lift <| return Sigma.mk candidate (addShrinks (n + 1) res)
-- Adaptation note:
-- The type ascription was not needed here before https://github.com/leanprover/lean4/pull/6104
let currentStep : OptionT Gen ((x : _) × TestResult (β (SampleableExt.interp x))) :=
OptionT.lift <| return Sigma.mk candidate (addShrinks (n + 1) res)
let nextStep := minimizeAux cfg var candidate (n + 1)
return ← (nextStep <|> currentStep)
if cfg.traceShrink then
Expand Down

0 comments on commit 479f69a

Please sign in to comment.