Skip to content

Commit

Permalink
fix(algebra/star/basic): more type classes that should be props (#12235)
Browse files Browse the repository at this point in the history
  • Loading branch information
dupuisf committed Feb 23, 2022
1 parent 98bcabb commit 515eefa
Showing 1 changed file with 2 additions and 2 deletions.
4 changes: 2 additions & 2 deletions src/algebra/star/basic.lean
Expand Up @@ -78,7 +78,7 @@ star_involutive.injective
/--
Typeclass for a trivial star operation. This is mostly meant for `ℝ`.
-/
class has_trivial_star (R : Type u) [has_star R] :=
class has_trivial_star (R : Type u) [has_star R] : Prop :=
(star_trivial : ∀ (r : R), star r = r)

export has_trivial_star (star_trivial)
Expand Down Expand Up @@ -337,7 +337,7 @@ the statement only requires `[has_star R] [has_star A] [has_scalar R A]`.
If used as `[comm_ring R] [star_ring R] [semiring A] [star_ring A] [algebra R A]`, this represents a
star algebra.
-/
class star_module (R : Type u) (A : Type v) [has_star R] [has_star A] [has_scalar R A] :=
class star_module (R : Type u) (A : Type v) [has_star R] [has_star A] [has_scalar R A] : Prop :=
(star_smul : ∀ (r : R) (a : A), star (r • a) = star r • star a)

export star_module (star_smul)
Expand Down

0 comments on commit 515eefa

Please sign in to comment.