Skip to content

Commit dacd3b1

Browse files
chore: move Int.coe_nat_strictMono (#13197)
1 parent b671156 commit dacd3b1

File tree

3 files changed

+7
-10
lines changed

3 files changed

+7
-10
lines changed

Mathlib/Algebra/Group/Int.lean

Lines changed: 1 addition & 6 deletions
Original file line numberDiff line numberDiff line change
@@ -4,7 +4,6 @@ Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Jeremy Avigad
55
-/
66
import Mathlib.Algebra.Group.Nat
7-
import Mathlib.Order.Monotone.Basic
87
import Mathlib.Tactic.Common
98

109
#align_import data.int.basic from "leanprover-community/mathlib"@"00d163e35035c3577c1c79fa53b68de17781ffc1"
@@ -19,8 +18,7 @@ See note [foundational algebra order theory].
1918
-/
2019

2120
assert_not_exists Ring
22-
-- TODO
23-
-- assert_not_exists DenselyOrdered
21+
assert_not_exists DenselyOrdered
2422

2523
open Nat
2624

@@ -79,9 +77,6 @@ lemma natAbs_pow (n : ℤ) (k : ℕ) : Int.natAbs (n ^ k) = Int.natAbs n ^ k :=
7977
· rw [_root_.pow_succ, natAbs_mul, Nat.pow_succ, ih, Nat.mul_comm]
8078
#align int.nat_abs_pow Int.natAbs_pow
8179

82-
theorem coe_nat_strictMono : StrictMono (· : ℕ → ℤ) := fun _ _ ↦ Int.ofNat_lt.2
83-
#align int.coe_nat_strict_mono Int.coe_nat_strictMono
84-
8580
section Multiplicative
8681

8782
open Multiplicative

Mathlib/Algebra/GroupPower/IterateHom.lean

Lines changed: 3 additions & 4 deletions
Original file line numberDiff line numberDiff line change
@@ -4,9 +4,8 @@ Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Yury Kudryashov
55
-/
66
import Mathlib.Algebra.Group.Int
7-
import Mathlib.Algebra.Group.Nat
87
import Mathlib.GroupTheory.GroupAction.Opposite
9-
import Mathlib.Tactic.Common
8+
import Mathlib.Logic.Function.Iterate
109

1110
#align_import algebra.hom.iterate from "leanprover-community/mathlib"@"792a2a264169d64986541c6f8f7e3bbb6acb6295"
1211

@@ -27,6 +26,8 @@ We also prove formulas for iterates of add/mul left/right.
2726
homomorphism, iterate
2827
-/
2928

29+
assert_not_exists DenselyOrdered
30+
assert_not_exists Ring
3031

3132
open Function
3233

@@ -192,5 +193,3 @@ theorem Commute.function_commute_mul_right (h : Commute a b) :
192193
#align add_commute.function_commute_add_right AddCommute.function_commute_add_right
193194

194195
end Semigroup
195-
196-
assert_not_exists Ring

Mathlib/Algebra/Order/Group/Int.lean

Lines changed: 3 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -34,6 +34,9 @@ open Function Nat
3434

3535
namespace Int
3636

37+
theorem coe_nat_strictMono : StrictMono (· : ℕ → ℤ) := fun _ _ ↦ Int.ofNat_lt.2
38+
#align int.coe_nat_strict_mono Int.coe_nat_strictMono
39+
3740
instance linearOrderedAddCommGroup : LinearOrderedAddCommGroup ℤ where
3841
__ := instLinearOrder
3942
__ := instAddCommGroup

0 commit comments

Comments
 (0)