Skip to content

Commit

Permalink
feat(algebra/order/complete_field): generalize ring_hom_monotone (#16147
Browse files Browse the repository at this point in the history
)

@alreadydone noticed that in the proof of ```ring_hom_monotone``` can be generalized to rings. 

Co-authored-by: Junyan Xu <junyanxumath@gmail.com>
  • Loading branch information
alreadydone committed Aug 20, 2022
1 parent 67488df commit ee26143
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion src/algebra/order/complete_field.lean
Expand Up @@ -313,7 +313,7 @@ end linear_ordered_field

section real

variables {R S : Type*} [linear_ordered_field R] [linear_ordered_field S]
variables {R S : Type*} [ordered_ring R] [linear_ordered_ring S]

lemma ring_hom_monotone (hR : ∀ r : R, 0 ≤ r → ∃ s : R, s^2 = r) (f : R →+* S) : monotone f :=
begin
Expand Down

0 comments on commit ee26143

Please sign in to comment.