Let a , b , c be three positive integers such that:
( lcm ( a , b ) ) ( lcm ( b , c ) ) ( lcm ( c , a ) ) = ( a b c ) g cd ( a , b , c ) ,
where “lcm” means “least common multiple” and “gcd” means “greatest common divisor.”
Given that no quotient of any two of a , b , c is an integer (that is, none of a , b , c is an integer multiple of any other of a , b , c ) , . find the minimum possible value of a + b + c .
This section requires Javascript.
You are seeing this because something didn't load right. We suggest you, (a) try
refreshing the page, (b) enabling javascript if it is disabled on your browser and,
finally, (c)
loading the
non-javascript version of this page
. We're sorry about the hassle.
Thank you.
Log in to reply
You're welcome. just shared some thoughts, as always. Not a real proof though
Any solution or thought is always welcomed, no worries.
let p be any prime, and suppose p r , p s , p t are the maximum prime powers that are factors of a , b , c respectively. Suppose r ≤ s ≤ t and isolating the powers of p yields:
( p s ) ( p t ) ( p t ) = ( p r + s + t ) ( p r ) ⟹ s + 2 t = 2 r + s + t ⟹ t = 2 r
Therefore, for any prime that appears as a factor in a , b , c , the greatest exponent of that prime (in a , b , or c ) must be exactly twice the exponent of that same prime in a , b , or c . In particular, if any prime divides one of a , b , and c , then it must divide all of them. We can't have a , b , or c all be a power of the same prime, since then clearly the smallest one would divide the largest one.
case 1 : Suppose that each of a , b , c are divisible by exactly two primes namely p and q .
We can not have one of a , b , c have the largest power of both primes simultaneously, since otherwise the other two numbers would divide it. So without loss of generosity, suppose that a has the largest power of p and b has the largest power of q . Since c does not divide a or b , we must have c has a higher power of q than a and a higher power of p than b . In other words, we can not have a = p 2 q and b = p q 2 which would imply that c = p 2 q 2 ⟹ a ∣ c and b ∣ c . The next smallest possibility is:
a = p 4 q 2 , b = p 2 q 4 , and c = p 3 q 3 . Plugging in the smallest possible primes p = 2 and q = 3 ⟹ a = 2 4 3 2 = 1 4 4 , b = 2 2 3 4 = 3 2 4 , c = 2 3 3 3 = 2 1 6 . The sum of a + b + c = 6 8 4 . This is the smallest possible sum with two primes.
case 2 : Now suppose that each of a , b , c are divisible by exactly three primes p , q , and r ⟹ a = p 2 q r , b = p q 2 r and c = p q r 2 . That is the smallest possibility that for each prime, two of the numbers are divisible by the prime and the third is divisible by the prime squared. Plugging in the smallest primes p = 2 , q = 3 , and r = 5 ⟹ a = 2 2 . 3 . 5 = 6 0 , b = 2 . 3 2 . 5 = 9 0 , c = 2 . 3 . 5 2 = 1 5 0 , giving a sum of a + b + c = 6 0 + 9 0 + 1 5 0 = 3 0 0 , indicating the smallest sum so far.
case 3 : If there are 4 or more primes, then each number must be at least 2 . 3 . 5 . 7 = 2 1 0 , so the sum must at least 630, which is larger than 300.
Thus, the smallest possible sum is 3 0 0 .
Problem Loading...
Note Loading...
Set Loading...
Note the notations [ a , b ] = l c m ( a , b ) and ( a , b ) = g c d ( a , b ) .
Using the relation [ a , b ] ( a , b ) = a . b one can re-write the equality, in the question, as below.
[ a , b ] [ b , c ] [ a , c ] = ( a , b ) ( b , c ) ( a , c ) a 2 b 2 c 2 = a b c ( a , b , c ) ⟹
a b c = ( a , b ) ( b , c ) ( a , c ) ( a , b , c ) ( ∗ )
Few facts (not hard to prove):
1- a , b , c = 0 , 1 , because non of them should divide the other one
2- a = b = c
We know that ( a , b , c ) = 1 , because, if a < b < c , then the RHS of ∗ would be a . b at most, which forces c to be 1 . Therefore ( a , b , c ) = t = 1 .
Also, one can notice that, given ( a , b ) = d and a = a ′ d , b = b ′ d and ( a ′ , b ′ ) = 1 , a ′ ∣ ( a , c ) ⟹ a ′ ∣ c . In a similar manner, b ′ ∣ c . Therefore, a ′ b ′ ∣ c and, by symmetry, we conclude that the parts of any of two integers x , y ∈ { a , b , c } , x = y , that are not included in ( x , y ) , should be included in z ∈ { a , b , c } z = x , z = y .
The first structure, that comes to mind, for the integers is a = p q t , b = p r t , c = r q t , such that p , q , r are pairwise coprimes. if we substitute in ∗ , we get
p q r = t
Hence, a = p 2 q 2 r , b = p 2 q r 2 , c = p q 2 r 2 . However, it is possible to come with yet better structure that leads to smaller integers: the following structure a = p 2 q r = p t , b = p q 2 r = q t , c = p q r 2 = r t , where t = p q r , such that what is discussed till this point is satisfied. So, we have a + b + c = p q r ( p + q + r ) We just need to take p , q , r to be the lowest possible, mutually coprime, positive integers ( p = 2 , q = 3 , r = 5 ).