Skip to content

Commit

Permalink
fix
Browse files Browse the repository at this point in the history
  • Loading branch information
FR-vdash-bot committed Jan 6, 2025
1 parent dbcd3d4 commit de602a1
Showing 1 changed file with 1 addition and 0 deletions.
1 change: 1 addition & 0 deletions Mathlib/Algebra/Order/Field/Canonical.lean
Original file line number Diff line number Diff line change
Expand Up @@ -19,6 +19,7 @@ variable {α : Type*} [Semifield α] [LinearOrder α] [CanonicallyOrderedAdd α]
abbrev CanonicallyOrderedAdd.toLinearOrderedCommGroupWithZero :
LinearOrderedCommGroupWithZero α :=
{ __ := ‹Semifield α›
__ := ‹LinearOrder α›
zero_le_one := zero_le_one
mul_le_mul_left := fun _ _ h _ ↦ mul_le_mul_of_nonneg_left h <| zero_le _ }

Expand Down

0 comments on commit de602a1

Please sign in to comment.