Skip to content

Commit

Permalink
bump to nightly-2023-05-21-11
Browse files Browse the repository at this point in the history
  • Loading branch information
leanprover-community-bot committed May 21, 2023
1 parent 6b18fd9 commit edafec7
Show file tree
Hide file tree
Showing 5 changed files with 172 additions and 6 deletions.
2 changes: 2 additions & 0 deletions Mathbin/Analysis/NormedSpace/Star/Basic.lean
Expand Up @@ -474,11 +474,13 @@ theorem starₗᵢ_apply {x : E} : starₗᵢ 𝕜 x = star x :=
rfl
#align starₗᵢ_apply starₗᵢ_apply

#print starₗᵢ_toContinuousLinearEquiv /-
@[simp]
theorem starₗᵢ_toContinuousLinearEquiv :
(starₗᵢ 𝕜 : E ≃ₗᵢ⋆[𝕜] E).toContinuousLinearEquiv = (starL 𝕜 : E ≃L⋆[𝕜] E) :=
ContinuousLinearEquiv.ext rfl
#align starₗᵢ_to_continuous_linear_equiv starₗᵢ_toContinuousLinearEquiv
-/

end starₗᵢ

Expand Down
24 changes: 24 additions & 0 deletions Mathbin/Analysis/NormedSpace/Star/Mul.lean

Large diffs are not rendered by default.

0 comments on commit edafec7

Please sign in to comment.