Zulip Chat Archive
Stream: general
Topic: Diamond with ordered rings
Wrenna Robson (Sep 02 2022 at 16:05):
I'm getting something that looks quite a lot like a diamond when trying to prove something on a type that is both a conditionally_complete_linear_order
and a linear_ordered_ring
.
In particular, it looks as though I am getting these two instances of has_le:
@has_le.le α
(@preorder.to_has_le α
(@partial_order.to_preorder α
(@semilattice_inf.to_partial_order α
(@lattice.to_semilattice_inf α
(@conditionally_complete_lattice.to_lattice α
(@conditionally_complete_linear_order.to_conditionally_complete_lattice α _inst_3))))))
and
@has_le.le α
(@preorder.to_has_le α
(@partial_order.to_preorder α
(@ordered_add_comm_group.to_partial_order α
(@ordered_ring.to_ordered_add_comm_group α (@linear_ordered_ring.to_ordered_ring α _inst_1)))))
And these are not, it seems, defeq. How can I avoid this problem: what is the right typeclass to use?
Eric Rodriguez (Sep 02 2022 at 16:09):
they both provide different le
s; you'd need to make a super-class that encompasses both
Wrenna Robson (Sep 02 2022 at 16:16):
Pfeh!
Wrenna Robson (Sep 02 2022 at 16:18):
So we don't have any way to talk about completeness properties of orders alongside orders on rings? (For context: was wanting to try and prove something like infi (fun x => floor (f x)) = floor (infi f).
Junyan Xu (Sep 02 2022 at 16:48):
You could mimic how src#conditionally_complete_linear_ordered_field is done.
Yaël Dillies (Sep 02 2022 at 22:05):
Aren't all conditionally complete linear ordered rings actually fields?
Yaël Dillies (Sep 02 2022 at 22:06):
Set a^-1 := infi (\la b, 1 <= a * b)
for positive a
.
Kevin Buzzard (Sep 02 2022 at 22:06):
Isn't the integers a counterexample?
Adam Topaz (Sep 02 2022 at 22:12):
Maybe some natural additional axiom is needed. A guess: add the condition that for all there exists some such that
Adam Topaz (Sep 02 2022 at 22:13):
One might call that condition "non-locally-discrete" or something
Yaël Dillies (Sep 02 2022 at 22:13):
Adam Topaz (Sep 02 2022 at 22:14):
:)
Adam Topaz (Sep 02 2022 at 22:14):
you order theorists named everything
Yaël Dillies (Sep 02 2022 at 22:14):
Eheheh
Kevin Buzzard (Sep 02 2022 at 22:17):
How about then?
Yaël Dillies (Sep 02 2022 at 22:19):
Is that really conditionally complete?
Kevin Buzzard (Sep 02 2022 at 22:20):
Oh good point! I doubt it. So maybe you're right.
Kevin Buzzard (Sep 02 2022 at 22:21):
I'm still a bit worried about stuff like (a polynomial ring) with infinitely small but positive.
Wrenna Robson (Sep 05 2022 at 13:14):
Yaël Dillies said:
Set
a^-1 := infi (\la b, 1 <= a * b)
for positivea
.
What if there is no such b?
Last updated: Dec 20 2023 at 11:08 UTC