Skip to content
This repository was archived by the owner on Jul 24, 2024. It is now read-only.

Commit 29d5700

Browse files
committed
chore(geometry/manifold/instances/sphere): speedup a proof (#18586)
This goes from 15s to 1.75 seconds. I've squeezed this in multiple steps to make the proof easier to follow.
1 parent 0111834 commit 29d5700

File tree

1 file changed

+9
-2
lines changed

1 file changed

+9
-2
lines changed

src/geometry/manifold/instances/sphere.lean

Lines changed: 9 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -398,8 +398,15 @@ begin
398398
have H₂ := (cont_diff_stereo_inv_fun_aux.comp
399399
(ℝ ∙ (v:E))ᗮ.subtypeL.cont_diff).comp U.symm.cont_diff,
400400
convert H₁.comp' (H₂.cont_diff_on : cont_diff_on ℝ ⊤ _ set.univ) using 1,
401-
ext,
402-
simp [sphere_ext_iff, stereographic'_symm_apply, real_inner_comm]
401+
-- squeezed from `ext, simp [sphere_ext_iff, stereographic'_symm_apply, real_inner_comm]`
402+
simp only [local_homeomorph.trans_to_local_equiv, local_homeomorph.symm_to_local_equiv,
403+
local_equiv.trans_source, local_equiv.symm_source, stereographic'_target,
404+
stereographic'_source],
405+
simp only [model_with_corners_self_coe, model_with_corners_self_coe_symm, set.preimage_id,
406+
set.range_id, set.inter_univ, set.univ_inter, set.compl_singleton_eq, set.preimage_set_of_eq],
407+
simp only [id.def, comp_apply, submodule.subtypeL_apply, local_homeomorph.coe_coe_symm,
408+
innerSL_apply, ne.def, sphere_ext_iff, real_inner_comm (v' : E)],
409+
refl,
403410
end
404411

405412
/-- The inclusion map (i.e., `coe`) from the sphere in `E` to `E` is smooth. -/

0 commit comments

Comments
 (0)