File tree Expand file tree Collapse file tree 2 files changed +4
-0
lines changed
Expand file tree Collapse file tree 2 files changed +4
-0
lines changed Original file line number Diff line number Diff line change @@ -50,6 +50,8 @@ protected theorem pow_ne_zero {n : Int} {m : Nat} : n ≠ 0 → n ^ m ≠ 0 := b
5050
5151instance {n : Int} {m : Nat} [NeZero n] : NeZero (n ^ m) := ⟨Int.pow_ne_zero (NeZero.ne _)⟩
5252
53+ instance {n : Int} : NeZero (n^0 ) := ⟨Int.one_ne_zero⟩
54+
5355-- This can't be removed until the next update-stage0
5456@[deprecated Nat.pow_pos (since := "2025-02-17")]
5557abbrev _root_.Nat.pos_pow_of_pos := @Nat.pow_pos
Original file line number Diff line number Diff line change @@ -801,6 +801,8 @@ protected theorem two_pow_pos (w : Nat) : 0 < 2^w := Nat.pow_pos (by decide)
801801instance {n m : Nat} [NeZero n] : NeZero (n^m) :=
802802 ⟨Nat.ne_zero_iff_zero_lt.mpr (Nat.pow_pos (pos_of_neZero _))⟩
803803
804+ instance {n : Nat} : NeZero (n^0 ) := ⟨Nat.one_ne_zero⟩
805+
804806protected theorem mul_pow (a b n : Nat) : (a * b) ^ n = a ^ n * b ^ n := by
805807 induction n with
806808 | zero => simp [Nat.pow_zero]
You can’t perform that action at this time.
0 commit comments