Skip to content

Commit

Permalink
Remove NormedGroup: one lemma is in mathlib already,
Browse files Browse the repository at this point in the history
the other can be inlined easily. It's just adding up two inequalities,
that should be golfed using a suitable tactic, not extracted into a lemma.
  • Loading branch information
grunweg committed Jan 24, 2024
1 parent 1461dc5 commit d91dd15
Show file tree
Hide file tree
Showing 3 changed files with 1 addition and 13 deletions.
1 change: 0 additions & 1 deletion SphereEversion.lean
Original file line number Diff line number Diff line change
Expand Up @@ -36,7 +36,6 @@ import SphereEversion.ToMathlib.Analysis.InnerProductSpace.CrossProduct
import SphereEversion.ToMathlib.Analysis.InnerProductSpace.Dual
import SphereEversion.ToMathlib.Analysis.InnerProductSpace.Projection
import SphereEversion.ToMathlib.Analysis.InnerProductSpace.Rotation
import SphereEversion.ToMathlib.Analysis.NormedGroup
import SphereEversion.ToMathlib.Analysis.NormedSpace.Misc
import SphereEversion.ToMathlib.Analysis.NormedSpace.OperatorNorm
import SphereEversion.ToMathlib.Data.Nat.Basic
Expand Down
3 changes: 1 addition & 2 deletions SphereEversion/Local/HPrinciple.lean
Original file line number Diff line number Diff line change
@@ -1,4 +1,3 @@
import SphereEversion.ToMathlib.Analysis.NormedGroup
import SphereEversion.ToMathlib.LinearAlgebra.Basis
import SphereEversion.Loops.Exists
import SphereEversion.Local.Corrugation
Expand Down Expand Up @@ -546,7 +545,7 @@ theorem RelLoc.FormalSol.improve (𝓕 : FormalSol R) (h_hol : ∀ᶠ x near L.C
simp only [ht, hHc0, HtpyJetSec.comp_of_le]
· simp only [ht, HtpyJetSec.comp_of_not_le, not_false_iff]
rw [← add_halves δ]
exact norm_sub_le_add_of_le (hN_close _ _) (hHc0 _ _)
exact (norm_sub_le_norm_sub_add_norm_sub _ _ _).trans <| add_le_add (hN_close _ _) (hHc0 _ _)
· -- formal solution
intro t
by_cases ht : t ≤ 1 / 2
Expand Down
10 changes: 0 additions & 10 deletions SphereEversion/ToMathlib/Analysis/NormedGroup.lean

This file was deleted.

0 comments on commit d91dd15

Please sign in to comment.