Skip to content

Commit

Permalink
chore: split Std.Data.Int.Lemmas (#534)
Browse files Browse the repository at this point in the history
  • Loading branch information
kim-em authored Jan 23, 2024
1 parent d3ccd13 commit 6ee0731
Show file tree
Hide file tree
Showing 6 changed files with 1,048 additions and 1,031 deletions.
1 change: 1 addition & 0 deletions Std/Data/Int.lean
Original file line number Diff line number Diff line change
Expand Up @@ -2,3 +2,4 @@ import Std.Data.Int.Basic
import Std.Data.Int.DivMod
import Std.Data.Int.Gcd
import Std.Data.Int.Lemmas
import Std.Data.Int.Order
2 changes: 1 addition & 1 deletion Std/Data/Int/DivMod.lean
Original file line number Diff line number Diff line change
Expand Up @@ -3,7 +3,7 @@ Copyright (c) 2016 Jeremy Avigad. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Jeremy Avigad, Mario Carneiro
-/
import Std.Data.Int.Lemmas
import Std.Data.Int.Order
import Std.Tactic.Change

/-!
Expand Down
Loading

0 comments on commit 6ee0731

Please sign in to comment.