![]() |
Metamath
Proof Explorer Theorem List (p. 155 of 426) | < Previous Next > |
Bad symbols? Try the
GIF version. |
||
Mirrors > Metamath Home Page > MPE Home Page > Theorem List Contents > Recent Proofs This page: Page List |
Color key: | ![]() (1-27775) |
![]() (27776-29300) |
![]() (29301-42551) |
Type | Label | Description |
---|---|---|
Statement | ||
Theorem | nprm 15401 | A product of two integers greater than one is composite. (Contributed by Mario Carneiro, 20-Jun-2015.) |
⊢ ((𝐴 ∈ (ℤ≥‘2) ∧ 𝐵 ∈ (ℤ≥‘2)) → ¬ (𝐴 · 𝐵) ∈ ℙ) | ||
Theorem | nprmi 15402 | An inference for compositeness. (Contributed by Mario Carneiro, 18-Feb-2014.) (Revised by Mario Carneiro, 20-Jun-2015.) |
⊢ 𝐴 ∈ ℕ & ⊢ 𝐵 ∈ ℕ & ⊢ 1 < 𝐴 & ⊢ 1 < 𝐵 & ⊢ (𝐴 · 𝐵) = 𝑁 ⇒ ⊢ ¬ 𝑁 ∈ ℙ | ||
Theorem | dvdsnprmd 15403 | If a number is divisible by an integer greater than 1 and less then the number, the number is not prime. (Contributed by AV, 24-Jul-2021.) |
⊢ (𝜑 → 1 < 𝐴) & ⊢ (𝜑 → 𝐴 < 𝑁) & ⊢ (𝜑 → 𝐴 ∥ 𝑁) ⇒ ⊢ (𝜑 → ¬ 𝑁 ∈ ℙ) | ||
Theorem | prm2orodd 15404 | A prime number is either 2 or odd. (Contributed by AV, 19-Jun-2021.) |
⊢ (𝑃 ∈ ℙ → (𝑃 = 2 ∨ ¬ 2 ∥ 𝑃)) | ||
Theorem | 2prm 15405 | 2 is a prime number. (Contributed by Paul Chapman, 22-Jun-2011.) (Proof shortened by Fan Zheng, 16-Jun-2016.) |
⊢ 2 ∈ ℙ | ||
Theorem | 3prm 15406 | 3 is a prime number. (Contributed by Paul Chapman, 22-Jun-2011.) |
⊢ 3 ∈ ℙ | ||
Theorem | 4nprm 15407 | 4 is not a prime number. (Contributed by Paul Chapman, 22-Jun-2011.) (Proof shortened by Mario Carneiro, 18-Feb-2014.) |
⊢ ¬ 4 ∈ ℙ | ||
Theorem | prmuz2 15408 | A prime number is an integer greater than or equal to 2. (Contributed by Paul Chapman, 17-Nov-2012.) |
⊢ (𝑃 ∈ ℙ → 𝑃 ∈ (ℤ≥‘2)) | ||
Theorem | prmgt1 15409 | A prime number is an integer greater than 1. (Contributed by Alexander van der Vekens, 17-May-2018.) |
⊢ (𝑃 ∈ ℙ → 1 < 𝑃) | ||
Theorem | prmm2nn0 15410 | Subtracting 2 from a prime number results in a nonnegative integer. (Contributed by Alexander van der Vekens, 30-Aug-2018.) |
⊢ (𝑃 ∈ ℙ → (𝑃 − 2) ∈ ℕ0) | ||
Theorem | oddprmgt2 15411 | An odd prime is greater than 2. (Contributed by AV, 20-Aug-2021.) |
⊢ (𝑃 ∈ (ℙ ∖ {2}) → 2 < 𝑃) | ||
Theorem | oddprmge3 15412 | An odd prime is greater than or equal to 3. (Contributed by Alexander van der Vekens, 7-Oct-2018.) (Revised by AV, 20-Aug-2021.) |
⊢ (𝑃 ∈ (ℙ ∖ {2}) → 𝑃 ∈ (ℤ≥‘3)) | ||
Theorem | prmn2uzge3OLD 15413 | Obsolete version of oddprmge3 15412 as of 20-Aug-2021. (Contributed by Alexander van der Vekens, 7-Oct-2018.) (Proof shortened by AV, 20-Aug-2021.) (New usage is discouraged.) (Proof modification is discouraged.) |
⊢ ((𝑃 ∈ ℙ ∧ 𝑃 ≠ 2) → 𝑃 ∈ (ℤ≥‘3)) | ||
Theorem | sqnprm 15414 | A square is never prime. (Contributed by Mario Carneiro, 20-Jun-2015.) |
⊢ (𝐴 ∈ ℤ → ¬ (𝐴↑2) ∈ ℙ) | ||
Theorem | dvdsprm 15415 | An integer greater than or equal to 2 divides a prime number iff it is equal to it. (Contributed by Paul Chapman, 26-Oct-2012.) |
⊢ ((𝑁 ∈ (ℤ≥‘2) ∧ 𝑃 ∈ ℙ) → (𝑁 ∥ 𝑃 ↔ 𝑁 = 𝑃)) | ||
Theorem | exprmfct 15416* | Every integer greater than or equal to 2 has a prime factor. (Contributed by Paul Chapman, 26-Oct-2012.) (Proof shortened by Mario Carneiro, 20-Jun-2015.) |
⊢ (𝑁 ∈ (ℤ≥‘2) → ∃𝑝 ∈ ℙ 𝑝 ∥ 𝑁) | ||
Theorem | prmdvdsfz 15417* | Each integer greater than 1 and less then or equal to a fixed number is divisible by a prime less then or equal to this fixed number. (Contributed by AV, 15-Aug-2020.) |
⊢ ((𝑁 ∈ ℕ ∧ 𝐼 ∈ (2...𝑁)) → ∃𝑝 ∈ ℙ (𝑝 ≤ 𝑁 ∧ 𝑝 ∥ 𝐼)) | ||
Theorem | nprmdvds1 15418 | No prime number divides 1. (Contributed by Paul Chapman, 17-Nov-2012.) (Proof shortened by Mario Carneiro, 2-Jul-2015.) |
⊢ (𝑃 ∈ ℙ → ¬ 𝑃 ∥ 1) | ||
Theorem | isprm5 15419* | One need only check prime divisors of 𝑃 up to √𝑃 in order to ensure primality. (Contributed by Mario Carneiro, 18-Feb-2014.) |
⊢ (𝑃 ∈ ℙ ↔ (𝑃 ∈ (ℤ≥‘2) ∧ ∀𝑧 ∈ ℙ ((𝑧↑2) ≤ 𝑃 → ¬ 𝑧 ∥ 𝑃))) | ||
Theorem | isprm7 15420* | One need only check prime divisors of 𝑃 up to √𝑃 in order to ensure primality. This version of isprm5 15419 combines the primality and bound on 𝑧 into a finite interval of prime numbers. (Contributed by Steve Rodriguez, 20-Jan-2020.) |
⊢ (𝑃 ∈ ℙ ↔ (𝑃 ∈ (ℤ≥‘2) ∧ ∀𝑧 ∈ ((2...(⌊‘(√‘𝑃))) ∩ ℙ) ¬ 𝑧 ∥ 𝑃)) | ||
Theorem | maxprmfct 15421* | The set of prime factors of an integer greater than or equal to 2 satisfies the conditions to have a supremum, and that supremum is a member of the set. (Contributed by Paul Chapman, 17-Nov-2012.) |
⊢ 𝑆 = {𝑧 ∈ ℙ ∣ 𝑧 ∥ 𝑁} ⇒ ⊢ (𝑁 ∈ (ℤ≥‘2) → ((𝑆 ⊆ ℤ ∧ 𝑆 ≠ ∅ ∧ ∃𝑥 ∈ ℤ ∀𝑦 ∈ 𝑆 𝑦 ≤ 𝑥) ∧ sup(𝑆, ℝ, < ) ∈ 𝑆)) | ||
Theorem | divgcdodd 15422 | Either 𝐴 / (𝐴 gcd 𝐵) is odd or 𝐵 / (𝐴 gcd 𝐵) is odd. (Contributed by Scott Fenton, 19-Apr-2014.) |
⊢ ((𝐴 ∈ ℕ ∧ 𝐵 ∈ ℕ) → (¬ 2 ∥ (𝐴 / (𝐴 gcd 𝐵)) ∨ ¬ 2 ∥ (𝐵 / (𝐴 gcd 𝐵)))) | ||
This section is about coprimality with respect to primes, and a special version of Euclid's lemma for primes is provided, see euclemma 15425. | ||
Theorem | coprm 15423 | A prime number either divides an integer or is coprime to it, but not both. Theorem 1.8 in [ApostolNT] p. 17. (Contributed by Paul Chapman, 22-Jun-2011.) |
⊢ ((𝑃 ∈ ℙ ∧ 𝑁 ∈ ℤ) → (¬ 𝑃 ∥ 𝑁 ↔ (𝑃 gcd 𝑁) = 1)) | ||
Theorem | prmrp 15424 | Unequal prime numbers are relatively prime. (Contributed by Mario Carneiro, 23-Feb-2014.) |
⊢ ((𝑃 ∈ ℙ ∧ 𝑄 ∈ ℙ) → ((𝑃 gcd 𝑄) = 1 ↔ 𝑃 ≠ 𝑄)) | ||
Theorem | euclemma 15425 | Euclid's lemma. A prime number divides the product of two integers iff it divides at least one of them. Theorem 1.9 in [ApostolNT] p. 17. (Contributed by Paul Chapman, 17-Nov-2012.) |
⊢ ((𝑃 ∈ ℙ ∧ 𝑀 ∈ ℤ ∧ 𝑁 ∈ ℤ) → (𝑃 ∥ (𝑀 · 𝑁) ↔ (𝑃 ∥ 𝑀 ∨ 𝑃 ∥ 𝑁))) | ||
Theorem | isprm6 15426* | A number is prime iff it satisfies Euclid's lemma euclemma 15425. (Contributed by Mario Carneiro, 6-Sep-2015.) |
⊢ (𝑃 ∈ ℙ ↔ (𝑃 ∈ (ℤ≥‘2) ∧ ∀𝑥 ∈ ℤ ∀𝑦 ∈ ℤ (𝑃 ∥ (𝑥 · 𝑦) → (𝑃 ∥ 𝑥 ∨ 𝑃 ∥ 𝑦)))) | ||
Theorem | prmdvdsexp 15427 | A prime divides a positive power of an integer iff it divides the integer. (Contributed by Mario Carneiro, 24-Feb-2014.) (Revised by Mario Carneiro, 17-Jul-2014.) |
⊢ ((𝑃 ∈ ℙ ∧ 𝐴 ∈ ℤ ∧ 𝑁 ∈ ℕ) → (𝑃 ∥ (𝐴↑𝑁) ↔ 𝑃 ∥ 𝐴)) | ||
Theorem | prmdvdsexpb 15428 | A prime divides a positive power of another iff they are equal. (Contributed by Paul Chapman, 30-Nov-2012.) (Revised by Mario Carneiro, 24-Feb-2014.) |
⊢ ((𝑃 ∈ ℙ ∧ 𝑄 ∈ ℙ ∧ 𝑁 ∈ ℕ) → (𝑃 ∥ (𝑄↑𝑁) ↔ 𝑃 = 𝑄)) | ||
Theorem | prmdvdsexpr 15429 | If a prime divides a nonnegative power of another, then they are equal. (Contributed by Mario Carneiro, 16-Jan-2015.) |
⊢ ((𝑃 ∈ ℙ ∧ 𝑄 ∈ ℙ ∧ 𝑁 ∈ ℕ0) → (𝑃 ∥ (𝑄↑𝑁) → 𝑃 = 𝑄)) | ||
Theorem | prmexpb 15430 | Two positive prime powers are equal iff the primes and the powers are equal. (Contributed by Paul Chapman, 30-Nov-2012.) |
⊢ (((𝑃 ∈ ℙ ∧ 𝑄 ∈ ℙ) ∧ (𝑀 ∈ ℕ ∧ 𝑁 ∈ ℕ)) → ((𝑃↑𝑀) = (𝑄↑𝑁) ↔ (𝑃 = 𝑄 ∧ 𝑀 = 𝑁))) | ||
Theorem | prmfac1 15431 | The factorial of a number only contains primes less than the base. (Contributed by Mario Carneiro, 6-Mar-2014.) |
⊢ ((𝑁 ∈ ℕ0 ∧ 𝑃 ∈ ℙ ∧ 𝑃 ∥ (!‘𝑁)) → 𝑃 ≤ 𝑁) | ||
Theorem | rpexp 15432 | If two numbers 𝐴 and 𝐵 are relatively prime, then they are still relatively prime if raised to a power. (Contributed by Mario Carneiro, 24-Feb-2014.) |
⊢ ((𝐴 ∈ ℤ ∧ 𝐵 ∈ ℤ ∧ 𝑁 ∈ ℕ) → (((𝐴↑𝑁) gcd 𝐵) = 1 ↔ (𝐴 gcd 𝐵) = 1)) | ||
Theorem | rpexp1i 15433 | Relative primality passes to asymmetric powers. (Contributed by Stefan O'Rear, 27-Sep-2014.) |
⊢ ((𝐴 ∈ ℤ ∧ 𝐵 ∈ ℤ ∧ 𝑀 ∈ ℕ0) → ((𝐴 gcd 𝐵) = 1 → ((𝐴↑𝑀) gcd 𝐵) = 1)) | ||
Theorem | rpexp12i 15434 | Relative primality passes to symmetric powers. (Contributed by Stefan O'Rear, 27-Sep-2014.) |
⊢ ((𝐴 ∈ ℤ ∧ 𝐵 ∈ ℤ ∧ (𝑀 ∈ ℕ0 ∧ 𝑁 ∈ ℕ0)) → ((𝐴 gcd 𝐵) = 1 → ((𝐴↑𝑀) gcd (𝐵↑𝑁)) = 1)) | ||
Theorem | prmndvdsfaclt 15435 | A prime number does not divide the factorial of a nonnegative integer less than the prime number. (Contributed by AV, 13-Jul-2021.) |
⊢ ((𝑃 ∈ ℙ ∧ 𝑁 ∈ ℕ0) → (𝑁 < 𝑃 → ¬ 𝑃 ∥ (!‘𝑁))) | ||
Theorem | ncoprmlnprm 15436 | If two positive integers are not coprime, the larger of them is not a prime number. (Contributed by AV, 9-Aug-2020.) |
⊢ ((𝐴 ∈ ℕ ∧ 𝐵 ∈ ℕ ∧ 𝐴 < 𝐵) → (1 < (𝐴 gcd 𝐵) → 𝐵 ∉ ℙ)) | ||
Theorem | cncongrprm 15437 | Corollary 2 of Cancellability of Congruences: Two products with a common factor are congruent modulo a prime number not dividing the common factor iff the other factors are congruent modulo the prime number. (Contributed by AV, 13-Jul-2021.) |
⊢ (((𝐴 ∈ ℤ ∧ 𝐵 ∈ ℤ ∧ 𝐶 ∈ ℤ) ∧ (𝑃 ∈ ℙ ∧ ¬ 𝑃 ∥ 𝐶)) → (((𝐴 · 𝐶) mod 𝑃) = ((𝐵 · 𝐶) mod 𝑃) ↔ (𝐴 mod 𝑃) = (𝐵 mod 𝑃))) | ||
Theorem | isevengcd2 15438 | The predicate "is an even number". An even number and 2 have 2 as greatest common divisor. (Contributed by AV, 1-Jul-2020.) (Revised by AV, 8-Aug-2021.) |
⊢ (𝑍 ∈ ℤ → (2 ∥ 𝑍 ↔ (2 gcd 𝑍) = 2)) | ||
Theorem | isoddgcd1 15439 | The predicate "is an odd number". An odd number and 2 have 1 as greatest common divisor. (Contributed by AV, 1-Jul-2020.) (Revised by AV, 8-Aug-2021.) |
⊢ (𝑍 ∈ ℤ → (¬ 2 ∥ 𝑍 ↔ (2 gcd 𝑍) = 1)) | ||
Theorem | 3lcm2e6 15440 | The least common multiple of three and two is six. The operands are unequal primes and thus coprime, so the result is (the absolute value of) their product. (Contributed by Steve Rodriguez, 20-Jan-2020.) (Proof shortened by AV, 27-Aug-2020.) |
⊢ (3 lcm 2) = 6 | ||
Syntax | cnumer 15441 | Extend class notation to include canonical numerator function. |
class numer | ||
Syntax | cdenom 15442 | Extend class notation to include canonical denominator function. |
class denom | ||
Definition | df-numer 15443* | The canonical numerator of a rational is the numerator of the rational's reduced fraction representation (no common factors, denominator positive). (Contributed by Stefan O'Rear, 13-Sep-2014.) |
⊢ numer = (𝑦 ∈ ℚ ↦ (1st ‘(℩𝑥 ∈ (ℤ × ℕ)(((1st ‘𝑥) gcd (2nd ‘𝑥)) = 1 ∧ 𝑦 = ((1st ‘𝑥) / (2nd ‘𝑥)))))) | ||
Definition | df-denom 15444* | The canonical denominator of a rational is the denominator of the rational's reduced fraction representation (no common factors, denominator positive). (Contributed by Stefan O'Rear, 13-Sep-2014.) |
⊢ denom = (𝑦 ∈ ℚ ↦ (2nd ‘(℩𝑥 ∈ (ℤ × ℕ)(((1st ‘𝑥) gcd (2nd ‘𝑥)) = 1 ∧ 𝑦 = ((1st ‘𝑥) / (2nd ‘𝑥)))))) | ||
Theorem | qnumval 15445* | Value of the canonical numerator function. (Contributed by Stefan O'Rear, 13-Sep-2014.) |
⊢ (𝐴 ∈ ℚ → (numer‘𝐴) = (1st ‘(℩𝑥 ∈ (ℤ × ℕ)(((1st ‘𝑥) gcd (2nd ‘𝑥)) = 1 ∧ 𝐴 = ((1st ‘𝑥) / (2nd ‘𝑥)))))) | ||
Theorem | qdenval 15446* | Value of the canonical denominator function. (Contributed by Stefan O'Rear, 13-Sep-2014.) |
⊢ (𝐴 ∈ ℚ → (denom‘𝐴) = (2nd ‘(℩𝑥 ∈ (ℤ × ℕ)(((1st ‘𝑥) gcd (2nd ‘𝑥)) = 1 ∧ 𝐴 = ((1st ‘𝑥) / (2nd ‘𝑥)))))) | ||
Theorem | qnumdencl 15447 | Lemma for qnumcl 15448 and qdencl 15449. (Contributed by Stefan O'Rear, 13-Sep-2014.) |
⊢ (𝐴 ∈ ℚ → ((numer‘𝐴) ∈ ℤ ∧ (denom‘𝐴) ∈ ℕ)) | ||
Theorem | qnumcl 15448 | The canonical numerator of a rational is an integer. (Contributed by Stefan O'Rear, 13-Sep-2014.) |
⊢ (𝐴 ∈ ℚ → (numer‘𝐴) ∈ ℤ) | ||
Theorem | qdencl 15449 | The canonical denominator is a positive integer. (Contributed by Stefan O'Rear, 13-Sep-2014.) |
⊢ (𝐴 ∈ ℚ → (denom‘𝐴) ∈ ℕ) | ||
Theorem | fnum 15450 | Canonical numerator defines a function. (Contributed by Stefan O'Rear, 13-Sep-2014.) |
⊢ numer:ℚ⟶ℤ | ||
Theorem | fden 15451 | Canonical denominator defines a function. (Contributed by Stefan O'Rear, 13-Sep-2014.) |
⊢ denom:ℚ⟶ℕ | ||
Theorem | qnumdenbi 15452 | Two numbers are the canonical representation of a rational iff they are coprime and have the right quotient. (Contributed by Stefan O'Rear, 13-Sep-2014.) |
⊢ ((𝐴 ∈ ℚ ∧ 𝐵 ∈ ℤ ∧ 𝐶 ∈ ℕ) → (((𝐵 gcd 𝐶) = 1 ∧ 𝐴 = (𝐵 / 𝐶)) ↔ ((numer‘𝐴) = 𝐵 ∧ (denom‘𝐴) = 𝐶))) | ||
Theorem | qnumdencoprm 15453 | The canonical representation of a rational is fully reduced. (Contributed by Stefan O'Rear, 13-Sep-2014.) |
⊢ (𝐴 ∈ ℚ → ((numer‘𝐴) gcd (denom‘𝐴)) = 1) | ||
Theorem | qeqnumdivden 15454 | Recover a rational number from its canonical representation. (Contributed by Stefan O'Rear, 13-Sep-2014.) |
⊢ (𝐴 ∈ ℚ → 𝐴 = ((numer‘𝐴) / (denom‘𝐴))) | ||
Theorem | qmuldeneqnum 15455 | Multiplying a rational by its denominator results in an integer. (Contributed by Stefan O'Rear, 13-Sep-2014.) |
⊢ (𝐴 ∈ ℚ → (𝐴 · (denom‘𝐴)) = (numer‘𝐴)) | ||
Theorem | divnumden 15456 | Calculate the reduced form of a quotient using gcd. (Contributed by Stefan O'Rear, 13-Sep-2014.) |
⊢ ((𝐴 ∈ ℤ ∧ 𝐵 ∈ ℕ) → ((numer‘(𝐴 / 𝐵)) = (𝐴 / (𝐴 gcd 𝐵)) ∧ (denom‘(𝐴 / 𝐵)) = (𝐵 / (𝐴 gcd 𝐵)))) | ||
Theorem | divdenle 15457 | Reducing a quotient never increases the denominator. (Contributed by Stefan O'Rear, 13-Sep-2014.) |
⊢ ((𝐴 ∈ ℤ ∧ 𝐵 ∈ ℕ) → (denom‘(𝐴 / 𝐵)) ≤ 𝐵) | ||
Theorem | qnumgt0 15458 | A rational is positive iff its canonical numerator is. (Contributed by Stefan O'Rear, 15-Sep-2014.) |
⊢ (𝐴 ∈ ℚ → (0 < 𝐴 ↔ 0 < (numer‘𝐴))) | ||
Theorem | qgt0numnn 15459 | A rational is positive iff its canonical numerator is a positive integer. (Contributed by Stefan O'Rear, 15-Sep-2014.) |
⊢ ((𝐴 ∈ ℚ ∧ 0 < 𝐴) → (numer‘𝐴) ∈ ℕ) | ||
Theorem | nn0gcdsq 15460 | Squaring commutes with GCD, in particular two coprime numbers have coprime squares. (Contributed by Stefan O'Rear, 15-Sep-2014.) |
⊢ ((𝐴 ∈ ℕ0 ∧ 𝐵 ∈ ℕ0) → ((𝐴 gcd 𝐵)↑2) = ((𝐴↑2) gcd (𝐵↑2))) | ||
Theorem | zgcdsq 15461 | nn0gcdsq 15460 extended to integers by symmetry. (Contributed by Stefan O'Rear, 15-Sep-2014.) |
⊢ ((𝐴 ∈ ℤ ∧ 𝐵 ∈ ℤ) → ((𝐴 gcd 𝐵)↑2) = ((𝐴↑2) gcd (𝐵↑2))) | ||
Theorem | numdensq 15462 | Squaring a rational squares its canonical components. (Contributed by Stefan O'Rear, 15-Sep-2014.) |
⊢ (𝐴 ∈ ℚ → ((numer‘(𝐴↑2)) = ((numer‘𝐴)↑2) ∧ (denom‘(𝐴↑2)) = ((denom‘𝐴)↑2))) | ||
Theorem | numsq 15463 | Square commutes with canonical numerator. (Contributed by Stefan O'Rear, 15-Sep-2014.) |
⊢ (𝐴 ∈ ℚ → (numer‘(𝐴↑2)) = ((numer‘𝐴)↑2)) | ||
Theorem | densq 15464 | Square commutes with canonical denominator. (Contributed by Stefan O'Rear, 15-Sep-2014.) |
⊢ (𝐴 ∈ ℚ → (denom‘(𝐴↑2)) = ((denom‘𝐴)↑2)) | ||
Theorem | qden1elz 15465 | A rational is an integer iff it has denominator 1. (Contributed by Stefan O'Rear, 15-Sep-2014.) |
⊢ (𝐴 ∈ ℚ → ((denom‘𝐴) = 1 ↔ 𝐴 ∈ ℤ)) | ||
Theorem | zsqrtelqelz 15466 | If an integer has a rational square root, that root is must be an integer. (Contributed by Stefan O'Rear, 15-Sep-2014.) |
⊢ ((𝐴 ∈ ℤ ∧ (√‘𝐴) ∈ ℚ) → (√‘𝐴) ∈ ℤ) | ||
Theorem | nonsq 15467 | Any integer strictly between two adjacent squares has an irrational square root. (Contributed by Stefan O'Rear, 15-Sep-2014.) |
⊢ (((𝐴 ∈ ℕ0 ∧ 𝐵 ∈ ℕ0) ∧ ((𝐵↑2) < 𝐴 ∧ 𝐴 < ((𝐵 + 1)↑2))) → ¬ (√‘𝐴) ∈ ℚ) | ||
Syntax | codz 15468 | Extend class notation with the order function on the class of integers mod N. |
class odℤ | ||
Syntax | cphi 15469 | Extend class notation with the Euler phi function. |
class ϕ | ||
Definition | df-odz 15470* | Define the order function on the class of integers mod N. (Contributed by Mario Carneiro, 23-Feb-2014.) (Revised by AV, 26-Sep-2020.) |
⊢ odℤ = (𝑛 ∈ ℕ ↦ (𝑥 ∈ {𝑥 ∈ ℤ ∣ (𝑥 gcd 𝑛) = 1} ↦ inf({𝑚 ∈ ℕ ∣ 𝑛 ∥ ((𝑥↑𝑚) − 1)}, ℝ, < ))) | ||
Definition | df-phi 15471* | Define the Euler phi function (also called _ Euler totient function_), which counts the number of integers less than 𝑛 and coprime to it, see definition in [ApostolNT] p. 25. (Contributed by Mario Carneiro, 23-Feb-2014.) |
⊢ ϕ = (𝑛 ∈ ℕ ↦ (#‘{𝑥 ∈ (1...𝑛) ∣ (𝑥 gcd 𝑛) = 1})) | ||
Theorem | phival 15472* | Value of the Euler ϕ function. (Contributed by Mario Carneiro, 23-Feb-2014.) |
⊢ (𝑁 ∈ ℕ → (ϕ‘𝑁) = (#‘{𝑥 ∈ (1...𝑁) ∣ (𝑥 gcd 𝑁) = 1})) | ||
Theorem | phicl2 15473 | Bounds and closure for the value of the Euler ϕ function. (Contributed by Mario Carneiro, 23-Feb-2014.) |
⊢ (𝑁 ∈ ℕ → (ϕ‘𝑁) ∈ (1...𝑁)) | ||
Theorem | phicl 15474 | Closure for the value of the Euler ϕ function. (Contributed by Mario Carneiro, 28-Feb-2014.) |
⊢ (𝑁 ∈ ℕ → (ϕ‘𝑁) ∈ ℕ) | ||
Theorem | phibndlem 15475* | Lemma for phibnd 15476. (Contributed by Mario Carneiro, 23-Feb-2014.) |
⊢ (𝑁 ∈ (ℤ≥‘2) → {𝑥 ∈ (1...𝑁) ∣ (𝑥 gcd 𝑁) = 1} ⊆ (1...(𝑁 − 1))) | ||
Theorem | phibnd 15476 | A slightly tighter bound on the value of the Euler ϕ function. (Contributed by Mario Carneiro, 23-Feb-2014.) |
⊢ (𝑁 ∈ (ℤ≥‘2) → (ϕ‘𝑁) ≤ (𝑁 − 1)) | ||
Theorem | phicld 15477 | Closure for the value of the Euler ϕ function. (Contributed by Mario Carneiro, 29-May-2016.) |
⊢ (𝜑 → 𝑁 ∈ ℕ) ⇒ ⊢ (𝜑 → (ϕ‘𝑁) ∈ ℕ) | ||
Theorem | phi1 15478 | Value of the Euler ϕ function at 1. (Contributed by Mario Carneiro, 23-Feb-2014.) |
⊢ (ϕ‘1) = 1 | ||
Theorem | dfphi2 15479* | Alternate definition of the Euler ϕ function. (Contributed by Mario Carneiro, 23-Feb-2014.) (Revised by Mario Carneiro, 2-May-2016.) |
⊢ (𝑁 ∈ ℕ → (ϕ‘𝑁) = (#‘{𝑥 ∈ (0..^𝑁) ∣ (𝑥 gcd 𝑁) = 1})) | ||
Theorem | hashdvds 15480* | The number of numbers in a given residue class in a finite set of integers. (Contributed by Mario Carneiro, 12-Mar-2014.) (Proof shortened by Mario Carneiro, 7-Jun-2016.) |
⊢ (𝜑 → 𝑁 ∈ ℕ) & ⊢ (𝜑 → 𝐴 ∈ ℤ) & ⊢ (𝜑 → 𝐵 ∈ (ℤ≥‘(𝐴 − 1))) & ⊢ (𝜑 → 𝐶 ∈ ℤ) ⇒ ⊢ (𝜑 → (#‘{𝑥 ∈ (𝐴...𝐵) ∣ 𝑁 ∥ (𝑥 − 𝐶)}) = ((⌊‘((𝐵 − 𝐶) / 𝑁)) − (⌊‘(((𝐴 − 1) − 𝐶) / 𝑁)))) | ||
Theorem | phiprmpw 15481 | Value of the Euler ϕ function at a prime power. Theorem 2.5(a) in [ApostolNT] p. 28. (Contributed by Mario Carneiro, 24-Feb-2014.) |
⊢ ((𝑃 ∈ ℙ ∧ 𝐾 ∈ ℕ) → (ϕ‘(𝑃↑𝐾)) = ((𝑃↑(𝐾 − 1)) · (𝑃 − 1))) | ||
Theorem | phiprm 15482 | Value of the Euler ϕ function at a prime. (Contributed by Mario Carneiro, 28-Feb-2014.) |
⊢ (𝑃 ∈ ℙ → (ϕ‘𝑃) = (𝑃 − 1)) | ||
Theorem | crth 15483* | The Chinese Remainder Theorem: the function that maps 𝑥 to its remainder classes mod 𝑀 and mod 𝑁 is 1-1 and onto when 𝑀 and 𝑁 are coprime. (Contributed by Mario Carneiro, 24-Feb-2014.) (Proof shortened by Mario Carneiro, 2-May-2016.) |
⊢ 𝑆 = (0..^(𝑀 · 𝑁)) & ⊢ 𝑇 = ((0..^𝑀) × (0..^𝑁)) & ⊢ 𝐹 = (𝑥 ∈ 𝑆 ↦ 〈(𝑥 mod 𝑀), (𝑥 mod 𝑁)〉) & ⊢ (𝜑 → (𝑀 ∈ ℕ ∧ 𝑁 ∈ ℕ ∧ (𝑀 gcd 𝑁) = 1)) ⇒ ⊢ (𝜑 → 𝐹:𝑆–1-1-onto→𝑇) | ||
Theorem | phimullem 15484* | Lemma for phimul 15485. (Contributed by Mario Carneiro, 24-Feb-2014.) |
⊢ 𝑆 = (0..^(𝑀 · 𝑁)) & ⊢ 𝑇 = ((0..^𝑀) × (0..^𝑁)) & ⊢ 𝐹 = (𝑥 ∈ 𝑆 ↦ 〈(𝑥 mod 𝑀), (𝑥 mod 𝑁)〉) & ⊢ (𝜑 → (𝑀 ∈ ℕ ∧ 𝑁 ∈ ℕ ∧ (𝑀 gcd 𝑁) = 1)) & ⊢ 𝑈 = {𝑦 ∈ (0..^𝑀) ∣ (𝑦 gcd 𝑀) = 1} & ⊢ 𝑉 = {𝑦 ∈ (0..^𝑁) ∣ (𝑦 gcd 𝑁) = 1} & ⊢ 𝑊 = {𝑦 ∈ 𝑆 ∣ (𝑦 gcd (𝑀 · 𝑁)) = 1} ⇒ ⊢ (𝜑 → (ϕ‘(𝑀 · 𝑁)) = ((ϕ‘𝑀) · (ϕ‘𝑁))) | ||
Theorem | phimul 15485 | The Euler ϕ function is a multiplicative function, meaning that it distributes over multiplication at relatively prime arguments. Theorem 2.5(c) in [ApostolNT] p. 28. (Contributed by Mario Carneiro, 24-Feb-2014.) |
⊢ ((𝑀 ∈ ℕ ∧ 𝑁 ∈ ℕ ∧ (𝑀 gcd 𝑁) = 1) → (ϕ‘(𝑀 · 𝑁)) = ((ϕ‘𝑀) · (ϕ‘𝑁))) | ||
Theorem | eulerthlem1 15486* | Lemma for eulerth 15488. (Contributed by Mario Carneiro, 8-May-2015.) |
⊢ (𝜑 → (𝑁 ∈ ℕ ∧ 𝐴 ∈ ℤ ∧ (𝐴 gcd 𝑁) = 1)) & ⊢ 𝑆 = {𝑦 ∈ (0..^𝑁) ∣ (𝑦 gcd 𝑁) = 1} & ⊢ 𝑇 = (1...(ϕ‘𝑁)) & ⊢ (𝜑 → 𝐹:𝑇–1-1-onto→𝑆) & ⊢ 𝐺 = (𝑥 ∈ 𝑇 ↦ ((𝐴 · (𝐹‘𝑥)) mod 𝑁)) ⇒ ⊢ (𝜑 → 𝐺:𝑇⟶𝑆) | ||
Theorem | eulerthlem2 15487* | Lemma for eulerth 15488. (Contributed by Mario Carneiro, 28-Feb-2014.) |
⊢ (𝜑 → (𝑁 ∈ ℕ ∧ 𝐴 ∈ ℤ ∧ (𝐴 gcd 𝑁) = 1)) & ⊢ 𝑆 = {𝑦 ∈ (0..^𝑁) ∣ (𝑦 gcd 𝑁) = 1} & ⊢ 𝑇 = (1...(ϕ‘𝑁)) & ⊢ (𝜑 → 𝐹:𝑇–1-1-onto→𝑆) & ⊢ 𝐺 = (𝑥 ∈ 𝑇 ↦ ((𝐴 · (𝐹‘𝑥)) mod 𝑁)) ⇒ ⊢ (𝜑 → ((𝐴↑(ϕ‘𝑁)) mod 𝑁) = (1 mod 𝑁)) | ||
Theorem | eulerth 15488 | Euler's theorem, a generalization of Fermat's little theorem. If 𝐴 and 𝑁 are coprime, then 𝐴↑ϕ(𝑁)≡1 (mod 𝑁). This is Metamath 100 proof #10. Also called Euler-Fermat theorem, see theorem 5.17 in [ApostolNT] p. 113. (Contributed by Mario Carneiro, 28-Feb-2014.) |
⊢ ((𝑁 ∈ ℕ ∧ 𝐴 ∈ ℤ ∧ (𝐴 gcd 𝑁) = 1) → ((𝐴↑(ϕ‘𝑁)) mod 𝑁) = (1 mod 𝑁)) | ||
Theorem | fermltl 15489 | Fermat's little theorem. When 𝑃 is prime, 𝐴↑𝑃≡𝐴 (mod 𝑃) for any 𝐴, see theorem 5.19 in [ApostolNT] p. 114. (Contributed by Mario Carneiro, 28-Feb-2014.) |
⊢ ((𝑃 ∈ ℙ ∧ 𝐴 ∈ ℤ) → ((𝐴↑𝑃) mod 𝑃) = (𝐴 mod 𝑃)) | ||
Theorem | prmdiv 15490 | Show an explicit expression for the modular inverse of 𝐴 mod 𝑃. (Contributed by Mario Carneiro, 24-Jan-2015.) |
⊢ 𝑅 = ((𝐴↑(𝑃 − 2)) mod 𝑃) ⇒ ⊢ ((𝑃 ∈ ℙ ∧ 𝐴 ∈ ℤ ∧ ¬ 𝑃 ∥ 𝐴) → (𝑅 ∈ (1...(𝑃 − 1)) ∧ 𝑃 ∥ ((𝐴 · 𝑅) − 1))) | ||
Theorem | prmdiveq 15491 | The modular inverse of 𝐴 mod 𝑃 is unique. (Contributed by Mario Carneiro, 24-Jan-2015.) |
⊢ 𝑅 = ((𝐴↑(𝑃 − 2)) mod 𝑃) ⇒ ⊢ ((𝑃 ∈ ℙ ∧ 𝐴 ∈ ℤ ∧ ¬ 𝑃 ∥ 𝐴) → ((𝑆 ∈ (0...(𝑃 − 1)) ∧ 𝑃 ∥ ((𝐴 · 𝑆) − 1)) ↔ 𝑆 = 𝑅)) | ||
Theorem | prmdivdiv 15492 | The (modular) inverse of the inverse of a number is itself. (Contributed by Mario Carneiro, 24-Jan-2015.) |
⊢ 𝑅 = ((𝐴↑(𝑃 − 2)) mod 𝑃) ⇒ ⊢ ((𝑃 ∈ ℙ ∧ 𝐴 ∈ (1...(𝑃 − 1))) → 𝐴 = ((𝑅↑(𝑃 − 2)) mod 𝑃)) | ||
Theorem | hashgcdlem 15493* | A correspondence between elements of specific GCD and relative primes in a smaller ring. (Contributed by Stefan O'Rear, 12-Sep-2015.) |
⊢ 𝐴 = {𝑦 ∈ (0..^(𝑀 / 𝑁)) ∣ (𝑦 gcd (𝑀 / 𝑁)) = 1} & ⊢ 𝐵 = {𝑧 ∈ (0..^𝑀) ∣ (𝑧 gcd 𝑀) = 𝑁} & ⊢ 𝐹 = (𝑥 ∈ 𝐴 ↦ (𝑥 · 𝑁)) ⇒ ⊢ ((𝑀 ∈ ℕ ∧ 𝑁 ∈ ℕ ∧ 𝑁 ∥ 𝑀) → 𝐹:𝐴–1-1-onto→𝐵) | ||
Theorem | hashgcdeq 15494* | Number of initial positive integers with specified divisors. (Contributed by Stefan O'Rear, 12-Sep-2015.) |
⊢ ((𝑀 ∈ ℕ ∧ 𝑁 ∈ ℕ) → (#‘{𝑥 ∈ (0..^𝑀) ∣ (𝑥 gcd 𝑀) = 𝑁}) = if(𝑁 ∥ 𝑀, (ϕ‘(𝑀 / 𝑁)), 0)) | ||
Theorem | phisum 15495* | The divisor sum identity of the totient function. Theorem 2.2 in [ApostolNT] p. 26. (Contributed by Stefan O'Rear, 12-Sep-2015.) |
⊢ (𝑁 ∈ ℕ → Σ𝑑 ∈ {𝑥 ∈ ℕ ∣ 𝑥 ∥ 𝑁} (ϕ‘𝑑) = 𝑁) | ||
Theorem | odzval 15496* | Value of the order function. This is a function of functions; the inner argument selects the base (i.e. mod 𝑁 for some 𝑁, often prime) and the outer argument selects the integer or equivalence class (if you want to think about it that way) from the integers mod 𝑁. In order to ensure the supremum is well-defined, we only define the expression when 𝐴 and 𝑁 are coprime. (Contributed by Mario Carneiro, 23-Feb-2014.) (Revised by AV, 26-Sep-2020.) |
⊢ ((𝑁 ∈ ℕ ∧ 𝐴 ∈ ℤ ∧ (𝐴 gcd 𝑁) = 1) → ((odℤ‘𝑁)‘𝐴) = inf({𝑛 ∈ ℕ ∣ 𝑁 ∥ ((𝐴↑𝑛) − 1)}, ℝ, < )) | ||
Theorem | odzcllem 15497 | - Lemma for odzcl 15498, showing existence of a recurrent point for the exponential. (Contributed by Mario Carneiro, 28-Feb-2014.) (Proof shortened by AV, 26-Sep-2020.) |
⊢ ((𝑁 ∈ ℕ ∧ 𝐴 ∈ ℤ ∧ (𝐴 gcd 𝑁) = 1) → (((odℤ‘𝑁)‘𝐴) ∈ ℕ ∧ 𝑁 ∥ ((𝐴↑((odℤ‘𝑁)‘𝐴)) − 1))) | ||
Theorem | odzcl 15498 | The order of a group element is an integer. (Contributed by Mario Carneiro, 28-Feb-2014.) |
⊢ ((𝑁 ∈ ℕ ∧ 𝐴 ∈ ℤ ∧ (𝐴 gcd 𝑁) = 1) → ((odℤ‘𝑁)‘𝐴) ∈ ℕ) | ||
Theorem | odzid 15499 | Any element raised to the power of its order is 1. (Contributed by Mario Carneiro, 28-Feb-2014.) |
⊢ ((𝑁 ∈ ℕ ∧ 𝐴 ∈ ℤ ∧ (𝐴 gcd 𝑁) = 1) → 𝑁 ∥ ((𝐴↑((odℤ‘𝑁)‘𝐴)) − 1)) | ||
Theorem | odzdvds 15500 | The only powers of 𝐴 that are congruent to 1 are the multiples of the order of 𝐴. (Contributed by Mario Carneiro, 28-Feb-2014.) (Proof shortened by AV, 26-Sep-2020.) |
⊢ (((𝑁 ∈ ℕ ∧ 𝐴 ∈ ℤ ∧ (𝐴 gcd 𝑁) = 1) ∧ 𝐾 ∈ ℕ0) → (𝑁 ∥ ((𝐴↑𝐾) − 1) ↔ ((odℤ‘𝑁)‘𝐴) ∥ 𝐾)) |
< Previous Next > |
Copyright terms: Public domain | < Previous Next > |