Skip to content

Commit a43628d

Browse files
revert spurious change
1 parent 3b118ae commit a43628d

File tree

1 file changed

+1
-2
lines changed

1 file changed

+1
-2
lines changed

Mathlib/Data/Nat/Factorial/Basic.lean

Lines changed: 1 addition & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -446,8 +446,7 @@ theorem descFactorial_lt_pow {n : ℕ} (hn : n ≠ 0) : ∀ {k : ℕ}, 2 ≤ k
446446
| 1 => by intro; contradiction
447447
| k + 2 => fun _ => by
448448
rw [descFactorial_succ, pow_succ', Nat.mul_comm, Nat.mul_comm n]
449-
exact Nat.mul_lt_mul_of_le_of_lt (descFactorial_le_pow _ _) (by lia)
450-
(Nat.pow_pos <| by lia)
449+
exact Nat.mul_lt_mul_of_le_of_lt (descFactorial_le_pow _ _) (by lia) (Nat.pow_pos <| by lia)
451450

452451
end DescFactorial
453452

0 commit comments

Comments
 (0)