Home | Intuitionistic Logic Explorer Theorem List (p. 103 of 142) | < Previous Next > |
Bad symbols? Try the
GIF version. |
||
Mirrors > Metamath Home Page > ILE Home Page > Theorem List Contents > Recent Proofs This page: Page List |
Type | Label | Description |
---|---|---|
Statement | ||
Theorem | qlelttric 10201 | Rational trichotomy. (Contributed by Jim Kingdon, 7-Oct-2021.) |
⊢ ((𝐴 ∈ ℚ ∧ 𝐵 ∈ ℚ) → (𝐴 ≤ 𝐵 ∨ 𝐵 < 𝐴)) | ||
Theorem | qltnle 10202 | 'Less than' expressed in terms of 'less than or equal to'. (Contributed by Jim Kingdon, 8-Oct-2021.) |
⊢ ((𝐴 ∈ ℚ ∧ 𝐵 ∈ ℚ) → (𝐴 < 𝐵 ↔ ¬ 𝐵 ≤ 𝐴)) | ||
Theorem | qdceq 10203 | Equality of rationals is decidable. (Contributed by Jim Kingdon, 11-Oct-2021.) |
⊢ ((𝐴 ∈ ℚ ∧ 𝐵 ∈ ℚ) → DECID 𝐴 = 𝐵) | ||
Theorem | exbtwnzlemstep 10204* | Lemma for exbtwnzlemex 10206. Induction step. (Contributed by Jim Kingdon, 10-May-2022.) |
⊢ (𝜑 → 𝐾 ∈ ℕ) & ⊢ (𝜑 → 𝐴 ∈ ℝ) & ⊢ ((𝜑 ∧ 𝑛 ∈ ℤ) → (𝑛 ≤ 𝐴 ∨ 𝐴 < 𝑛)) ⇒ ⊢ ((𝜑 ∧ ∃𝑚 ∈ ℤ (𝑚 ≤ 𝐴 ∧ 𝐴 < (𝑚 + (𝐾 + 1)))) → ∃𝑚 ∈ ℤ (𝑚 ≤ 𝐴 ∧ 𝐴 < (𝑚 + 𝐾))) | ||
Theorem | exbtwnzlemshrink 10205* | Lemma for exbtwnzlemex 10206. Shrinking the range around 𝐴. (Contributed by Jim Kingdon, 10-May-2022.) |
⊢ (𝜑 → 𝐽 ∈ ℕ) & ⊢ (𝜑 → 𝐴 ∈ ℝ) & ⊢ ((𝜑 ∧ 𝑛 ∈ ℤ) → (𝑛 ≤ 𝐴 ∨ 𝐴 < 𝑛)) ⇒ ⊢ ((𝜑 ∧ ∃𝑚 ∈ ℤ (𝑚 ≤ 𝐴 ∧ 𝐴 < (𝑚 + 𝐽))) → ∃𝑥 ∈ ℤ (𝑥 ≤ 𝐴 ∧ 𝐴 < (𝑥 + 1))) | ||
Theorem | exbtwnzlemex 10206* |
Existence of an integer so that a given real number is between the
integer and its successor. The real number must satisfy the
𝑛
≤ 𝐴 ∨ 𝐴 < 𝑛 hypothesis. For example either a
rational number or
a number which is irrational (in the sense of being apart from any
rational number) will meet this condition.
The proof starts by finding two integers which are less than and greater than 𝐴. Then this range can be shrunk by choosing an integer in between the endpoints of the range and then deciding which half of the range to keep based on the 𝑛 ≤ 𝐴 ∨ 𝐴 < 𝑛 hypothesis, and iterating until the range consists of two consecutive integers. (Contributed by Jim Kingdon, 8-Oct-2021.) |
⊢ (𝜑 → 𝐴 ∈ ℝ) & ⊢ ((𝜑 ∧ 𝑛 ∈ ℤ) → (𝑛 ≤ 𝐴 ∨ 𝐴 < 𝑛)) ⇒ ⊢ (𝜑 → ∃𝑥 ∈ ℤ (𝑥 ≤ 𝐴 ∧ 𝐴 < (𝑥 + 1))) | ||
Theorem | exbtwnz 10207* | If a real number is between an integer and its successor, there is a unique greatest integer less than or equal to the real number. (Contributed by Jim Kingdon, 10-May-2022.) |
⊢ (𝜑 → ∃𝑥 ∈ ℤ (𝑥 ≤ 𝐴 ∧ 𝐴 < (𝑥 + 1))) & ⊢ (𝜑 → 𝐴 ∈ ℝ) ⇒ ⊢ (𝜑 → ∃!𝑥 ∈ ℤ (𝑥 ≤ 𝐴 ∧ 𝐴 < (𝑥 + 1))) | ||
Theorem | qbtwnz 10208* | There is a unique greatest integer less than or equal to a rational number. (Contributed by Jim Kingdon, 8-Oct-2021.) |
⊢ (𝐴 ∈ ℚ → ∃!𝑥 ∈ ℤ (𝑥 ≤ 𝐴 ∧ 𝐴 < (𝑥 + 1))) | ||
Theorem | rebtwn2zlemstep 10209* | Lemma for rebtwn2z 10211. Induction step. (Contributed by Jim Kingdon, 13-Oct-2021.) |
⊢ ((𝐾 ∈ (ℤ≥‘2) ∧ 𝐴 ∈ ℝ ∧ ∃𝑚 ∈ ℤ (𝑚 < 𝐴 ∧ 𝐴 < (𝑚 + (𝐾 + 1)))) → ∃𝑚 ∈ ℤ (𝑚 < 𝐴 ∧ 𝐴 < (𝑚 + 𝐾))) | ||
Theorem | rebtwn2zlemshrink 10210* | Lemma for rebtwn2z 10211. Shrinking the range around the given real number. (Contributed by Jim Kingdon, 13-Oct-2021.) |
⊢ ((𝐴 ∈ ℝ ∧ 𝐽 ∈ (ℤ≥‘2) ∧ ∃𝑚 ∈ ℤ (𝑚 < 𝐴 ∧ 𝐴 < (𝑚 + 𝐽))) → ∃𝑥 ∈ ℤ (𝑥 < 𝐴 ∧ 𝐴 < (𝑥 + 2))) | ||
Theorem | rebtwn2z 10211* |
A real number can be bounded by integers above and below which are two
apart.
The proof starts by finding two integers which are less than and greater than the given real number. Then this range can be shrunk by choosing an integer in between the endpoints of the range and then deciding which half of the range to keep based on weak linearity, and iterating until the range consists of integers which are two apart. (Contributed by Jim Kingdon, 13-Oct-2021.) |
⊢ (𝐴 ∈ ℝ → ∃𝑥 ∈ ℤ (𝑥 < 𝐴 ∧ 𝐴 < (𝑥 + 2))) | ||
Theorem | qbtwnrelemcalc 10212 | Lemma for qbtwnre 10213. Calculations involved in showing the constructed rational number is less than 𝐵. (Contributed by Jim Kingdon, 14-Oct-2021.) |
⊢ (𝜑 → 𝑀 ∈ ℤ) & ⊢ (𝜑 → 𝑁 ∈ ℕ) & ⊢ (𝜑 → 𝐴 ∈ ℝ) & ⊢ (𝜑 → 𝐵 ∈ ℝ) & ⊢ (𝜑 → 𝑀 < (𝐴 · (2 · 𝑁))) & ⊢ (𝜑 → (1 / 𝑁) < (𝐵 − 𝐴)) ⇒ ⊢ (𝜑 → ((𝑀 + 2) / (2 · 𝑁)) < 𝐵) | ||
Theorem | qbtwnre 10213* | The rational numbers are dense in ℝ: any two real numbers have a rational between them. Exercise 6 of [Apostol] p. 28. (Contributed by NM, 18-Nov-2004.) |
⊢ ((𝐴 ∈ ℝ ∧ 𝐵 ∈ ℝ ∧ 𝐴 < 𝐵) → ∃𝑥 ∈ ℚ (𝐴 < 𝑥 ∧ 𝑥 < 𝐵)) | ||
Theorem | qbtwnxr 10214* | The rational numbers are dense in ℝ*: any two extended real numbers have a rational between them. (Contributed by NM, 6-Feb-2007.) (Proof shortened by Mario Carneiro, 23-Aug-2015.) |
⊢ ((𝐴 ∈ ℝ* ∧ 𝐵 ∈ ℝ* ∧ 𝐴 < 𝐵) → ∃𝑥 ∈ ℚ (𝐴 < 𝑥 ∧ 𝑥 < 𝐵)) | ||
Theorem | qavgle 10215 | The average of two rational numbers is less than or equal to at least one of them. (Contributed by Jim Kingdon, 3-Nov-2021.) |
⊢ ((𝐴 ∈ ℚ ∧ 𝐵 ∈ ℚ) → (((𝐴 + 𝐵) / 2) ≤ 𝐴 ∨ ((𝐴 + 𝐵) / 2) ≤ 𝐵)) | ||
Theorem | ioo0 10216 | An empty open interval of extended reals. (Contributed by NM, 6-Feb-2007.) |
⊢ ((𝐴 ∈ ℝ* ∧ 𝐵 ∈ ℝ*) → ((𝐴(,)𝐵) = ∅ ↔ 𝐵 ≤ 𝐴)) | ||
Theorem | ioom 10217* | An open interval of extended reals is inhabited iff the lower argument is less than the upper argument. (Contributed by Jim Kingdon, 27-Nov-2021.) |
⊢ ((𝐴 ∈ ℝ* ∧ 𝐵 ∈ ℝ*) → (∃𝑥 𝑥 ∈ (𝐴(,)𝐵) ↔ 𝐴 < 𝐵)) | ||
Theorem | ico0 10218 | An empty open interval of extended reals. (Contributed by FL, 30-May-2014.) |
⊢ ((𝐴 ∈ ℝ* ∧ 𝐵 ∈ ℝ*) → ((𝐴[,)𝐵) = ∅ ↔ 𝐵 ≤ 𝐴)) | ||
Theorem | ioc0 10219 | An empty open interval of extended reals. (Contributed by FL, 30-May-2014.) |
⊢ ((𝐴 ∈ ℝ* ∧ 𝐵 ∈ ℝ*) → ((𝐴(,]𝐵) = ∅ ↔ 𝐵 ≤ 𝐴)) | ||
Theorem | dfrp2 10220 | Alternate definition of the positive real numbers. (Contributed by Thierry Arnoux, 4-May-2020.) |
⊢ ℝ+ = (0(,)+∞) | ||
Theorem | elicod 10221 | Membership in a left-closed right-open interval. (Contributed by Glauco Siliprandi, 11-Dec-2019.) |
⊢ (𝜑 → 𝐴 ∈ ℝ*) & ⊢ (𝜑 → 𝐵 ∈ ℝ*) & ⊢ (𝜑 → 𝐶 ∈ ℝ*) & ⊢ (𝜑 → 𝐴 ≤ 𝐶) & ⊢ (𝜑 → 𝐶 < 𝐵) ⇒ ⊢ (𝜑 → 𝐶 ∈ (𝐴[,)𝐵)) | ||
Theorem | icogelb 10222 | An element of a left-closed right-open interval is greater than or equal to its lower bound. (Contributed by Glauco Siliprandi, 11-Dec-2019.) |
⊢ ((𝐴 ∈ ℝ* ∧ 𝐵 ∈ ℝ* ∧ 𝐶 ∈ (𝐴[,)𝐵)) → 𝐴 ≤ 𝐶) | ||
Theorem | elicore 10223 | A member of a left-closed right-open interval of reals is real. (Contributed by Glauco Siliprandi, 11-Dec-2019.) |
⊢ ((𝐴 ∈ ℝ ∧ 𝐶 ∈ (𝐴[,)𝐵)) → 𝐶 ∈ ℝ) | ||
Syntax | cfl 10224 | Extend class notation with floor (greatest integer) function. |
class ⌊ | ||
Syntax | cceil 10225 | Extend class notation to include the ceiling function. |
class ⌈ | ||
Definition | df-fl 10226* |
Define the floor (greatest integer less than or equal to) function. See
flval 10228 for its value, flqlelt 10232 for its basic property, and flqcl 10229 for
its closure. For example, (⌊‘(3 / 2)) =
1 while
(⌊‘-(3 / 2)) = -2 (ex-fl 13760).
Although we define this on real numbers so that notations are similar to the Metamath Proof Explorer, in the absence of excluded middle few theorems will be possible for all real numbers. Imagine a real number which is around 2.99995 or 3.00001 . In order to determine whether its floor is 2 or 3, it would be necessary to compute the number to arbitrary precision. The term "floor" was coined by Ken Iverson. He also invented a mathematical notation for floor, consisting of an L-shaped left bracket and its reflection as a right bracket. In APL, the left-bracket alone is used, and we borrow this idea. (Thanks to Paul Chapman for this information.) (Contributed by NM, 14-Nov-2004.) |
⊢ ⌊ = (𝑥 ∈ ℝ ↦ (℩𝑦 ∈ ℤ (𝑦 ≤ 𝑥 ∧ 𝑥 < (𝑦 + 1)))) | ||
Definition | df-ceil 10227 |
The ceiling (least integer greater than or equal to) function. Defined in
ISO 80000-2:2009(E) operation 2-9.18 and the "NIST Digital Library of
Mathematical Functions" , front introduction, "Common Notations
and
Definitions" section at http://dlmf.nist.gov/front/introduction#Sx4.
See ceilqval 10262 for its value, ceilqge 10266 and ceilqm1lt 10268 for its basic
properties, and ceilqcl 10264 for its closure. For example,
(⌈‘(3 / 2)) = 2 while (⌈‘-(3 / 2)) = -1
(ex-ceil 13761).
As described in df-fl 10226 most theorems are only for rationals, not reals. The symbol ⌈ is inspired by the gamma shaped left bracket of the usual notation. (Contributed by David A. Wheeler, 19-May-2015.) |
⊢ ⌈ = (𝑥 ∈ ℝ ↦ -(⌊‘-𝑥)) | ||
Theorem | flval 10228* | Value of the floor (greatest integer) function. The floor of 𝐴 is the (unique) integer less than or equal to 𝐴 whose successor is strictly greater than 𝐴. (Contributed by NM, 14-Nov-2004.) (Revised by Mario Carneiro, 2-Nov-2013.) |
⊢ (𝐴 ∈ ℝ → (⌊‘𝐴) = (℩𝑥 ∈ ℤ (𝑥 ≤ 𝐴 ∧ 𝐴 < (𝑥 + 1)))) | ||
Theorem | flqcl 10229 | The floor (greatest integer) function yields an integer when applied to a rational (closure law). For a similar closure law for real numbers apart from any integer, see flapcl 10231. (Contributed by Jim Kingdon, 8-Oct-2021.) |
⊢ (𝐴 ∈ ℚ → (⌊‘𝐴) ∈ ℤ) | ||
Theorem | apbtwnz 10230* | There is a unique greatest integer less than or equal to a real number which is apart from all integers. (Contributed by Jim Kingdon, 11-May-2022.) |
⊢ ((𝐴 ∈ ℝ ∧ ∀𝑛 ∈ ℤ 𝐴 # 𝑛) → ∃!𝑥 ∈ ℤ (𝑥 ≤ 𝐴 ∧ 𝐴 < (𝑥 + 1))) | ||
Theorem | flapcl 10231* | The floor (greatest integer) function yields an integer when applied to a real number apart from any integer. For example, an irrational number (see for example sqrt2irrap 12134) would satisfy this condition. (Contributed by Jim Kingdon, 11-May-2022.) |
⊢ ((𝐴 ∈ ℝ ∧ ∀𝑛 ∈ ℤ 𝐴 # 𝑛) → (⌊‘𝐴) ∈ ℤ) | ||
Theorem | flqlelt 10232 | A basic property of the floor (greatest integer) function. (Contributed by Jim Kingdon, 8-Oct-2021.) |
⊢ (𝐴 ∈ ℚ → ((⌊‘𝐴) ≤ 𝐴 ∧ 𝐴 < ((⌊‘𝐴) + 1))) | ||
Theorem | flqcld 10233 | The floor (greatest integer) function is an integer (closure law). (Contributed by Jim Kingdon, 8-Oct-2021.) |
⊢ (𝜑 → 𝐴 ∈ ℚ) ⇒ ⊢ (𝜑 → (⌊‘𝐴) ∈ ℤ) | ||
Theorem | flqle 10234 | A basic property of the floor (greatest integer) function. (Contributed by Jim Kingdon, 8-Oct-2021.) |
⊢ (𝐴 ∈ ℚ → (⌊‘𝐴) ≤ 𝐴) | ||
Theorem | flqltp1 10235 | A basic property of the floor (greatest integer) function. (Contributed by Jim Kingdon, 8-Oct-2021.) |
⊢ (𝐴 ∈ ℚ → 𝐴 < ((⌊‘𝐴) + 1)) | ||
Theorem | qfraclt1 10236 | The fractional part of a rational number is less than one. (Contributed by Jim Kingdon, 8-Oct-2021.) |
⊢ (𝐴 ∈ ℚ → (𝐴 − (⌊‘𝐴)) < 1) | ||
Theorem | qfracge0 10237 | The fractional part of a rational number is nonnegative. (Contributed by Jim Kingdon, 8-Oct-2021.) |
⊢ (𝐴 ∈ ℚ → 0 ≤ (𝐴 − (⌊‘𝐴))) | ||
Theorem | flqge 10238 | The floor function value is the greatest integer less than or equal to its argument. (Contributed by Jim Kingdon, 8-Oct-2021.) |
⊢ ((𝐴 ∈ ℚ ∧ 𝐵 ∈ ℤ) → (𝐵 ≤ 𝐴 ↔ 𝐵 ≤ (⌊‘𝐴))) | ||
Theorem | flqlt 10239 | The floor function value is less than the next integer. (Contributed by Jim Kingdon, 8-Oct-2021.) |
⊢ ((𝐴 ∈ ℚ ∧ 𝐵 ∈ ℤ) → (𝐴 < 𝐵 ↔ (⌊‘𝐴) < 𝐵)) | ||
Theorem | flid 10240 | An integer is its own floor. (Contributed by NM, 15-Nov-2004.) |
⊢ (𝐴 ∈ ℤ → (⌊‘𝐴) = 𝐴) | ||
Theorem | flqidm 10241 | The floor function is idempotent. (Contributed by Jim Kingdon, 8-Oct-2021.) |
⊢ (𝐴 ∈ ℚ → (⌊‘(⌊‘𝐴)) = (⌊‘𝐴)) | ||
Theorem | flqidz 10242 | A rational number equals its floor iff it is an integer. (Contributed by Jim Kingdon, 9-Oct-2021.) |
⊢ (𝐴 ∈ ℚ → ((⌊‘𝐴) = 𝐴 ↔ 𝐴 ∈ ℤ)) | ||
Theorem | flqltnz 10243 | If A is not an integer, then the floor of A is less than A. (Contributed by Jim Kingdon, 9-Oct-2021.) |
⊢ ((𝐴 ∈ ℚ ∧ ¬ 𝐴 ∈ ℤ) → (⌊‘𝐴) < 𝐴) | ||
Theorem | flqwordi 10244 | Ordering relationship for the greatest integer function. (Contributed by Jim Kingdon, 9-Oct-2021.) |
⊢ ((𝐴 ∈ ℚ ∧ 𝐵 ∈ ℚ ∧ 𝐴 ≤ 𝐵) → (⌊‘𝐴) ≤ (⌊‘𝐵)) | ||
Theorem | flqword2 10245 | Ordering relationship for the greatest integer function. (Contributed by Jim Kingdon, 9-Oct-2021.) |
⊢ ((𝐴 ∈ ℚ ∧ 𝐵 ∈ ℚ ∧ 𝐴 ≤ 𝐵) → (⌊‘𝐵) ∈ (ℤ≥‘(⌊‘𝐴))) | ||
Theorem | flqbi 10246 | A condition equivalent to floor. (Contributed by Jim Kingdon, 9-Oct-2021.) |
⊢ ((𝐴 ∈ ℚ ∧ 𝐵 ∈ ℤ) → ((⌊‘𝐴) = 𝐵 ↔ (𝐵 ≤ 𝐴 ∧ 𝐴 < (𝐵 + 1)))) | ||
Theorem | flqbi2 10247 | A condition equivalent to floor. (Contributed by Jim Kingdon, 9-Oct-2021.) |
⊢ ((𝑁 ∈ ℤ ∧ 𝐹 ∈ ℚ) → ((⌊‘(𝑁 + 𝐹)) = 𝑁 ↔ (0 ≤ 𝐹 ∧ 𝐹 < 1))) | ||
Theorem | adddivflid 10248 | The floor of a sum of an integer and a fraction is equal to the integer iff the denominator of the fraction is less than the numerator. (Contributed by AV, 14-Jul-2021.) |
⊢ ((𝐴 ∈ ℤ ∧ 𝐵 ∈ ℕ0 ∧ 𝐶 ∈ ℕ) → (𝐵 < 𝐶 ↔ (⌊‘(𝐴 + (𝐵 / 𝐶))) = 𝐴)) | ||
Theorem | flqge0nn0 10249 | The floor of a number greater than or equal to 0 is a nonnegative integer. (Contributed by Jim Kingdon, 10-Oct-2021.) |
⊢ ((𝐴 ∈ ℚ ∧ 0 ≤ 𝐴) → (⌊‘𝐴) ∈ ℕ0) | ||
Theorem | flqge1nn 10250 | The floor of a number greater than or equal to 1 is a positive integer. (Contributed by Jim Kingdon, 10-Oct-2021.) |
⊢ ((𝐴 ∈ ℚ ∧ 1 ≤ 𝐴) → (⌊‘𝐴) ∈ ℕ) | ||
Theorem | fldivnn0 10251 | The floor function of a division of a nonnegative integer by a positive integer is a nonnegative integer. (Contributed by Alexander van der Vekens, 14-Apr-2018.) |
⊢ ((𝐾 ∈ ℕ0 ∧ 𝐿 ∈ ℕ) → (⌊‘(𝐾 / 𝐿)) ∈ ℕ0) | ||
Theorem | divfl0 10252 | The floor of a fraction is 0 iff the denominator is less than the numerator. (Contributed by AV, 8-Jul-2021.) |
⊢ ((𝐴 ∈ ℕ0 ∧ 𝐵 ∈ ℕ) → (𝐴 < 𝐵 ↔ (⌊‘(𝐴 / 𝐵)) = 0)) | ||
Theorem | flqaddz 10253 | An integer can be moved in and out of the floor of a sum. (Contributed by Jim Kingdon, 10-Oct-2021.) |
⊢ ((𝐴 ∈ ℚ ∧ 𝑁 ∈ ℤ) → (⌊‘(𝐴 + 𝑁)) = ((⌊‘𝐴) + 𝑁)) | ||
Theorem | flqzadd 10254 | An integer can be moved in and out of the floor of a sum. (Contributed by Jim Kingdon, 10-Oct-2021.) |
⊢ ((𝑁 ∈ ℤ ∧ 𝐴 ∈ ℚ) → (⌊‘(𝑁 + 𝐴)) = (𝑁 + (⌊‘𝐴))) | ||
Theorem | flqmulnn0 10255 | Move a nonnegative integer in and out of a floor. (Contributed by Jim Kingdon, 10-Oct-2021.) |
⊢ ((𝑁 ∈ ℕ0 ∧ 𝐴 ∈ ℚ) → (𝑁 · (⌊‘𝐴)) ≤ (⌊‘(𝑁 · 𝐴))) | ||
Theorem | btwnzge0 10256 | A real bounded between an integer and its successor is nonnegative iff the integer is nonnegative. Second half of Lemma 13-4.1 of [Gleason] p. 217. (Contributed by NM, 12-Mar-2005.) |
⊢ (((𝐴 ∈ ℝ ∧ 𝑁 ∈ ℤ) ∧ (𝑁 ≤ 𝐴 ∧ 𝐴 < (𝑁 + 1))) → (0 ≤ 𝐴 ↔ 0 ≤ 𝑁)) | ||
Theorem | 2tnp1ge0ge0 10257 | Two times an integer plus one is not negative iff the integer is not negative. (Contributed by AV, 19-Jun-2021.) |
⊢ (𝑁 ∈ ℤ → (0 ≤ ((2 · 𝑁) + 1) ↔ 0 ≤ 𝑁)) | ||
Theorem | flhalf 10258 | Ordering relation for the floor of half of an integer. (Contributed by NM, 1-Jan-2006.) (Proof shortened by Mario Carneiro, 7-Jun-2016.) |
⊢ (𝑁 ∈ ℤ → 𝑁 ≤ (2 · (⌊‘((𝑁 + 1) / 2)))) | ||
Theorem | fldivnn0le 10259 | The floor function of a division of a nonnegative integer by a positive integer is less than or equal to the division. (Contributed by Alexander van der Vekens, 14-Apr-2018.) |
⊢ ((𝐾 ∈ ℕ0 ∧ 𝐿 ∈ ℕ) → (⌊‘(𝐾 / 𝐿)) ≤ (𝐾 / 𝐿)) | ||
Theorem | flltdivnn0lt 10260 | The floor function of a division of a nonnegative integer by a positive integer is less than the division of a greater dividend by the same positive integer. (Contributed by Alexander van der Vekens, 14-Apr-2018.) |
⊢ ((𝐾 ∈ ℕ0 ∧ 𝑁 ∈ ℕ0 ∧ 𝐿 ∈ ℕ) → (𝐾 < 𝑁 → (⌊‘(𝐾 / 𝐿)) < (𝑁 / 𝐿))) | ||
Theorem | fldiv4p1lem1div2 10261 | The floor of an integer equal to 3 or greater than 4, increased by 1, is less than or equal to the half of the integer minus 1. (Contributed by AV, 8-Jul-2021.) |
⊢ ((𝑁 = 3 ∨ 𝑁 ∈ (ℤ≥‘5)) → ((⌊‘(𝑁 / 4)) + 1) ≤ ((𝑁 − 1) / 2)) | ||
Theorem | ceilqval 10262 | The value of the ceiling function. (Contributed by Jim Kingdon, 10-Oct-2021.) |
⊢ (𝐴 ∈ ℚ → (⌈‘𝐴) = -(⌊‘-𝐴)) | ||
Theorem | ceiqcl 10263 | The ceiling function returns an integer (closure law). (Contributed by Jim Kingdon, 11-Oct-2021.) |
⊢ (𝐴 ∈ ℚ → -(⌊‘-𝐴) ∈ ℤ) | ||
Theorem | ceilqcl 10264 | Closure of the ceiling function. (Contributed by Jim Kingdon, 11-Oct-2021.) |
⊢ (𝐴 ∈ ℚ → (⌈‘𝐴) ∈ ℤ) | ||
Theorem | ceiqge 10265 | The ceiling of a real number is greater than or equal to that number. (Contributed by Jim Kingdon, 11-Oct-2021.) |
⊢ (𝐴 ∈ ℚ → 𝐴 ≤ -(⌊‘-𝐴)) | ||
Theorem | ceilqge 10266 | The ceiling of a real number is greater than or equal to that number. (Contributed by Jim Kingdon, 11-Oct-2021.) |
⊢ (𝐴 ∈ ℚ → 𝐴 ≤ (⌈‘𝐴)) | ||
Theorem | ceiqm1l 10267 | One less than the ceiling of a real number is strictly less than that number. (Contributed by Jim Kingdon, 11-Oct-2021.) |
⊢ (𝐴 ∈ ℚ → (-(⌊‘-𝐴) − 1) < 𝐴) | ||
Theorem | ceilqm1lt 10268 | One less than the ceiling of a real number is strictly less than that number. (Contributed by Jim Kingdon, 11-Oct-2021.) |
⊢ (𝐴 ∈ ℚ → ((⌈‘𝐴) − 1) < 𝐴) | ||
Theorem | ceiqle 10269 | The ceiling of a real number is the smallest integer greater than or equal to it. (Contributed by Jim Kingdon, 11-Oct-2021.) |
⊢ ((𝐴 ∈ ℚ ∧ 𝐵 ∈ ℤ ∧ 𝐴 ≤ 𝐵) → -(⌊‘-𝐴) ≤ 𝐵) | ||
Theorem | ceilqle 10270 | The ceiling of a real number is the smallest integer greater than or equal to it. (Contributed by Jim Kingdon, 11-Oct-2021.) |
⊢ ((𝐴 ∈ ℚ ∧ 𝐵 ∈ ℤ ∧ 𝐴 ≤ 𝐵) → (⌈‘𝐴) ≤ 𝐵) | ||
Theorem | ceilid 10271 | An integer is its own ceiling. (Contributed by AV, 30-Nov-2018.) |
⊢ (𝐴 ∈ ℤ → (⌈‘𝐴) = 𝐴) | ||
Theorem | ceilqidz 10272 | A rational number equals its ceiling iff it is an integer. (Contributed by Jim Kingdon, 11-Oct-2021.) |
⊢ (𝐴 ∈ ℚ → (𝐴 ∈ ℤ ↔ (⌈‘𝐴) = 𝐴)) | ||
Theorem | flqleceil 10273 | The floor of a rational number is less than or equal to its ceiling. (Contributed by Jim Kingdon, 11-Oct-2021.) |
⊢ (𝐴 ∈ ℚ → (⌊‘𝐴) ≤ (⌈‘𝐴)) | ||
Theorem | flqeqceilz 10274 | A rational number is an integer iff its floor equals its ceiling. (Contributed by Jim Kingdon, 11-Oct-2021.) |
⊢ (𝐴 ∈ ℚ → (𝐴 ∈ ℤ ↔ (⌊‘𝐴) = (⌈‘𝐴))) | ||
Theorem | intqfrac2 10275 | Decompose a real into integer and fractional parts. (Contributed by Jim Kingdon, 18-Oct-2021.) |
⊢ 𝑍 = (⌊‘𝐴) & ⊢ 𝐹 = (𝐴 − 𝑍) ⇒ ⊢ (𝐴 ∈ ℚ → (0 ≤ 𝐹 ∧ 𝐹 < 1 ∧ 𝐴 = (𝑍 + 𝐹))) | ||
Theorem | intfracq 10276 | Decompose a rational number, expressed as a ratio, into integer and fractional parts. The fractional part has a tighter bound than that of intqfrac2 10275. (Contributed by NM, 16-Aug-2008.) |
⊢ 𝑍 = (⌊‘(𝑀 / 𝑁)) & ⊢ 𝐹 = ((𝑀 / 𝑁) − 𝑍) ⇒ ⊢ ((𝑀 ∈ ℤ ∧ 𝑁 ∈ ℕ) → (0 ≤ 𝐹 ∧ 𝐹 ≤ ((𝑁 − 1) / 𝑁) ∧ (𝑀 / 𝑁) = (𝑍 + 𝐹))) | ||
Theorem | flqdiv 10277 | Cancellation of the embedded floor of a real divided by an integer. (Contributed by Jim Kingdon, 18-Oct-2021.) |
⊢ ((𝐴 ∈ ℚ ∧ 𝑁 ∈ ℕ) → (⌊‘((⌊‘𝐴) / 𝑁)) = (⌊‘(𝐴 / 𝑁))) | ||
Syntax | cmo 10278 | Extend class notation with the modulo operation. |
class mod | ||
Definition | df-mod 10279* | Define the modulo (remainder) operation. See modqval 10280 for its value. For example, (5 mod 3) = 2 and (-7 mod 2) = 1. As with df-fl 10226 we define this for first and second arguments which are real and positive real, respectively, even though many theorems will need to be more restricted (for example, specify rational arguments). (Contributed by NM, 10-Nov-2008.) |
⊢ mod = (𝑥 ∈ ℝ, 𝑦 ∈ ℝ+ ↦ (𝑥 − (𝑦 · (⌊‘(𝑥 / 𝑦))))) | ||
Theorem | modqval 10280 | The value of the modulo operation. The modulo congruence notation of number theory, 𝐽≡𝐾 (modulo 𝑁), can be expressed in our notation as (𝐽 mod 𝑁) = (𝐾 mod 𝑁). Definition 1 in Knuth, The Art of Computer Programming, Vol. I (1972), p. 38. Knuth uses "mod" for the operation and "modulo" for the congruence. Unlike Knuth, we restrict the second argument to positive numbers to simplify certain theorems. (This also gives us future flexibility to extend it to any one of several different conventions for a zero or negative second argument, should there be an advantage in doing so.) As with flqcl 10229 we only prove this for rationals although other particular kinds of real numbers may be possible. (Contributed by Jim Kingdon, 16-Oct-2021.) |
⊢ ((𝐴 ∈ ℚ ∧ 𝐵 ∈ ℚ ∧ 0 < 𝐵) → (𝐴 mod 𝐵) = (𝐴 − (𝐵 · (⌊‘(𝐴 / 𝐵))))) | ||
Theorem | modqvalr 10281 | The value of the modulo operation (multiplication in reversed order). (Contributed by Jim Kingdon, 16-Oct-2021.) |
⊢ ((𝐴 ∈ ℚ ∧ 𝐵 ∈ ℚ ∧ 0 < 𝐵) → (𝐴 mod 𝐵) = (𝐴 − ((⌊‘(𝐴 / 𝐵)) · 𝐵))) | ||
Theorem | modqcl 10282 | Closure law for the modulo operation. (Contributed by Jim Kingdon, 16-Oct-2021.) |
⊢ ((𝐴 ∈ ℚ ∧ 𝐵 ∈ ℚ ∧ 0 < 𝐵) → (𝐴 mod 𝐵) ∈ ℚ) | ||
Theorem | flqpmodeq 10283 | Partition of a division into its integer part and the remainder. (Contributed by Jim Kingdon, 16-Oct-2021.) |
⊢ ((𝐴 ∈ ℚ ∧ 𝐵 ∈ ℚ ∧ 0 < 𝐵) → (((⌊‘(𝐴 / 𝐵)) · 𝐵) + (𝐴 mod 𝐵)) = 𝐴) | ||
Theorem | modqcld 10284 | Closure law for the modulo operation. (Contributed by Jim Kingdon, 16-Oct-2021.) |
⊢ (𝜑 → 𝐴 ∈ ℚ) & ⊢ (𝜑 → 𝐵 ∈ ℚ) & ⊢ (𝜑 → 0 < 𝐵) ⇒ ⊢ (𝜑 → (𝐴 mod 𝐵) ∈ ℚ) | ||
Theorem | modq0 10285 | 𝐴 mod 𝐵 is zero iff 𝐴 is evenly divisible by 𝐵. (Contributed by Jim Kingdon, 17-Oct-2021.) |
⊢ ((𝐴 ∈ ℚ ∧ 𝐵 ∈ ℚ ∧ 0 < 𝐵) → ((𝐴 mod 𝐵) = 0 ↔ (𝐴 / 𝐵) ∈ ℤ)) | ||
Theorem | mulqmod0 10286 | The product of an integer and a positive rational number is 0 modulo the positive real number. (Contributed by Jim Kingdon, 18-Oct-2021.) |
⊢ ((𝐴 ∈ ℤ ∧ 𝑀 ∈ ℚ ∧ 0 < 𝑀) → ((𝐴 · 𝑀) mod 𝑀) = 0) | ||
Theorem | negqmod0 10287 | 𝐴 is divisible by 𝐵 iff its negative is. (Contributed by Jim Kingdon, 18-Oct-2021.) |
⊢ ((𝐴 ∈ ℚ ∧ 𝐵 ∈ ℚ ∧ 0 < 𝐵) → ((𝐴 mod 𝐵) = 0 ↔ (-𝐴 mod 𝐵) = 0)) | ||
Theorem | modqge0 10288 | The modulo operation is nonnegative. (Contributed by Jim Kingdon, 18-Oct-2021.) |
⊢ ((𝐴 ∈ ℚ ∧ 𝐵 ∈ ℚ ∧ 0 < 𝐵) → 0 ≤ (𝐴 mod 𝐵)) | ||
Theorem | modqlt 10289 | The modulo operation is less than its second argument. (Contributed by Jim Kingdon, 18-Oct-2021.) |
⊢ ((𝐴 ∈ ℚ ∧ 𝐵 ∈ ℚ ∧ 0 < 𝐵) → (𝐴 mod 𝐵) < 𝐵) | ||
Theorem | modqelico 10290 | Modular reduction produces a half-open interval. (Contributed by Jim Kingdon, 18-Oct-2021.) |
⊢ ((𝐴 ∈ ℚ ∧ 𝐵 ∈ ℚ ∧ 0 < 𝐵) → (𝐴 mod 𝐵) ∈ (0[,)𝐵)) | ||
Theorem | modqdiffl 10291 | The modulo operation differs from 𝐴 by an integer multiple of 𝐵. (Contributed by Jim Kingdon, 18-Oct-2021.) |
⊢ ((𝐴 ∈ ℚ ∧ 𝐵 ∈ ℚ ∧ 0 < 𝐵) → ((𝐴 − (𝐴 mod 𝐵)) / 𝐵) = (⌊‘(𝐴 / 𝐵))) | ||
Theorem | modqdifz 10292 | The modulo operation differs from 𝐴 by an integer multiple of 𝐵. (Contributed by Jim Kingdon, 18-Oct-2021.) |
⊢ ((𝐴 ∈ ℚ ∧ 𝐵 ∈ ℚ ∧ 0 < 𝐵) → ((𝐴 − (𝐴 mod 𝐵)) / 𝐵) ∈ ℤ) | ||
Theorem | modqfrac 10293 | The fractional part of a number is the number modulo 1. (Contributed by Jim Kingdon, 18-Oct-2021.) |
⊢ (𝐴 ∈ ℚ → (𝐴 mod 1) = (𝐴 − (⌊‘𝐴))) | ||
Theorem | flqmod 10294 | The floor function expressed in terms of the modulo operation. (Contributed by Jim Kingdon, 18-Oct-2021.) |
⊢ (𝐴 ∈ ℚ → (⌊‘𝐴) = (𝐴 − (𝐴 mod 1))) | ||
Theorem | intqfrac 10295 | Break a number into its integer part and its fractional part. (Contributed by Jim Kingdon, 18-Oct-2021.) |
⊢ (𝐴 ∈ ℚ → 𝐴 = ((⌊‘𝐴) + (𝐴 mod 1))) | ||
Theorem | zmod10 10296 | An integer modulo 1 is 0. (Contributed by Paul Chapman, 22-Jun-2011.) |
⊢ (𝑁 ∈ ℤ → (𝑁 mod 1) = 0) | ||
Theorem | zmod1congr 10297 | Two arbitrary integers are congruent modulo 1, see example 4 in [ApostolNT] p. 107. (Contributed by AV, 21-Jul-2021.) |
⊢ ((𝐴 ∈ ℤ ∧ 𝐵 ∈ ℤ) → (𝐴 mod 1) = (𝐵 mod 1)) | ||
Theorem | modqmulnn 10298 | Move a positive integer in and out of a floor in the first argument of a modulo operation. (Contributed by Jim Kingdon, 18-Oct-2021.) |
⊢ ((𝑁 ∈ ℕ ∧ 𝐴 ∈ ℚ ∧ 𝑀 ∈ ℕ) → ((𝑁 · (⌊‘𝐴)) mod (𝑁 · 𝑀)) ≤ ((⌊‘(𝑁 · 𝐴)) mod (𝑁 · 𝑀))) | ||
Theorem | modqvalp1 10299 | The value of the modulo operation (expressed with sum of denominator and nominator). (Contributed by Jim Kingdon, 20-Oct-2021.) |
⊢ ((𝐴 ∈ ℚ ∧ 𝐵 ∈ ℚ ∧ 0 < 𝐵) → ((𝐴 + 𝐵) − (((⌊‘(𝐴 / 𝐵)) + 1) · 𝐵)) = (𝐴 mod 𝐵)) | ||
Theorem | zmodcl 10300 | Closure law for the modulo operation restricted to integers. (Contributed by NM, 27-Nov-2008.) |
⊢ ((𝐴 ∈ ℤ ∧ 𝐵 ∈ ℕ) → (𝐴 mod 𝐵) ∈ ℕ0) |
< Previous Next > |
Copyright terms: Public domain | < Previous Next > |