File tree Expand file tree Collapse file tree 3 files changed +551
-3
lines changed Expand file tree Collapse file tree 3 files changed +551
-3
lines changed Original file line number Diff line number Diff line change @@ -8,6 +8,7 @@ import Mathlib.Data.ByteArray
8
8
import Mathlib.Data.Char
9
9
import Mathlib.Data.Equiv.Basic
10
10
import Mathlib.Data.Equiv.Functor
11
+ import Mathlib.Data.Int.Basic
11
12
import Mathlib.Data.List.Basic
12
13
import Mathlib.Data.Nat.Basic
13
14
import Mathlib.Data.Nat.Gcd
Original file line number Diff line number Diff line change 1
1
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"
2
3
import Mathlib.Tactic.Spread
3
4
4
5
/-!
@@ -60,9 +61,6 @@ end nat_action
60
61
61
62
section int_action
62
63
63
- -- TODO -- this should be in a prelude
64
- notation "ℤ" => Int
65
-
66
64
/-- The fundamental scalar multiplication in an additive group. `gsmul_rec n a = a+a+...+a` n
67
65
times, for integer `n`. Use instead `n • a`, which has better definitional behavior. -/
68
66
def gsmul_rec {G : Type u} [Zero G] [Add G] [Neg G]: ℤ → G → G
You can’t perform that action at this time.
0 commit comments