Skip to content

Commit

Permalink
doc(analysis/normed_space): fixed normed_star_monoid doc-string (#12296)
Browse files Browse the repository at this point in the history


Co-authored-by: Scott Morrison <scott.morrison@gmail.com>
  • Loading branch information
semorrison and semorrison committed Feb 26, 2022
1 parent 05d8188 commit 43fb516
Showing 1 changed file with 2 additions and 1 deletion.
3 changes: 2 additions & 1 deletion src/analysis/normed_space/star/basic.lean
Expand Up @@ -35,7 +35,8 @@ open_locale topological_space

local postfix `⋆`:std.prec.max_plus := star

/-- A normed star ring is a star ring endowed with a norm such that `star` is isometric. -/
/-- A normed star monoid is an additive monoid with a star,
endowed with a norm such that `star` is isometric. -/
class normed_star_monoid (E : Type*) [normed_group E] [star_add_monoid E] : Prop :=
(norm_star : ∀ {x : E}, ∥x⋆∥ = ∥x∥)

Expand Down

0 comments on commit 43fb516

Please sign in to comment.