Skip to content

Commit ac21cca

Browse files
committed
Remove useless intermediate have.
1 parent e7efe2b commit ac21cca

File tree

1 file changed

+1
-2
lines changed

1 file changed

+1
-2
lines changed

SphereEversion/ToMathlib/Analysis/InnerProductSpace/Rotation.lean

Lines changed: 1 addition & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -147,7 +147,7 @@ theorem injOn_rot_of_ne (t : ℝ) {x : E} (hx : x ≠ 0) : Set.InjOn (ω.rot (t,
147147
simp_rw [← pow_two, norm_smul, mul_pow] at hy
148148
change _ + _ * ‖x×₃(⟨y, hy'⟩ : (span ℝ {x})ᗮ)‖ ^ 2 = ‖(0 : E)‖ ^ 2 at hy
149149
rw [norm_crossProduct] at hy
150-
simp (config := {decide := true}) only [norm_eq_abs, Even.pow_abs, coe_mk, norm_zero, zero_pow,
150+
simp (config := {decide := true}) only [norm_eq_abs, Even.pow_abs, coe_mk, norm_zero, zero_pow,
151151
Ne, Nat.one_ne_zero, not_false_iff] at hy
152152
change _ + _ * (_ * ‖y‖) ^ 2 = 0 at hy
153153
rw [mul_pow, ← mul_assoc, ← add_mul, mul_eq_zero, or_iff_not_imp_left] at hy
@@ -156,7 +156,6 @@ theorem injOn_rot_of_ne (t : ℝ) {x : E} (hx : x ≠ 0) : Set.InjOn (ω.rot (t,
156156
rw [cos_sq']
157157
rw [show (1 : ℝ) - sin (t * π) ^ 2 + sin (t * π) ^ 2 * ‖x‖ ^ 2 = (1 : ℝ) + sin (t * π) ^ 2 * (‖x‖ ^ 2 - 1)
158158
by ring]
159-
have I₁ : ‖x‖ ^ 2 - 1 > -1 := by linarith
160159
have I₂ : sin (t * π) ^ 21 := sin_sq_le_one (t * π)
161160
have I₃ : (0 : ℝ) ≤ sin (t * π) ^ 2 := sq_nonneg _
162161
rcases I₃.eq_or_lt with (H | H)

0 commit comments

Comments
 (0)