Skip to content

Commit 9a4a3ba

Browse files
authored
feat(Data/Int): port data.int.basic from the lean3 prelude (#23)
* port lean3 core's int/basic.lean * refactor(Int): undo my strange naming * add coe_nat_inj which I apparantly forgot about * minor cleanup * add missing imports * cleanup proofs, implementing kevin's suggestions Co-authored-by: Deniz Aydin <40861512+BeesNation@users.noreply.github.com>
1 parent 93b0fef commit 9a4a3ba

File tree

3 files changed

+551
-3
lines changed

3 files changed

+551
-3
lines changed

Mathlib.lean

Lines changed: 1 addition & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -8,6 +8,7 @@ import Mathlib.Data.ByteArray
88
import Mathlib.Data.Char
99
import Mathlib.Data.Equiv.Basic
1010
import Mathlib.Data.Equiv.Functor
11+
import Mathlib.Data.Int.Basic
1112
import Mathlib.Data.List.Basic
1213
import Mathlib.Data.Nat.Basic
1314
import Mathlib.Data.Nat.Gcd

Mathlib/Algebra/Group/Defs.lean

Lines changed: 1 addition & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -1,4 +1,5 @@
11
import Mathlib.Data.Nat.Basic -- *only* for notation ℕ which should be in a "prelude"
2+
import Mathlib.Data.Int.Basic -- *only* for notation ℤ which should be in a "prelude"
23
import Mathlib.Tactic.Spread
34

45
/-!
@@ -60,9 +61,6 @@ end nat_action
6061

6162
section int_action
6263

63-
-- TODO -- this should be in a prelude
64-
notation "ℤ" => Int
65-
6664
/-- The fundamental scalar multiplication in an additive group. `gsmul_rec n a = a+a+...+a` n
6765
times, for integer `n`. Use instead `n • a`, which has better definitional behavior. -/
6866
def gsmul_rec {G : Type u} [Zero G] [Add G] [Neg G]: ℤ → G → G

0 commit comments

Comments
 (0)