Skip to content

Commit

Permalink
Add a fix for a test
Browse files Browse the repository at this point in the history
  • Loading branch information
Vierkantor committed Dec 6, 2023
1 parent 13e1627 commit c485120
Showing 1 changed file with 2 additions and 1 deletion.
3 changes: 2 additions & 1 deletion test/positivity.lean
Original file line number Diff line number Diff line change
Expand Up @@ -323,7 +323,8 @@ example {r : ℝ≥0} (hr : 0 < r) : (0 : ℝ) < r := by positivity

/- ## Other extensions -/

example [Zero β] [PartialOrder β] [NonnegHomClass F α β] (f : F) (x : α) : 0 ≤ f x := by positivity
example [Zero β] [PartialOrder β] [NDFunLike F α β] [NonnegHomClass F α β]
(f : F) (x : α) : 0 ≤ f x := by positivity

example [OrderedSemiring S] [Semiring R] (abv : R → S) [IsAbsoluteValue abv] (x : R) :
0 ≤ abv x := by
Expand Down

0 comments on commit c485120

Please sign in to comment.