Skip to content

Commit

Permalink
hrm...
Browse files Browse the repository at this point in the history
  • Loading branch information
kim-em committed May 10, 2024
1 parent da48ba0 commit 2cb0ebf
Show file tree
Hide file tree
Showing 2 changed files with 6 additions and 4 deletions.
6 changes: 3 additions & 3 deletions Mathlib/Analysis/NormedSpace/OperatorNorm/Bilinear.lean
Original file line number Diff line number Diff line change
Expand Up @@ -159,7 +159,7 @@ def flip (f : E →SL[σ₁₃] F →SL[σ₂₃] G) : F →SL[σ₂₃] E →SL
#align continuous_linear_map.flip ContinuousLinearMap.flip

private theorem le_norm_flip (f : E →SL[σ₁₃] F →SL[σ₂₃] G) : ‖f‖ ≤ ‖flip f‖ :=
f.opNorm_le_bound₂ (norm_nonneg _) fun x y => by
f.opNorm_le_bound₂ (norm_nonneg f.flip) fun x y => by
rw [mul_right_comm]
exact (flip f).le_opNorm₂ y x

Expand Down Expand Up @@ -297,7 +297,7 @@ theorem norm_compSL_le :
-- Currently, this cannot be synthesized because it violated `synthPendingDepth` restrictions
-- see leanprover/lean4#3927
letI : Norm ((F →SL[σ₂₃] G) →L[𝕜₃] (E →SL[σ₁₂] F) →SL[σ₂₃] E →SL[σ₁₃] G) :=
hasOpNorm (E := F →SL[σ₂₃] G) (F := (E →SL[σ₁₂] F) →SL[σ₂₃] E →SL[σ₁₃] G)
hasOpNorm (𝕜₂ := 𝕜₃) (E := F →SL[σ₂₃] G) (F := (E →SL[σ₁₂] F) →SL[σ₂₃] E →SL[σ₁₃] G)
‖compSL E F G σ₁₂ σ₂₃‖ ≤ 1 :=
LinearMap.mkContinuous₂_norm_le _ zero_le_one _
#align continuous_linear_map.norm_compSL_le ContinuousLinearMap.norm_compSL_le
Expand Down Expand Up @@ -334,7 +334,7 @@ theorem norm_compL_le :
-- Currently, this cannot be synthesized because it violated `synthPendingDepth` restrictions
-- see leanprover/lean4#3927
letI : Norm ((Fₗ →L[𝕜] Gₗ) →L[𝕜] (E →L[𝕜] Fₗ) →L[𝕜] E →L[𝕜] Gₗ) :=
hasOpNorm (E := Fₗ →L[𝕜] Gₗ) (F := (E →L[𝕜] Fₗ) →L[𝕜] E →L[𝕜] Gₗ)
hasOpNorm (𝕜₂ := 𝕜) (E := Fₗ →L[𝕜] Gₗ) (F := (E →L[𝕜] Fₗ) →L[𝕜] E →L[𝕜] Gₗ)
‖compL 𝕜 E Fₗ Gₗ‖ ≤ 1 :=
norm_compSL_le _ _ _ _ _
#align continuous_linear_map.norm_compL_le ContinuousLinearMap.norm_compL_le
Expand Down
4 changes: 3 additions & 1 deletion Mathlib/LinearAlgebra/Orientation.lean
Original file line number Diff line number Diff line change
Expand Up @@ -374,7 +374,9 @@ theorem eq_or_eq_neg (x₁ x₂ : Orientation R M ι) (h : Fintype.card ι = fin
letI := Classical.decEq ι
-- Porting note: this needs to be made explicit for the simp below
have orientation_neg_neg :
∀ f : Basis ι R M, - -Basis.orientation f = Basis.orientation f := by simp
∀ f : Basis ι R M, - -Basis.orientation f = Basis.orientation f := by
intro f
rw [neg_neg f.orientation]
rcases e.orientation_eq_or_eq_neg x₁ with (h₁ | h₁) <;>
rcases e.orientation_eq_or_eq_neg x₂ with (h₂ | h₂) <;> simp [h₁, h₂, orientation_neg_neg]
#align orientation.eq_or_eq_neg Orientation.eq_or_eq_neg
Expand Down

0 comments on commit 2cb0ebf

Please sign in to comment.