Skip to content

Commit

Permalink
chore: remove LazyInitExtension
Browse files Browse the repository at this point in the history
  • Loading branch information
Kha committed Oct 8, 2024
1 parent 7c29c3f commit 9807459
Show file tree
Hide file tree
Showing 3 changed files with 0 additions and 44 deletions.
1 change: 0 additions & 1 deletion src/Lean.lean
Original file line number Diff line number Diff line change
Expand Up @@ -30,7 +30,6 @@ import Lean.Server
import Lean.ScopedEnvExtension
import Lean.DocString
import Lean.DeclarationRange
import Lean.LazyInitExtension
import Lean.LoadDynlib
import Lean.Widget
import Lean.Log
Expand Down
42 changes: 0 additions & 42 deletions src/Lean/LazyInitExtension.lean

This file was deleted.

1 change: 0 additions & 1 deletion src/Lean/Meta/Tactic/SplitIf.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,6 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Leonardo de Moura
-/
prelude
import Lean.LazyInitExtension
import Lean.Meta.Tactic.Cases
import Lean.Meta.Tactic.Simp.Main

Expand Down

0 comments on commit 9807459

Please sign in to comment.