Skip to content

Commit

Permalink
fix(analysis/normed_space/star/basic): make prop type classes props (#…
Browse files Browse the repository at this point in the history
…12233)

The type classes `normed_star_monoid` and `cstar_ring` are now properly declared as prop.
  • Loading branch information
dupuisf committed Feb 23, 2022
1 parent 264dd7f commit e77675d
Showing 1 changed file with 3 additions and 3 deletions.
6 changes: 3 additions & 3 deletions src/analysis/normed_space/star/basic.lean
Expand Up @@ -35,18 +35,18 @@ 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. -/
class normed_star_monoid (E : Type*) [normed_group E] [star_add_monoid E] :=
class normed_star_monoid (E : Type*) [normed_group E] [star_add_monoid E] : Prop :=
(norm_star : ∀ {x : E}, ∥x⋆∥ = ∥x∥)

export normed_star_monoid (norm_star)
attribute [simp] norm_star

/-- A C*-ring is a normed star ring that satifies the stronger condition `∥x⋆ * x∥ = ∥x∥^2`
for every `x`. -/
class cstar_ring (E : Type*) [normed_ring E] [star_ring E] :=
class cstar_ring (E : Type*) [normed_ring E] [star_ring E] : Prop :=
(norm_star_mul_self : ∀ {x : E}, ∥x⋆ * x∥ = ∥x∥ * ∥x∥)

noncomputable instance : cstar_ring ℝ :=
instance : cstar_ring ℝ :=
{ norm_star_mul_self := λ x, by simp only [star, id.def, norm_mul] }

variables {𝕜 E α : Type*}
Expand Down

0 comments on commit e77675d

Please sign in to comment.