File tree Expand file tree Collapse file tree 1 file changed +4
-1
lines changed
Mathlib/Geometry/Manifold/IsManifold Expand file tree Collapse file tree 1 file changed +4
-1
lines changed Original file line number Diff line number Diff line change @@ -690,11 +690,14 @@ theorem isManifold_of_contDiffOn {𝕜 : Type*} [NontriviallyNormedField 𝕜]
690
690
alias smoothManifoldWithCorners_of_contDiffOn := isManifold_of_contDiffOn
691
691
692
692
/-- For any model with corners, the model space is a `C^n` manifold -/
693
- instance intIsManifoldModelSpace {𝕜 : Type *} [NontriviallyNormedField 𝕜] {E : Type *}
693
+ instance instIsManifoldModelSpace {𝕜 : Type *} [NontriviallyNormedField 𝕜] {E : Type *}
694
694
[NormedAddCommGroup E] [NormedSpace 𝕜 E] {H : Type *} [TopologicalSpace H]
695
695
{I : ModelWithCorners 𝕜 E H} {n : WithTop ℕ∞} : IsManifold I n H :=
696
696
{ hasGroupoid_model_space _ _ with }
697
697
698
+ @[deprecated (since := "2025-04-22")]
699
+ alias intIsManifoldModelSpace := instIsManifoldModelSpace
700
+
698
701
end IsManifold
699
702
700
703
namespace IsManifold
You can’t perform that action at this time.
0 commit comments