We read every piece of feedback, and take your input very seriously.
To see all available qualifiers, see our documentation.
There was an error while loading. Please reload this page.
1 parent cf06366 commit 7fa953eCopy full SHA for 7fa953e
Mathlib/Data/Int/Interval.lean
@@ -57,7 +57,7 @@ instance instLocallyFiniteOrder : LocallyFiniteOrder ℤ where
57
· lia
58
· intro
59
use (x - (a + 1)).toNat
60
- lia
+ omega
61
finset_mem_Ioo a b x := by
62
simp_rw [mem_map, mem_range, Function.Embedding.trans_apply, Nat.castEmbedding_apply,
63
addLeftEmbedding_apply]
0 commit comments