Home | Intuitionistic Logic Explorer Theorem List (p. 120 of 141) | < Previous Next > |
Browser slow? Try the
Unicode version. |
||
Mirrors > Metamath Home Page > ILE Home Page > Theorem List Contents > Recent Proofs This page: Page List |
Type | Label | Description |
---|---|---|
Statement | ||
Theorem | gcdval 11901* | The value of the operator. is the greatest common divisor of and . If and are both , the result is defined conventionally as . (Contributed by Paul Chapman, 21-Mar-2011.) (Revised by Mario Carneiro, 10-Nov-2013.) |
Theorem | gcd0val 11902 | The value, by convention, of the operator when both operands are 0. (Contributed by Paul Chapman, 21-Mar-2011.) |
Theorem | gcdn0val 11903* | The value of the operator when at least one operand is nonzero. (Contributed by Paul Chapman, 21-Mar-2011.) |
Theorem | gcdn0cl 11904 | Closure of the operator. (Contributed by Paul Chapman, 21-Mar-2011.) |
Theorem | gcddvds 11905 | The gcd of two integers divides each of them. (Contributed by Paul Chapman, 21-Mar-2011.) |
Theorem | dvdslegcd 11906 | An integer which divides both operands of the operator is bounded by it. (Contributed by Paul Chapman, 21-Mar-2011.) |
Theorem | nndvdslegcd 11907 | A positive integer which divides both positive operands of the operator is bounded by it. (Contributed by AV, 9-Aug-2020.) |
Theorem | gcdcl 11908 | Closure of the operator. (Contributed by Paul Chapman, 21-Mar-2011.) |
Theorem | gcdnncl 11909 | Closure of the operator. (Contributed by Thierry Arnoux, 2-Feb-2020.) |
Theorem | gcdcld 11910 | Closure of the operator. (Contributed by Mario Carneiro, 29-May-2016.) |
Theorem | gcd2n0cl 11911 | Closure of the operator if the second operand is not 0. (Contributed by AV, 10-Jul-2021.) |
Theorem | zeqzmulgcd 11912* | An integer is the product of an integer and the gcd of it and another integer. (Contributed by AV, 11-Jul-2021.) |
Theorem | divgcdz 11913 | An integer divided by the gcd of it and a nonzero integer is an integer. (Contributed by AV, 11-Jul-2021.) |
Theorem | gcdf 11914 | Domain and codomain of the operator. (Contributed by Paul Chapman, 31-Mar-2011.) (Revised by Mario Carneiro, 16-Nov-2013.) |
Theorem | gcdcom 11915 | The operator is commutative. Theorem 1.4(a) in [ApostolNT] p. 16. (Contributed by Paul Chapman, 21-Mar-2011.) |
Theorem | gcdcomd 11916 | The operator is commutative, deduction version. (Contributed by SN, 24-Aug-2024.) |
Theorem | divgcdnn 11917 | A positive integer divided by the gcd of it and another integer is a positive integer. (Contributed by AV, 10-Jul-2021.) |
Theorem | divgcdnnr 11918 | A positive integer divided by the gcd of it and another integer is a positive integer. (Contributed by AV, 10-Jul-2021.) |
Theorem | gcdeq0 11919 | The gcd of two integers is zero iff they are both zero. (Contributed by Paul Chapman, 21-Mar-2011.) |
Theorem | gcdn0gt0 11920 | The gcd of two integers is positive (nonzero) iff they are not both zero. (Contributed by Paul Chapman, 22-Jun-2011.) |
Theorem | gcd0id 11921 | The gcd of 0 and an integer is the integer's absolute value. (Contributed by Paul Chapman, 21-Mar-2011.) |
Theorem | gcdid0 11922 | The gcd of an integer and 0 is the integer's absolute value. Theorem 1.4(d)2 in [ApostolNT] p. 16. (Contributed by Paul Chapman, 31-Mar-2011.) |
Theorem | nn0gcdid0 11923 | The gcd of a nonnegative integer with 0 is itself. (Contributed by Paul Chapman, 31-Mar-2011.) |
Theorem | gcdneg 11924 | Negating one operand of the operator does not alter the result. (Contributed by Paul Chapman, 21-Mar-2011.) |
Theorem | neggcd 11925 | Negating one operand of the operator does not alter the result. (Contributed by Paul Chapman, 22-Jun-2011.) |
Theorem | gcdaddm 11926 | Adding a multiple of one operand of the operator to the other does not alter the result. (Contributed by Paul Chapman, 31-Mar-2011.) |
Theorem | gcdadd 11927 | The GCD of two numbers is the same as the GCD of the left and their sum. (Contributed by Scott Fenton, 20-Apr-2014.) |
Theorem | gcdid 11928 | The gcd of a number and itself is its absolute value. (Contributed by Paul Chapman, 31-Mar-2011.) |
Theorem | gcd1 11929 | The gcd of a number with 1 is 1. Theorem 1.4(d)1 in [ApostolNT] p. 16. (Contributed by Mario Carneiro, 19-Feb-2014.) |
Theorem | gcdabs 11930 | The gcd of two integers is the same as that of their absolute values. (Contributed by Paul Chapman, 31-Mar-2011.) |
Theorem | gcdabs1 11931 | of the absolute value of the first operator. (Contributed by Scott Fenton, 2-Apr-2014.) (Revised by Mario Carneiro, 19-Apr-2014.) |
Theorem | gcdabs2 11932 | of the absolute value of the second operator. (Contributed by Scott Fenton, 2-Apr-2014.) (Revised by Mario Carneiro, 19-Apr-2014.) |
Theorem | modgcd 11933 | The gcd remains unchanged if one operand is replaced with its remainder modulo the other. (Contributed by Paul Chapman, 31-Mar-2011.) |
Theorem | 1gcd 11934 | The GCD of one and an integer is one. (Contributed by Scott Fenton, 17-Apr-2014.) (Revised by Mario Carneiro, 19-Apr-2014.) |
Theorem | gcdmultipled 11935 | The greatest common divisor of a nonnegative integer and a multiple of it is itself. (Contributed by Rohan Ridenour, 3-Aug-2023.) |
Theorem | dvdsgcdidd 11936 | The greatest common divisor of a positive integer and another integer it divides is itself. (Contributed by Rohan Ridenour, 3-Aug-2023.) |
Theorem | 6gcd4e2 11937 | The greatest common divisor of six and four is two. To calculate this gcd, a simple form of Euclid's algorithm is used: and . (Contributed by AV, 27-Aug-2020.) |
Theorem | bezoutlemnewy 11938* | Lemma for Bézout's identity. The is-bezout predicate holds for . (Contributed by Jim Kingdon, 6-Jan-2022.) |
Theorem | bezoutlemstep 11939* | Lemma for Bézout's identity. This is the induction step for the proof by induction. (Contributed by Jim Kingdon, 3-Jan-2022.) |
Theorem | bezoutlemmain 11940* | Lemma for Bézout's identity. This is the main result which we prove by induction and which represents the application of the Extended Euclidean algorithm. (Contributed by Jim Kingdon, 30-Dec-2021.) |
Theorem | bezoutlema 11941* | Lemma for Bézout's identity. The is-bezout condition is satisfied by . (Contributed by Jim Kingdon, 30-Dec-2021.) |
Theorem | bezoutlemb 11942* | Lemma for Bézout's identity. The is-bezout condition is satisfied by . (Contributed by Jim Kingdon, 30-Dec-2021.) |
Theorem | bezoutlemex 11943* | Lemma for Bézout's identity. Existence of a number which we will later show to be the greater common divisor and its decomposition into cofactors. (Contributed by Mario Carneiro and Jim Kingdon, 3-Jan-2022.) |
Theorem | bezoutlemzz 11944* | Lemma for Bézout's identity. Like bezoutlemex 11943 but where ' z ' is any integer, not just a nonnegative one. (Contributed by Mario Carneiro and Jim Kingdon, 8-Jan-2022.) |
Theorem | bezoutlemaz 11945* | Lemma for Bézout's identity. Like bezoutlemzz 11944 but where ' A ' can be any integer, not just a nonnegative one. (Contributed by Mario Carneiro and Jim Kingdon, 8-Jan-2022.) |
Theorem | bezoutlembz 11946* | Lemma for Bézout's identity. Like bezoutlemaz 11945 but where ' B ' can be any integer, not just a nonnegative one. (Contributed by Mario Carneiro and Jim Kingdon, 8-Jan-2022.) |
Theorem | bezoutlembi 11947* | Lemma for Bézout's identity. Like bezoutlembz 11946 but the greatest common divisor condition is a biconditional, not just an implication. (Contributed by Mario Carneiro and Jim Kingdon, 8-Jan-2022.) |
Theorem | bezoutlemmo 11948* | Lemma for Bézout's identity. There is at most one nonnegative integer meeting the greatest common divisor condition. (Contributed by Mario Carneiro and Jim Kingdon, 9-Jan-2022.) |
Theorem | bezoutlemeu 11949* | Lemma for Bézout's identity. There is exactly one nonnegative integer meeting the greatest common divisor condition. (Contributed by Mario Carneiro and Jim Kingdon, 9-Jan-2022.) |
Theorem | bezoutlemle 11950* | Lemma for Bézout's identity. The number satisfying the greatest common divisor condition is the largest number which divides both and . (Contributed by Mario Carneiro and Jim Kingdon, 9-Jan-2022.) |
Theorem | bezoutlemsup 11951* | Lemma for Bézout's identity. The number satisfying the greatest common divisor condition is the supremum of divisors of both and . (Contributed by Mario Carneiro and Jim Kingdon, 9-Jan-2022.) |
Theorem | dfgcd3 11952* | Alternate definition of the operator. (Contributed by Jim Kingdon, 31-Dec-2021.) |
Theorem | bezout 11953* |
Bézout's identity: For any integers and , there are
integers such that
. This
is Metamath 100 proof #60.
The proof is constructive, in the sense that it applies the Extended Euclidian Algorithm to constuct a number which can be shown to be and which satisfies the rest of the theorem. In the presence of excluded middle, it is common to prove Bézout's identity by taking the smallest number which satisfies the Bézout condition, and showing it is the greatest common divisor. But we do not have the ability to show that number exists other than by providing a way to determine it. (Contributed by Mario Carneiro, 22-Feb-2014.) |
Theorem | dvdsgcd 11954 | An integer which divides each of two others also divides their gcd. (Contributed by Paul Chapman, 22-Jun-2011.) (Revised by Mario Carneiro, 30-May-2014.) |
Theorem | dvdsgcdb 11955 | Biconditional form of dvdsgcd 11954. (Contributed by Scott Fenton, 2-Apr-2014.) (Revised by Mario Carneiro, 19-Apr-2014.) |
Theorem | dfgcd2 11956* | Alternate definition of the operator, see definition in [ApostolNT] p. 15. (Contributed by AV, 8-Aug-2021.) |
Theorem | gcdass 11957 | Associative law for operator. Theorem 1.4(b) in [ApostolNT] p. 16. (Contributed by Scott Fenton, 2-Apr-2014.) (Revised by Mario Carneiro, 19-Apr-2014.) |
Theorem | mulgcd 11958 | Distribute multiplication by a nonnegative integer over gcd. (Contributed by Paul Chapman, 22-Jun-2011.) (Proof shortened by Mario Carneiro, 30-May-2014.) |
Theorem | absmulgcd 11959 | Distribute absolute value of multiplication over gcd. Theorem 1.4(c) in [ApostolNT] p. 16. (Contributed by Paul Chapman, 22-Jun-2011.) |
Theorem | mulgcdr 11960 | Reverse distribution law for the operator. (Contributed by Scott Fenton, 2-Apr-2014.) (Revised by Mario Carneiro, 19-Apr-2014.) |
Theorem | gcddiv 11961 | Division law for GCD. (Contributed by Scott Fenton, 18-Apr-2014.) (Revised by Mario Carneiro, 19-Apr-2014.) |
Theorem | gcdmultiple 11962 | The GCD of a multiple of a number is the number itself. (Contributed by Scott Fenton, 12-Apr-2014.) (Revised by Mario Carneiro, 19-Apr-2014.) |
Theorem | gcdmultiplez 11963 | Extend gcdmultiple 11962 so can be an integer. (Contributed by Scott Fenton, 18-Apr-2014.) (Revised by Mario Carneiro, 19-Apr-2014.) |
Theorem | gcdzeq 11964 | A positive integer is equal to its gcd with an integer if and only if divides . Generalization of gcdeq 11965. (Contributed by AV, 1-Jul-2020.) |
Theorem | gcdeq 11965 | is equal to its gcd with if and only if divides . (Contributed by Mario Carneiro, 23-Feb-2014.) (Proof shortened by AV, 8-Aug-2021.) |
Theorem | dvdssqim 11966 | Unidirectional form of dvdssq 11973. (Contributed by Scott Fenton, 19-Apr-2014.) |
Theorem | dvdsmulgcd 11967 | Relationship between the order of an element and that of a multiple. (a divisibility equivalent). (Contributed by Stefan O'Rear, 6-Sep-2015.) |
Theorem | rpmulgcd 11968 | If and are relatively prime, then the GCD of and is the GCD of and . (Contributed by Scott Fenton, 12-Apr-2014.) (Revised by Mario Carneiro, 19-Apr-2014.) |
Theorem | rplpwr 11969 | If and are relatively prime, then so are and . (Contributed by Scott Fenton, 12-Apr-2014.) (Revised by Mario Carneiro, 19-Apr-2014.) |
Theorem | rppwr 11970 | If and are relatively prime, then so are and . (Contributed by Scott Fenton, 12-Apr-2014.) (Revised by Mario Carneiro, 19-Apr-2014.) |
Theorem | sqgcd 11971 | Square distributes over gcd. (Contributed by Scott Fenton, 18-Apr-2014.) (Revised by Mario Carneiro, 19-Apr-2014.) |
Theorem | dvdssqlem 11972 | Lemma for dvdssq 11973. (Contributed by Scott Fenton, 18-Apr-2014.) (Revised by Mario Carneiro, 19-Apr-2014.) |
Theorem | dvdssq 11973 | Two numbers are divisible iff their squares are. (Contributed by Scott Fenton, 18-Apr-2014.) (Revised by Mario Carneiro, 19-Apr-2014.) |
Theorem | bezoutr 11974 | Partial converse to bezout 11953. Existence of a linear combination does not set the GCD, but it does upper bound it. (Contributed by Stefan O'Rear, 23-Sep-2014.) |
Theorem | bezoutr1 11975 | Converse of bezout 11953 for when the greater common divisor is one (sufficient condition for relative primality). (Contributed by Stefan O'Rear, 23-Sep-2014.) |
Theorem | nnmindc 11976* | An inhabited decidable subset of the natural numbers has a minimum. (Contributed by Jim Kingdon, 23-Sep-2024.) |
DECID inf | ||
Theorem | nnminle 11977* | The infimum of a decidable subset of the natural numbers is less than an element of the set. The infimum is also a minimum as shown at nnmindc 11976. (Contributed by Jim Kingdon, 26-Sep-2024.) |
DECID inf | ||
Theorem | nnwodc 11978* | Well-ordering principle: any inhabited decidable set of positive integers has a least element. Theorem I.37 (well-ordering principle) of [Apostol] p. 34. (Contributed by NM, 17-Aug-2001.) (Revised by Jim Kingdon, 23-Oct-2024.) |
DECID | ||
Theorem | uzwodc 11979* | Well-ordering principle: any inhabited decidable subset of an upper set of integers has a least element. (Contributed by NM, 8-Oct-2005.) (Revised by Jim Kingdon, 22-Oct-2024.) |
DECID | ||
Theorem | nnwofdc 11980* | Well-ordering principle: any inhabited decidable set of positive integers has a least element. This version allows and to be present in as long as they are effectively not free. (Contributed by NM, 17-Aug-2001.) (Revised by Mario Carneiro, 15-Oct-2016.) |
DECID | ||
Theorem | nnwosdc 11981* | Well-ordering principle: any inhabited decidable set of positive integers has a least element (schema form). (Contributed by NM, 17-Aug-2001.) (Revised by Jim Kingdon, 25-Oct-2024.) |
DECID | ||
Theorem | nn0seqcvgd 11982* | A strictly-decreasing nonnegative integer sequence with initial term reaches zero by the th term. Deduction version. (Contributed by Paul Chapman, 31-Mar-2011.) |
Theorem | ialgrlem1st 11983 | Lemma for ialgr0 11985. Expressing algrflemg 6206 in a form suitable for theorems such as seq3-1 10403 or seqf 10404. (Contributed by Jim Kingdon, 22-Jul-2021.) |
Theorem | ialgrlemconst 11984 | Lemma for ialgr0 11985. Closure of a constant function, in a form suitable for theorems such as seq3-1 10403 or seqf 10404. (Contributed by Jim Kingdon, 22-Jul-2021.) |
Theorem | ialgr0 11985 | The value of the algorithm iterator at is the initial state . (Contributed by Paul Chapman, 31-Mar-2011.) (Revised by Jim Kingdon, 12-Mar-2023.) |
Theorem | algrf 11986 |
An algorithm is a step function on a state space .
An algorithm acts on an initial state by
iteratively applying
to give , , and so
on. An algorithm is said to halt if a fixed point of is reached
after a finite number of iterations.
The algorithm iterator "runs" the algorithm so that is the state after iterations of on the initial state . Domain and codomain of the algorithm iterator . (Contributed by Paul Chapman, 31-Mar-2011.) (Revised by Mario Carneiro, 28-May-2014.) |
Theorem | algrp1 11987 | The value of the algorithm iterator at . (Contributed by Paul Chapman, 31-Mar-2011.) (Revised by Jim Kingdon, 12-Mar-2023.) |
Theorem | alginv 11988* | If is an invariant of , then its value is unchanged after any number of iterations of . (Contributed by Paul Chapman, 31-Mar-2011.) |
Theorem | algcvg 11989* |
One way to prove that an algorithm halts is to construct a countdown
function whose value is guaranteed to decrease for
each iteration of until it reaches . That is, if
is not a fixed point of , then
.
If is a countdown function for algorithm , the sequence reaches after at most steps, where is the value of for the initial state . (Contributed by Paul Chapman, 22-Jun-2011.) |
Theorem | algcvgblem 11990 | Lemma for algcvgb 11991. (Contributed by Paul Chapman, 31-Mar-2011.) |
Theorem | algcvgb 11991 | Two ways of expressing that is a countdown function for algorithm . The first is used in these theorems. The second states the condition more intuitively as a conjunction: if the countdown function's value is currently nonzero, it must decrease at the next step; if it has reached zero, it must remain zero at the next step. (Contributed by Paul Chapman, 31-Mar-2011.) |
Theorem | algcvga 11992* | The countdown function remains after steps. (Contributed by Paul Chapman, 22-Jun-2011.) |
Theorem | algfx 11993* | If reaches a fixed point when the countdown function reaches , remains fixed after steps. (Contributed by Paul Chapman, 22-Jun-2011.) |
Theorem | eucalgval2 11994* | The value of the step function for Euclid's Algorithm on an ordered pair. (Contributed by Paul Chapman, 31-Mar-2011.) (Revised by Mario Carneiro, 28-May-2014.) |
Theorem | eucalgval 11995* |
Euclid's Algorithm eucalg 12000 computes the greatest common divisor of two
nonnegative integers by repeatedly replacing the larger of them with its
remainder modulo the smaller until the remainder is 0.
The value of the step function for Euclid's Algorithm. (Contributed by Paul Chapman, 31-Mar-2011.) (Revised by Mario Carneiro, 28-May-2014.) |
Theorem | eucalgf 11996* | Domain and codomain of the step function for Euclid's Algorithm. (Contributed by Paul Chapman, 31-Mar-2011.) (Revised by Mario Carneiro, 28-May-2014.) |
Theorem | eucalginv 11997* | The invariant of the step function for Euclid's Algorithm is the operator applied to the state. (Contributed by Paul Chapman, 31-Mar-2011.) (Revised by Mario Carneiro, 29-May-2014.) |
Theorem | eucalglt 11998* | The second member of the state decreases with each iteration of the step function for Euclid's Algorithm. (Contributed by Paul Chapman, 31-Mar-2011.) (Revised by Mario Carneiro, 29-May-2014.) |
Theorem | eucalgcvga 11999* | Once Euclid's Algorithm halts after steps, the second element of the state remains 0 . (Contributed by Paul Chapman, 22-Jun-2011.) (Revised by Mario Carneiro, 29-May-2014.) |
Theorem | eucalg 12000* |
Euclid's Algorithm computes the greatest common divisor of two
nonnegative integers by repeatedly replacing the larger of them with its
remainder modulo the smaller until the remainder is 0. Theorem 1.15 in
[ApostolNT] p. 20.
Upon halting, the 1st member of the final state is equal to the gcd of the values comprising the input state . This is Metamath 100 proof #69 (greatest common divisor algorithm). (Contributed by Paul Chapman, 31-Mar-2011.) (Proof shortened by Mario Carneiro, 29-May-2014.) |
< Previous Next > |
Copyright terms: Public domain | < Previous Next > |