Skip to content

Commit

Permalink
wip tinkering
Browse files Browse the repository at this point in the history
  • Loading branch information
grunweg committed Feb 17, 2025
1 parent ce49515 commit 113d0cf
Showing 1 changed file with 10 additions and 0 deletions.
10 changes: 10 additions & 0 deletions Mathlib/Geometry/Manifold/Bordisms.lean
Original file line number Diff line number Diff line change
Expand Up @@ -216,6 +216,15 @@ def trivial (hequiv : H ≃ₜ EuclideanSpace ℝ (Fin n)) [h: Fact (finrank ℝ
f := fun _ ↦ PUnit.unit
hf := continuous_const

variable (α : Type*)
#synth TopologicalSpace (WithLp 2 α)

def WithLp.prodEquivSum (α β 𝕜 : Type*) [NontriviallyNormedField 𝕜] :
(WithLp 2 (PiLp 2 (fun _ : α ↦ 𝕜))) × (EuclideanSpace 𝕜 β) ≃ₜ EuclideanSpace 𝕜 (α ⊕ β) where
toEquiv := (Equiv.sumArrowEquivProdArrow α β 𝕜).symm
continuous_toFun := sorry
continuous_invFun := sorry

def EuclideanSpace.prodEquivSum (α β 𝕜 : Type*) [NontriviallyNormedField 𝕜] :
(EuclideanSpace 𝕜 α) × (EuclideanSpace 𝕜 β) ≃ₜ EuclideanSpace 𝕜 (α ⊕ β) where
toEquiv := (Equiv.sumArrowEquivProdArrow α β 𝕜).symm
Expand Down Expand Up @@ -262,6 +271,7 @@ instance {n : ℕ} (s t : SingularNManifold X n k) :
haveI := ChartedSpace.comp (EuclideanSpace ℝ (Fin n)) t.H t.M
infer_instance

-- missing: if M is a manifold w.r.t. I over (E, H), this transfer across a homeo
instance {n : ℕ} (s t : SingularNManifold X n k) : IsManifold (𝓡 n) k (s.M ⊕ t.M) := sorry

/-- The disjoint union of two singular `n`-manifolds on `X` is a singular `n`-manifold on `X`. -/
Expand Down

0 comments on commit 113d0cf

Please sign in to comment.