From e0ccbbe6213c4c7c56e6f664ce0c818d44451037 Mon Sep 17 00:00:00 2001 From: Michael Rothgang Date: Mon, 22 Jul 2024 19:12:47 +0200 Subject: [PATCH] Fix a few lean3 names. --- SphereEversion/ToMathlib/Analysis/ContDiff.lean | 2 +- SphereEversion/ToMathlib/Analysis/Convex/Basic.lean | 2 +- .../ToMathlib/Analysis/InnerProductSpace/CrossProduct.lean | 2 +- SphereEversion/ToMathlib/LinearAlgebra/Basic.lean | 2 +- 4 files changed, 4 insertions(+), 4 deletions(-) diff --git a/SphereEversion/ToMathlib/Analysis/ContDiff.lean b/SphereEversion/ToMathlib/Analysis/ContDiff.lean index d8330fef..3f59b92f 100644 --- a/SphereEversion/ToMathlib/Analysis/ContDiff.lean +++ b/SphereEversion/ToMathlib/Analysis/ContDiff.lean @@ -230,7 +230,7 @@ variable {๐•œ : Type*} [RCLike ๐•œ] variable {E : Type*} [NormedAddCommGroup E] [InnerProductSpace ๐•œ E] [CompleteSpace E] --- variant of `orthogonal_projection_singleton` +-- variant of `orthogonalProjection_singleton` theorem orthogonalProjection_singleton' {v : E} : (๐•œ โˆ™ v).subtypeL.comp (orthogonalProjection (๐•œ โˆ™ v)) = (1 / (โ€–vโ€– : ๐•œ) ^ 2) โ€ข .toSpanSingleton ๐•œ v โˆ˜L InnerProductSpace.toDual ๐•œ E v := by diff --git a/SphereEversion/ToMathlib/Analysis/Convex/Basic.lean b/SphereEversion/ToMathlib/Analysis/Convex/Basic.lean index f6a0564b..bb00c91d 100644 --- a/SphereEversion/ToMathlib/Analysis/Convex/Basic.lean +++ b/SphereEversion/ToMathlib/Analysis/Convex/Basic.lean @@ -103,7 +103,7 @@ theorem reallyConvexHull_mono : Monotone (reallyConvexHull ๐•œ : Set E โ†’ Set rintro s t h _ โŸจw, w_pos, supp_w, sum_w, rflโŸฉ exact โŸจw, w_pos, supp_w.trans h, sum_w, rflโŸฉ -/-- Generalization of `convex` to semirings. We only add the `s = โˆ…` clause if `๐•œ` is trivial. -/ +/-- Generalization of `Convex` to semirings. We only add the `s = โˆ…` clause if `๐•œ` is trivial. -/ def ReallyConvex (๐•œ : Type*) {E : Type*} [OrderedSemiring ๐•œ] [AddCommMonoid E] [Module ๐•œ E] (s : Set E) : Prop := s = โˆ… โˆจ โˆ€ w : E โ†’ ๐•œ, 0 โ‰ค w โ†’ support w โŠ† s โ†’ โˆ‘แถ  x, w x = 1 โ†’ โˆ‘แถ  x, w x โ€ข x โˆˆ s diff --git a/SphereEversion/ToMathlib/Analysis/InnerProductSpace/CrossProduct.lean b/SphereEversion/ToMathlib/Analysis/InnerProductSpace/CrossProduct.lean index 662092f6..fe0bd9c2 100644 --- a/SphereEversion/ToMathlib/Analysis/InnerProductSpace/CrossProduct.lean +++ b/SphereEversion/ToMathlib/Analysis/InnerProductSpace/CrossProduct.lean @@ -71,7 +71,7 @@ theorem inner_crossProduct_apply_apply_self (u : E) (v : (โ„ โˆ™ u)แ—ฎ) : โŸชu rw [ฯ‰.inner_crossProduct_apply u v v] exact ฯ‰.volumeForm.map_eq_zero_of_eq ![u, v, v] (by simp) (by norm_num; decide : (1 : Fin 3) โ‰  2) -/-- The map `cross_product`, upgraded from linear to continuous-linear; useful for calculus. -/ +/-- The map `crossProduct`, upgraded from linear to continuous-linear; useful for calculus. -/ def crossProduct' : E โ†’L[โ„] E โ†’L[โ„] E := LinearMap.toContinuousLinearMap (โ†‘(LinearMap.toContinuousLinearMap : (E โ†’โ‚—[โ„] E) โ‰ƒโ‚—[โ„] E โ†’L[โ„] E) โˆ˜โ‚— ฯ‰.crossProduct) diff --git a/SphereEversion/ToMathlib/LinearAlgebra/Basic.lean b/SphereEversion/ToMathlib/LinearAlgebra/Basic.lean index 0a901e26..28080f7b 100644 --- a/SphereEversion/ToMathlib/LinearAlgebra/Basic.lean +++ b/SphereEversion/ToMathlib/LinearAlgebra/Basic.lean @@ -1,6 +1,6 @@ import Mathlib.LinearAlgebra.Span -/-! Note: some results should go to `linear_algebra.span`. -/ +/-! Note: some results should go to `LinearAlgebra.Span`. -/ open Submodule Function