Skip to content

Commit

Permalink
chore: cleanup (#4494)
Browse files Browse the repository at this point in the history
closes #4287
closes #4288
  • Loading branch information
leodemoura authored Jun 18, 2024
1 parent 1677719 commit 294b1d5
Show file tree
Hide file tree
Showing 2 changed files with 1 addition and 4 deletions.
2 changes: 1 addition & 1 deletion src/Init/Prelude.lean
Original file line number Diff line number Diff line change
Expand Up @@ -2976,7 +2976,7 @@ def MonadExcept.ofExcept [Monad m] [MonadExcept ε m] : Except ε α → m α

export MonadExcept (throw tryCatch ofExcept)

instance (ε : outParam (Type u)) (m : Type v → Type w) [MonadExceptOf ε m] : MonadExcept ε m where
instance (ε : Type u) (m : Type v → Type w) [MonadExceptOf ε m] : MonadExcept ε m where
throw := throwThe ε
tryCatch := tryCatchThe ε

Expand Down
3 changes: 0 additions & 3 deletions src/Lean/Meta/SynthInstance.lean
Original file line number Diff line number Diff line change
Expand Up @@ -194,9 +194,6 @@ def checkSystem : SynthM Unit := do
Core.checkInterrupted
Core.checkMaxHeartbeatsCore "typeclass" `synthInstance.maxHeartbeats (← read).maxHeartbeats

@[inline] def mapMetaM (f : forall {α}, MetaM α → MetaM α) {α} : SynthM α → SynthM α :=
monadMap @f

instance : Inhabited (SynthM α) where
default := fun _ _ => default

Expand Down

0 comments on commit 294b1d5

Please sign in to comment.