Skip to content

Commit

Permalink
zeta := false forever
Browse files Browse the repository at this point in the history
  • Loading branch information
PatrickMassot committed Sep 13, 2023
1 parent fb95368 commit 1e945bb
Showing 1 changed file with 1 addition and 4 deletions.
5 changes: 1 addition & 4 deletions SphereEversion/Loops/Exists.lean
Original file line number Diff line number Diff line change
Expand Up @@ -77,10 +77,7 @@ theorem exist_loops_aux1 (hK : IsCompact K) (hΩ_op : IsOpen Ω) (hb : 𝒞 ∞
rw [← h0ε₁, add_halves']
refine' (ball_subset_thickening (mem_image_of_mem _ hx.2) _).trans hεΩ
· rintro x ⟨-, -⟩ t s
-- Porting note: should be `simp [h2ε]`
simp only [Loop.transform_apply]
simp only [dist_self_add_left]
simp only [h2ε]
simp (config := {zeta := false}) [h2ε]

/- Some remarks about `exist_loops_aux2`:
`δ`: loop after smoothing
Expand Down

0 comments on commit 1e945bb

Please sign in to comment.