Zulip Chat Archive
Stream: general
Topic: Clearly finite bounded set, but how can prove finiteness?
SnO2WMaN (Feb 13 2025 at 04:22):
import Mathlib.Data.Finite.Defs
example : Set.Finite { Nat.toFloat x | x ≤ 2 } := by sorry;
This might be very oblivious, but I didn't find good way to prove. How can prove? and I hope that tauto_set
will solve like this trivial problems...
Zhang Qinchuan (Feb 13 2025 at 04:50):
You can write your set as Nat.toFloat '' Set.Icc 0 2
, then it is trivial:
import Mathlib
example : Set.Finite <| Nat.toFloat '' Set.Icc 0 2 := by
exact Set.toFinite ..
SnO2WMaN (Feb 13 2025 at 05:38):
It works, I didn't import Mathlib.Order.Interval.Finset.Nat
. Thanks.
Last updated: May 02 2025 at 03:31 UTC