diff --git "a/putnam_solving_format_unified.jsonl" "b/putnam_solving_format_unified.jsonl" --- "a/putnam_solving_format_unified.jsonl" +++ "b/putnam_solving_format_unified.jsonl" @@ -1,5 +1,5 @@ {"informal_problem": "Find every real-valued function $f$ whose domain is an interval $I$ (finite or infinite) having 0 as a left-hand endpoint, such that for every positive member $x$ of $I$ the average of $f$ over the closed interval $[0, x]$ is equal to the geometric mean of the numbers $f(0)$ and $f(x)$.", "informal_answer": "the set of functions $f(x) = \\frac{a}{(1 - c x)^2}$ where $a \\geq 0$", "informal_solution": "Show that \\[ f(x) = \\frac{a}{(1 - cx)^2} \\begin{cases} \\text{for } 0 \\le x < \\frac{1}{c}, & \\text{if } c > 0\\\\ \\text{for } 0 \\le x < \\infty, & \\text{if } c \\le 0, \\end{cases} \\] where $a > 0$.", "header": "open MeasureTheory Set", "intros": [], "formal_answer": "@Eq (Set (Real → Real)) answer\n (@setOf (Real → Real) fun (f : Real → Real) =>\n @Exists Real fun (a : Real) =>\n @Exists Real fun (c : Real) =>\n And (@GE.ge Real Real.instLE a (@OfNat.ofNat Real (nat_lit 0) (@Zero.toOfNat0 Real Real.instZero)))\n (@Eq (Real → Real) f fun (x : Real) =>\n @HDiv.hDiv Real Real Real (@instHDiv Real (@DivInvMonoid.toDiv Real Real.instDivInvMonoid)) a\n (@HPow.hPow Real Nat Real (@instHPow Real Nat (@Monoid.toNatPow Real Real.instMonoid))\n (@HSub.hSub Real Real Real (@instHSub Real Real.instSub)\n (@OfNat.ofNat Real (nat_lit 1) (@One.toOfNat1 Real Real.instOne))\n (@HMul.hMul Real Real Real (@instHMul Real Real.instMul) c x))\n (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))))))", "formal_answer_type": "Set (ℝ → ℝ)", "outros": [{"t": "Set ℝ → (ℝ → ℝ) → Prop", "v": null, "name": "P"}, {"t": "∀ s f, P s f ↔ 0 ≤ f ∧ ∀ x ∈ s, ⨍ t in Ico 0 x, f t = √(f 0 * f x)", "v": null, "name": "P_def"}, {"t": "answer = {f : ℝ → ℝ | P (Ioi 0) f ∨ (∃ e > 0, P (Ioo 0 e) f)}", "v": null, "name": "h_answer"}]} -{"informal_problem": "Evaluate in closed form \\[ \\sum_{k=1}^n {n \\choose k} k^2. \\]", "informal_answer": "$n(n+1)2^{n-2}$", "informal_solution": "Show that the expression equals $n(n+1)2^{n-2}$.", "header": null, "intros": [], "formal_answer": "@Eq (Nat → Nat) answer fun (n_1 : Nat) =>\n @HMul.hMul Nat Nat Nat (@instHMul Nat instMulNat)\n (@HMul.hMul Nat Nat Nat (@instHMul Nat instMulNat) n_1\n (@HAdd.hAdd Nat Nat Nat (@instHAdd Nat instAddNat) n_1 (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1)))))\n (@HPow.hPow Nat Nat Nat (@instHPow Nat Nat (@Monoid.toNatPow Nat Nat.instMonoid))\n (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))\n (@HSub.hSub Nat Nat Nat (@instHSub Nat instSubNat) n_1 (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))))", "formal_answer_type": "ℕ → ℕ", "outros": [{"t": "ℕ", "v": null, "name": "n"}, {"t": "n ≥ 2", "v": null, "name": "hn"}, {"t": "answer n = ∑ k in Finset.Icc 1 n, Nat.choose n k * k^2", "v": null, "name": "h_answer"}]} +{"informal_problem": "Evaluate in closed form \\[ \\sum_{k=1}^n {n \\choose k} k^2. \\]", "informal_answer": "$n(n+1)2^{n-2}$", "informal_solution": "Show that the expression equals $n(n+1)2^{n-2}$.", "header": "open BigOperators Real Nat Topology", "intros": [], "formal_answer": "@Eq (Nat → Nat) answer fun (n_1 : Nat) =>\n @HMul.hMul Nat Nat Nat (@instHMul Nat instMulNat)\n (@HMul.hMul Nat Nat Nat (@instHMul Nat instMulNat) n_1\n (@HAdd.hAdd Nat Nat Nat (@instHAdd Nat instAddNat) n_1 (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1)))))\n (@HPow.hPow Nat Nat Nat (@instHPow Nat Nat (@Monoid.toNatPow Nat Nat.instMonoid))\n (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))\n (@HSub.hSub Nat Nat Nat (@instHSub Nat instSubNat) n_1 (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))))", "formal_answer_type": "ℕ → ℕ", "outros": [{"t": "ℕ", "v": null, "name": "n"}, {"t": "n ≥ 2", "v": null, "name": "hn"}, {"t": "answer n = ∑ k in Finset.Icc 1 n, Nat.choose n k * k^2", "v": null, "name": "h_answer"}]} {"informal_problem": "Find an integral formula (i.e., a function $z$ such that $y(x) = \\int_{1}^{x} z(t) dt$) for the solution of the differential equation $$\\delta (\\delta - 1) (\\delta - 2) \\cdots (\\delta - n + 1) y = f(x)$$ with the initial conditions $y(1) = y'(1) = \\cdots = y^{(n-1)}(1) = 0$, where $n \\in \\mathbb{N}$, $f$ is continuous for all $x \\ge 1$, and $\\delta$ denotes $x\\frac{d}{dx}$.", "informal_answer": "$(x - t)^{n-1} \\cdot f(t) / ((n-1)! \\cdot t^n)$", "informal_solution": "Show that the solution is $$y(x) = \\int_{1}^{x} \\frac{(x - t)^{n - 1} f(t)}{(n - 1)!t^n} dt$$.", "header": "open Nat Set Topology Filter", "intros": [], "formal_answer": "@Eq ((Real → Real) → Nat → Real → Real → Real) answer fun (f_1 : Real → Real) (n_1 : Nat) (x t : Real) =>\n @HDiv.hDiv Real Real Real (@instHDiv Real (@DivInvMonoid.toDiv Real Real.instDivInvMonoid))\n (@HMul.hMul Real Real Real (@instHMul Real Real.instMul)\n (@HPow.hPow Real Nat Real (@instHPow Real Nat (@Monoid.toNatPow Real Real.instMonoid))\n (@HSub.hSub Real Real Real (@instHSub Real Real.instSub) x t)\n (@HSub.hSub Nat Nat Nat (@instHSub Nat instSubNat) n_1\n (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1)))))\n (f_1 t))\n (@HMul.hMul Real Real Real (@instHMul Real Real.instMul)\n (@Nat.cast Real Real.instNatCast\n (Nat.factorial\n (@HSub.hSub Nat Nat Nat (@instHSub Nat instSubNat) n_1\n (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1))))))\n (@HPow.hPow Real Nat Real (@instHPow Real Nat (@Monoid.toNatPow Real Real.instMonoid)) t n_1))", "formal_answer_type": "(ℝ → ℝ) → ℕ → ℝ → ℝ → ℝ", "outros": [{"t": "ℕ → (ℝ → ℝ) → (ℝ → ℝ)", "v": null, "name": "P"}, {"t": "P 0 = id ∧ ∀ i y, P (i + 1) y = P i (fun x ↦ x * deriv y x - i * y x)", "v": null, "name": "hP"}, {"t": "ℕ", "v": null, "name": "n"}, {"t": "0 < n", "v": null, "name": "hn"}, {"t": "ℝ → ℝ", "v": null, "name": "f"}, {"t": "ℝ → ℝ", "v": null, "name": "y"}, {"t": "ContinuousOn f (Ici 1)", "v": null, "name": "hf"}, {"t": "ContDiffOn ℝ n y (Ici 1)", "v": null, "name": "hy"}, {"t": "∀ x ≥ 1, y x = ∫ t in (1 : ℝ)..x, answer f n x t", "v": null, "name": "h_answer"}]} {"informal_problem": "For what integer $a$ does $x^2-x+a$ divide $x^{13}+x+90$?", "informal_answer": "2", "informal_solution": "Show that $a=2$.", "header": "open Topology Filter Polynomial", "intros": [], "formal_answer": "@Eq Int answer (@OfNat.ofNat Int (nat_lit 2) (@instOfNat (nat_lit 2)))", "formal_answer_type": "ℤ", "outros": [{"t": "ℤ", "v": null, "name": "a"}, {"t": "Polynomial.X^2 - Polynomial.X + (Polynomial.C a) ∣ (Polynomial.X ^ 13 + Polynomial.X + (Polynomial.C 90))", "v": null, "name": "h_div"}, {"t": "answer = a", "v": null, "name": "h_answer"}]} {"informal_problem": "Let $S$ be the set of all numbers of the form $2^m3^n$, where $m$ and $n$ are integers, and let $P$ be the set of all positive real numbers. Is $S$ dense in $P$?", "informal_answer": "True", "informal_solution": "Show that $S$ is dense in $P$.", "header": "open Topology Filter Polynomial", "intros": [], "formal_answer": "@Eq Prop answer True", "formal_answer_type": "Prop", "outros": [{"t": "Set ℝ", "v": null, "name": "S"}, {"t": "S = {2 ^ m * 3 ^ n | (m : ℤ) (n : ℤ)}", "v": null, "name": "hS"}, {"t": "answer = (closure S ⊇ Set.Ioi (0 : ℝ))", "v": null, "name": "h_answer"}]} @@ -37,14 +37,14 @@ {"informal_problem": "Let $H$ be a subgroup of the additive group of ordered pairs of integers under componentwise addition. If $H$ is generated by the elements $(3, 8)$, $(4, -1)$, and $(5, 4)$, then $H$ is also generated by two elements $(1, b)$ and $(0, a)$ for some integer $b$ and positive integer $a$. Find $a$.", "informal_answer": "7", "informal_solution": "$a$ must equal $7$.", "header": "open Polynomial Real Complex", "intros": [], "formal_answer": "@Eq Int answer (@OfNat.ofNat Int (nat_lit 7) (@instOfNat (nat_lit 7)))", "formal_answer_type": "ℤ", "outros": [{"t": "Set (ℤ × ℤ)", "v": null, "name": "H"}, {"t": "H = {h : (ℤ × ℤ) | ∃ u v w : ℤ, h = (u*3 + v*4 + w*5, u*8 + v*(-1) + w*4)}", "v": null, "name": "hH"}, {"t": "(∃ b : ℤ, H = {h : (ℤ × ℤ) | ∃ u v : ℤ, h = (u, u*b + v*answer)}) ∧ answer > 0", "v": null, "name": "h_answer"}]} {"informal_problem": "Let $s_k (a_1, a_2, \\dots, a_n)$ denote the $k$-th elementary symmetric function; that is, the sum of all $k$-fold products of the $a_i$. For example, $s_1 (a_1, \\dots, a_n) = \\sum_{i=1}^{n} a_i$, and $s_2 (a_1, a_2, a_3) = a_1a_2 + a_2a_3 + a_1a_3$. Find the supremum $M_k$ (which is never attained) of $$\\frac{s_k (a_1, a_2, \\dots, a_n)}{(s_1 (a_1, a_2, \\dots, a_n))^k}$$ across all $n$-tuples $(a_1, a_2, \\dots, a_n)$ of positive real numbers with $n \\ge k$.", "informal_answer": "fun k : ℕ => (1: ℝ)/(Nat.factorial k)", "informal_solution": "The supremum $M_k$ is $\\frac{1}{k!}$.", "header": "open Polynomial Real Complex Matrix Filter Topology Multiset", "intros": [], "formal_answer": "@Eq (Nat → Real) answer fun (k : Nat) =>\n @HDiv.hDiv Real Real Real (@instHDiv Real (@DivInvMonoid.toDiv Real Real.instDivInvMonoid))\n (@OfNat.ofNat Real (nat_lit 1) (@One.toOfNat1 Real Real.instOne))\n (@Nat.cast Real Real.instNatCast (Nat.factorial k))", "formal_answer_type": "ℕ → ℝ", "outros": [{"t": "∀ k : ℕ, k > 0 → (∀ a : Multiset ℝ, (∀ i ∈ a, i > 0) ∧ card a ≥ k →\n(esymm a k)/(esymm a 1)^k ≤ answer k) ∧\n∀ M : ℝ, M < answer k → (∃ a : Multiset ℝ, (∀ i ∈ a, i > 0) ∧ card a ≥ k ∧\n(esymm a k)/(esymm a 1)^k > M)", "v": null, "name": "h_answer"}]} {"informal_problem": "Let $C = \\{(x, y) \\in \\mathbb{R}^2 : x^2 + y^2 = 1\\}$ denote the unit circle. Does there exist $B \\subseteq C$ for which $B$ is topologically closed and contains exactly one point from each pair of diametrically opposite points in $C$?", "informal_answer": "False", "informal_solution": "Such $B$ does not exist.", "header": "open Polynomial Real Complex Matrix Filter Topology Multiset", "intros": [], "formal_answer": "@Eq Prop answer False", "formal_answer_type": "Prop", "outros": [{"t": "ℝ × ℝ → Prop", "v": null, "name": "P"}, {"t": "P = fun (x, y) => x^2 + y^2 = 1", "v": null, "name": "hP"}, {"t": "(∃ B ⊆ setOf P, IsClosed B ∧ ∀ x y : ℝ, P (x, y) → Xor' ((x, y) ∈ B) ((-x, -y) ∈ B)) ↔ answer", "v": null, "name": "h_answer"}]} -{"informal_problem": "Find all integer solutions $(p, r, q, s)$ of the equation $|p^r - q^s| = 1$, where $p$ and $q$ are prime and $r$ and $s$ are greater than $1$.", "informal_answer": "{(3, 2, 2, 3), (2, 3, 3, 2)}", "informal_solution": "The only solutions are $(p, r, q, s) = (3, 2, 2, 3)$ and $(p, r, q, s) = (2, 3, 3, 2)$.", "header": null, "intros": [], "formal_answer": "@Eq (Set (Prod Nat (Prod Nat (Prod Nat Nat)))) answer\n (@Insert.insert (Prod Nat (Prod Nat (Prod Nat Nat))) (Set (Prod Nat (Prod Nat (Prod Nat Nat))))\n (@Set.instInsert (Prod Nat (Prod Nat (Prod Nat Nat))))\n (@Prod.mk Nat (Prod Nat (Prod Nat Nat)) (@OfNat.ofNat Nat (nat_lit 3) (instOfNatNat (nat_lit 3)))\n (@Prod.mk Nat (Prod Nat Nat) (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))\n (@Prod.mk Nat Nat (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))\n (@OfNat.ofNat Nat (nat_lit 3) (instOfNatNat (nat_lit 3))))))\n (@Singleton.singleton (Prod Nat (Prod Nat (Prod Nat Nat))) (Set (Prod Nat (Prod Nat (Prod Nat Nat))))\n (@Set.instSingletonSet (Prod Nat (Prod Nat (Prod Nat Nat))))\n (@Prod.mk Nat (Prod Nat (Prod Nat Nat)) (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))\n (@Prod.mk Nat (Prod Nat Nat) (@OfNat.ofNat Nat (nat_lit 3) (instOfNatNat (nat_lit 3)))\n (@Prod.mk Nat Nat (@OfNat.ofNat Nat (nat_lit 3) (instOfNatNat (nat_lit 3)))\n (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))))))))", "formal_answer_type": "Set (ℕ × ℕ × ℕ × ℕ)", "outros": [{"t": "{a : ℕ × ℕ × ℕ × ℕ | Nat.Prime a.1 ∧ Nat.Prime a.2.2.1 ∧ a.2.1 > 1 ∧ a.2.2.2 > 1 ∧ |(a.1^a.2.1 : ℤ) - a.2.2.1^a.2.2.2| = 1} = answer", "v": null, "name": "h_answer"}]} +{"informal_problem": "Find all integer solutions $(p, r, q, s)$ of the equation $|p^r - q^s| = 1$, where $p$ and $q$ are prime and $r$ and $s$ are greater than $1$.", "informal_answer": "{(3, 2, 2, 3), (2, 3, 3, 2)}", "informal_solution": "The only solutions are $(p, r, q, s) = (3, 2, 2, 3)$ and $(p, r, q, s) = (2, 3, 3, 2)$.", "header": "open BigOperators Real Nat Topology", "intros": [], "formal_answer": "@Eq (Set (Prod Nat (Prod Nat (Prod Nat Nat)))) answer\n (@Insert.insert (Prod Nat (Prod Nat (Prod Nat Nat))) (Set (Prod Nat (Prod Nat (Prod Nat Nat))))\n (@Set.instInsert (Prod Nat (Prod Nat (Prod Nat Nat))))\n (@Prod.mk Nat (Prod Nat (Prod Nat Nat)) (@OfNat.ofNat Nat (nat_lit 3) (instOfNatNat (nat_lit 3)))\n (@Prod.mk Nat (Prod Nat Nat) (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))\n (@Prod.mk Nat Nat (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))\n (@OfNat.ofNat Nat (nat_lit 3) (instOfNatNat (nat_lit 3))))))\n (@Singleton.singleton (Prod Nat (Prod Nat (Prod Nat Nat))) (Set (Prod Nat (Prod Nat (Prod Nat Nat))))\n (@Set.instSingletonSet (Prod Nat (Prod Nat (Prod Nat Nat))))\n (@Prod.mk Nat (Prod Nat (Prod Nat Nat)) (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))\n (@Prod.mk Nat (Prod Nat Nat) (@OfNat.ofNat Nat (nat_lit 3) (instOfNatNat (nat_lit 3)))\n (@Prod.mk Nat Nat (@OfNat.ofNat Nat (nat_lit 3) (instOfNatNat (nat_lit 3)))\n (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))))))))", "formal_answer_type": "Set (ℕ × ℕ × ℕ × ℕ)", "outros": [{"t": "{a : ℕ × ℕ × ℕ × ℕ | Nat.Prime a.1 ∧ Nat.Prime a.2.2.1 ∧ a.2.1 > 1 ∧ a.2.2.2 > 1 ∧ |(a.1^a.2.1 : ℤ) - a.2.2.1^a.2.2.2| = 1} = answer", "v": null, "name": "h_answer"}]} {"informal_problem": "Let $r$ be a real root of $P(x) = x^3 + ax^2 + bx - 1$, where $a$ and $b$ are integers and $P$ is irreducible over the rationals. Suppose that $r + 1$ is a root of $x^3 + cx^2 + dx + 1$, where $c$ and $d$ are also integers. Express another root $s$ of $P$ as a function of $r$ that does not depend on the values of $a$, $b$, $c$, or $d$.", "informal_answer": "$\\left(-\\frac{1}{r + 1}, -\\frac{r + 1}{r}\\right)$", "informal_solution": "The possible answers are $s = -\\frac{1}{r + 1}$ and $s = -\\frac{r + 1}{r}$.", "header": "open Polynomial", "intros": [], "formal_answer": "@Eq (Prod (Real → Real) (Real → Real)) answer\n (@Prod.mk (Real → Real) (Real → Real)\n (fun (r_1 : Real) =>\n @HDiv.hDiv Real Real Real (@instHDiv Real (@DivInvMonoid.toDiv Real Real.instDivInvMonoid))\n (@Neg.neg Real Real.instNeg (@OfNat.ofNat Real (nat_lit 1) (@One.toOfNat1 Real Real.instOne)))\n (@HAdd.hAdd Real Real Real (@instHAdd Real Real.instAdd) r_1\n (@OfNat.ofNat Real (nat_lit 1) (@One.toOfNat1 Real Real.instOne))))\n fun (r_1 : Real) =>\n @HDiv.hDiv Real Real Real (@instHDiv Real (@DivInvMonoid.toDiv Real Real.instDivInvMonoid))\n (@Neg.neg Real Real.instNeg\n (@HAdd.hAdd Real Real Real (@instHAdd Real Real.instAdd) r_1\n (@OfNat.ofNat Real (nat_lit 1) (@One.toOfNat1 Real Real.instOne))))\n r_1)", "formal_answer_type": "(ℝ → ℝ) × (ℝ → ℝ)", "outros": [{"t": "ℤ", "v": null, "name": "a"}, {"t": "ℤ", "v": null, "name": "b"}, {"t": "ℤ", "v": null, "name": "c"}, {"t": "ℤ", "v": null, "name": "d"}, {"t": "ℝ", "v": null, "name": "r"}, {"t": "Polynomial ℚ", "v": null, "name": "P"}, {"t": "Polynomial ℚ", "v": null, "name": "Q"}, {"t": "P = Polynomial.X^3 + (Polynomial.C (a : ℚ))*Polynomial.X^2 + (Polynomial.C (b : ℚ))*Polynomial.X - (Polynomial.C 1) ∧ Polynomial.aeval r P = 0 ∧ Irreducible P", "v": null, "name": "hP"}, {"t": "Q = Polynomial.X^3 + (Polynomial.C (c : ℚ))*Polynomial.X^2 + (Polynomial.C (d : ℚ))*Polynomial.X + (Polynomial.C 1) ∧ Polynomial.aeval (r + 1) Q = 0", "v": null, "name": "hQ"}, {"t": "∃ s : ℝ, Polynomial.aeval s P = 0 ∧ (s = answer.1 r ∨ s = answer.2 r)", "v": null, "name": "h_answer"}]} {"informal_problem": "Find $$\\lim_{n \\to \\infty} \\frac{1}{n} \\sum_{k=1}^{n}\\left(\\left\\lfloor \\frac{2n}{k} \\right\\rfloor - 2\\left\\lfloor \\frac{n}{k} \\right\\rfloor\\right).$$ Your answer should be in the form $\\ln(a) - b$, where $a$ and $b$ are positive integers.", "informal_answer": "ln(4) - 1", "informal_solution": "The limit equals $\\ln(4) - 1$, so $a = 4$ and $b = 1$.", "header": "open Polynomial Filter Topology", "intros": [], "formal_answer": "@Eq (Prod Nat Nat) answer\n (@Prod.mk Nat Nat (@OfNat.ofNat Nat (nat_lit 4) (instOfNatNat (nat_lit 4)))\n (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1))))", "formal_answer_type": "ℕ × ℕ", "outros": [{"t": "Tendsto (fun n : ℕ => ((1 : ℝ)/n)*∑ k in Finset.Icc (1 : ℤ) n, (Int.floor ((2*n)/k) - 2*Int.floor (n/k))) atTop\n (𝓝 (Real.log answer.1 - answer.2))", "v": null, "name": "h_answer"}]} {"informal_problem": "Let $G$ be a group generated by two elements $A$ and $B$; i.e., every element of $G$ can be expressed as a finite word $A^{n_1}B^{n_2} \\cdots A^{n_{k-1}}B^{n_k}$, where the $n_i$ can assume any integer values and $A^0 = B^0 = 1$. Further assume that $A^4 = B^7 = ABA^{-1}B = 1$, but $A^2 \\ne 1$ and $B \\ne 1$. Find the number of elements of $G$ than can be written as $C^2$ for some $C \\in G$ and express each such square as a word in $A$ and $B$.", "informal_answer": "(8, {[(0, 0)], [(2, 0)], [(0, 1)], [(0, 2)], [(0, 3)], [(0, 4)], [(0, 5)], [(0, 6)]})", "informal_solution": "There are $8$ such squares: $1$, $A^2$, $B$, $B^2$, $B^3$, $B^4$, $B^5$, and $B^6$.", "header": "open Polynomial Filter Topology", "intros": [], "formal_answer": "@Eq (Prod Nat (Set (List (Prod Int Int)))) answer\n (@Prod.mk Nat (Set (List (Prod Int Int))) (@OfNat.ofNat Nat (nat_lit 8) (instOfNatNat (nat_lit 8)))\n (@Insert.insert (List (Prod Int Int)) (Set (List (Prod Int Int))) (@Set.instInsert (List (Prod Int Int)))\n (@List.cons (Prod Int Int)\n (@Prod.mk Int Int (@OfNat.ofNat Int (nat_lit 0) (@instOfNat (nat_lit 0)))\n (@OfNat.ofNat Int (nat_lit 0) (@instOfNat (nat_lit 0))))\n (@List.nil (Prod Int Int)))\n (@Insert.insert (List (Prod Int Int)) (Set (List (Prod Int Int))) (@Set.instInsert (List (Prod Int Int)))\n (@List.cons (Prod Int Int)\n (@Prod.mk Int Int (@OfNat.ofNat Int (nat_lit 2) (@instOfNat (nat_lit 2)))\n (@OfNat.ofNat Int (nat_lit 0) (@instOfNat (nat_lit 0))))\n (@List.nil (Prod Int Int)))\n (@Insert.insert (List (Prod Int Int)) (Set (List (Prod Int Int))) (@Set.instInsert (List (Prod Int Int)))\n (@List.cons (Prod Int Int)\n (@Prod.mk Int Int (@OfNat.ofNat Int (nat_lit 0) (@instOfNat (nat_lit 0)))\n (@OfNat.ofNat Int (nat_lit 1) (@instOfNat (nat_lit 1))))\n (@List.nil (Prod Int Int)))\n (@Insert.insert (List (Prod Int Int)) (Set (List (Prod Int Int))) (@Set.instInsert (List (Prod Int Int)))\n (@List.cons (Prod Int Int)\n (@Prod.mk Int Int (@OfNat.ofNat Int (nat_lit 0) (@instOfNat (nat_lit 0)))\n (@OfNat.ofNat Int (nat_lit 2) (@instOfNat (nat_lit 2))))\n (@List.nil (Prod Int Int)))\n (@Insert.insert (List (Prod Int Int)) (Set (List (Prod Int Int))) (@Set.instInsert (List (Prod Int Int)))\n (@List.cons (Prod Int Int)\n (@Prod.mk Int Int (@OfNat.ofNat Int (nat_lit 0) (@instOfNat (nat_lit 0)))\n (@OfNat.ofNat Int (nat_lit 3) (@instOfNat (nat_lit 3))))\n (@List.nil (Prod Int Int)))\n (@Insert.insert (List (Prod Int Int)) (Set (List (Prod Int Int))) (@Set.instInsert (List (Prod Int Int)))\n (@List.cons (Prod Int Int)\n (@Prod.mk Int Int (@OfNat.ofNat Int (nat_lit 0) (@instOfNat (nat_lit 0)))\n (@OfNat.ofNat Int (nat_lit 4) (@instOfNat (nat_lit 4))))\n (@List.nil (Prod Int Int)))\n (@Insert.insert (List (Prod Int Int)) (Set (List (Prod Int Int)))\n (@Set.instInsert (List (Prod Int Int)))\n (@List.cons (Prod Int Int)\n (@Prod.mk Int Int (@OfNat.ofNat Int (nat_lit 0) (@instOfNat (nat_lit 0)))\n (@OfNat.ofNat Int (nat_lit 5) (@instOfNat (nat_lit 5))))\n (@List.nil (Prod Int Int)))\n (@Singleton.singleton (List (Prod Int Int)) (Set (List (Prod Int Int)))\n (@Set.instSingletonSet (List (Prod Int Int)))\n (@List.cons (Prod Int Int)\n (@Prod.mk Int Int (@OfNat.ofNat Int (nat_lit 0) (@instOfNat (nat_lit 0)))\n (@OfNat.ofNat Int (nat_lit 6) (@instOfNat (nat_lit 6))))\n (@List.nil (Prod Int Int))))))))))))", "formal_answer_type": "ℕ × Set (List (ℤ × ℤ))", "outros": [{"t": "Type*", "v": null, "name": "G"}, {"t": "Group G", "v": null, "name": null}, {"t": "G", "v": null, "name": "A"}, {"t": "G", "v": null, "name": "B"}, {"t": "List (ℤ × ℤ) → G", "v": null, "name": "word"}, {"t": "word = fun w : List (ℤ × ℤ) => (List.map (fun t : ℤ × ℤ => A^(t.1)*B^(t.2)) w).prod", "v": null, "name": "hword"}, {"t": "∀ g : G, ∃ w : List (ℤ × ℤ), g = word w", "v": null, "name": "hG"}, {"t": "A^4 = 1 ∧ A^2 ≠ 1", "v": null, "name": "hA"}, {"t": "B^7 = 1 ∧ B ≠ 1", "v": null, "name": "hB"}, {"t": "A*B*A^(-(1 : ℤ))*B = 1", "v": null, "name": "h1"}, {"t": "Set G", "v": null, "name": "S"}, {"t": "S = {g : G | ∃ C : G, C^2 = g}", "v": null, "name": "hS"}, {"t": "S.ncard = answer.1 ∧ S = {word w | w ∈ answer.2}", "v": null, "name": "h_answer"}]} {"informal_problem": "Find $$\\sum_{k=0}^{n} (-1)^k {n \\choose k} (x - k)^n.$$", "informal_answer": "fun n => C (Nat.factorial n)", "informal_solution": "The sum equals $n!$.", "header": "open Polynomial Filter Topology ProbabilityTheory MeasureTheory", "intros": [], "formal_answer": "@Eq (Nat → @Polynomial Int Int.instSemiring) answer fun (n : Nat) =>\n @DFunLike.coe\n (@RingHom Int (@Polynomial Int Int.instSemiring) (@Semiring.toNonAssocSemiring Int Int.instSemiring)\n (@Semiring.toNonAssocSemiring (@Polynomial Int Int.instSemiring) (@Polynomial.semiring Int Int.instSemiring)))\n Int (fun (x : Int) => @Polynomial Int Int.instSemiring)\n (@RingHom.instFunLike Int (@Polynomial Int Int.instSemiring) (@Semiring.toNonAssocSemiring Int Int.instSemiring)\n (@Semiring.toNonAssocSemiring (@Polynomial Int Int.instSemiring) (@Polynomial.semiring Int Int.instSemiring)))\n (@Polynomial.C Int Int.instSemiring) (@Nat.cast Int instNatCastInt (Nat.factorial n))", "formal_answer_type": "ℕ → Polynomial ℤ", "outros": [{"t": "∀ n : ℕ, ∑ k in Finset.range (n + 1), C ((-(1 : ℤ))^k * Nat.choose n k) * (X - (C (k : ℤ)))^n = answer n", "v": null, "name": "h_answer"}]} -{"informal_problem": "Show that if four distinct points of the curve $y = 2x^4 + 7x^3 + 3x - 5$ are collinear, then their average $x$-coordinate is some constant $k$. Find $k$.", "informal_answer": "$-7/8$", "informal_solution": "Prove that $k = -\\frac{7}{8}$.", "header": null, "intros": [], "formal_answer": "@Eq Real answer\n (@HDiv.hDiv Real Real Real (@instHDiv Real (@DivInvMonoid.toDiv Real Real.instDivInvMonoid))\n (@Neg.neg Real Real.instNeg\n (@OfNat.ofNat Real (nat_lit 7)\n (@instOfNatAtLeastTwo Real (nat_lit 7) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 5) (instOfNatNat (nat_lit 5)))))))\n (@OfNat.ofNat Real (nat_lit 8)\n (@instOfNatAtLeastTwo Real (nat_lit 8) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 6) (instOfNatNat (nat_lit 6)))))))", "formal_answer_type": "ℝ", "outros": [{"t": "ℝ → ℝ", "v": null, "name": "y"}, {"t": "y = fun x ↦ 2 * x ^ 4 + 7 * x ^ 3 + 3 * x - 5", "v": null, "name": "hy"}, {"t": "Finset ℝ", "v": null, "name": "S"}, {"t": "S.card = 4", "v": null, "name": "hS"}, {"t": "Collinear ℝ {P : Fin 2 → ℝ | P 0 ∈ S ∧ P 1 = y (P 0)}", "v": null, "name": "h_collinear"}, {"t": "(∑ x in S, x) / 4 = answer", "v": null, "name": "h_answer"}]} -{"informal_problem": "Find all real solutions $(a, b, c, d)$ to the equations $a + b + c = d$, $\\frac{1}{a} + \\frac{1}{b} + \\frac{1}{c} = \\frac{1}{d}$.", "informal_answer": "$d = a \\land b = -c \\lor d = b \\land a = -c \\lor d = c \\land a = -b$", "informal_solution": "Prove that the solutions are $d = a$ and $b = -c$, $d = b$ and $a = -c$, or $d = c$ and $a = -b$, with $a, b, c, d$ nonzero.", "header": null, "intros": [], "formal_answer": "@Eq (Real → Real → Real → Real → Prop) answer fun (a_1 b_1 c_1 d_1 : Real) =>\n Or (And (@Eq Real d_1 a_1) (@Eq Real b_1 (@Neg.neg Real Real.instNeg c_1)))\n (Or (And (@Eq Real d_1 b_1) (@Eq Real a_1 (@Neg.neg Real Real.instNeg c_1)))\n (And (@Eq Real d_1 c_1) (@Eq Real a_1 (@Neg.neg Real Real.instNeg b_1))))", "formal_answer_type": "ℝ → ℝ → ℝ → ℝ → Prop", "outros": [{"t": "ℝ", "v": null, "name": "a"}, {"t": "ℝ", "v": null, "name": "b"}, {"t": "ℝ", "v": null, "name": "c"}, {"t": "ℝ", "v": null, "name": "d"}, {"t": "answer a b c d ↔\n a ≠ 0 → b ≠ 0 → c ≠ 0 → d ≠ 0 → (a + b + c = d ∧ 1 / a + 1 / b + 1 / c = 1 / d)", "v": null, "name": "h_answer"}]} -{"informal_problem": "Let $f, g, h$ be functions $\\mathbb{R} \\to \\mathbb{R}$. Find an expression for $h(x)$ in terms of $f$ and $g$ such that $f(x) = \\frac{h(x + 1) + h(x - 1)}{2}$ and $g(x) = \\frac{h(x + 4) + h(x - 4)}{2}$.", "informal_answer": "$h(x) = g(x) - f(x - 3) + f(x - 1) + f(x + 1) - f(x + 3)$", "informal_solution": "Prove that $h(x) = g(x) - f(x - 3) + f(x - 1) + f(x + 1) - f(x + 3)$ suffices.", "header": null, "intros": [], "formal_answer": "@Eq ((Real → Real) → (Real → Real) → Real → Real) answer fun (f_1 g_1 : Real → Real) (x : Real) =>\n @HSub.hSub Real Real Real (@instHSub Real Real.instSub)\n (@HAdd.hAdd Real Real Real (@instHAdd Real Real.instAdd)\n (@HAdd.hAdd Real Real Real (@instHAdd Real Real.instAdd)\n (@HSub.hSub Real Real Real (@instHSub Real Real.instSub) (g_1 x)\n (f_1\n (@HSub.hSub Real Real Real (@instHSub Real Real.instSub) x\n (@OfNat.ofNat Real (nat_lit 3)\n (@instOfNatAtLeastTwo Real (nat_lit 3) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1)))))))))\n (f_1\n (@HSub.hSub Real Real Real (@instHSub Real Real.instSub) x\n (@OfNat.ofNat Real (nat_lit 1) (@One.toOfNat1 Real Real.instOne)))))\n (f_1\n (@HAdd.hAdd Real Real Real (@instHAdd Real Real.instAdd) x\n (@OfNat.ofNat Real (nat_lit 1) (@One.toOfNat1 Real Real.instOne)))))\n (f_1\n (@HAdd.hAdd Real Real Real (@instHAdd Real Real.instAdd) x\n (@OfNat.ofNat Real (nat_lit 3)\n (@instOfNatAtLeastTwo Real (nat_lit 3) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1))))))))", "formal_answer_type": "(ℝ → ℝ) → (ℝ → ℝ) → (ℝ → ℝ)", "outros": [{"t": "ℝ → ℝ", "v": null, "name": "f"}, {"t": "ℝ → ℝ", "v": null, "name": "g"}, {"t": "ℝ → ℝ", "v": null, "name": "h"}, {"t": "∀ x, f x = (h (x + 1) + h (x - 1)) / 2", "v": null, "name": "hf"}, {"t": "∀ x, g x = (h (x + 4) + h (x - 4)) / 2", "v": null, "name": "hg"}, {"t": "h = answer f g", "v": null, "name": "h_answer"}]} +{"informal_problem": "Show that if four distinct points of the curve $y = 2x^4 + 7x^3 + 3x - 5$ are collinear, then their average $x$-coordinate is some constant $k$. Find $k$.", "informal_answer": "$-7/8$", "informal_solution": "Prove that $k = -\\frac{7}{8}$.", "header": "open BigOperators Real Nat Topology", "intros": [], "formal_answer": "@Eq Real answer\n (@HDiv.hDiv Real Real Real (@instHDiv Real (@DivInvMonoid.toDiv Real Real.instDivInvMonoid))\n (@Neg.neg Real Real.instNeg\n (@OfNat.ofNat Real (nat_lit 7)\n (@instOfNatAtLeastTwo Real (nat_lit 7) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 5) (instOfNatNat (nat_lit 5)))))))\n (@OfNat.ofNat Real (nat_lit 8)\n (@instOfNatAtLeastTwo Real (nat_lit 8) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 6) (instOfNatNat (nat_lit 6)))))))", "formal_answer_type": "ℝ", "outros": [{"t": "ℝ → ℝ", "v": null, "name": "y"}, {"t": "y = fun x ↦ 2 * x ^ 4 + 7 * x ^ 3 + 3 * x - 5", "v": null, "name": "hy"}, {"t": "Finset ℝ", "v": null, "name": "S"}, {"t": "S.card = 4", "v": null, "name": "hS"}, {"t": "Collinear ℝ {P : Fin 2 → ℝ | P 0 ∈ S ∧ P 1 = y (P 0)}", "v": null, "name": "h_collinear"}, {"t": "(∑ x in S, x) / 4 = answer", "v": null, "name": "h_answer"}]} +{"informal_problem": "Find all real solutions $(a, b, c, d)$ to the equations $a + b + c = d$, $\\frac{1}{a} + \\frac{1}{b} + \\frac{1}{c} = \\frac{1}{d}$.", "informal_answer": "$d = a \\land b = -c \\lor d = b \\land a = -c \\lor d = c \\land a = -b$", "informal_solution": "Prove that the solutions are $d = a$ and $b = -c$, $d = b$ and $a = -c$, or $d = c$ and $a = -b$, with $a, b, c, d$ nonzero.", "header": "open BigOperators Real Nat Topology", "intros": [], "formal_answer": "@Eq (Real → Real → Real → Real → Prop) answer fun (a_1 b_1 c_1 d_1 : Real) =>\n Or (And (@Eq Real d_1 a_1) (@Eq Real b_1 (@Neg.neg Real Real.instNeg c_1)))\n (Or (And (@Eq Real d_1 b_1) (@Eq Real a_1 (@Neg.neg Real Real.instNeg c_1)))\n (And (@Eq Real d_1 c_1) (@Eq Real a_1 (@Neg.neg Real Real.instNeg b_1))))", "formal_answer_type": "ℝ → ℝ → ℝ → ℝ → Prop", "outros": [{"t": "ℝ", "v": null, "name": "a"}, {"t": "ℝ", "v": null, "name": "b"}, {"t": "ℝ", "v": null, "name": "c"}, {"t": "ℝ", "v": null, "name": "d"}, {"t": "answer a b c d ↔\n a ≠ 0 → b ≠ 0 → c ≠ 0 → d ≠ 0 → (a + b + c = d ∧ 1 / a + 1 / b + 1 / c = 1 / d)", "v": null, "name": "h_answer"}]} +{"informal_problem": "Let $f, g, h$ be functions $\\mathbb{R} \\to \\mathbb{R}$. Find an expression for $h(x)$ in terms of $f$ and $g$ such that $f(x) = \\frac{h(x + 1) + h(x - 1)}{2}$ and $g(x) = \\frac{h(x + 4) + h(x - 4)}{2}$.", "informal_answer": "$h(x) = g(x) - f(x - 3) + f(x - 1) + f(x + 1) - f(x + 3)$", "informal_solution": "Prove that $h(x) = g(x) - f(x - 3) + f(x - 1) + f(x + 1) - f(x + 3)$ suffices.", "header": "open BigOperators Real Nat Topology", "intros": [], "formal_answer": "@Eq ((Real → Real) → (Real → Real) → Real → Real) answer fun (f_1 g_1 : Real → Real) (x : Real) =>\n @HSub.hSub Real Real Real (@instHSub Real Real.instSub)\n (@HAdd.hAdd Real Real Real (@instHAdd Real Real.instAdd)\n (@HAdd.hAdd Real Real Real (@instHAdd Real Real.instAdd)\n (@HSub.hSub Real Real Real (@instHSub Real Real.instSub) (g_1 x)\n (f_1\n (@HSub.hSub Real Real Real (@instHSub Real Real.instSub) x\n (@OfNat.ofNat Real (nat_lit 3)\n (@instOfNatAtLeastTwo Real (nat_lit 3) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1)))))))))\n (f_1\n (@HSub.hSub Real Real Real (@instHSub Real Real.instSub) x\n (@OfNat.ofNat Real (nat_lit 1) (@One.toOfNat1 Real Real.instOne)))))\n (f_1\n (@HAdd.hAdd Real Real Real (@instHAdd Real Real.instAdd) x\n (@OfNat.ofNat Real (nat_lit 1) (@One.toOfNat1 Real Real.instOne)))))\n (f_1\n (@HAdd.hAdd Real Real Real (@instHAdd Real Real.instAdd) x\n (@OfNat.ofNat Real (nat_lit 3)\n (@instOfNatAtLeastTwo Real (nat_lit 3) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1))))))))", "formal_answer_type": "(ℝ → ℝ) → (ℝ → ℝ) → (ℝ → ℝ)", "outros": [{"t": "ℝ → ℝ", "v": null, "name": "f"}, {"t": "ℝ → ℝ", "v": null, "name": "g"}, {"t": "ℝ → ℝ", "v": null, "name": "h"}, {"t": "∀ x, f x = (h (x + 1) + h (x - 1)) / 2", "v": null, "name": "hf"}, {"t": "∀ x, g x = (h (x + 4) + h (x - 4)) / 2", "v": null, "name": "hg"}, {"t": "h = answer f g", "v": null, "name": "h_answer"}]} {"informal_problem": "Find $\\sum_{n=0}^{\\infty} \\frac{x^{2^n}}{1 - x^{2^{n+1}}}$ as a rational function of $x$ for $x \\in (0, 1)$.", "informal_answer": "$\\frac{x}{1 - x}$", "informal_solution": "Prove that the sum equals $\\frac{x}{1 - x}$.", "header": "open RingHom Set", "intros": [], "formal_answer": "@Eq (@RatFunc Real Real.commRing) answer\n (@HDiv.hDiv (@RatFunc Real Real.commRing) (@RatFunc Real Real.commRing) (@RatFunc Real Real.commRing)\n (@instHDiv (@RatFunc Real Real.commRing) (@RatFunc.instDiv Real Real.commRing Real.instIsDomain))\n (@RatFunc.X Real Real.commRing Real.instIsDomain)\n (@HSub.hSub (@RatFunc Real Real.commRing) (@RatFunc Real Real.commRing) (@RatFunc Real Real.commRing)\n (@instHSub (@RatFunc Real Real.commRing) (@RatFunc.instSub Real Real.commRing))\n (@OfNat.ofNat (@RatFunc Real Real.commRing) (nat_lit 1)\n (@One.toOfNat1 (@RatFunc Real Real.commRing) (@RatFunc.instOne Real Real.commRing)))\n (@RatFunc.X Real Real.commRing Real.instIsDomain)))", "formal_answer_type": "RatFunc ℝ", "outros": [{"t": "ℝ", "v": null, "name": "x"}, {"t": "x ∈ Ioo 0 1", "v": null, "name": "hx"}, {"t": "answer.eval (id ℝ) x = ∑' n : ℕ, x ^ 2 ^ n / (1 - x ^ 2 ^ (n + 1))", "v": null, "name": "h_answer"}]} {"informal_problem": "Let $X$ be the square $[0, 1] \\times [0, 1]$, and let $f : X \\to \\mathbb{R}$ be continuous. If $\\int_Y f(x, y) \\, dx \\, dy = 0$ for all squares $Y$ such that\n\\begin{itemize}\n\\item[(1)] $Y \\subseteq X$,\n\\item[(2)] $Y$ has sides parallel to those of $X$,\n\\item[(3)] at least one of $Y$'s sides is contained in the boundary of $X$,\n\\end{itemize}\nis it true that $f(x, y) = 0$ for all $x, y$?", "informal_answer": "True", "informal_solution": "Prove that $f(x,y)$ must be identically zero.", "header": "open RingHom Set Nat", "intros": [], "formal_answer": "@Eq Prop answer True", "formal_answer_type": "Prop", "outros": [{"t": "Set (ℝ × ℝ)", "v": null, "name": "X"}, {"t": "X = Set.prod (Icc 0 1) (Icc 0 1)", "v": null, "name": "hX"}, {"t": "(ℝ × ℝ) → ℝ", "v": null, "name": "room"}, {"t": "room = fun (a,b) ↦ min (min a (1 - a)) (min b (1 - b))", "v": null, "name": "hroom"}, {"t": "(∀ f : (ℝ × ℝ) → ℝ, Continuous f → (∀ P ∈ X, ∫ x in (P.1 - room P)..(P.1 + room P), ∫ y in (P.2 - room P)..(P.2 + room P), f (x, y) = 0) → (∀ P ∈ X, f P = 0)) ↔ answer", "v": null, "name": "h_answer"}]} {"informal_problem": "Find $\\prod_{n=2}^{\\infty} \\frac{(n^3 - 1)}{(n^3 + 1)}$.", "informal_answer": "2/3", "informal_solution": "Prove that the product equals $\\frac{2}{3}$.", "header": "open RingHom Set Nat Filter Topology", "intros": [], "formal_answer": "@Eq Real answer\n (@HDiv.hDiv Real Real Real (@instHDiv Real (@DivInvMonoid.toDiv Real Real.instDivInvMonoid))\n (@OfNat.ofNat Real (nat_lit 2)\n (@instOfNatAtLeastTwo Real (nat_lit 2) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 0) (instOfNatNat (nat_lit 0))))))\n (@OfNat.ofNat Real (nat_lit 3)\n (@instOfNatAtLeastTwo Real (nat_lit 3) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1)))))))", "formal_answer_type": "ℝ", "outros": [{"t": "Tendsto (fun N ↦ ∏ n in Finset.Icc (2 : ℤ) N, ((n : ℝ) ^ 3 - 1) / (n ^ 3 + 1)) atTop (𝓝 answer)", "v": null, "name": "h_answer"}]} @@ -52,17 +52,17 @@ {"informal_problem": "Let $p(x) = 2(x^6 + 1) + 4(x^5 + x) + 3(x^4 + x^2) + 5x^3$. For $k$ with $0 < k < 5$, let\n\\[\nI_k = \\int_0^{\\infty} \\frac{x^k}{p(x)} \\, dx.\n\\]\nFor which $k$ is $I_k$ smallest?", "informal_answer": "2", "informal_solution": "Show that $I_k$ is smallest for $k = 2$.", "header": "open Set Polynomial", "intros": [], "formal_answer": "@Eq Nat answer (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))", "formal_answer_type": "ℕ", "outros": [{"t": "Polynomial ℝ", "v": null, "name": "p"}, {"t": "p = 2 * (Polynomial.X ^ 6 + 1) + 4 * (Polynomial.X ^ 5 + Polynomial.X) + 3 * (Polynomial.X ^ 4 + Polynomial.X ^ 2) + 5 * Polynomial.X ^ 3", "v": null, "name": "hp"}, {"t": "ℕ → ℝ", "v": null, "name": "I"}, {"t": "I = fun k ↦ ∫ x in Ioi 0, x ^ k / p.eval x", "v": null, "name": "hI"}, {"t": "IsLeast {y | ∃ k ∈ Ioo 0 5, I k = y} answer", "v": null, "name": "h_answer"}]} {"informal_problem": "Find\n\\[\n\\sum_{i=1}^{\\infty} \\sum_{j=1}^{\\infty} \\frac{1}{i^2j + 2ij + ij^2}.\n\\]", "informal_answer": "7 / 4", "informal_solution": "Prove that the sum evaluates to $\\frac{7}{4}$.", "header": "open Set Real", "intros": [], "formal_answer": "@Eq Rat answer\n (@HDiv.hDiv Rat Rat Rat (@instHDiv Rat Rat.instDiv) (@OfNat.ofNat Rat (nat_lit 7) (@Rat.instOfNat (nat_lit 7)))\n (@OfNat.ofNat Rat (nat_lit 4) (@Rat.instOfNat (nat_lit 4))))", "formal_answer_type": "ℚ", "outros": [{"t": "(∑' i : ℕ+, ∑' j : ℕ+, (1 : ℚ) / (i ^ 2 * j + 2 * i * j + i * j ^ 2)) = answer", "v": null, "name": "h_answer"}]} {"informal_problem": "Find the real polynomial $p(x)$ of degree $4$ with largest possible coefficient of $x^4$ such that $p([-1, 1]) \\subseteq [0, 1]$.", "informal_answer": "$4x^4 - 4x^2 + 1$", "informal_solution": "Prove that $p(x) = 4x^4 - 4x^2 + 1$.", "header": "open Set Real Filter Topology Polynomial", "intros": [], "formal_answer": "@Eq (@Polynomial Real Real.semiring) answer\n (@HAdd.hAdd (@Polynomial Real Real.semiring) (@Polynomial Real Real.semiring) (@Polynomial Real Real.semiring)\n (@instHAdd (@Polynomial Real Real.semiring) (@Polynomial.add' Real Real.semiring))\n (@HSub.hSub (@Polynomial Real Real.semiring) (@Polynomial Real Real.semiring) (@Polynomial Real Real.semiring)\n (@instHSub (@Polynomial Real Real.semiring) (@Polynomial.sub Real Real.instRing))\n (@HMul.hMul (@Polynomial Real Real.semiring) (@Polynomial Real Real.semiring) (@Polynomial Real Real.semiring)\n (@instHMul (@Polynomial Real Real.semiring) (@Polynomial.mul' Real Real.semiring))\n (@OfNat.ofNat (@Polynomial Real Real.semiring) (nat_lit 4)\n (@instOfNatAtLeastTwo (@Polynomial Real Real.semiring) (nat_lit 4)\n (@Polynomial.instNatCast Real Real.semiring)\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))))))\n (@HPow.hPow (@Polynomial Real Real.semiring) Nat (@Polynomial Real Real.semiring)\n (@instHPow (@Polynomial Real Real.semiring) Nat\n (@Monoid.toNatPow (@Polynomial Real Real.semiring)\n (@MonoidWithZero.toMonoid (@Polynomial Real Real.semiring)\n (@Semiring.toMonoidWithZero (@Polynomial Real Real.semiring)\n (@Polynomial.semiring Real Real.semiring)))))\n (@Polynomial.X Real Real.semiring) (@OfNat.ofNat Nat (nat_lit 4) (instOfNatNat (nat_lit 4)))))\n (@HMul.hMul (@Polynomial Real Real.semiring) (@Polynomial Real Real.semiring) (@Polynomial Real Real.semiring)\n (@instHMul (@Polynomial Real Real.semiring) (@Polynomial.mul' Real Real.semiring))\n (@OfNat.ofNat (@Polynomial Real Real.semiring) (nat_lit 4)\n (@instOfNatAtLeastTwo (@Polynomial Real Real.semiring) (nat_lit 4)\n (@Polynomial.instNatCast Real Real.semiring)\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))))))\n (@HPow.hPow (@Polynomial Real Real.semiring) Nat (@Polynomial Real Real.semiring)\n (@instHPow (@Polynomial Real Real.semiring) Nat\n (@Monoid.toNatPow (@Polynomial Real Real.semiring)\n (@MonoidWithZero.toMonoid (@Polynomial Real Real.semiring)\n (@Semiring.toMonoidWithZero (@Polynomial Real Real.semiring)\n (@Polynomial.semiring Real Real.semiring)))))\n (@Polynomial.X Real Real.semiring) (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))))))\n (@OfNat.ofNat (@Polynomial Real Real.semiring) (nat_lit 1)\n (@One.toOfNat1 (@Polynomial Real Real.semiring) (@Polynomial.one Real Real.semiring))))", "formal_answer_type": "Polynomial ℝ", "outros": [{"t": "Set (Polynomial ℝ)", "v": null, "name": "S"}, {"t": "S = {p : Polynomial ℝ | p.degree = 4 ∧ ∀ x ∈ Icc (-1 : ℝ) 1, p.eval x ∈ Icc 0 1}", "v": null, "name": "hS"}, {"t": "answer ∈ S ∧ (∀ p ∈ S, p.coeff 4 ≤ answer.coeff 4)", "v": null, "name": "h_answer"}]} -{"informal_problem": "For which positive integers $n$ and $a_1, a_2, \\dots, a_n$ with $\\sum_{i = 1}^{n} a_i = 1979$ does $\\prod_{i = 1}^{n} a_i$ attain the greatest value?", "informal_answer": "Multiset.replicate 659 3 + {2}", "informal_solution": "$n$ equals $660$; all but one of the $a_i$ equal $3$ and the remaining $a_i$ equals $2$.", "header": null, "intros": [], "formal_answer": "@Eq (Multiset Nat) answer\n (@HAdd.hAdd (Multiset Nat) (Multiset Nat) (Multiset Nat) (@instHAdd (Multiset Nat) (@Multiset.instAdd Nat))\n (@Multiset.replicate Nat (@OfNat.ofNat Nat (nat_lit 659) (instOfNatNat (nat_lit 659)))\n (@OfNat.ofNat Nat (nat_lit 3) (instOfNatNat (nat_lit 3))))\n (@Singleton.singleton Nat (Multiset Nat) (@Multiset.instSingleton Nat)\n (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))))", "formal_answer_type": "Multiset ℕ", "outros": [{"t": "Multiset ℕ → Prop", "v": null, "name": "P"}, {"t": "∀ a, P a ↔ Multiset.card a > 0 ∧ (∀ i ∈ a, i > 0) ∧ a.sum = 1979", "v": null, "name": "hP"}, {"t": "P answer ∧ ∀ a : Multiset ℕ, P a → answer.prod ≥ a.prod", "v": null, "name": "h_answer"}]} -{"informal_problem": "For which real numbers $k$ does there exist a continuous function $f : \\mathbb{R} \\to \\mathbb{R}$ such that $f(f(x)) = kx^9$ for all real $x$?", "informal_answer": "$k \\geq 0$", "informal_solution": "Such a function exists if and only if $k \\ge 0$.", "header": null, "intros": [], "formal_answer": "@Eq (Real → Prop) answer fun (k_1 : Real) =>\n @GE.ge Real Real.instLE k_1 (@OfNat.ofNat Real (nat_lit 0) (@Zero.toOfNat0 Real Real.instZero))", "formal_answer_type": "ℝ → Prop", "outros": [{"t": "ℝ", "v": null, "name": "k"}, {"t": "answer k ↔ ∃ f : ℝ → ℝ, Continuous f ∧ ∀ x : ℝ, f (f x) = k * x^9", "v": null, "name": "h_answer"}]} -{"informal_problem": "Let $x_1, x_2, x_3, \\dots$ be a sequence of nonzero real numbers such that $$x_n = \\frac{x_{n-2}x_{n-1}}{2x_{n-2}-x_{n-1}}$$ for all $n \\ge 3$. For which real values of $x_1$ and $x_2$ does $x_n$ attain integer values for infinitely many $n$?", "informal_answer": "fun (a, b) => ∃ m : ℤ, a = m ∧ b = m", "informal_solution": "We must have $x_1 = x_2 = m$ for some integer $m$.", "header": null, "intros": [], "formal_answer": "@Eq (Prod Real Real → Prop) answer fun (x_1 : Prod Real Real) =>\n _example.match_1 (fun (x_2 : Prod Real Real) => Prop) x_1 fun (a b : Real) =>\n @Exists Int fun (m : Int) =>\n And (@Eq Real a (@Int.cast Real Real.instIntCast m)) (@Eq Real b (@Int.cast Real Real.instIntCast m))", "formal_answer_type": "(ℝ × ℝ) → Prop", "outros": [{"t": "ℕ → ℝ", "v": null, "name": "x"}, {"t": "∀ n : ℕ, x n ≠ 0 ∧ (n ≥ 3 → x n = (x (n - 2))*(x (n - 1))/(2*(x (n - 2)) - (x (n - 1))))", "v": null, "name": "hx"}, {"t": "(∀ m : ℕ, ∃ n : ℕ, n > m ∧ ∃ a : ℤ, a = x n) ↔ answer (x 1, x 2)", "v": null, "name": "h_answer"}]} +{"informal_problem": "For which positive integers $n$ and $a_1, a_2, \\dots, a_n$ with $\\sum_{i = 1}^{n} a_i = 1979$ does $\\prod_{i = 1}^{n} a_i$ attain the greatest value?", "informal_answer": "Multiset.replicate 659 3 + {2}", "informal_solution": "$n$ equals $660$; all but one of the $a_i$ equal $3$ and the remaining $a_i$ equals $2$.", "header": "open BigOperators Real Nat Topology", "intros": [], "formal_answer": "@Eq (Multiset Nat) answer\n (@HAdd.hAdd (Multiset Nat) (Multiset Nat) (Multiset Nat) (@instHAdd (Multiset Nat) (@Multiset.instAdd Nat))\n (@Multiset.replicate Nat (@OfNat.ofNat Nat (nat_lit 659) (instOfNatNat (nat_lit 659)))\n (@OfNat.ofNat Nat (nat_lit 3) (instOfNatNat (nat_lit 3))))\n (@Singleton.singleton Nat (Multiset Nat) (@Multiset.instSingleton Nat)\n (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))))", "formal_answer_type": "Multiset ℕ", "outros": [{"t": "Multiset ℕ → Prop", "v": null, "name": "P"}, {"t": "∀ a, P a ↔ Multiset.card a > 0 ∧ (∀ i ∈ a, i > 0) ∧ a.sum = 1979", "v": null, "name": "hP"}, {"t": "P answer ∧ ∀ a : Multiset ℕ, P a → answer.prod ≥ a.prod", "v": null, "name": "h_answer"}]} +{"informal_problem": "For which real numbers $k$ does there exist a continuous function $f : \\mathbb{R} \\to \\mathbb{R}$ such that $f(f(x)) = kx^9$ for all real $x$?", "informal_answer": "$k \\geq 0$", "informal_solution": "Such a function exists if and only if $k \\ge 0$.", "header": "open BigOperators Real Nat Topology", "intros": [], "formal_answer": "@Eq (Real → Prop) answer fun (k_1 : Real) =>\n @GE.ge Real Real.instLE k_1 (@OfNat.ofNat Real (nat_lit 0) (@Zero.toOfNat0 Real Real.instZero))", "formal_answer_type": "ℝ → Prop", "outros": [{"t": "ℝ", "v": null, "name": "k"}, {"t": "answer k ↔ ∃ f : ℝ → ℝ, Continuous f ∧ ∀ x : ℝ, f (f x) = k * x^9", "v": null, "name": "h_answer"}]} +{"informal_problem": "Let $x_1, x_2, x_3, \\dots$ be a sequence of nonzero real numbers such that $$x_n = \\frac{x_{n-2}x_{n-1}}{2x_{n-2}-x_{n-1}}$$ for all $n \\ge 3$. For which real values of $x_1$ and $x_2$ does $x_n$ attain integer values for infinitely many $n$?", "informal_answer": "fun (a, b) => ∃ m : ℤ, a = m ∧ b = m", "informal_solution": "We must have $x_1 = x_2 = m$ for some integer $m$.", "header": "open BigOperators Real Nat Topology", "intros": [], "formal_answer": "@Eq (Prod Real Real → Prop) answer fun (x_1 : Prod Real Real) =>\n _example.match_1 (fun (x_2 : Prod Real Real) => Prop) x_1 fun (a b : Real) =>\n @Exists Int fun (m : Int) =>\n And (@Eq Real a (@Int.cast Real Real.instIntCast m)) (@Eq Real b (@Int.cast Real Real.instIntCast m))", "formal_answer_type": "(ℝ × ℝ) → Prop", "outros": [{"t": "ℕ → ℝ", "v": null, "name": "x"}, {"t": "∀ n : ℕ, x n ≠ 0 ∧ (n ≥ 3 → x n = (x (n - 2))*(x (n - 1))/(2*(x (n - 2)) - (x (n - 1))))", "v": null, "name": "hx"}, {"t": "(∀ m : ℕ, ∃ n : ℕ, n > m ∧ ∃ a : ℤ, a = x n) ↔ answer (x 1, x 2)", "v": null, "name": "h_answer"}]} {"informal_problem": "Let $A$ be a set of $2n$ points in the plane, $n$ colored red and $n$ colored blue, such that no three points in $A$ are collinear. Must there exist $n$ closed straight line segments, each connecting one red and one blue point in $A$, such that no two of the $n$ line segments intersect?", "informal_answer": "True", "informal_solution": "Such line segments must exist.", "header": "open Set", "intros": [], "formal_answer": "@Eq Prop answer True", "formal_answer_type": "Prop", "outros": [{"t": "Finset (Fin 2 → ℝ) × Finset (Fin 2 → ℝ) → Prop", "v": null, "name": "A"}, {"t": "A = fun (R, B) => R.card = B.card ∧ R ∩ B = ∅ ∧\n ∀ u : Finset (Fin 2 → ℝ), u ⊆ R ∪ B → u.card = 3 → ¬Collinear ℝ (u : Set (Fin 2 → ℝ))", "v": null, "name": "hA"}, {"t": "(Fin 2 → ℝ) × (Fin 2 → ℝ) → ℝ → (Fin 2 → ℝ)", "v": null, "name": "w"}, {"t": "w = fun (P, Q) => fun x : ℝ => fun i : Fin 2 => x * P i + (1 - x) * Q i", "v": null, "name": "hw"}, {"t": "answer ↔\n (∀ R B, A (R, B) →\n ∃ v : Finset ((Fin 2 → ℝ) × (Fin 2 → ℝ)),\n (∀ L ∈ v, ∀ M ∈ v, L ≠ M → ∀ x ∈ Icc 0 1, ∀ y ∈ Icc 0 1,\n Real.sqrt ((w (L.1, L.2) x 0 - w (M.1, M.2) y 0)^2 + (w (L.1, L.2) x 1 - w (M.1, M.2) y 1)^2) ≠ 0) ∧\n v.card = R.card ∧ ∀ L ∈ v, L.1 ∈ R ∧ L.2 ∈ B)", "v": null, "name": "h_answer"}]} {"informal_problem": "If $0 < a < b$, find $$\\lim_{t \\to 0} \\left( \\int_{0}^{1}(bx + a(1-x))^t dx \\right)^{\\frac{1}{t}}$$ in terms of $a$ and $b$.", "informal_answer": "fun (a, b) => (Real.exp (-1))*(b^b/a^a)^(1/(b-a))", "informal_solution": "The limit equals $$e^{-1}\\left(\\frac{b^b}{a^a}\\right)^{\\frac{1}{b-a}}.$$", "header": "open Set Topology Filter", "intros": [], "formal_answer": "@Eq (Prod Real Real → Real) answer fun (x : Prod Real Real) =>\n _example.match_1 (fun (x_1 : Prod Real Real) => Real) x fun (a b : Real) =>\n @HMul.hMul Real Real Real (@instHMul Real Real.instMul)\n (Real.exp (@Neg.neg Real Real.instNeg (@OfNat.ofNat Real (nat_lit 1) (@One.toOfNat1 Real Real.instOne))))\n (@HPow.hPow Real Real Real (@instHPow Real Real Real.instPow)\n (@HDiv.hDiv Real Real Real (@instHDiv Real (@DivInvMonoid.toDiv Real Real.instDivInvMonoid))\n (@HPow.hPow Real Real Real (@instHPow Real Real Real.instPow) b b)\n (@HPow.hPow Real Real Real (@instHPow Real Real Real.instPow) a a))\n (@HDiv.hDiv Real Real Real (@instHDiv Real (@DivInvMonoid.toDiv Real Real.instDivInvMonoid))\n (@OfNat.ofNat Real (nat_lit 1) (@One.toOfNat1 Real Real.instOne))\n (@HSub.hSub Real Real Real (@instHSub Real Real.instSub) b a)))", "formal_answer_type": "ℝ × ℝ → ℝ", "outros": [{"t": "∀ a b : ℝ, 0 < a ∧ a < b → Tendsto (fun t : ℝ => (∫ x in Icc 0 1, (b*x + a*(1 - x))^t)^(1/t)) (𝓝[≠] 0) (𝓝 (answer (a, b)))", "v": null, "name": "h_answer"}]} {"informal_problem": "Let $F$ be a finite field with $n$ elements, and assume $n$ is odd. Suppose $x^2 + bx + c$ is an irreducible polynomial over $F$. For how many elements $d \\in F$ is $x^2 + bx + c + d$ irreducible?", "informal_answer": "fun n : ℕ ↦ (n - (1 : ℤ)) / 2", "informal_solution": "Show that there are $\\frac{n - 1}{2}$ such elements $d$.", "header": "open Set Topology Filter Polynomial", "intros": [], "formal_answer": "@Eq (Nat → Int) answer fun (n_1 : Nat) =>\n @HDiv.hDiv Int Int Int (@instHDiv Int Int.instDiv)\n (@HSub.hSub Int Int Int (@instHSub Int Int.instSub) (@Nat.cast Int instNatCastInt n_1)\n (@OfNat.ofNat Int (nat_lit 1) (@instOfNat (nat_lit 1))))\n (@OfNat.ofNat Int (nat_lit 2) (@instOfNat (nat_lit 2)))", "formal_answer_type": "ℕ → ℤ", "outros": [{"t": "Type*", "v": null, "name": "F"}, {"t": "Field F", "v": null, "name": null}, {"t": "Fintype F", "v": null, "name": null}, {"t": "ℕ", "v": null, "name": "n"}, {"t": "n = Fintype.card F", "v": null, "name": "hn"}, {"t": "Odd n", "v": null, "name": "nodd"}, {"t": "F", "v": null, "name": "b"}, {"t": "F", "v": null, "name": "c"}, {"t": "Polynomial F", "v": null, "name": "p"}, {"t": "p = X ^ 2 + (C b) * X + (C c) ∧ Irreducible p", "v": null, "name": "hp"}, {"t": "{d : F | Irreducible (p + (C d))}.ncard = answer n", "v": null, "name": "h_answer"}]} -{"informal_problem": "Let $r$ and $s$ be positive integers. Derive a formula for the number of ordered quadruples $(a,b,c,d)$ of positive integers such that $3^r \\cdot 7^s=\\text{lcm}[a,b,c]=\\text{lcm}[a,b,d]=\\text{lcm}[a,c,d]=\\text{lcm}[b,c,d]$. The answer should be a function of $r$ and $s$. (Note that $\\text{lcm}[x,y,z]$ denotes the least common multiple of $x,y,z$.)", "informal_answer": "(fun r s : ℕ => (1 + 4 * r + 6 * r ^ 2) * (1 + 4 * s + 6 * s ^ 2))", "informal_solution": "Show that the number is $(1+4r+6r^2)(1+4s+6s^2)$.", "header": null, "intros": [], "formal_answer": "@Eq (Nat → Nat → Nat) answer fun (r_1 s_1 : Nat) =>\n @HMul.hMul Nat Nat Nat (@instHMul Nat instMulNat)\n (@HAdd.hAdd Nat Nat Nat (@instHAdd Nat instAddNat)\n (@HAdd.hAdd Nat Nat Nat (@instHAdd Nat instAddNat) (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1)))\n (@HMul.hMul Nat Nat Nat (@instHMul Nat instMulNat) (@OfNat.ofNat Nat (nat_lit 4) (instOfNatNat (nat_lit 4)))\n r_1))\n (@HMul.hMul Nat Nat Nat (@instHMul Nat instMulNat) (@OfNat.ofNat Nat (nat_lit 6) (instOfNatNat (nat_lit 6)))\n (@HPow.hPow Nat Nat Nat (@instHPow Nat Nat (@Monoid.toNatPow Nat Nat.instMonoid)) r_1\n (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))))))\n (@HAdd.hAdd Nat Nat Nat (@instHAdd Nat instAddNat)\n (@HAdd.hAdd Nat Nat Nat (@instHAdd Nat instAddNat) (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1)))\n (@HMul.hMul Nat Nat Nat (@instHMul Nat instMulNat) (@OfNat.ofNat Nat (nat_lit 4) (instOfNatNat (nat_lit 4)))\n s_1))\n (@HMul.hMul Nat Nat Nat (@instHMul Nat instMulNat) (@OfNat.ofNat Nat (nat_lit 6) (instOfNatNat (nat_lit 6)))\n (@HPow.hPow Nat Nat Nat (@instHPow Nat Nat (@Monoid.toNatPow Nat Nat.instMonoid)) s_1\n (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))))))", "formal_answer_type": "ℕ → ℕ → ℕ", "outros": [{"t": "ℕ", "v": null, "name": "r"}, {"t": "ℕ", "v": null, "name": "s"}, {"t": "ℕ → ℕ → ℕ → ℕ → Prop", "v": null, "name": "abcdlcm"}, {"t": "r > 0 ∧ s > 0", "v": null, "name": "rspos"}, {"t": "∀ a b c d : ℕ, abcdlcm a b c d ↔\n (a > 0 ∧ b > 0 ∧ c > 0 ∧ d > 0 ∧\n (3 ^ r * 7 ^ s = Nat.lcm (Nat.lcm a b) c) ∧\n (3 ^ r * 7 ^ s = Nat.lcm (Nat.lcm a b) d) ∧\n (3 ^ r * 7 ^ s = Nat.lcm (Nat.lcm a c) d) ∧\n (3 ^ r * 7 ^ s = Nat.lcm (Nat.lcm b c) d))", "v": null, "name": "habcdlcm"}, {"t": "{h : ℕ × ℕ × ℕ × ℕ | abcdlcm h.1 h.2.1 h.2.2.1 h.2.2.2}.encard = answer r s", "v": null, "name": "h_answer"}]} -{"informal_problem": "Evaluate $\\int_0^{\\pi/2}\\frac{dx}{1+(\\tan x)^{\\sqrt{2}}}$.", "informal_answer": "$\\pi / 4$", "informal_solution": "Show that the integral is $\\pi/4$.", "header": null, "intros": [], "formal_answer": "@Eq Real answer\n (@HDiv.hDiv Real Real Real (@instHDiv Real (@DivInvMonoid.toDiv Real Real.instDivInvMonoid)) Real.pi\n (@OfNat.ofNat Real (nat_lit 4)\n (@instOfNatAtLeastTwo Real (nat_lit 4) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))))))", "formal_answer_type": "ℝ", "outros": [{"t": "answer = ∫ x in Set.Ioo 0 (Real.pi / 2), 1 / (1 + (Real.tan x) ^ (Real.sqrt 2))", "v": null, "name": "h_answer"}]} -{"informal_problem": "Let $C$ be the class of all real valued continuously differentiable functions $f$ on the interval $0 \\leq x \\leq 1$ with $f(0)=0$ and $f(1)=1$. Determine the largest real number $u$ such that $u \\leq \\int_0^1|f'(x)-f(x)|\\,dx$ for all $f$ in $C$.", "informal_answer": "$1/e$", "informal_solution": "Show that $u=1/e$.", "header": null, "intros": [], "formal_answer": "@Eq Real answer\n (@HDiv.hDiv Real Real Real (@instHDiv Real (@DivInvMonoid.toDiv Real Real.instDivInvMonoid))\n (@OfNat.ofNat Real (nat_lit 1) (@One.toOfNat1 Real Real.instOne))\n (Real.exp (@OfNat.ofNat Real (nat_lit 1) (@One.toOfNat1 Real Real.instOne))))", "formal_answer_type": "ℝ", "outros": [{"t": "Set (ℝ → ℝ)", "v": null, "name": "C"}, {"t": "C = {f : ℝ → ℝ | ContDiffOn ℝ 1 f (Set.Icc 0 1) ∧ f 0 = 0 ∧ f 1 = 1}", "v": null, "name": "hC"}, {"t": "IsGreatest {u : ℝ | ∀ f ∈ C, u ≤ (∫ x in Set.Ioo 0 1, |deriv f x - f x|)} answer", "v": null, "name": "h_answer"}]} +{"informal_problem": "Let $r$ and $s$ be positive integers. Derive a formula for the number of ordered quadruples $(a,b,c,d)$ of positive integers such that $3^r \\cdot 7^s=\\text{lcm}[a,b,c]=\\text{lcm}[a,b,d]=\\text{lcm}[a,c,d]=\\text{lcm}[b,c,d]$. The answer should be a function of $r$ and $s$. (Note that $\\text{lcm}[x,y,z]$ denotes the least common multiple of $x,y,z$.)", "informal_answer": "(fun r s : ℕ => (1 + 4 * r + 6 * r ^ 2) * (1 + 4 * s + 6 * s ^ 2))", "informal_solution": "Show that the number is $(1+4r+6r^2)(1+4s+6s^2)$.", "header": "open BigOperators Real Nat Topology", "intros": [], "formal_answer": "@Eq (Nat → Nat → Nat) answer fun (r_1 s_1 : Nat) =>\n @HMul.hMul Nat Nat Nat (@instHMul Nat instMulNat)\n (@HAdd.hAdd Nat Nat Nat (@instHAdd Nat instAddNat)\n (@HAdd.hAdd Nat Nat Nat (@instHAdd Nat instAddNat) (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1)))\n (@HMul.hMul Nat Nat Nat (@instHMul Nat instMulNat) (@OfNat.ofNat Nat (nat_lit 4) (instOfNatNat (nat_lit 4)))\n r_1))\n (@HMul.hMul Nat Nat Nat (@instHMul Nat instMulNat) (@OfNat.ofNat Nat (nat_lit 6) (instOfNatNat (nat_lit 6)))\n (@HPow.hPow Nat Nat Nat (@instHPow Nat Nat (@Monoid.toNatPow Nat Nat.instMonoid)) r_1\n (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))))))\n (@HAdd.hAdd Nat Nat Nat (@instHAdd Nat instAddNat)\n (@HAdd.hAdd Nat Nat Nat (@instHAdd Nat instAddNat) (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1)))\n (@HMul.hMul Nat Nat Nat (@instHMul Nat instMulNat) (@OfNat.ofNat Nat (nat_lit 4) (instOfNatNat (nat_lit 4)))\n s_1))\n (@HMul.hMul Nat Nat Nat (@instHMul Nat instMulNat) (@OfNat.ofNat Nat (nat_lit 6) (instOfNatNat (nat_lit 6)))\n (@HPow.hPow Nat Nat Nat (@instHPow Nat Nat (@Monoid.toNatPow Nat Nat.instMonoid)) s_1\n (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))))))", "formal_answer_type": "ℕ → ℕ → ℕ", "outros": [{"t": "ℕ", "v": null, "name": "r"}, {"t": "ℕ", "v": null, "name": "s"}, {"t": "ℕ → ℕ → ℕ → ℕ → Prop", "v": null, "name": "abcdlcm"}, {"t": "r > 0 ∧ s > 0", "v": null, "name": "rspos"}, {"t": "∀ a b c d : ℕ, abcdlcm a b c d ↔\n (a > 0 ∧ b > 0 ∧ c > 0 ∧ d > 0 ∧\n (3 ^ r * 7 ^ s = Nat.lcm (Nat.lcm a b) c) ∧\n (3 ^ r * 7 ^ s = Nat.lcm (Nat.lcm a b) d) ∧\n (3 ^ r * 7 ^ s = Nat.lcm (Nat.lcm a c) d) ∧\n (3 ^ r * 7 ^ s = Nat.lcm (Nat.lcm b c) d))", "v": null, "name": "habcdlcm"}, {"t": "{h : ℕ × ℕ × ℕ × ℕ | abcdlcm h.1 h.2.1 h.2.2.1 h.2.2.2}.encard = answer r s", "v": null, "name": "h_answer"}]} +{"informal_problem": "Evaluate $\\int_0^{\\pi/2}\\frac{dx}{1+(\\tan x)^{\\sqrt{2}}}$.", "informal_answer": "$\\pi / 4$", "informal_solution": "Show that the integral is $\\pi/4$.", "header": "open BigOperators Real Nat Topology", "intros": [], "formal_answer": "@Eq Real answer\n (@HDiv.hDiv Real Real Real (@instHDiv Real (@DivInvMonoid.toDiv Real Real.instDivInvMonoid)) Real.pi\n (@OfNat.ofNat Real (nat_lit 4)\n (@instOfNatAtLeastTwo Real (nat_lit 4) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))))))", "formal_answer_type": "ℝ", "outros": [{"t": "answer = ∫ x in Set.Ioo 0 (Real.pi / 2), 1 / (1 + (Real.tan x) ^ (Real.sqrt 2))", "v": null, "name": "h_answer"}]} +{"informal_problem": "Let $C$ be the class of all real valued continuously differentiable functions $f$ on the interval $0 \\leq x \\leq 1$ with $f(0)=0$ and $f(1)=1$. Determine the largest real number $u$ such that $u \\leq \\int_0^1|f'(x)-f(x)|\\,dx$ for all $f$ in $C$.", "informal_answer": "$1/e$", "informal_solution": "Show that $u=1/e$.", "header": "open BigOperators Real Nat Topology", "intros": [], "formal_answer": "@Eq Real answer\n (@HDiv.hDiv Real Real Real (@instHDiv Real (@DivInvMonoid.toDiv Real Real.instDivInvMonoid))\n (@OfNat.ofNat Real (nat_lit 1) (@One.toOfNat1 Real Real.instOne))\n (Real.exp (@OfNat.ofNat Real (nat_lit 1) (@One.toOfNat1 Real Real.instOne))))", "formal_answer_type": "ℝ", "outros": [{"t": "Set (ℝ → ℝ)", "v": null, "name": "C"}, {"t": "C = {f : ℝ → ℝ | ContDiffOn ℝ 1 f (Set.Icc 0 1) ∧ f 0 = 0 ∧ f 1 = 1}", "v": null, "name": "hC"}, {"t": "IsGreatest {u : ℝ | ∀ f ∈ C, u ≤ (∫ x in Set.Ioo 0 1, |deriv f x - f x|)} answer", "v": null, "name": "h_answer"}]} {"informal_problem": "For which real numbers $c$ is $(e^x+e^{-x})/2 \\leq e^{cx^2}$ for all real $x$?", "informal_answer": "$\\{c : \\mathbb{R} \\mid c \\geq 1/2\\}$", "informal_solution": "Show that the inequality holds if and only if $c \\geq 1/2$.", "header": "open Real", "intros": [], "formal_answer": "@Eq (Set Real) answer\n (@setOf Real fun (c_1 : Real) =>\n @GE.ge Real Real.instLE c_1\n (@HDiv.hDiv Real Real Real (@instHDiv Real (@DivInvMonoid.toDiv Real Real.instDivInvMonoid))\n (@OfNat.ofNat Real (nat_lit 1) (@One.toOfNat1 Real Real.instOne))\n (@OfNat.ofNat Real (nat_lit 2)\n (@instOfNatAtLeastTwo Real (nat_lit 2) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 0) (instOfNatNat (nat_lit 0))))))))", "formal_answer_type": "Set ℝ", "outros": [{"t": "ℝ", "v": null, "name": "c"}, {"t": "∀ x : ℝ, (exp x + exp (-x)) / 2 ≤ exp (c * x ^ 2) ↔ c ∈ answer", "v": null, "name": "h_answer"}]} -{"informal_problem": "For which real numbers $a$ does the sequence defined by the initial condition $u_0=a$ and the recursion $u_{n+1}=2u_n-n^2$ have $u_n>0$ for all $n \\geq 0$? (Express the answer in the simplest form.)", "informal_answer": "$\\{a : \\mathbb{R} \\mid a \\geq 3\\}$", "informal_solution": "Show that $u_n>0$ for all $n \\geq 0$ if and only if $a \\geq 3$.", "header": null, "intros": [], "formal_answer": "@Eq (Set Real) answer\n (@setOf Real fun (a_1 : Real) =>\n @GE.ge Real Real.instLE a_1\n (@OfNat.ofNat Real (nat_lit 3)\n (@instOfNatAtLeastTwo Real (nat_lit 3) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1)))))))", "formal_answer_type": "Set ℝ", "outros": [{"t": "ℝ", "v": null, "name": "a"}, {"t": "ℕ → ℝ", "v": null, "name": "u"}, {"t": "u 0 = a ∧ (∀ n : ℕ, u (n + 1) = 2 * u n - n ^ 2)", "v": null, "name": "hu"}, {"t": "(∀ n : ℕ, u n > 0) ↔ a ∈ answer", "v": null, "name": "h_answer"}]} +{"informal_problem": "For which real numbers $a$ does the sequence defined by the initial condition $u_0=a$ and the recursion $u_{n+1}=2u_n-n^2$ have $u_n>0$ for all $n \\geq 0$? (Express the answer in the simplest form.)", "informal_answer": "$\\{a : \\mathbb{R} \\mid a \\geq 3\\}$", "informal_solution": "Show that $u_n>0$ for all $n \\geq 0$ if and only if $a \\geq 3$.", "header": "open BigOperators Real Nat Topology", "intros": [], "formal_answer": "@Eq (Set Real) answer\n (@setOf Real fun (a_1 : Real) =>\n @GE.ge Real Real.instLE a_1\n (@OfNat.ofNat Real (nat_lit 3)\n (@instOfNatAtLeastTwo Real (nat_lit 3) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1)))))))", "formal_answer_type": "Set ℝ", "outros": [{"t": "ℝ", "v": null, "name": "a"}, {"t": "ℕ → ℝ", "v": null, "name": "u"}, {"t": "u 0 = a ∧ (∀ n : ℕ, u (n + 1) = 2 * u n - n ^ 2)", "v": null, "name": "hu"}, {"t": "(∀ n : ℕ, u n > 0) ↔ a ∈ answer", "v": null, "name": "h_answer"}]} {"informal_problem": "A function $f$ is convex on $[0, 1]$ if and only if $$f(su + (1-s)v) \\le sf(u) + (1 - s)f(v)$$ for all $s \\in [0, 1]$.\nLet $S_t$ denote the set of all nonnegative increasing convex continuous functions $f : [0, 1] \\rightarrow \\mathbb{R}$ such that $$f(1) - 2f\\left(\\frac{2}{3}\\right) + f\\left(\\frac{1}{3}\\right) \\ge t\\left(f\\left(\\frac{2}{3}\\right) - 2f\\left(\\frac{1}{3}\\right) + f(0)\\right).$$\nFor which real numbers $t \\ge 0$ is $S_t$ closed under multiplication?", "informal_answer": "$t \\le 1$", "informal_solution": "$S_t$ is closed under multiplication if and only if $1 \\ge t$.", "header": "open Set", "intros": [], "formal_answer": "@Eq (Real → Prop) answer fun (t_1 : Real) =>\n @LE.le Real Real.instLE t_1 (@OfNat.ofNat Real (nat_lit 1) (@One.toOfNat1 Real Real.instOne))", "formal_answer_type": "ℝ → Prop", "outros": [{"t": "Set ℝ", "v": null, "name": "T"}, {"t": "T = Icc 0 1", "v": null, "name": "hT"}, {"t": "ℝ → (ℝ → ℝ) → Prop", "v": null, "name": "P"}, {"t": "(ℝ → ℝ) → Prop", "v": null, "name": "IsConvex"}, {"t": "ℝ → Set (ℝ → ℝ)", "v": null, "name": "S"}, {"t": "∀ t f, P t f ↔ f 1 - 2*f (2/3) + f (1/3) ≥ t*(f (2/3) - 2*f (1/3) + f 0)", "v": null, "name": "P_def"}, {"t": "∀ f, IsConvex f ↔ ∀ u ∈ T, ∀ v ∈ T, ∀ s ∈ T, f (s*u + (1 - s)*v) ≤ s*(f u) + (1 - s)*(f v)", "v": null, "name": "IsConvex_def"}, {"t": "S = fun t : ℝ => {f : ℝ → ℝ | (∀ x ∈ T, f x ≥ 0) ∧ StrictMonoOn f T ∧ IsConvex f ∧ ContinuousOn f T ∧ P t f}", "v": null, "name": "hS"}, {"t": "ℝ", "v": null, "name": "t"}, {"t": "t ≥ 0", "v": null, "name": "ht"}, {"t": "answer t ↔ (∀ f ∈ S t, ∀ g ∈ S t, f * g ∈ S t)", "v": null, "name": "h_answer"}]} {"informal_problem": "Let $E(n)$ be the greatest integer $k$ such that $5^k$ divides $1^1 2^2 3^3 \\cdots n^n$. Find $\\lim_{n \\rightarrow \\infty} \\frac{E(n)}{n^2}$.", "informal_answer": "$\\frac{1}{8}$", "informal_solution": "The limit equals $\\frac{1}{8}$.", "header": "open Topology Filter Set Polynomial Function", "intros": [], "formal_answer": "@Eq Real answer\n (@HDiv.hDiv Real Real Real (@instHDiv Real (@DivInvMonoid.toDiv Real Real.instDivInvMonoid))\n (@OfNat.ofNat Real (nat_lit 1) (@One.toOfNat1 Real Real.instOne))\n (@OfNat.ofNat Real (nat_lit 8)\n (@instOfNatAtLeastTwo Real (nat_lit 8) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 6) (instOfNatNat (nat_lit 6)))))))", "formal_answer_type": "ℝ", "outros": [{"t": "ℕ → ℕ → Prop", "v": null, "name": "P"}, {"t": "∀ n k, P n k ↔ 5^k ∣ ∏ m in Finset.Icc 1 n, (m^m : ℤ)", "v": null, "name": "hP"}, {"t": "ℕ → ℕ", "v": null, "name": "E"}, {"t": "∀ n ∈ Ici 1, P n (E n) ∧ ∀ k : ℕ, P n k → k ≤ E n", "v": null, "name": "hE"}, {"t": "Tendsto (fun n : ℕ => ((E n) : ℝ)/n^2) atTop (𝓝 answer)", "v": null, "name": "h_answer"}]} {"informal_problem": "Does the limit $$lim_{t \\rightarrow \\infty}e^{-t}\\int_{0}^{t}\\int_{0}^{t}\\frac{e^x - e^y}{x - y} dx dy$$exist?", "informal_answer": "False", "informal_solution": "The limit does not exist.", "header": "open Topology Filter Set Polynomial Function", "intros": [], "formal_answer": "@Eq Prop answer False", "formal_answer_type": "Prop", "outros": [{"t": "ℝ → ℝ", "v": null, "name": "f"}, {"t": "f = fun t : ℝ => Real.exp (-t) * ∫ y in (Ico 0 t), ∫ x in (Ico 0 t), (Real.exp x - Real.exp y) / (x - y)", "v": null, "name": "hf"}, {"t": "(∃ L : ℝ, Tendsto f atTop (𝓝 L)) ↔ answer", "v": null, "name": "h_answer"}]} @@ -77,12 +77,12 @@ {"informal_problem": "Let $A(x, y)$ denote the number of points $(m, n)$ with integer coordinates $m$ and $n$ where $m^2 + n^2 \\le x^2 + y^2$. Also, let $g = \\sum_{k = 0}^{\\infty} e^{-k^2}$. Express the value $$\\int_{-\\infty}^{\\infty}\\int_{-\\infty}^{\\infty} A(x, y)e^{-x^2 - y^2} dx dy$$ as a polynomial in $g$.", "informal_answer": "C Real.pi * (2*X - 1)^2", "informal_solution": "The desired polynomial is $\\pi(2g - 1)^2$.", "header": "open Set Function Filter Topology Polynomial Real", "intros": [], "formal_answer": "@Eq (@Polynomial Real Real.semiring) answer\n (@HMul.hMul (@Polynomial Real Real.semiring) (@Polynomial Real Real.semiring) (@Polynomial Real Real.semiring)\n (@instHMul (@Polynomial Real Real.semiring) (@Polynomial.mul' Real Real.semiring))\n (@DFunLike.coe\n (@RingHom Real (@Polynomial Real Real.semiring) (@Semiring.toNonAssocSemiring Real Real.semiring)\n (@Semiring.toNonAssocSemiring (@Polynomial Real Real.semiring) (@Polynomial.semiring Real Real.semiring)))\n Real (fun (x : Real) => @Polynomial Real Real.semiring)\n (@RingHom.instFunLike Real (@Polynomial Real Real.semiring) (@Semiring.toNonAssocSemiring Real Real.semiring)\n (@Semiring.toNonAssocSemiring (@Polynomial Real Real.semiring) (@Polynomial.semiring Real Real.semiring)))\n (@Polynomial.C Real Real.semiring) Real.pi)\n (@HPow.hPow (@Polynomial Real Real.semiring) Nat (@Polynomial Real Real.semiring)\n (@instHPow (@Polynomial Real Real.semiring) Nat\n (@Monoid.toNatPow (@Polynomial Real Real.semiring)\n (@MonoidWithZero.toMonoid (@Polynomial Real Real.semiring)\n (@Semiring.toMonoidWithZero (@Polynomial Real Real.semiring) (@Polynomial.semiring Real Real.semiring)))))\n (@HSub.hSub (@Polynomial Real Real.semiring) (@Polynomial Real Real.semiring) (@Polynomial Real Real.semiring)\n (@instHSub (@Polynomial Real Real.semiring) (@Polynomial.sub Real Real.instRing))\n (@HMul.hMul (@Polynomial Real Real.semiring) (@Polynomial Real Real.semiring) (@Polynomial Real Real.semiring)\n (@instHMul (@Polynomial Real Real.semiring) (@Polynomial.mul' Real Real.semiring))\n (@OfNat.ofNat (@Polynomial Real Real.semiring) (nat_lit 2)\n (@instOfNatAtLeastTwo (@Polynomial Real Real.semiring) (nat_lit 2)\n (@Polynomial.instNatCast Real Real.semiring)\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 0) (instOfNatNat (nat_lit 0))))))\n (@Polynomial.X Real Real.semiring))\n (@OfNat.ofNat (@Polynomial Real Real.semiring) (nat_lit 1)\n (@One.toOfNat1 (@Polynomial Real Real.semiring) (@Polynomial.one Real Real.semiring))))\n (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))))", "formal_answer_type": "Polynomial ℝ", "outros": [{"t": "ℝ × ℝ → ℕ", "v": null, "name": "A"}, {"t": "ℝ", "v": null, "name": "g"}, {"t": "ℝ", "v": null, "name": "I"}, {"t": "A = fun (x, y) => {a : ℤ × ℤ | a.1^2 + a.2^2 ≤ x^2 + y^2}.ncard", "v": null, "name": "hA"}, {"t": "g = ∑' k : ℕ, Real.exp (-k^2)", "v": null, "name": "hg"}, {"t": "I = ∫ y : ℝ, ∫ x : ℝ, A (x, y) * Real.exp (-x^2 - y^2)", "v": null, "name": "hI"}, {"t": "I = answer.eval g", "v": null, "name": "h_answer"}]} {"informal_problem": "Let $p_n$ denote the probability that $c + d$ will be a perfect square if $c$ and $d$ are selected independently and uniformly at random from $\\{1, 2, 3, \\dots, n\\}$. Express $\\lim_{n \\rightarrow \\infty} p_n \\sqrt{n}$ in the form $r(\\sqrt{s} - t)$ for integers $s$ and $t$ and rational $r$.", "informal_answer": "4/3 * (Real.sqrt 2 - 1)", "informal_solution": "The limit equals $\\frac{4}{3}(\\sqrt{2} - 1)$.", "header": "open Set Function Filter Topology Polynomial Real", "intros": [], "formal_answer": "@Eq Real answer\n (@HMul.hMul Real Real Real (@instHMul Real Real.instMul)\n (@HDiv.hDiv Real Real Real (@instHDiv Real (@DivInvMonoid.toDiv Real Real.instDivInvMonoid))\n (@OfNat.ofNat Real (nat_lit 4)\n (@instOfNatAtLeastTwo Real (nat_lit 4) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))))))\n (@OfNat.ofNat Real (nat_lit 3)\n (@instOfNatAtLeastTwo Real (nat_lit 3) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1)))))))\n (@HSub.hSub Real Real Real (@instHSub Real Real.instSub)\n (Real.sqrt\n (@OfNat.ofNat Real (nat_lit 2)\n (@instOfNatAtLeastTwo Real (nat_lit 2) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 0) (instOfNatNat (nat_lit 0)))))))\n (@OfNat.ofNat Real (nat_lit 1) (@One.toOfNat1 Real Real.instOne))))", "formal_answer_type": "ℝ", "outros": [{"t": "ℕ → ℝ", "v": null, "name": "p"}, {"t": "p = fun n : ℕ => ({c : Finset.Icc 1 n × Finset.Icc 1 n | ∃ m : ℕ, m^2 = c.1 + c.2}.ncard : ℝ) / n^2", "v": null, "name": "hp"}, {"t": "Tendsto (fun n : ℕ => p n * Real.sqrt n) atTop (𝓝 answer)", "v": null, "name": "h_answer"}]} {"informal_problem": "Let $n_1, n_2, \\dots, n_s$ be distinct integers such that, for every integer $k$, $n_1n_2\\cdots n_s$ divides $(n_1 + k)(n_2 + k) \\cdots (n_s + k)$. Prove or provide a counterexample to the following claims:\n\\begin{enumerate}\n\\item\nFor some $i$, $|n_i| = 1$.\n\\item\nIf all $n_i$ are positive, then $\\{n_1, n_2, \\dots, n_s\\} = \\{1, 2, \\dots, s\\}$.\n\\end{enumerate}", "informal_answer": "(True, True)", "informal_solution": "Both claims are true.", "header": "open Set Function Filter Topology Polynomial Real", "intros": [], "formal_answer": "@Eq (Prod Prop Prop) answer (@Prod.mk Prop Prop True True)", "formal_answer_type": "Prop × Prop", "outros": [{"t": "Finset ℤ → Prop", "v": null, "name": "P"}, {"t": "∀ n, P n ↔ n.Nonempty ∧ ∀ k, ∏ i in n, i ∣ ∏ i in n, (i + k)", "v": null, "name": "P_def"}, {"t": "((∀ n, P n → 1 ∈ n ∨ -1 ∈ n) ↔ answer.1) ∧\n ((∀ n, P n → (∀ i ∈ n, 0 < i) → n = Finset.Icc (1 : ℤ) n.card) ↔ answer.2)", "v": null, "name": "h_answer"}]} -{"informal_problem": "How many positive integers $n$ are there such that $n$ is an exact divisor of at least one of the numbers $10^{40},20^{30}$?", "informal_answer": "2301", "informal_solution": "Show that the desired count is $2301$.", "header": null, "intros": [], "formal_answer": "@Eq Nat answer (@OfNat.ofNat Nat (nat_lit 2301) (instOfNatNat (nat_lit 2301)))", "formal_answer_type": "ℕ", "outros": [{"t": "{n : ℤ | n > 0 ∧ (n ∣ 10 ^ 40 ∨ n ∣ 20 ^ 30)}.encard = answer", "v": null, "name": "h_answer"}]} +{"informal_problem": "How many positive integers $n$ are there such that $n$ is an exact divisor of at least one of the numbers $10^{40},20^{30}$?", "informal_answer": "2301", "informal_solution": "Show that the desired count is $2301$.", "header": "open BigOperators Real Nat Topology", "intros": [], "formal_answer": "@Eq Nat answer (@OfNat.ofNat Nat (nat_lit 2301) (instOfNatNat (nat_lit 2301)))", "formal_answer_type": "ℕ", "outros": [{"t": "{n : ℤ | n > 0 ∧ (n ∣ 10 ^ 40 ∨ n ∣ 20 ^ 30)}.encard = answer", "v": null, "name": "h_answer"}]} {"informal_problem": "Prove or disprove that there exists a positive real number $\\alpha$ such that $[\\alpha_n] - n$ is even for all integers $n > 0$. (Here $[x]$ denotes the greatest integer less than or equal to $x$.)", "informal_answer": "True", "informal_solution": "Prove that such an $\\alpha$ exists.", "header": "open Nat", "intros": [], "formal_answer": "@Eq Prop answer True", "formal_answer_type": "Prop", "outros": [{"t": "answer ↔ (∃ α : ℝ, α > 0 ∧ ∀ n : ℕ, n > 0 → Even (⌊α ^ n⌋ - n))", "v": null, "name": "h_answer"}]} {"informal_problem": "Let $T$ be the triangle with vertices $(0, 0)$, $(a, 0)$, and $(0, a)$. Find $\\lim_{a \\to \\infty} a^4 \\exp(-a^3) \\int_T \\exp(x^3+y^3) \\, dx \\, dy$.", "informal_answer": "2 / 9", "informal_solution": "Show that the integral evaluates to $\\frac{2}{9}$.", "header": "open Nat Filter Topology Real", "intros": [], "formal_answer": "@Eq Real answer\n (@HDiv.hDiv Real Real Real (@instHDiv Real (@DivInvMonoid.toDiv Real Real.instDivInvMonoid))\n (@OfNat.ofNat Real (nat_lit 2)\n (@instOfNatAtLeastTwo Real (nat_lit 2) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 0) (instOfNatNat (nat_lit 0))))))\n (@OfNat.ofNat Real (nat_lit 9)\n (@instOfNatAtLeastTwo Real (nat_lit 9) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 7) (instOfNatNat (nat_lit 7)))))))", "formal_answer_type": "ℝ", "outros": [{"t": "ℝ → ℝ", "v": null, "name": "F"}, {"t": "F = fun a ↦ (a ^ 4 / exp (a ^ 3)) * ∫ x in (0)..a, ∫ y in (0)..(a - x), exp (x ^ 3 + y ^ 3)", "v": null, "name": "hF"}, {"t": "Tendsto F atTop (𝓝 answer)", "v": null, "name": "h_answer"}]} {"informal_problem": "Let $f(n)$ be the number of ways of representing $n$ as a sum of powers of $2$ with no power being used more than $3$ times. For example, $f(7) = 4$ (the representations are $4 + 2 + 1$, $4 + 1 + 1 + 1$, $2 + 2 + 2 + 1$, $2 + 2 + 1 + 1 + 1$). Can we find a real polynomial $p(x)$ such that $f(n) = [p(n)]$, where $[u]$ denotes the greatest integer less than or equal to $u$?", "informal_answer": "True", "informal_solution": "Prove that such a polynomial exists.", "header": "open Nat Filter Topology Real", "intros": [], "formal_answer": "@Eq Prop answer True", "formal_answer_type": "Prop", "outros": [{"t": "ℕ+ → ℕ", "v": null, "name": "f"}, {"t": "f = fun (n : ℕ+) ↦\n Set.ncard {M : Multiset ℕ |\n (∀ m ∈ M, ∃ k : ℕ, m = (2 ^ k : ℤ)) ∧ \n (∀ m ∈ M, M.count m ≤ 3) ∧ \n (M.sum : ℤ) = n}", "v": null, "name": "hf"}, {"t": "answer ↔ (∃ p : Polynomial ℝ, ∀ n : ℕ+, ⌊p.eval (n : ℝ)⌋ = f n)", "v": null, "name": "h_answer"}]} {"informal_problem": "Define $\\left\\lVert x \\right\\rVert$ as the distance from $x$ to the nearest integer. Find $\\lim_{n \\to \\infty} \\frac{1}{n} \\int_{1}^{n} \\left\\lVert \\frac{n}{x} \\right\\rVert \\, dx$. You may assume that $\\prod_{n=1}^{\\infty} \\frac{2n}{(2n-1)} \\cdot \\frac{2n}{(2n+1)} = \\frac{\\pi}{2}$.", "informal_answer": "$\\log \\left(\\frac{4}{\\pi}\\right)$", "informal_solution": "Show that the limit equals $\\ln \\left( \\frac{4}{\\pi} \\right)$.", "header": "open Nat Filter Topology Real", "intros": [], "formal_answer": "@Eq Real answer\n (Real.log\n (@HDiv.hDiv Real Real Real (@instHDiv Real (@DivInvMonoid.toDiv Real Real.instDivInvMonoid))\n (@OfNat.ofNat Real (nat_lit 4)\n (@instOfNatAtLeastTwo Real (nat_lit 4) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))))))\n Real.pi))", "formal_answer_type": "ℝ", "outros": [{"t": "ℝ → ℝ", "v": null, "name": "dist_fun"}, {"t": "dist_fun = fun (x : ℝ) ↦ min (x - ⌊x⌋) (⌈x⌉ - x)", "v": null, "name": "hdist_fun"}, {"t": "Tendsto (fun N ↦ ∏ n in Finset.Icc 1 N, (2 * n / (2 * n - 1)) * (2 * n / (2 * n + 1)) : ℕ → ℝ) atTop (𝓝 (Real.pi / 2))", "v": null, "name": "fact"}, {"t": "Tendsto (fun n ↦ (1 / n) * ∫ x in (1)..n, dist_fun (n / x) : ℕ → ℝ) atTop (𝓝 answer)", "v": null, "name": "h_answer"}]} -{"informal_problem": "Express $\\sum_{k=1}^\\infty (6^k/(3^{k+1}-2^{k+1})(3^k-2^k))$ as a rational number.", "informal_answer": "2", "informal_solution": "Show that the sum converges to $2$.", "header": null, "intros": [], "formal_answer": "@Eq Rat answer (@OfNat.ofNat Rat (nat_lit 2) (@Rat.instOfNat (nat_lit 2)))", "formal_answer_type": "ℚ", "outros": [{"t": "∑' k : Set.Ici 1, (6 ^ (k : ℕ) / ((3 ^ ((k : ℕ) + 1) - 2 ^ ((k : ℕ) + 1)) * (3 ^ (k : ℕ) - 2 ^ (k : ℕ)))) = answer", "v": null, "name": "h_answer"}]} +{"informal_problem": "Express $\\sum_{k=1}^\\infty (6^k/(3^{k+1}-2^{k+1})(3^k-2^k))$ as a rational number.", "informal_answer": "2", "informal_solution": "Show that the sum converges to $2$.", "header": "open BigOperators Real Nat Topology", "intros": [], "formal_answer": "@Eq Rat answer (@OfNat.ofNat Rat (nat_lit 2) (@Rat.instOfNat (nat_lit 2)))", "formal_answer_type": "ℚ", "outros": [{"t": "∑' k : Set.Ici 1, (6 ^ (k : ℕ) / ((3 ^ ((k : ℕ) + 1) - 2 ^ ((k : ℕ) + 1)) * (3 ^ (k : ℕ) - 2 ^ (k : ℕ)))) = answer", "v": null, "name": "h_answer"}]} {"informal_problem": "Let $n$ be a positive integer. Let $a,b,x$ be real numbers, with $a \\neq b$, and let $M_n$ denote the $2n \\times 2n$ matrix whose $(i,j)$ entry $m_{ij}$ is given by\n\\[\nm_{ij}=\\begin{cases}\nx & \\text{if }i=j, \\\\\na & \\text{if }i \\neq j\\text{ and }i+j\\text{ is even}, \\\\\nb & \\text{if }i \\neq j\\text{ and }i+j\\text{ is odd}.\n\\end{cases}\n\\]\nThus, for example, $M_2=\\begin{pmatrix} x & b & a & b \\\\ b & x & b & a \\\\ a & b & x & b \\\\ b & a & b & x \\end{pmatrix}$. Express $\\lim_{x \\to a} \\det M_n/(x-a)^{2n-2}$ as a polynomial in $a$, $b$, and $n$, where $\\det M_n$ denotes the determinant of $M_n$.", "informal_answer": "$(X_2)^2 \\cdot ((X_0)^2 - (X_1)^2)$", "informal_solution": "Show that $\\lim_{x \\to a} \\frac{\\det M_n}{(x-a)^{2n-2}}=n^2(a^2-b^2)$.", "header": "open Topology Filter", "intros": [], "formal_answer": "@Eq (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 3) (instOfNatNat (nat_lit 3)))) Real Real.instCommSemiring) answer\n (@HMul.hMul (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 3) (instOfNatNat (nat_lit 3)))) Real Real.instCommSemiring)\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 3) (instOfNatNat (nat_lit 3)))) Real Real.instCommSemiring)\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 3) (instOfNatNat (nat_lit 3)))) Real Real.instCommSemiring)\n (@instHMul\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 3) (instOfNatNat (nat_lit 3)))) Real Real.instCommSemiring)\n (@Distrib.toMul\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 3) (instOfNatNat (nat_lit 3)))) Real Real.instCommSemiring)\n (@NonUnitalNonAssocSemiring.toDistrib\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 3) (instOfNatNat (nat_lit 3)))) Real Real.instCommSemiring)\n (@NonUnitalNonAssocCommSemiring.toNonUnitalNonAssocSemiring\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 3) (instOfNatNat (nat_lit 3)))) Real Real.instCommSemiring)\n (@NonUnitalNonAssocCommRing.toNonUnitalNonAssocCommSemiring\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 3) (instOfNatNat (nat_lit 3)))) Real Real.instCommSemiring)\n (@NonUnitalCommRing.toNonUnitalNonAssocCommRing\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 3) (instOfNatNat (nat_lit 3)))) Real\n Real.instCommSemiring)\n (@CommRing.toNonUnitalCommRing\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 3) (instOfNatNat (nat_lit 3)))) Real\n Real.instCommSemiring)\n (@MvPolynomial.instCommRingMvPolynomial Real\n (Fin (@OfNat.ofNat Nat (nat_lit 3) (instOfNatNat (nat_lit 3)))) Real.commRing))))))))\n (@HPow.hPow\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 3) (instOfNatNat (nat_lit 3)))) Real Real.instCommSemiring) Nat\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 3) (instOfNatNat (nat_lit 3)))) Real Real.instCommSemiring)\n (@instHPow\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 3) (instOfNatNat (nat_lit 3)))) Real Real.instCommSemiring) Nat\n (@Monoid.toNatPow\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 3) (instOfNatNat (nat_lit 3)))) Real Real.instCommSemiring)\n (@MonoidWithZero.toMonoid\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 3) (instOfNatNat (nat_lit 3)))) Real Real.instCommSemiring)\n (@Semiring.toMonoidWithZero\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 3) (instOfNatNat (nat_lit 3)))) Real Real.instCommSemiring)\n (@CommSemiring.toSemiring\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 3) (instOfNatNat (nat_lit 3)))) Real\n Real.instCommSemiring)\n (@MvPolynomial.commSemiring Real (Fin (@OfNat.ofNat Nat (nat_lit 3) (instOfNatNat (nat_lit 3))))\n Real.instCommSemiring))))))\n (@MvPolynomial.X Real (Fin (@OfNat.ofNat Nat (nat_lit 3) (instOfNatNat (nat_lit 3)))) Real.instCommSemiring\n (@OfNat.ofNat (Fin (@OfNat.ofNat Nat (nat_lit 3) (instOfNatNat (nat_lit 3)))) (nat_lit 2)\n (@Fin.instOfNat (@OfNat.ofNat Nat (nat_lit 3) (instOfNatNat (nat_lit 3)))\n (@Nat.instNeZeroSucc (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) (nat_lit 2))))\n (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))))\n (@HSub.hSub\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 3) (instOfNatNat (nat_lit 3)))) Real Real.instCommSemiring)\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 3) (instOfNatNat (nat_lit 3)))) Real Real.instCommSemiring)\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 3) (instOfNatNat (nat_lit 3)))) Real Real.instCommSemiring)\n (@instHSub\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 3) (instOfNatNat (nat_lit 3)))) Real Real.instCommSemiring)\n (@SubNegMonoid.toSub\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 3) (instOfNatNat (nat_lit 3)))) Real Real.instCommSemiring)\n (@AddGroup.toSubNegMonoid\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 3) (instOfNatNat (nat_lit 3)))) Real Real.instCommSemiring)\n (@AddGroupWithOne.toAddGroup\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 3) (instOfNatNat (nat_lit 3)))) Real Real.instCommSemiring)\n (@Ring.toAddGroupWithOne\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 3) (instOfNatNat (nat_lit 3)))) Real\n Real.instCommSemiring)\n (@CommRing.toRing\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 3) (instOfNatNat (nat_lit 3)))) Real\n Real.instCommSemiring)\n (@MvPolynomial.instCommRingMvPolynomial Real\n (Fin (@OfNat.ofNat Nat (nat_lit 3) (instOfNatNat (nat_lit 3)))) Real.commRing)))))))\n (@HPow.hPow\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 3) (instOfNatNat (nat_lit 3)))) Real Real.instCommSemiring) Nat\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 3) (instOfNatNat (nat_lit 3)))) Real Real.instCommSemiring)\n (@instHPow\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 3) (instOfNatNat (nat_lit 3)))) Real Real.instCommSemiring) Nat\n (@Monoid.toNatPow\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 3) (instOfNatNat (nat_lit 3)))) Real Real.instCommSemiring)\n (@MonoidWithZero.toMonoid\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 3) (instOfNatNat (nat_lit 3)))) Real Real.instCommSemiring)\n (@Semiring.toMonoidWithZero\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 3) (instOfNatNat (nat_lit 3)))) Real\n Real.instCommSemiring)\n (@CommSemiring.toSemiring\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 3) (instOfNatNat (nat_lit 3)))) Real\n Real.instCommSemiring)\n (@MvPolynomial.commSemiring Real (Fin (@OfNat.ofNat Nat (nat_lit 3) (instOfNatNat (nat_lit 3))))\n Real.instCommSemiring))))))\n (@MvPolynomial.X Real (Fin (@OfNat.ofNat Nat (nat_lit 3) (instOfNatNat (nat_lit 3)))) Real.instCommSemiring\n (@OfNat.ofNat (Fin (@OfNat.ofNat Nat (nat_lit 3) (instOfNatNat (nat_lit 3)))) (nat_lit 0)\n (@Fin.instOfNat (@OfNat.ofNat Nat (nat_lit 3) (instOfNatNat (nat_lit 3)))\n (@Nat.instNeZeroSucc (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) (nat_lit 0))))\n (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))))\n (@HPow.hPow\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 3) (instOfNatNat (nat_lit 3)))) Real Real.instCommSemiring) Nat\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 3) (instOfNatNat (nat_lit 3)))) Real Real.instCommSemiring)\n (@instHPow\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 3) (instOfNatNat (nat_lit 3)))) Real Real.instCommSemiring) Nat\n (@Monoid.toNatPow\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 3) (instOfNatNat (nat_lit 3)))) Real Real.instCommSemiring)\n (@MonoidWithZero.toMonoid\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 3) (instOfNatNat (nat_lit 3)))) Real Real.instCommSemiring)\n (@Semiring.toMonoidWithZero\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 3) (instOfNatNat (nat_lit 3)))) Real\n Real.instCommSemiring)\n (@CommSemiring.toSemiring\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 3) (instOfNatNat (nat_lit 3)))) Real\n Real.instCommSemiring)\n (@MvPolynomial.commSemiring Real (Fin (@OfNat.ofNat Nat (nat_lit 3) (instOfNatNat (nat_lit 3))))\n Real.instCommSemiring))))))\n (@MvPolynomial.X Real (Fin (@OfNat.ofNat Nat (nat_lit 3) (instOfNatNat (nat_lit 3)))) Real.instCommSemiring\n (@OfNat.ofNat (Fin (@OfNat.ofNat Nat (nat_lit 3) (instOfNatNat (nat_lit 3)))) (nat_lit 1)\n (@Fin.instOfNat (@OfNat.ofNat Nat (nat_lit 3) (instOfNatNat (nat_lit 3)))\n (@Nat.instNeZeroSucc (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) (nat_lit 1))))\n (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))))))", "formal_answer_type": "MvPolynomial (Fin 3) ℝ", "outros": [{"t": "ℕ", "v": null, "name": "n"}, {"t": "ℝ", "v": null, "name": "a"}, {"t": "ℝ", "v": null, "name": "b"}, {"t": "ℝ → Matrix (Fin (2 * n)) (Fin (2 * n)) ℝ", "v": null, "name": "Mn"}, {"t": "Fin 3 → ℝ", "v": null, "name": "polyabn"}, {"t": "n > 0", "v": null, "name": "npos"}, {"t": "a ≠ b", "v": null, "name": "aneb"}, {"t": "Mn = fun x : ℝ => fun i j : Fin (2 * n) => if i = j then x else if Even (i.1 + j.1) then a else b", "v": null, "name": "hMn"}, {"t": "polyabn 0 = a ∧ polyabn 1 = b ∧ polyabn 2 = n", "v": null, "name": "hpolyabn"}, {"t": "Tendsto (fun x : ℝ => (Mn x).det / (x - a) ^ (2 * n - 2)) (𝓝[≠] a) (𝓝 (MvPolynomial.eval polyabn answer))", "v": null, "name": "h_answer"}]} {"informal_problem": "Let $R$ be the region consisting of all triples $(x,y,z)$ of nonnegative real numbers satisfying $x+y+z \\leq 1$. Let $w=1-x-y-z$. Express the value of the triple integral $\\iiint_R x^1y^9z^8w^4\\,dx\\,dy\\,dz$ in the form $a!b!c!d!/n!$, where $a$, $b$, $c$, $d$, and $n$ are positive integers.", "informal_answer": "(1, 9, 8, 4, 25)", "informal_solution": "Show that the integral we desire is $1!9!8!4!/25!$.", "header": "open Topology Filter Nat", "intros": [], "formal_answer": "@Eq (Prod Nat (Prod Nat (Prod Nat (Prod Nat Nat)))) answer\n (@Prod.mk Nat (Prod Nat (Prod Nat (Prod Nat Nat))) (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1)))\n (@Prod.mk Nat (Prod Nat (Prod Nat Nat)) (@OfNat.ofNat Nat (nat_lit 9) (instOfNatNat (nat_lit 9)))\n (@Prod.mk Nat (Prod Nat Nat) (@OfNat.ofNat Nat (nat_lit 8) (instOfNatNat (nat_lit 8)))\n (@Prod.mk Nat Nat (@OfNat.ofNat Nat (nat_lit 4) (instOfNatNat (nat_lit 4)))\n (@OfNat.ofNat Nat (nat_lit 25) (instOfNatNat (nat_lit 25)))))))", "formal_answer_type": "ℕ × ℕ × ℕ × ℕ × ℕ", "outros": [{"t": "Set (Fin 3 → ℝ)", "v": null, "name": "R"}, {"t": "(Fin 3 → ℝ) → ℝ", "v": null, "name": "w"}, {"t": "R = {p | (∀ i : Fin 3, p i ≥ 0) ∧ p 0 + p 1 + p 2 ≤ 1}", "v": null, "name": "hR"}, {"t": "∀ p, w p = 1 - p 0 - p 1 - p 2", "v": null, "name": "hw"}, {"t": "ℕ", "v": null, "name": "a"}, {"t": "ℕ", "v": null, "name": "b"}, {"t": "ℕ", "v": null, "name": "c"}, {"t": "ℕ", "v": null, "name": "d"}, {"t": "ℕ", "v": null, "name": "n"}, {"t": "answer = (a, b, c, d, n)", "v": null, "name": "h_answer"}, {"t": "a > 0 ∧ b > 0 ∧ c > 0 ∧ d > 0 ∧ n > 0", "v": null, "name": "h_pos"}, {"t": "(∫ p in R, (p 0) ^ 1 * (p 1) ^ 9 * (p 2) ^ 8 * (w p) ^ 4 = ((a)! * (b)! * (c)! * (d)! : ℝ) / (n)!)", "v": null, "name": "h_integral"}]} {"informal_problem": "Let $n$ be a positive integer, and let $f(n)$ denote the last nonzero digit in the decimal expansion of $n!$. For instance, $f(5)=2$.\n\\begin{enumerate}\n\\item[(a)] Show that if $a_1,a_2,\\dots,a_k$ are \\emph{distinct} nonnegative integers, then $f(5^{a_1}+5^{a_2}+\\dots+5^{a_k})$ depends only on the sum $a_1+a_2+\\dots+a_k$.\n\\item[(b)] Assuming part (a), we can define $g(s)=f(5^{a_1}+5^{a_2}+\\dots+5^{a_k})$, where $s=a_1+a_2+\\dots+a_k$. Find the least positive integer $p$ for which $g(s)=g(s + p)$, for all $s \\geq 1$, or else show that no such $p$ exists.\n\\end{enumerate}", "informal_answer": "4", "informal_solution": "Show that the least such $p$ is $p=4$.", "header": "open Topology Filter Function Nat", "intros": [], "formal_answer": "@Eq Nat answer (@OfNat.ofNat Nat (nat_lit 4) (instOfNatNat (nat_lit 4)))", "formal_answer_type": "ℕ", "outros": [{"t": "ℕ → ℕ", "v": null, "name": "f"}, {"t": "∀ n, some (f n) = (Nat.digits 10 (n !)).find? (fun d ↦ d ≠ 0)", "v": null, "name": "hf"}, {"t": "ℕ → (ℕ → ℕ) → ℕ → Prop", "v": null, "name": "IsPeriodicFrom"}, {"t": "∀ x f p, IsPeriodicFrom x f p ↔ Periodic (f ∘ (· + x)) p", "v": null, "name": "IsPeriodicFrom_def"}, {"t": "ℕ → (ℕ → ℕ) → ℕ → Prop", "v": null, "name": "P"}, {"t": "∀ x g p, P x g p ↔ if p = 0 then (∀ q > 0, ¬ IsPeriodicFrom x g q) else\n IsLeast {q | 0 < q ∧ IsPeriodicFrom x g q} p", "v": null, "name": "P_def"}, {"t": "∃ g : ℕ → ℕ,\n (∀ᵉ (k > 0) (a : Fin k → ℕ) (ha : Injective a), f (∑ i, 5 ^ (a i)) = g (∑ i, a i)) ∧\n P 1 g answer", "v": null, "name": "h_answer"}]} @@ -98,8 +98,8 @@ {"informal_problem": "Let $k$ be the smallest positive integer for which there exist distinct integers $m_1, m_2, m_3, m_4, m_5$ such that the polynomial\n\\[\np(x) = (x-m_1)(x-m_2)(x-m_3)(x-m_4)(x-m_5)\n\\]\nhas exactly $k$ nonzero coefficients. Find, with proof, a set of integers $m_1, m_2, m_3, m_4, m_5$ for which this minimum $k$ is achieved.", "informal_answer": "fun i : Fin 5 ↦ ↑i - (2 : ℤ)", "informal_solution": "Show that the minimum $k = 3$ is obtained for $\\{m_1, m_2, m_3, m_4, m_5\\} = \\{-2, -1, 0, 1, 2\\}$.", "header": "open Set Filter Topology Real Polynomial Function", "intros": [], "formal_answer": "@Eq (Fin (@OfNat.ofNat Nat (nat_lit 5) (instOfNatNat (nat_lit 5))) → Int) answer\n fun (i : Fin (@OfNat.ofNat Nat (nat_lit 5) (instOfNatNat (nat_lit 5)))) =>\n @HSub.hSub Int Int Int (@instHSub Int Int.instSub)\n (@Nat.cast Int instNatCastInt (@Fin.val (@OfNat.ofNat Nat (nat_lit 5) (instOfNatNat (nat_lit 5))) i))\n (@OfNat.ofNat Int (nat_lit 2) (@instOfNat (nat_lit 2)))", "formal_answer_type": "Fin 5 → ℤ", "outros": [{"t": "(Fin 5 → ℤ) → (Polynomial ℝ)", "v": null, "name": "p"}, {"t": "p = fun m ↦ ∏ i : Fin 5, ((X : Polynomial ℝ) - m i)", "v": null, "name": "hp"}, {"t": "Polynomial ℝ → ℕ", "v": null, "name": "numnzcoeff"}, {"t": "numnzcoeff = fun p ↦ {j ∈ Finset.range (p.natDegree + 1) | coeff p j ≠ 0}.card", "v": null, "name": "hnumnzcoeff"}, {"t": "(Injective answer ∧ ∀ m : Fin 5 → ℤ, Injective m → numnzcoeff (p answer) ≤ numnzcoeff (p m))", "v": null, "name": "h_answer"}]} {"informal_problem": "Define polynomials $f_n(x)$ for $n \\geq 0$ by $f_0(x)=1$, $f_n(0)=0$ for $n \\geq 1$, and\n\\[\n\\frac{d}{dx} f_{n+1}(x) = (n+1)f_n(x+1)\n\\]\nfor $n \\geq 0$. Find, with proof, the explicit factorization of $f_{100}(1)$ into powers of distinct primes.", "informal_answer": "99 if $n = 101$, otherwise 0", "informal_solution": "Show that $f_{100}(1) = 101^{99}$.", "header": "open Set Filter Topology Real Polynomial Function", "intros": [], "formal_answer": "@Eq (Nat → Nat) answer fun (n : Nat) =>\n @ite Nat (@Eq Nat n (@OfNat.ofNat Nat (nat_lit 101) (instOfNatNat (nat_lit 101))))\n (instDecidableEqNat n (@OfNat.ofNat Nat (nat_lit 101) (instOfNatNat (nat_lit 101))))\n (@OfNat.ofNat Nat (nat_lit 99) (instOfNatNat (nat_lit 99)))\n (@OfNat.ofNat Nat (nat_lit 0) (instOfNatNat (nat_lit 0)))", "formal_answer_type": "ℕ → ℕ", "outros": [{"t": "ℕ -> Polynomial ℕ", "v": null, "name": "f"}, {"t": "f 0 = 1", "v": null, "name": "hf0x"}, {"t": "∀ n ≥ 1, (f n).eval 0 = 0", "v": null, "name": "hfn0"}, {"t": "∀ n : ℕ, derivative (f (n + 1)) = (n + 1) * (Polynomial.comp (f n) (X + 1))", "v": null, "name": "hfderiv"}, {"t": "Nat.factorization ((f 100).eval 1) = answer", "v": null, "name": "h_answer"}]} {"informal_problem": "Evaluate $\\int_0^\\infty t^{-1/2}e^{-1985(t+t^{-1})}\\,dt$. You may assume that $\\int_{-\\infty}^\\infty e^{-x^2}\\,dx = \\sqrt{\\pi}$.", "informal_answer": "$\\sqrt{\\pi / 1985} \\cdot e^{-3970}$", "informal_solution": "Show that the integral evaluates to $\\sqrt{\\frac{\\pi}{1985}}e^{-3970}$.", "header": "open Set Filter Topology Real Polynomial Function", "intros": [], "formal_answer": "@Eq Real answer\n (@HMul.hMul Real Real Real (@instHMul Real Real.instMul)\n (Real.sqrt\n (@HDiv.hDiv Real Real Real (@instHDiv Real (@DivInvMonoid.toDiv Real Real.instDivInvMonoid)) Real.pi\n (@OfNat.ofNat Real (nat_lit 1985)\n (@instOfNatAtLeastTwo Real (nat_lit 1985) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 1983) (instOfNatNat (nat_lit 1983))))))))\n (Real.exp\n (@Neg.neg Real Real.instNeg\n (@OfNat.ofNat Real (nat_lit 3970)\n (@instOfNatAtLeastTwo Real (nat_lit 3970) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 3968) (instOfNatNat (nat_lit 3968)))))))))", "formal_answer_type": "ℝ", "outros": [{"t": "∫ x in Set.univ, Real.exp (- x ^ 2) = Real.sqrt Real.pi", "v": null, "name": "fact"}, {"t": "∫ t in Set.Ioi 0, t ^ (- (1 : ℝ) / 2) * Real.exp (-1985 * (t + t ^ (-(1 : ℝ)))) = answer", "v": null, "name": "h_answer"}]} -{"informal_problem": "Find, with explanation, the maximum value of $f(x)=x^3-3x$ on the set of all real numbers $x$ satisfying $x^4+36 \\leq 13x^2$.", "informal_answer": "18", "informal_solution": "Show that the maximum value is $18$.", "header": null, "intros": [], "formal_answer": "@Eq Real answer\n (@OfNat.ofNat Real (nat_lit 18)\n (@instOfNatAtLeastTwo Real (nat_lit 18) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 16) (instOfNatNat (nat_lit 16))))))", "formal_answer_type": "ℝ", "outros": [{"t": "Set ℝ", "v": null, "name": "S"}, {"t": "ℝ → ℝ", "v": null, "name": "f"}, {"t": "S = {x : ℝ | x ^ 4 + 36 ≤ 13 * x ^ 2}", "v": null, "name": "hS"}, {"t": "f = fun x ↦ x ^ 3 - 3 * x", "v": null, "name": "hf"}, {"t": "IsGreatest {f x | x ∈ S} answer", "v": null, "name": "h_answer"}]} -{"informal_problem": "What is the units (i.e., rightmost) digit of\n\\[\n\\left\\lfloor \\frac{10^{20000}}{10^{100}+3}\\right\\rfloor ?\n\\]", "informal_answer": "3", "informal_solution": "Show that the answer is $3$.", "header": null, "intros": [], "formal_answer": "@Eq Nat answer (@OfNat.ofNat Nat (nat_lit 3) (instOfNatNat (nat_lit 3)))", "formal_answer_type": "ℕ", "outros": [{"t": "Nat.floor ((10 ^ 20000 : ℝ) / (10 ^ 100 + 3)) % 10 = answer", "v": null, "name": "h_answer"}]} +{"informal_problem": "Find, with explanation, the maximum value of $f(x)=x^3-3x$ on the set of all real numbers $x$ satisfying $x^4+36 \\leq 13x^2$.", "informal_answer": "18", "informal_solution": "Show that the maximum value is $18$.", "header": "open BigOperators Real Nat Topology", "intros": [], "formal_answer": "@Eq Real answer\n (@OfNat.ofNat Real (nat_lit 18)\n (@instOfNatAtLeastTwo Real (nat_lit 18) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 16) (instOfNatNat (nat_lit 16))))))", "formal_answer_type": "ℝ", "outros": [{"t": "Set ℝ", "v": null, "name": "S"}, {"t": "ℝ → ℝ", "v": null, "name": "f"}, {"t": "S = {x : ℝ | x ^ 4 + 36 ≤ 13 * x ^ 2}", "v": null, "name": "hS"}, {"t": "f = fun x ↦ x ^ 3 - 3 * x", "v": null, "name": "hf"}, {"t": "IsGreatest {f x | x ∈ S} answer", "v": null, "name": "h_answer"}]} +{"informal_problem": "What is the units (i.e., rightmost) digit of\n\\[\n\\left\\lfloor \\frac{10^{20000}}{10^{100}+3}\\right\\rfloor ?\n\\]", "informal_answer": "3", "informal_solution": "Show that the answer is $3$.", "header": "open BigOperators Real Nat Topology", "intros": [], "formal_answer": "@Eq Nat answer (@OfNat.ofNat Nat (nat_lit 3) (instOfNatNat (nat_lit 3)))", "formal_answer_type": "ℕ", "outros": [{"t": "Nat.floor ((10 ^ 20000 : ℝ) / (10 ^ 100 + 3)) % 10 = answer", "v": null, "name": "h_answer"}]} {"informal_problem": "Evaluate $\\sum_{n=0}^\\infty \\mathrm{Arccot}(n^2+n+1)$, where $\\mathrm{Arccot}\\,t$ for $t \\geq 0$ denotes the number $\\theta$ in the interval $0 < \\theta \\leq \\pi/2$ with $\\cot \\theta = t$.", "informal_answer": "π / 2", "informal_solution": "Show that the sum equals $\\pi/2$.", "header": "open Real", "intros": [], "formal_answer": "@Eq Real answer\n (@HDiv.hDiv Real Real Real (@instHDiv Real (@DivInvMonoid.toDiv Real Real.instDivInvMonoid)) Real.pi\n (@OfNat.ofNat Real (nat_lit 2)\n (@instOfNatAtLeastTwo Real (nat_lit 2) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 0) (instOfNatNat (nat_lit 0)))))))", "formal_answer_type": "ℝ", "outros": [{"t": "ℝ → ℝ", "v": null, "name": "cot"}, {"t": "cot = fun θ ↦ Real.cos θ / Real.sin θ", "v": null, "name": "fcot"}, {"t": "ℝ → ℝ", "v": null, "name": "arccot"}, {"t": "∀ t : ℝ, t ≥ 0 → arccot t ∈ Set.Ioc 0 (Real.pi / 2) ∧ cot (arccot t) = t", "v": null, "name": "harccot"}, {"t": "(∑' n : ℕ, arccot (n ^ 2 + n + 1)) = answer", "v": null, "name": "h_answer"}]} {"informal_problem": "A \\emph{transversal} of an $n\\times n$ matrix $A$ consists of $n$ entries of $A$, no two in the same row or column. Let $f(n)$ be the number of $n \\times n$ matrices $A$ satisfying the following two conditions:\n\\begin{enumerate}\n\\item[(a)] Each entry $\\alpha_{i,j}$ of $A$ is in the set\n$\\{-1,0,1\\}$.\n\\item[(b)] The sum of the $n$ entries of a transversal is the same for all transversals of $A$.\n\\end{enumerate}\nAn example of such a matrix $A$ is\n\\[\nA = \\left( \\begin{array}{ccc} -1 & 0 & -1 \\\\ 0 & 1 & 0 \\\\ 0 & 1 & 0\n\\end{array}\n\\right).\n\\]\nDetermine with proof a formula for $f(n)$ of the form\n\\[\nf(n) = a_1 b_1^n + a_2 b_2^n + a_3 b_3^n + a_4,\n\\]\nwhere the $a_i$'s and $b_i$'s are rational numbers.", "informal_answer": "(1, 4, 2, 3, -4, 2, 1)", "informal_solution": "Prove that $f(n) = 4^n + 2 \\cdot 3^n - 4 \\cdot 2^n + 1$.", "header": "open Real Equiv", "intros": [], "formal_answer": "@Eq (Prod Rat (Prod Rat (Prod Rat (Prod Rat (Prod Rat (Prod Rat Rat)))))) answer\n (@Prod.mk Rat (Prod Rat (Prod Rat (Prod Rat (Prod Rat (Prod Rat Rat)))))\n (@OfNat.ofNat Rat (nat_lit 1) (@Rat.instOfNat (nat_lit 1)))\n (@Prod.mk Rat (Prod Rat (Prod Rat (Prod Rat (Prod Rat Rat))))\n (@OfNat.ofNat Rat (nat_lit 4) (@Rat.instOfNat (nat_lit 4)))\n (@Prod.mk Rat (Prod Rat (Prod Rat (Prod Rat Rat))) (@OfNat.ofNat Rat (nat_lit 2) (@Rat.instOfNat (nat_lit 2)))\n (@Prod.mk Rat (Prod Rat (Prod Rat Rat)) (@OfNat.ofNat Rat (nat_lit 3) (@Rat.instOfNat (nat_lit 3)))\n (@Prod.mk Rat (Prod Rat Rat)\n (@Neg.neg Rat Rat.instNeg (@OfNat.ofNat Rat (nat_lit 4) (@Rat.instOfNat (nat_lit 4))))\n (@Prod.mk Rat Rat (@OfNat.ofNat Rat (nat_lit 2) (@Rat.instOfNat (nat_lit 2)))\n (@OfNat.ofNat Rat (nat_lit 1) (@Rat.instOfNat (nat_lit 1)))))))))", "formal_answer_type": "ℚ × ℚ × ℚ × ℚ × ℚ × ℚ × ℚ", "outros": [{"t": "ℕ → ℕ", "v": null, "name": "f"}, {"t": "f = fun n ↦\n Set.ncard {A : Matrix (Fin n) (Fin n) ℤ |\n (∀ i j : Fin n, A i j ∈ ({-1, 0, 1} : Set ℤ)) ∧\n ∃ S : ℤ, ∀ ϕ : Perm (Fin n), ∑ i : Fin n, A i (ϕ i) = S}", "v": null, "name": "hf"}, {"t": "let (a1, b1, a2, b2, a3, b3, a4) := answer;\n (∀ n > 0, f n = a1 * b1 ^ n + a2 * b2 ^ n + a3 * b3 ^ n + a4)", "v": null, "name": "h_answer"}]} {"informal_problem": "Let $a_1, a_2, \\dots, a_n$ be real numbers, and let $b_1, b_2, \\dots, b_n$ be distinct positive integers. Suppose that there is a polynomial $f(x)$ satisfying the identity\n\\[\n(1-x)^n f(x) = 1 + \\sum_{i=1}^n a_i x^{b_i}.\n\\]\nFind a simple expression (not involving any sums) for $f(1)$ in terms of $b_1, b_2, \\dots, b_n$ and $n$ (but independent of $a_1, a_2, \\dots, a_n$).", "informal_answer": "fun b n ↦ (∏ i : Finset.Icc 1 n, b i) / Nat.factorial n", "informal_solution": "Show that $f(1) = b_1 b_2 \\dots b_n / n!$.", "header": "open Real Equiv", "intros": [], "formal_answer": "@Eq ((Nat → Nat) → Nat → Real) answer fun (b_1 : Nat → Nat) (n_1 : Nat) =>\n @HDiv.hDiv Real Real Real (@instHDiv Real (@DivInvMonoid.toDiv Real Real.instDivInvMonoid))\n (@Nat.cast Real Real.instNatCast\n (@Finset.prod\n (@Subtype Nat fun (x : Nat) =>\n @Membership.mem Nat (Finset Nat) (@Finset.instMembership Nat)\n (@Finset.Icc Nat Nat.instPreorder Nat.instLocallyFiniteOrder\n (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1))) n_1)\n x)\n Nat Nat.instCommMonoid\n (@Finset.univ\n (@Subtype Nat fun (x : Nat) =>\n @Membership.mem Nat (Finset Nat) (@Finset.instMembership Nat)\n (@Finset.Icc Nat Nat.instPreorder Nat.instLocallyFiniteOrder\n (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1))) n_1)\n x)\n (@Finset.Subtype.fintype Nat\n (@Finset.Icc Nat Nat.instPreorder Nat.instLocallyFiniteOrder\n (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1))) n_1)))\n fun\n (i :\n @Subtype Nat fun (x : Nat) =>\n @Membership.mem Nat (Finset Nat) (@Finset.instMembership Nat)\n (@Finset.Icc Nat Nat.instPreorder Nat.instLocallyFiniteOrder\n (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1))) n_1)\n x) =>\n b_1\n (@Subtype.val Nat\n (fun (x : Nat) =>\n @Membership.mem Nat (Finset Nat) (@Finset.instMembership Nat)\n (@Finset.Icc Nat Nat.instPreorder Nat.instLocallyFiniteOrder\n (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1))) n_1)\n x)\n i)))\n (@Nat.cast Real Real.instNatCast (Nat.factorial n_1))", "formal_answer_type": "(ℕ → ℕ) → ℕ → ℝ", "outros": [{"t": "ℕ", "v": null, "name": "n"}, {"t": "n > 0", "v": null, "name": "npos"}, {"t": "ℕ → ℝ", "v": null, "name": "a"}, {"t": "ℕ → ℕ", "v": null, "name": "b"}, {"t": "∀ i ∈ Finset.Icc 1 n, b i > 0", "v": null, "name": "bpos"}, {"t": "∀ i ∈ Finset.Icc 1 n, ∀ j ∈ Finset.Icc 1 n, b i = b j → i = j", "v": null, "name": "binj"}, {"t": "Polynomial ℝ", "v": null, "name": "f"}, {"t": "∀ x : ℝ, (1 - x) ^ n * f.eval x = 1 + ∑ i : Finset.Icc 1 n, (a i) * x ^ (b i)", "v": null, "name": "hf"}, {"t": "f.eval 1 = answer b n", "v": null, "name": "h_answer"}]} @@ -107,9 +107,9 @@ {"informal_problem": "Prove that there are only a finite number of possibilities for the ordered triple $T=(x-y,y-z,z-x)$, where $x,y,z$ are complex numbers satisfying the simultaneous equations\n\\[\nx(x-1)+2yz = y(y-1)+2zx = z(z-1)+2xy,\n\\]\nand list all such triples $T$.", "informal_answer": "{(0, 0, 0), (0, -1, 1), (1, 0, -1), (-1, 1, 0)}", "informal_solution": "Show that the possibilities for $T$ are $(0, 0, 0), \\, (0, -1, 1), \\, (1, 0, -1), \\, (-1, 1, 0)$.", "header": "open Real Equiv", "intros": [], "formal_answer": "@Eq (Finset (Prod Complex (Prod Complex Complex))) answer\n (@Insert.insert (Prod Complex (Prod Complex Complex)) (Finset (Prod Complex (Prod Complex Complex)))\n (@Finset.instInsert (Prod Complex (Prod Complex Complex)) fun (a b : Prod Complex (Prod Complex Complex)) =>\n @instDecidableEqProd Complex (Prod Complex Complex) Complex.instDecidableEq\n (fun (a_1 b_1 : Prod Complex Complex) =>\n @instDecidableEqProd Complex Complex Complex.instDecidableEq Complex.instDecidableEq a_1 b_1)\n a b)\n (@Prod.mk Complex (Prod Complex Complex)\n (@OfNat.ofNat Complex (nat_lit 0) (@Zero.toOfNat0 Complex Complex.instZero))\n (@Prod.mk Complex Complex (@OfNat.ofNat Complex (nat_lit 0) (@Zero.toOfNat0 Complex Complex.instZero))\n (@OfNat.ofNat Complex (nat_lit 0) (@Zero.toOfNat0 Complex Complex.instZero))))\n (@Insert.insert (Prod Complex (Prod Complex Complex)) (Finset (Prod Complex (Prod Complex Complex)))\n (@Finset.instInsert (Prod Complex (Prod Complex Complex)) fun (a b : Prod Complex (Prod Complex Complex)) =>\n @instDecidableEqProd Complex (Prod Complex Complex) Complex.instDecidableEq\n (fun (a_1 b_1 : Prod Complex Complex) =>\n @instDecidableEqProd Complex Complex Complex.instDecidableEq Complex.instDecidableEq a_1 b_1)\n a b)\n (@Prod.mk Complex (Prod Complex Complex)\n (@OfNat.ofNat Complex (nat_lit 0) (@Zero.toOfNat0 Complex Complex.instZero))\n (@Prod.mk Complex Complex\n (@Neg.neg Complex Complex.instNeg (@OfNat.ofNat Complex (nat_lit 1) (@One.toOfNat1 Complex Complex.instOne)))\n (@OfNat.ofNat Complex (nat_lit 1) (@One.toOfNat1 Complex Complex.instOne))))\n (@Insert.insert (Prod Complex (Prod Complex Complex)) (Finset (Prod Complex (Prod Complex Complex)))\n (@Finset.instInsert (Prod Complex (Prod Complex Complex)) fun (a b : Prod Complex (Prod Complex Complex)) =>\n @instDecidableEqProd Complex (Prod Complex Complex) Complex.instDecidableEq\n (fun (a_1 b_1 : Prod Complex Complex) =>\n @instDecidableEqProd Complex Complex Complex.instDecidableEq Complex.instDecidableEq a_1 b_1)\n a b)\n (@Prod.mk Complex (Prod Complex Complex)\n (@OfNat.ofNat Complex (nat_lit 1) (@One.toOfNat1 Complex Complex.instOne))\n (@Prod.mk Complex Complex (@OfNat.ofNat Complex (nat_lit 0) (@Zero.toOfNat0 Complex Complex.instZero))\n (@Neg.neg Complex Complex.instNeg\n (@OfNat.ofNat Complex (nat_lit 1) (@One.toOfNat1 Complex Complex.instOne)))))\n (@Singleton.singleton (Prod Complex (Prod Complex Complex)) (Finset (Prod Complex (Prod Complex Complex)))\n (@Finset.instSingleton (Prod Complex (Prod Complex Complex)))\n (@Prod.mk Complex (Prod Complex Complex)\n (@Neg.neg Complex Complex.instNeg\n (@OfNat.ofNat Complex (nat_lit 1) (@One.toOfNat1 Complex Complex.instOne)))\n (@Prod.mk Complex Complex (@OfNat.ofNat Complex (nat_lit 1) (@One.toOfNat1 Complex Complex.instOne))\n (@OfNat.ofNat Complex (nat_lit 0) (@Zero.toOfNat0 Complex Complex.instZero))))))))", "formal_answer_type": "Finset (ℂ × ℂ × ℂ)", "outros": [{"t": "{T : ℂ × ℂ × ℂ | ∃ x y z : ℂ, T = (x - y, y - z, z - x) ∧ x * (x - 1) + 2 * y * z = y * (y - 1) + 2 * z * x ∧ y * (y - 1) + 2 * z * x = z * (z - 1) + 2 * x * y} = answer", "v": null, "name": "h_answer"}]} {"informal_problem": "For a positive real number $r$, let $G(r)$ be the minimum value of $|r - \\sqrt{m^2+2n^2}|$ for all integers $m$ and $n$. Prove or disprove the assertion that $\\lim_{r\\to \\infty}G(r)$ exists and equals $0$.", "informal_answer": "True", "informal_solution": "Show that the limit exists and equals $0$.", "header": "open Real Equiv Polynomial Filter Topology", "intros": [], "formal_answer": "@Eq Prop answer True", "formal_answer_type": "Prop", "outros": [{"t": "ℝ → ℝ", "v": null, "name": "G"}, {"t": "∀ r : ℝ, ∃ m n : ℤ, G r = |r - Real.sqrt (m ^ 2 + 2 * n ^ 2)|", "v": null, "name": "hGeq"}, {"t": "∀ r : ℝ, ∀ m n : ℤ, G r ≤ |r - Real.sqrt (m ^ 2 + 2 * n ^ 2)|", "v": null, "name": "hGlb"}, {"t": "answer ↔ Tendsto G atTop (𝓝 0)", "v": null, "name": "h_answer"}]} {"informal_problem": "Let $f(x,y,z) = x^2+y^2+z^2+xyz$. Let $p(x,y,z), q(x,y,z)$, $r(x,y,z)$ be polynomials with real coefficients satisfying\n\\[\nf(p(x,y,z), q(x,y,z), r(x,y,z)) = f(x,y,z).\n\\]\nProve or disprove the assertion that the sequence $p,q,r$ consists of some permutation of $\\pm x, \\pm y, \\pm z$, where the number of minus signs is $0$ or $2$.", "informal_answer": "False", "informal_solution": "Prove that the assertion is false.", "header": "open Real Equiv Polynomial Filter Topology MvPolynomial", "intros": [], "formal_answer": "@Eq Prop answer False", "formal_answer_type": "Prop", "outros": [{"t": "MvPolynomial (Fin 3) ℝ", "v": null, "name": "f"}, {"t": "Set (Set (MvPolynomial (Fin 3) ℝ))", "v": null, "name": "perms"}, {"t": "f = (X 0) ^ 2 + (X 1) ^ 2 + (X 2) ^ 2 + (X 0) * (X 1) * (X 2)", "v": null, "name": "hf"}, {"t": "perms = {{X 0, X 1, X 2}, {X 0, -X 1, -X 2}, {-X 0, X 1, -X 2}, {-X 0, -X 1, X 2}}", "v": null, "name": "hperms"}, {"t": "answer ↔ (∀ pqr : Fin 3 → MvPolynomial (Fin 3) ℝ,\n (∀ xyz : Fin 3 → ℝ, MvPolynomial.eval (fun i ↦ MvPolynomial.eval xyz (pqr i)) f = MvPolynomial.eval xyz f) →\n ({pqr 0, pqr 1, pqr 2} ∈ perms))", "v": null, "name": "h_answer"}]} -{"informal_problem": "The sequence of digits $123456789101112131415161718192021 \\dots$ is obtained by writing the positive integers in order. If the $10^n$-th digit in this sequence occurs in the part of the sequence in which the $m$-digit numbers are placed, define $f(n)$ to be $m$. For example, $f(2)=2$ because the $100$th digit enters the sequence in the placement of the two-digit integer $55$. Find, with proof, $f(1987)$.", "informal_answer": "1984", "informal_solution": "Show that the value of $f(1987)$ is $1984$.", "header": null, "intros": [], "formal_answer": "@Eq Nat answer (@OfNat.ofNat Nat (nat_lit 1984) (instOfNatNat (nat_lit 1984)))", "formal_answer_type": "ℕ", "outros": [{"t": "ℕ → ℕ", "v": null, "name": "seqind"}, {"t": "ℕ → ℕ", "v": null, "name": "seqsize"}, {"t": "ℕ → ℕ", "v": null, "name": "f"}, {"t": "seqind 1 = 1 ∧ ∀ i ≥ 2, seqind i = seqind (i - 1) + (Nat.digits 10 (i - 1)).length", "v": null, "name": "hseqind"}, {"t": "∀ i ≥ 1, ∀ j : Fin ((Nat.digits 10 i).length), seqsize (seqind i + j) = (Nat.digits 10 i).length", "v": null, "name": "hseqsize"}, {"t": "∀ n : ℕ, f n = seqsize (10 ^ n)", "v": null, "name": "hf"}, {"t": "f 1987 = answer", "v": null, "name": "h_answer"}]} +{"informal_problem": "The sequence of digits $123456789101112131415161718192021 \\dots$ is obtained by writing the positive integers in order. If the $10^n$-th digit in this sequence occurs in the part of the sequence in which the $m$-digit numbers are placed, define $f(n)$ to be $m$. For example, $f(2)=2$ because the $100$th digit enters the sequence in the placement of the two-digit integer $55$. Find, with proof, $f(1987)$.", "informal_answer": "1984", "informal_solution": "Show that the value of $f(1987)$ is $1984$.", "header": "open BigOperators Real Nat Topology", "intros": [], "formal_answer": "@Eq Nat answer (@OfNat.ofNat Nat (nat_lit 1984) (instOfNatNat (nat_lit 1984)))", "formal_answer_type": "ℕ", "outros": [{"t": "ℕ → ℕ", "v": null, "name": "seqind"}, {"t": "ℕ → ℕ", "v": null, "name": "seqsize"}, {"t": "ℕ → ℕ", "v": null, "name": "f"}, {"t": "seqind 1 = 1 ∧ ∀ i ≥ 2, seqind i = seqind (i - 1) + (Nat.digits 10 (i - 1)).length", "v": null, "name": "hseqind"}, {"t": "∀ i ≥ 1, ∀ j : Fin ((Nat.digits 10 i).length), seqsize (seqind i + j) = (Nat.digits 10 i).length", "v": null, "name": "hseqsize"}, {"t": "∀ n : ℕ, f n = seqsize (10 ^ n)", "v": null, "name": "hf"}, {"t": "f 1987 = answer", "v": null, "name": "h_answer"}]} {"informal_problem": "Let $P$ be a polynomial, with real coefficients, in three variables and $F$ be a function of two variables such that\n\\[\nP(ux, uy, uz) = u^2 F(y-x,z-x) \\quad \\mbox{for all real $x,y,z,u$},\n\\]\nand such that $P(1,0,0)=4$, $P(0,1,0)=5$, and $P(0,0,1)=6$. Also let $A,B,C$ be complex numbers with $P(A,B,C)=0$ and $|B-A|=10$. Find $|C-A|$.", "informal_answer": "$\\frac{5}{3}\\sqrt{30}$", "informal_solution": "Prove that $|C - A| = \\frac{5}{3}\\sqrt{30}$.", "header": "open MvPolynomial Real", "intros": [], "formal_answer": "@Eq Complex answer\n (@HMul.hMul Complex Complex Complex (@instHMul Complex Complex.instMul)\n (@HDiv.hDiv Complex Complex Complex (@instHDiv Complex (@DivInvMonoid.toDiv Complex Complex.instDivInvMonoid))\n (@OfNat.ofNat Complex (nat_lit 5)\n (@instOfNatAtLeastTwo Complex (nat_lit 5)\n (@AddMonoidWithOne.toNatCast Complex (@AddGroupWithOne.toAddMonoidWithOne Complex Complex.addGroupWithOne))\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 3) (instOfNatNat (nat_lit 3))))))\n (@OfNat.ofNat Complex (nat_lit 3)\n (@instOfNatAtLeastTwo Complex (nat_lit 3)\n (@AddMonoidWithOne.toNatCast Complex (@AddGroupWithOne.toAddMonoidWithOne Complex Complex.addGroupWithOne))\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1)))))))\n ↑(Real.sqrt\n (@OfNat.ofNat Real (nat_lit 30)\n (@instOfNatAtLeastTwo Real (nat_lit 30) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 28) (instOfNatNat (nat_lit 28))))))))", "formal_answer_type": "ℂ", "outros": [{"t": "MvPolynomial (Fin 3) ℂ", "v": null, "name": "P"}, {"t": "∀ i : Fin 3 →₀ ℕ, (coeff i P).im = 0", "v": null, "name": "hPreal"}, {"t": "ℝ → ℝ → ℝ", "v": null, "name": "F"}, {"t": "ℂ → ℂ → ℂ → (Fin 3 → ℂ)", "v": null, "name": "vars"}, {"t": "vars = fun a b c ↦ fun i ↦ ite (i = 0) a (ite (i = 1) b c)", "v": null, "name": "hvars"}, {"t": "∀ x y z u : ℝ, eval (vars (u * x) (u * y) (u * z)) P = u ^ 2 * F (y - x) (z - x)", "v": null, "name": "h"}, {"t": "eval (vars 1 0 0) P = 4 ∧ eval (vars 0 1 0) P = 5 ∧ eval (vars 0 0 1) P = 6", "v": null, "name": "hPval"}, {"t": "ℂ", "v": null, "name": "A"}, {"t": "ℂ", "v": null, "name": "B"}, {"t": "ℂ", "v": null, "name": "C"}, {"t": "eval (vars A B C) P = 0", "v": null, "name": "hPABC"}, {"t": "‖B - A‖ = 10", "v": null, "name": "habs"}, {"t": "‖C - A‖ = answer", "v": null, "name": "h_answer"}]} -{"informal_problem": "Let $\\vec{G}(x,y)=\\left(\\frac{-y}{x^2+4y^2},\\frac{x}{x^2+4y^2},0\\right)$. Prove or disprove that there is a vector-valued function $\\vec{F}(x,y,z)=(M(x,y,z),N(x,y,z),P(x,y,z))$ with the following properties:\n\\begin{enumerate}\n\\item[(i)] $M$, $N$, $P$ have continuous partial derivatives for all $(x,y,z) \\neq (0,0,0)$;\n\\item[(ii)] $\\text{Curl}\\,\\vec{F}=\\vec{0}$ for all $(x,y,z) \\neq (0,0,0)$;\n\\item[(iii)] $\\vec{F}(x,y,0)=\\vec{G}(x,y)$.\n\\end{enumerate}", "informal_answer": "False", "informal_solution": "Show that there is no such $\\vec{F}$.", "header": null, "intros": [], "formal_answer": "@Eq Prop answer False", "formal_answer_type": "Prop", "outros": [{"t": "((Fin 3 → ℝ) → (Fin 3 → ℝ)) → ((Fin 3 → ℝ) → (Fin 3 → ℝ))", "v": null, "name": "curl"}, {"t": "∀ f x, curl f x = ![\n fderiv ℝ f x (Pi.single 1 1) 2 - fderiv ℝ f x (Pi.single 2 1) 1,\n fderiv ℝ f x (Pi.single 2 1) 0 - fderiv ℝ f x (Pi.single 0 1) 2,\n fderiv ℝ f x (Pi.single 0 1) 1 - fderiv ℝ f x (Pi.single 1 1) 0]", "v": null, "name": "curl_def"}, {"t": "(Fin 2 → ℝ) → (Fin 3 → ℝ)", "v": null, "name": "G"}, {"t": "∀ x y, G ![x, y] = ![(-y / (x ^ 2 + 4 * y ^ 2)), (x / (x ^ 2 + 4 * y ^ 2)), 0]", "v": null, "name": "G_def"}, {"t": "(∃ F : (Fin 3 → ℝ) → (Fin 3 → ℝ),\n ContDiffOn ℝ 1 F {v | v ≠ ![0,0,0]} ∧\n (∀ x, x ≠ 0 → curl F x = 0) ∧\n ∀ x y, F ![x, y, 0] = G ![x, y]) ↔ answer", "v": null, "name": "h_answer"}]} +{"informal_problem": "Let $\\vec{G}(x,y)=\\left(\\frac{-y}{x^2+4y^2},\\frac{x}{x^2+4y^2},0\\right)$. Prove or disprove that there is a vector-valued function $\\vec{F}(x,y,z)=(M(x,y,z),N(x,y,z),P(x,y,z))$ with the following properties:\n\\begin{enumerate}\n\\item[(i)] $M$, $N$, $P$ have continuous partial derivatives for all $(x,y,z) \\neq (0,0,0)$;\n\\item[(ii)] $\\text{Curl}\\,\\vec{F}=\\vec{0}$ for all $(x,y,z) \\neq (0,0,0)$;\n\\item[(iii)] $\\vec{F}(x,y,0)=\\vec{G}(x,y)$.\n\\end{enumerate}", "informal_answer": "False", "informal_solution": "Show that there is no such $\\vec{F}$.", "header": "open BigOperators Real Nat Topology", "intros": [], "formal_answer": "@Eq Prop answer False", "formal_answer_type": "Prop", "outros": [{"t": "((Fin 3 → ℝ) → (Fin 3 → ℝ)) → ((Fin 3 → ℝ) → (Fin 3 → ℝ))", "v": null, "name": "curl"}, {"t": "∀ f x, curl f x = ![\n fderiv ℝ f x (Pi.single 1 1) 2 - fderiv ℝ f x (Pi.single 2 1) 1,\n fderiv ℝ f x (Pi.single 2 1) 0 - fderiv ℝ f x (Pi.single 0 1) 2,\n fderiv ℝ f x (Pi.single 0 1) 1 - fderiv ℝ f x (Pi.single 1 1) 0]", "v": null, "name": "curl_def"}, {"t": "(Fin 2 → ℝ) → (Fin 3 → ℝ)", "v": null, "name": "G"}, {"t": "∀ x y, G ![x, y] = ![(-y / (x ^ 2 + 4 * y ^ 2)), (x / (x ^ 2 + 4 * y ^ 2)), 0]", "v": null, "name": "G_def"}, {"t": "(∃ F : (Fin 3 → ℝ) → (Fin 3 → ℝ),\n ContDiffOn ℝ 1 F {v | v ≠ ![0,0,0]} ∧\n (∀ x, x ≠ 0 → curl F x = 0) ∧\n ∀ x y, F ![x, y, 0] = G ![x, y]) ↔ answer", "v": null, "name": "h_answer"}]} {"informal_problem": "For each positive integer $n$, let $a(n)$ be the number of zeroes in the base $3$ representation of $n$. For which positive real numbers $x$ does the series\n\\[\n\\sum_{n=1}^\\infty \\frac{x^{a(n)}}{n^3}\n\\]\nconverge?", "informal_answer": "the set of positive real numbers $x$ such that $0 < x < 25$", "informal_solution": "Show that for positive $x$, the series converges if and only if $x < 25$.", "header": "open MvPolynomial Real Nat", "intros": [], "formal_answer": "@Eq (Set Real) answer\n (@setOf Real fun (x : Real) =>\n And (@GT.gt Real Real.instLT x (@OfNat.ofNat Real (nat_lit 0) (@Zero.toOfNat0 Real Real.instZero)))\n (@LT.lt Real Real.instLT x\n (@OfNat.ofNat Real (nat_lit 25)\n (@instOfNatAtLeastTwo Real (nat_lit 25) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 23) (instOfNatNat (nat_lit 23))))))))", "formal_answer_type": "Set ℝ", "outros": [{"t": "ℕ → ℕ", "v": null, "name": "a"}, {"t": "a = fun n ↦ {i | (digits 3 n).get i = 0}.ncard", "v": null, "name": "ha"}, {"t": "{x : ℝ | x > 0 ∧ Summable (fun n ↦ x ^ (a n) / (n ^ 3))} = answer", "v": null, "name": "h_answer"}]} {"informal_problem": "Evaluate\n\\[\n\\int_2^4 \\frac{\\sqrt{\\ln(9-x)}\\,dx}{\\sqrt{\\ln(9-x)}+\\sqrt{\\ln(x+3)}}.\n\\]", "informal_answer": "1", "informal_solution": "Prove that the integral evaluates to $1$.", "header": "open MvPolynomial Real Nat", "intros": [], "formal_answer": "@Eq Real answer (@OfNat.ofNat Real (nat_lit 1) (@One.toOfNat1 Real Real.instOne))", "formal_answer_type": "ℝ", "outros": [{"t": "answer = ∫ x in (2)..4, sqrt (log (9 - x)) / (sqrt (log (9 - x)) + sqrt (log (x + 3)))", "v": null, "name": "h_answer"}]} {"informal_problem": "Let $(x_1,y_1) = (0.8, 0.6)$ and let $x_{n+1} = x_n \\cos y_n - y_n \\sin y_n$ and $y_{n+1}= x_n \\sin y_n + y_n \\cos y_n$ for $n=1,2,3,\\dots$. For each of $\\lim_{n\\to \\infty} x_n$ and $\\lim_{n \\to \\infty} y_n$, prove that the limit exists and find it or prove that the limit does not exist.", "informal_answer": "(True, -1, True, 0)", "informal_solution": "Show that $\\lim_{n \\to \\infty} x_n = -1$ and $\\lim_{n \\to \\infty} y_n = 0$.", "header": "open MvPolynomial Real Nat Filter Topology", "intros": [], "formal_answer": "@Eq (Prod Prop (Prod Real (Prod Prop Real))) answer\n (@Prod.mk Prop (Prod Real (Prod Prop Real)) True\n (@Prod.mk Real (Prod Prop Real)\n (@Neg.neg Real Real.instNeg (@OfNat.ofNat Real (nat_lit 1) (@One.toOfNat1 Real Real.instOne)))\n (@Prod.mk Prop Real True (@OfNat.ofNat Real (nat_lit 0) (@Zero.toOfNat0 Real Real.instZero)))))", "formal_answer_type": "Prop × ℝ × Prop × ℝ", "outros": [{"t": "ℕ → ℝ", "v": null, "name": "x"}, {"t": "ℕ → ℝ", "v": null, "name": "y"}, {"t": "(x 1, y 1) = (0.8, 0.6)", "v": null, "name": "hxy1"}, {"t": "∀ n ≥ 1, x (n + 1) = (x n) * cos (y n) - (y n) * sin (y n)", "v": null, "name": "hx"}, {"t": "∀ n ≥ 1, y (n + 1) = (x n) * sin (y n) + (y n) * cos (y n)", "v": null, "name": "hy"}, {"t": "let (existsx, limx, existsy, limy) := answer\n((∃ c : ℝ, Tendsto x atTop (𝓝 c)) → existsx) ∧\n(existsx → Tendsto x atTop (𝓝 limx)) ∧\n((∃ c : ℝ, Tendsto y atTop (𝓝 c)) → existsy) ∧\n(existsy → Tendsto y atTop (𝓝 limy))", "v": null, "name": "h_answer"}]} @@ -121,8 +121,8 @@ {"informal_problem": "Prove or disprove: If $x$ and $y$ are real numbers with $y \\geq 0$ and $y(y+1) \\leq (x+1)^2$, then $y(y-1) \\leq x^2$.", "informal_answer": "True", "informal_solution": "Show that this is true.", "header": "open Set Filter Topology", "intros": [], "formal_answer": "@Eq Prop answer True", "formal_answer_type": "Prop", "outros": [{"t": "ℝ", "v": null, "name": "x"}, {"t": "ℝ", "v": null, "name": "y"}, {"t": "y ≥ 0", "v": null, "name": "h_y_nonneg"}, {"t": "y * (y + 1) ≤ (x + 1) ^ 2", "v": null, "name": "h_ineq"}, {"t": "answer = (y * (y - 1) ≤ x ^ 2)", "v": null, "name": "h_answer"}]} {"informal_problem": "For every $n$ in the set $N=\\{1,2,\\dots\\}$ of positive integers, let $r_n$ be the minimum value of $|c-d \\sqrt{3}|$ for all nonnegative integers $c$ and $d$ with $c+d=n$. Find, with proof, the smallest positive real number $g$ with $r_n \\leq g$ for all $n \\in N$.", "informal_answer": "(1 + √3) / 2", "informal_solution": "Show that the smallest such $g$ is $(1+\\sqrt{3})/2$.", "header": "open Set Filter Topology", "intros": [], "formal_answer": "@Eq Real answer\n (@HDiv.hDiv Real Real Real (@instHDiv Real (@DivInvMonoid.toDiv Real Real.instDivInvMonoid))\n (@HAdd.hAdd Real Real Real (@instHAdd Real Real.instAdd)\n (@OfNat.ofNat Real (nat_lit 1) (@One.toOfNat1 Real Real.instOne))\n (Real.sqrt\n (@OfNat.ofNat Real (nat_lit 3)\n (@instOfNatAtLeastTwo Real (nat_lit 3) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1))))))))\n (@OfNat.ofNat Real (nat_lit 2)\n (@instOfNatAtLeastTwo Real (nat_lit 2) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 0) (instOfNatNat (nat_lit 0)))))))", "formal_answer_type": "ℝ", "outros": [{"t": "ℤ → ℝ", "v": null, "name": "r"}, {"t": "∀ n ≥ 1,\n (∃ c d : ℤ,\n (c ≥ 0 ∧ d ≥ 0) ∧\n c + d = n ∧ r n = |c - d * Real.sqrt 3|) ∧\n (∀ c d : ℤ, (c ≥ 0 ∧ d ≥ 0 ∧ c + d = n) → |c - d * Real.sqrt 3| ≥ r n)", "v": null, "name": "hr"}, {"t": "IsLeast {g : ℝ | g > 0 ∧ (∀ n : ℤ, n ≥ 1 → r n ≤ g)} answer", "v": null, "name": "h_answer"}]} {"informal_problem": "For positive integers $n$, let $M_n$ be the $2n+1$ by $2n+1$ skew-symmetric matrix for which each entry in the first $n$ subdiagonals below the main diagonal is $1$ and each of the remaining entries below the main diagonal is $-1$. Find, with proof, the rank of $M_n$. (According to one definition, the rank of a matrix is the largest $k$ such that there is a $k \\times k$ submatrix with nonzero determinant.) One may note that\n\\begin{align*}\nM_1&=\\begin{pmatrix} 0 & -1 & 1 \\\\ 1 & 0 & -1 \\\\ -1 & 1 & 0 \\end{pmatrix} \\\\\nM_2&=\\begin{pmatrix} 0 & -1 & -1 & 1 & 1 \\\\ 1 & 0 & -1 & -1 & 1 \\\\ 1 & 1 & 0 & -1 & -1 \\\\ -1 & 1 & 1 & 0 & -1 \\\\ -1 & -1 & 1 & 1 & 0 \\end{pmatrix}.\n\\end{align*}", "informal_answer": "2n", "informal_solution": "Show that the rank of $M_n$ equals $2n$.", "header": "open Set Filter Topology", "intros": [], "formal_answer": "@Eq (Nat → Nat) answer fun (n_1 : Nat) =>\n @HMul.hMul Nat Nat Nat (@instHMul Nat instMulNat) (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))) n_1", "formal_answer_type": "ℕ → ℕ", "outros": [{"t": "ℕ", "v": null, "name": "n"}, {"t": "n > 0", "v": null, "name": "hn"}, {"t": "Matrix (Fin (2 * n + 1)) (Fin (2 * n + 1)) ℝ", "v": null, "name": "Mn"}, {"t": "∀ i j, Mn i j = -(Mn j i)", "v": null, "name": "Mnskewsymm"}, {"t": "∀ i j, (1 ≤ (i.1 : ℤ) - j.1 ∧ (i.1 : ℤ) - j.1 ≤ n) → Mn i j = 1", "v": null, "name": "hMn1"}, {"t": "∀ i j, (i.1 : ℤ) - j.1 > n → Mn i j = -1", "v": null, "name": "hMnn1"}, {"t": "Mn.rank = answer n", "v": null, "name": "h_answer"}]} -{"informal_problem": "How many primes among the positive integers, written as usual in base $10$, are alternating $1$'s and $0$'s, beginning and ending with $1$?", "informal_answer": "1", "informal_solution": "Show that there is only one such prime.", "header": null, "intros": [], "formal_answer": "@Eq ENat answer\n (@OfNat.ofNat ENat (nat_lit 1)\n (@One.toOfNat1 ENat\n (@AddMonoidWithOne.toOne ENat\n (@AddCommMonoidWithOne.toAddMonoidWithOne ENat\n (@NonAssocSemiring.toAddCommMonoidWithOne ENat\n (@Semiring.toNonAssocSemiring ENat\n (@OrderedSemiring.toSemiring ENat\n (@OrderedCommSemiring.toOrderedSemiring ENat\n (@CanonicallyOrderedCommSemiring.toOrderedCommSemiring ENat\n instENatCanonicallyOrderedCommSemiring)))))))))", "formal_answer_type": "ℕ∞", "outros": [{"t": "List ℕ → Prop", "v": null, "name": "pdigalt"}, {"t": "∀ l, pdigalt l ↔ Odd l.length ∧ (∀ i, l.get i = if Even (i : ℕ) then 1 else 0)", "v": null, "name": "hpdigalt"}, {"t": "{p : ℕ | p.Prime ∧ pdigalt (Nat.digits 10 p)}.encard = answer", "v": null, "name": "h_answer"}]} -{"informal_problem": "Evaluate $\\int_0^a \\int_0^b e^{\\max\\{b^2x^2,a^2y^2\\}}\\,dy\\,dx$ where $a$ and $b$ are positive.", "informal_answer": "$\\frac{e^{a^2 b^2} - 1}{a b}$", "informal_solution": "Show that the value of the integral is $(e^{a^2b^2}-1)/(ab)$.", "header": null, "intros": [], "formal_answer": "@Eq (Real → Real → Real) answer fun (a_1 b_1 : Real) =>\n @HDiv.hDiv Real Real Real (@instHDiv Real (@DivInvMonoid.toDiv Real Real.instDivInvMonoid))\n (@HSub.hSub Real Real Real (@instHSub Real Real.instSub)\n (Real.exp\n (@HMul.hMul Real Real Real (@instHMul Real Real.instMul)\n (@HPow.hPow Real Nat Real (@instHPow Real Nat (@Monoid.toNatPow Real Real.instMonoid)) a_1\n (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))))\n (@HPow.hPow Real Nat Real (@instHPow Real Nat (@Monoid.toNatPow Real Real.instMonoid)) b_1\n (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))))))\n (@OfNat.ofNat Real (nat_lit 1) (@One.toOfNat1 Real Real.instOne)))\n (@HMul.hMul Real Real Real (@instHMul Real Real.instMul) a_1 b_1)", "formal_answer_type": "ℝ → ℝ → ℝ", "outros": [{"t": "ℝ", "v": null, "name": "a"}, {"t": "ℝ", "v": null, "name": "b"}, {"t": "a > 0 ∧ b > 0", "v": null, "name": "abpos"}, {"t": "∫ x in Set.Ioo 0 a, ∫ y in Set.Ioo 0 b, Real.exp (max (b ^ 2 * x ^ 2) (a ^ 2 * y ^ 2)) = answer a b", "v": null, "name": "h_answer"}]} +{"informal_problem": "How many primes among the positive integers, written as usual in base $10$, are alternating $1$'s and $0$'s, beginning and ending with $1$?", "informal_answer": "1", "informal_solution": "Show that there is only one such prime.", "header": "open BigOperators Real Nat Topology", "intros": [], "formal_answer": "@Eq ENat answer\n (@OfNat.ofNat ENat (nat_lit 1)\n (@One.toOfNat1 ENat\n (@AddMonoidWithOne.toOne ENat\n (@AddCommMonoidWithOne.toAddMonoidWithOne ENat\n (@NonAssocSemiring.toAddCommMonoidWithOne ENat\n (@Semiring.toNonAssocSemiring ENat\n (@OrderedSemiring.toSemiring ENat\n (@OrderedCommSemiring.toOrderedSemiring ENat\n (@CanonicallyOrderedCommSemiring.toOrderedCommSemiring ENat\n instENatCanonicallyOrderedCommSemiring)))))))))", "formal_answer_type": "ℕ∞", "outros": [{"t": "List ℕ → Prop", "v": null, "name": "pdigalt"}, {"t": "∀ l, pdigalt l ↔ Odd l.length ∧ (∀ i, l.get i = if Even (i : ℕ) then 1 else 0)", "v": null, "name": "hpdigalt"}, {"t": "{p : ℕ | p.Prime ∧ pdigalt (Nat.digits 10 p)}.encard = answer", "v": null, "name": "h_answer"}]} +{"informal_problem": "Evaluate $\\int_0^a \\int_0^b e^{\\max\\{b^2x^2,a^2y^2\\}}\\,dy\\,dx$ where $a$ and $b$ are positive.", "informal_answer": "$\\frac{e^{a^2 b^2} - 1}{a b}$", "informal_solution": "Show that the value of the integral is $(e^{a^2b^2}-1)/(ab)$.", "header": "open BigOperators Real Nat Topology", "intros": [], "formal_answer": "@Eq (Real → Real → Real) answer fun (a_1 b_1 : Real) =>\n @HDiv.hDiv Real Real Real (@instHDiv Real (@DivInvMonoid.toDiv Real Real.instDivInvMonoid))\n (@HSub.hSub Real Real Real (@instHSub Real Real.instSub)\n (Real.exp\n (@HMul.hMul Real Real Real (@instHMul Real Real.instMul)\n (@HPow.hPow Real Nat Real (@instHPow Real Nat (@Monoid.toNatPow Real Real.instMonoid)) a_1\n (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))))\n (@HPow.hPow Real Nat Real (@instHPow Real Nat (@Monoid.toNatPow Real Real.instMonoid)) b_1\n (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))))))\n (@OfNat.ofNat Real (nat_lit 1) (@One.toOfNat1 Real Real.instOne)))\n (@HMul.hMul Real Real Real (@instHMul Real Real.instMul) a_1 b_1)", "formal_answer_type": "ℝ → ℝ → ℝ", "outros": [{"t": "ℝ", "v": null, "name": "a"}, {"t": "ℝ", "v": null, "name": "b"}, {"t": "a > 0 ∧ b > 0", "v": null, "name": "abpos"}, {"t": "∫ x in Set.Ioo 0 a, ∫ y in Set.Ioo 0 b, Real.exp (max (b ^ 2 * x ^ 2) (a ^ 2 * y ^ 2)) = answer a b", "v": null, "name": "h_answer"}]} {"informal_problem": "A dart, thrown at random, hits a square target. Assuming that any two parts of the target of equal area are equally likely to be hit, find the probability that the point hit is nearer to the center than to any edge. Express your answer in the form $(a\\sqrt{b}+c)/d$, where $a$, $b$, $c$, $d$ are integers and $b$, $d$ are positive.", "informal_answer": "(4, 2, -5, 3)", "informal_solution": "Show that the probability is $(4\\sqrt{2}-5)/3$.", "header": "open Nat MeasureTheory", "intros": [], "formal_answer": "@Eq (Prod Int (Prod Int (Prod Int Int))) answer\n (@Prod.mk Int (Prod Int (Prod Int Int)) (@OfNat.ofNat Int (nat_lit 4) (@instOfNat (nat_lit 4)))\n (@Prod.mk Int (Prod Int Int) (@OfNat.ofNat Int (nat_lit 2) (@instOfNat (nat_lit 2)))\n (@Prod.mk Int Int (@Neg.neg Int Int.instNegInt (@OfNat.ofNat Int (nat_lit 5) (@instOfNat (nat_lit 5))))\n (@OfNat.ofNat Int (nat_lit 3) (@instOfNat (nat_lit 3))))))", "formal_answer_type": "ℤ × ℤ × ℤ × ℤ", "outros": [{"t": "Set (EuclideanSpace ℝ (Fin 2))", "v": null, "name": "square"}, {"t": "Set (EuclideanSpace ℝ (Fin 2))", "v": null, "name": "Scloser"}, {"t": "Set (EuclideanSpace ℝ (Fin 2))", "v": null, "name": "perimeter"}, {"t": "EuclideanSpace ℝ (Fin 2)", "v": null, "name": "center"}, {"t": "square = {p | ∀ i : Fin 2, p i ∈ Set.Icc 0 1}", "v": null, "name": "square_def"}, {"t": "perimeter = {p ∈ square | p 0 = 0 ∨ p 0 = 1 ∨ p 1 = 0 ∨ p 1 = 1}", "v": null, "name": "perimeter_def"}, {"t": "center = (fun i : Fin 2 => 1 / 2)", "v": null, "name": "center_def"}, {"t": "Scloser = {p ∈ square | ∀ q ∈ perimeter, dist p center < dist p q}", "v": null, "name": "hScloser"}, {"t": "let (a, b, c, d) := answer;\n b > 0 ∧ d > 0 ∧ (¬∃ n : ℤ, n^2 = b) ∧\n (volume Scloser).toReal / (volume square).toReal = (a * Real.sqrt b + c) / d", "v": null, "name": "h_answer"}]} {"informal_problem": "Let $S$ be a non-empty set with an associative operation that is left and right cancellative ($xy=xz$ implies $y=z$, and $yx=zx$ implies $y=z$). Assume that for every $a$ in $S$ the set $\\{a^n:\\,n=1, 2, 3, \\ldots\\}$ is finite. Must $S$ be a group?", "informal_answer": "True", "informal_solution": "Prove that $S$ must be a group.", "header": "open Nat", "intros": [], "formal_answer": "@Eq Prop answer True", "formal_answer_type": "Prop", "outros": [{"t": "(∀ (S : Type) [Nonempty S] [Semigroup S] [IsCancelMul S]\n (h_fin : ∀ a : S, {(a * ·)^[n] a | n : ℕ}.Finite),\n ∃ e : S, ∀ x, e * x = x ∧ x * e = x ∧ ∃ y, x * y = e ∧ y * x = e) ↔\n answer", "v": null, "name": "h_answer"}]} {"informal_problem": "Let $f$ be a function on $[0,\\infty)$, differentiable and satisfying\n\\[\nf'(x)=-3f(x)+6f(2x)\n\\]\nfor $x>0$. Assume that $|f(x)|\\le e^{-\\sqrt{x}}$ for $x\\ge 0$ (so that $f(x)$ tends rapidly to $0$ as $x$ increases). For $n$ a non-negative integer, define\n\\[\n\\mu_n=\\int_0^\\infty x^n f(x)\\,dx\n\\]\n(sometimes called the $n$th moment of $f$).\n\\begin{enumerate}\n\\item[a)] Express $\\mu_n$ in terms of $\\mu_0$.\n\\item[b)] Prove that the sequence $\\{\\mu_n \\frac{3^n}{n!}\\}$ always converges, and that the limit is $0$ only if $\\mu_0=0$.\n\\end{enumerate}", "informal_answer": "fun n c ↦ c * n ! / (3 ^ n * ∏ m in Finset.Icc (1 : ℤ) n, (1 - 2 ^ (-m)))", "informal_solution": "Show that for each $n \\geq 0$, $\\mu_n = \\frac{n!}{3^n} \\left( \\prod_{m=1}^{n}(1 - 2^{-m}) \\right)^{-1} \\mu_0$.", "header": "open Nat Filter Topology", "intros": [], "formal_answer": "@Eq (Nat → Real → Real) answer fun (n : Nat) (c : Real) =>\n @HDiv.hDiv Real Real Real (@instHDiv Real (@DivInvMonoid.toDiv Real Real.instDivInvMonoid))\n (@HMul.hMul Real Real Real (@instHMul Real Real.instMul) c (@Nat.cast Real Real.instNatCast (Nat.factorial n)))\n (@HMul.hMul Real Real Real (@instHMul Real Real.instMul)\n (@HPow.hPow Real Nat Real (@instHPow Real Nat (@Monoid.toNatPow Real Real.instMonoid))\n (@OfNat.ofNat Real (nat_lit 3)\n (@instOfNatAtLeastTwo Real (nat_lit 3) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1))))))\n n)\n (@Finset.prod Int Real Real.instCommMonoid\n (@Finset.Icc Int\n (@PartialOrder.toPreorder Int\n (@OrderedAddCommGroup.toPartialOrder Int\n (@StrictOrderedRing.toOrderedAddCommGroup Int\n (@LinearOrderedRing.toStrictOrderedRing Int\n (@LinearOrderedCommRing.toLinearOrderedRing Int Int.instLinearOrderedCommRing)))))\n Int.instLocallyFiniteOrder (@OfNat.ofNat Int (nat_lit 1) (@instOfNat (nat_lit 1)))\n (@Nat.cast Int instNatCastInt n))\n fun (m : Int) =>\n @HSub.hSub Real Real Real (@instHSub Real Real.instSub)\n (@OfNat.ofNat Real (nat_lit 1) (@One.toOfNat1 Real Real.instOne))\n (@HPow.hPow Real Int Real (@instHPow Real Int (@DivInvMonoid.toZPow Real Real.instDivInvMonoid))\n (@OfNat.ofNat Real (nat_lit 2)\n (@instOfNatAtLeastTwo Real (nat_lit 2) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 0) (instOfNatNat (nat_lit 0))))))\n (@Neg.neg Int Int.instNegInt m))))", "formal_answer_type": "ℕ → ℝ → ℝ", "outros": [{"t": "ℝ → ℝ", "v": null, "name": "f"}, {"t": "Differentiable ℝ f", "v": null, "name": "hfdiff"}, {"t": "∀ x > 0, deriv f x = -3 * f x + 6 * f (2 * x)", "v": null, "name": "hfderiv"}, {"t": "∀ x ≥ 0, |f x| ≤ Real.exp (- √x)", "v": null, "name": "hdecay"}, {"t": "ℕ → ℝ", "v": null, "name": "μ"}, {"t": "∀ n, μ n = ∫ x in Set.Ioi 0, x ^ n * f x", "v": null, "name": "μ_def"}, {"t": "(∀ n, μ n = answer n (μ 0)) ∧\n (∃ L, Tendsto (fun n ↦ (μ n) * 3 ^ n / n !) atTop (𝓝 L)) ∧\n (Tendsto (fun n ↦ (μ n) * 3 ^ n / n !) atTop (𝓝 0) → μ 0 = 0)", "v": null, "name": "h_answer"}]} @@ -149,9 +149,9 @@ {"informal_problem": "For any pair $(x,y)$ of real numbers, a sequence $(a_n(x,y))_{n \\geq 0}$ is defined as follows:\n\\begin{align*}\na_0(x,y)&=x, \\\\\na_{n+1}(x,y)&=\\frac{(a_n(x,y))^2+y^2}{2},\\text{ for $n \\geq 0$.}\n\\end{align*}\nFind the area of the region $\\{(x,y) \\mid (a_n(x,y))_{n \\geq 0}\\text{ converges}\\}$.", "informal_answer": "4 + π", "informal_solution": "Show that the area is $4+\\pi$.", "header": "open Topology Filter Nat Function Polynomial", "intros": [], "formal_answer": "@Eq Real answer\n (@HAdd.hAdd Real Real Real (@instHAdd Real Real.instAdd)\n (@OfNat.ofNat Real (nat_lit 4)\n (@instOfNatAtLeastTwo Real (nat_lit 4) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))))))\n Real.pi)", "formal_answer_type": "ℝ", "outros": [{"t": "(Fin 2 → ℝ) → (ℕ → ℝ)", "v": null, "name": "a"}, {"t": "∀ p, (a p) 0 = p 0 ∧ (∀ n, (a p) (n + 1) = (((a p) n) ^ 2 + (p 1) ^ 2) / 2)", "v": null, "name": "ha"}, {"t": "answer = (MeasureTheory.volume {p | ∃ L, Tendsto (a p) atTop (𝓝 L)}).toReal", "v": null, "name": "h_answer"}]} {"informal_problem": "Let $p(x)$ be a nonzero polynomial of degree less than $1992$ having no nonconstant factor in common with $x^3 - x$. Let\n\\[\n\\frac{d^{1992}}{dx^{1992}} \\left( \\frac{p(x)}{x^3 - x} \\right) = \\frac{f(x)}{g(x)}\n\\]\nfor polynomials $f(x)$ and $g(x)$. Find the smallest possible degree of $f(x)$.", "informal_answer": "3984", "informal_solution": "Show that the minimum degree is $3984$.", "header": "open Topology Filter Nat Function Polynomial", "intros": [], "formal_answer": "@Eq Nat answer (@OfNat.ofNat Nat (nat_lit 3984) (instOfNatNat (nat_lit 3984)))", "formal_answer_type": "ℕ", "outros": [{"t": "Polynomial ℝ → Prop", "v": null, "name": "IsValid"}, {"t": "Polynomial ℝ → Polynomial ℝ → Prop", "v": null, "name": "pair"}, {"t": "∀ p, IsValid p ↔ p ≠ 0 ∧ p.degree < 1992 ∧ IsCoprime p (X ^ 3 - X)", "v": null, "name": "IsValid_def"}, {"t": "∀ p f, pair p f ↔ ∃ g : Polynomial ℝ, iteratedDeriv 1992 (fun x ↦ p.eval x / (x ^ 3 - x)) = fun x ↦ f.eval x / g.eval x", "v": null, "name": "hpair"}, {"t": "IsLeast {k : ℕ | ∃ p f, IsValid p ∧ pair p f ∧ k = f.degree} answer", "v": null, "name": "h_answer"}]} {"informal_problem": "Let $D_n$ denote the value of the $(n-1) \\times (n-1)$ determinant\n\\[\n\\left[\n\\begin{array}{cccccc}\n3 & 1 & 1 & 1 & \\cdots & 1 \\\\\n1 & 4 & 1 & 1 & \\cdots & 1 \\\\\n1 & 1 & 5 & 1 & \\cdots & 1 \\\\\n1 & 1 & 1 & 6 & \\cdots & 1 \\\\\n\\vdots & \\vdots & \\vdots & \\vdots & \\ddots & \\vdots \\\\\n1 & 1 & 1 & 1 & \\cdots & n+1\n\\end{array}\n\\right].\n\\]\nIs the set $\\left\\{ \\frac{D_n}{n!} \\right\\}_{n \\geq 2}$ bounded?", "informal_answer": "False", "informal_solution": "Prove that the set is not bounded.", "header": "open Topology Filter Nat Function Polynomial", "intros": [], "formal_answer": "@Eq Prop answer False", "formal_answer_type": "Prop", "outros": [{"t": "ℕ → ℚ", "v": null, "name": "D"}, {"t": "∀ n, D n = Matrix.det (fun i j : Fin (n - 1) ↦ ite (i = j) ((i : ℕ) + 3 : ℚ) 1)", "v": null, "name": "hD"}, {"t": "answer ↔ (Bornology.IsBounded {x | ∃ n ≥ 2, D n / factorial n = x})", "v": null, "name": "h_answer"}]} -{"informal_problem": "The horizontal line $y=c$ intersects the curve $y=2x-3x^3$ in the first quadrant as in the figure. Find $c$ so that the areas of the two shaded regions are equal. [Figure not included. The first region is bounded by the $y$-axis, the line $y=c$ and the curve; the other lies under the curve and above the line $y=c$ between their two points of intersection.]", "informal_answer": "4/9", "informal_solution": "Show that the area of the two regions are equal when $c=4/9$.", "header": null, "intros": [], "formal_answer": "@Eq Real answer\n (@HDiv.hDiv Real Real Real (@instHDiv Real (@DivInvMonoid.toDiv Real Real.instDivInvMonoid))\n (@OfNat.ofNat Real (nat_lit 4)\n (@instOfNatAtLeastTwo Real (nat_lit 4) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))))))\n (@OfNat.ofNat Real (nat_lit 9)\n (@instOfNatAtLeastTwo Real (nat_lit 9) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 7) (instOfNatNat (nat_lit 7)))))))", "formal_answer_type": "ℝ", "outros": [{"t": "0 < answer ∧ answer < (4 * Real.sqrt 2) / 9 ∧\n (∫ x in Set.Ioo 0 ((Real.sqrt 2) / 3), max (answer - (2 * x - 3 * x ^ 3)) 0) =\n (∫ x in Set.Ioo 0 ((Real.sqrt 6) / 3), max ((2 * x - 3 * x ^ 3) - answer) 0)", "v": null, "name": "h_answer"}]} -{"informal_problem": "Find the smallest positive integer $n$ such that for every integer $m$ with $0\n Or\n (And (@LE.le Int Int.instLEInt (@OfNat.ofNat Int (nat_lit 315) (@instOfNat (nat_lit 315))) n_1)\n (@LE.le Int Int.instLEInt n_1 (@OfNat.ofNat Int (nat_lit 325) (@instOfNat (nat_lit 325)))))\n (And (@LE.le Int Int.instLEInt (@OfNat.ofNat Int (nat_lit 332) (@instOfNat (nat_lit 332))) n_1)\n (@LE.le Int Int.instLEInt n_1 (@OfNat.ofNat Int (nat_lit 350) (@instOfNat (nat_lit 350))))))", "formal_answer_type": "Set ℤ", "outros": [{"t": "ℤ", "v": null, "name": "n"}, {"t": "n ∈ answer ↔ (0 < n ∧ {m : ℕ | |n - m ^ 2| ≤ 250}.encard = 15)", "v": null, "name": "h_answer"}]} {"informal_problem": "For which real numbers $c$ is there a straight line that intersects the curve $x^4+9x^3+cx^2+9x+4$ in four distinct points?", "informal_answer": "{c : ℝ | c < 243 / 8}", "informal_solution": "Show that there exists such a line if and only if $c<243/8$.", "header": "open Filter Topology", "intros": [], "formal_answer": "@Eq (Set Real) answer\n (@setOf Real fun (c_1 : Real) =>\n @LT.lt Real Real.instLT c_1\n (@HDiv.hDiv Real Real Real (@instHDiv Real (@DivInvMonoid.toDiv Real Real.instDivInvMonoid))\n (@OfNat.ofNat Real (nat_lit 243)\n (@instOfNatAtLeastTwo Real (nat_lit 243) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 241) (instOfNatNat (nat_lit 241))))))\n (@OfNat.ofNat Real (nat_lit 8)\n (@instOfNatAtLeastTwo Real (nat_lit 8) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 6) (instOfNatNat (nat_lit 6))))))))", "formal_answer_type": "Set ℝ", "outros": [{"t": "ℝ", "v": null, "name": "c"}, {"t": "answer = {c : ℝ | (∃ m b : ℝ,\n {x : ℝ | m * x + b = x ^ 4 + 9 * x ^ 3 + c * x ^ 2 + 9 * x + 4}.encard = 4)}", "v": null, "name": "h_answer"}]} {"informal_problem": "Find the set of all real numbers $k$ with the following property: For any positive, differentiable function $f$ that satisfies $f'(x)>f(x)$ for all $x$, there is some number $N$ such that $f(x)>e^{kx}$ for all $x>N$.", "informal_answer": "the set of all real numbers less than 1", "informal_solution": "Show that the desired set is $(-\\infty,1)$.", "header": "open Filter Topology", "intros": [], "formal_answer": "@Eq (Set Real) answer\n (@Set.Iio Real Real.instPreorder (@OfNat.ofNat Real (nat_lit 1) (@One.toOfNat1 Real Real.instOne)))", "formal_answer_type": "Set ℝ", "outros": [{"t": "{k | ∀ f (hf : (∀ x, 0 < f x ∧ f x < deriv f x) ∧ Differentiable ℝ f),\n ∃ N, ∀ x > N, Real.exp (k * x) < f x} = answer", "v": null, "name": "h_answer"}]} @@ -160,7 +160,7 @@ {"informal_problem": "To each positive integer with $n^{2}$ decimal digits, we associate the determinant of the matrix obtained by writing the digits in order across the rows. For example, for $n=2$, to the integer 8617 we associate $\\det \\left( \\begin{array}{cc} 8 & 6 \\ 1 & 7 \\end{array} \\right) = 50$. Find, as a function of $n$, the sum of all the determinants associated with $n^{2}$-digit integers. (Leading digits are assumed to be nonzero; for example, for $n=2$, there are 9000 determinants.)", "informal_answer": "45 if n = 1, 10 * 45² if n = 2, and 0 otherwise", "informal_solution": "Show that the solution is $45$ if $n = 1$, $45^2*10$ if $n = 2$, and $0$ if $n$ is greater than 2.", "header": "open Filter Topology Real Nat", "intros": [], "formal_answer": "@Eq (Nat → Int) answer fun (n_1 : Nat) =>\n @ite Int (@Eq Nat n_1 (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1))))\n (instDecidableEqNat n_1 (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1))))\n (@OfNat.ofNat Int (nat_lit 45) (@instOfNat (nat_lit 45)))\n (@ite Int (@Eq Nat n_1 (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))))\n (instDecidableEqNat n_1 (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))))\n (@HMul.hMul Int Int Int (@instHMul Int Int.instMul) (@OfNat.ofNat Int (nat_lit 10) (@instOfNat (nat_lit 10)))\n (@HPow.hPow Int Nat Int (@instHPow Int Nat (@Monoid.toNatPow Int Int.instMonoid))\n (@OfNat.ofNat Int (nat_lit 45) (@instOfNat (nat_lit 45)))\n (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))))\n (@OfNat.ofNat Int (nat_lit 0) (@instOfNat (nat_lit 0))))", "formal_answer_type": "ℕ → ℤ", "outros": [{"t": "ℕ", "v": null, "name": "n"}, {"t": "n > 0", "v": null, "name": "hn"}, {"t": "Set (ℕ → ℕ)", "v": null, "name": "digits_set"}, {"t": "digits_set = {f | f 0 ≠ 0 ∧ (∀ i : Fin (n ^ 2), f i ≤ 9) ∧ (∀ i ≥ n ^ 2, f i = 0)}", "v": null, "name": "hdigits_set"}, {"t": "(ℕ → ℕ) → Matrix (Fin n) (Fin n) ℤ", "v": null, "name": "digits_to_matrix"}, {"t": "digits_to_matrix = fun f => (fun i j => f (i.1 * n + j.1))", "v": null, "name": "hdigits_to_matrix"}, {"t": "∑' f : digits_set, (digits_to_matrix f).det = answer n", "v": null, "name": "h_answer"}]} {"informal_problem": "Evaluate \\[ \\sqrt[8]{2207 - \\frac{1}{2207-\\frac{1}{2207-\\dots}}}. \\] Express your answer in the form $\\frac{a+b\\sqrt{c}}{d}$, where $a,b,c,d$ are integers.", "informal_answer": "⟨3,1,5,2⟩", "informal_solution": "Show that the solution is $(3 + 1*\\sqrt{5})/2.", "header": "open Filter Topology Real Nat", "intros": [], "formal_answer": "@Eq (Prod Int (Prod Int (Prod Int Int))) answer\n (@Prod.mk Int (Prod Int (Prod Int Int)) (@OfNat.ofNat Int (nat_lit 3) (@instOfNat (nat_lit 3)))\n (@Prod.mk Int (Prod Int Int) (@OfNat.ofNat Int (nat_lit 1) (@instOfNat (nat_lit 1)))\n (@Prod.mk Int Int (@OfNat.ofNat Int (nat_lit 5) (@instOfNat (nat_lit 5)))\n (@OfNat.ofNat Int (nat_lit 2) (@instOfNat (nat_lit 2))))))", "formal_answer_type": "ℤ × ℤ × ℤ × ℤ", "outros": [{"t": "ℝ", "v": null, "name": "contfrac"}, {"t": "contfrac = 2207 - 1 / contfrac", "v": null, "name": "hcontfrac"}, {"t": "1 < contfrac", "v": null, "name": "hcontfrac'"}, {"t": "let ⟨a, b, c, d⟩ := answer;\n contfrac ^ ((1 : ℝ) / 8) = (a + b * sqrt c) / d", "v": null, "name": "h_answer"}]} {"informal_problem": "Let $C_1$ and $C_2$ be circles whose centers are $10$ units apart, and whose radii are $1$ and $3$. Find, with proof, the locus of all points $M$ for which there exist points $X$ on $C_1$ and $Y$ on $C_2$ such that $M$ is the midpoint of the line segment $XY$.", "informal_answer": "the set of points $p$ such that the distance from $p$ to the midpoint of $O_1$ and $O_2$ is between 1 and 2", "informal_solution": "Let $O_1$ and $O_2$ be the centers of $C_1$ and $C_2$, respectively. Then show that the desired locus is an annulus centered at the midpoint $O$ of $O_1O_2$, with inner radius $1$ and outer radius $2$.", "header": "open Metric", "intros": [], "formal_answer": "@Eq\n (EuclideanSpace Real (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) →\n EuclideanSpace Real (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) →\n Set (EuclideanSpace Real (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))))))\n answer fun (O1_1 O2_1 : EuclideanSpace Real (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))))) =>\n @setOf (EuclideanSpace Real (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))))\n fun (p : EuclideanSpace Real (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))))) =>\n And\n (@GE.ge Real Real.instLE\n (@Dist.dist (EuclideanSpace Real (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))))\n (@PiLp.instDist\n (@OfNat.ofNat ENNReal (nat_lit 2)\n (@instOfNatAtLeastTwo ENNReal (nat_lit 2)\n (@AddMonoidWithOne.toNatCast ENNReal\n (@AddCommMonoidWithOne.toAddMonoidWithOne ENNReal instENNRealAddCommMonoidWithOne))\n EuclideanSpace.proof_1))\n (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))))\n (fun (x : Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) => Real)\n (Fin.fintype (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))))\n fun (i : Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) =>\n @PseudoMetricSpace.toDist Real Real.pseudoMetricSpace)\n p\n (@midpoint Real (EuclideanSpace Real (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))))\n (EuclideanSpace Real (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))))) Real.instRing\n (@invertibleTwo Real Real.instDivisionRing (@RCLike.charZero_rclike Real Real.instRCLike))\n (@WithLp.instAddCommGroup\n (@OfNat.ofNat ENNReal (nat_lit 2)\n (@instOfNatAtLeastTwo ENNReal (nat_lit 2)\n (@AddMonoidWithOne.toNatCast ENNReal\n (@AddCommMonoidWithOne.toAddMonoidWithOne ENNReal instENNRealAddCommMonoidWithOne))\n EuclideanSpace.proof_1))\n ((i : Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) →\n (fun (x : Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) => Real) i)\n (@Pi.addCommGroup (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))))\n (fun (x : Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) => Real)\n fun (i : Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) => Real.instAddCommGroup))\n (@WithLp.instModule\n (@OfNat.ofNat ENNReal (nat_lit 2)\n (@instOfNatAtLeastTwo ENNReal (nat_lit 2)\n (@AddMonoidWithOne.toNatCast ENNReal\n (@AddCommMonoidWithOne.toAddMonoidWithOne ENNReal instENNRealAddCommMonoidWithOne))\n EuclideanSpace.proof_1))\n Real\n ((i : Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) →\n (fun (x : Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) => Real) i)\n (@Ring.toSemiring Real Real.instRing)\n (@Pi.addCommGroup (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))))\n (fun (x : Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) => Real)\n fun (i : Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) => Real.instAddCommGroup)\n (@Pi.Function.module (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real Real\n (@Ring.toSemiring Real Real.instRing)\n (@NonUnitalNonAssocSemiring.toAddCommMonoid Real\n (@NonUnitalSemiring.toNonUnitalNonAssocSemiring Real\n (@Semiring.toNonUnitalSemiring Real (@Ring.toSemiring Real Real.instRing))))\n (@NormedSpace.toModule Real Real Real.normedField\n (@NonUnitalSeminormedRing.toSeminormedAddCommGroup Real\n (@NonUnitalSeminormedCommRing.toNonUnitalSeminormedRing Real\n (@SeminormedCommRing.toNonUnitalSeminormedCommRing Real\n (@NormedCommRing.toSeminormedCommRing Real Real.normedCommRing))))\n (@InnerProductSpace.toNormedSpace Real Real Real.instRCLike\n (@NonUnitalSeminormedRing.toSeminormedAddCommGroup Real\n (@NonUnitalSeminormedCommRing.toNonUnitalSeminormedRing Real\n (@SeminormedCommRing.toNonUnitalSeminormedCommRing Real\n (@NormedCommRing.toSeminormedCommRing Real Real.normedCommRing))))\n (@RCLike.toInnerProductSpaceReal Real Real.instRCLike)))))\n (@NormedAddTorsor.toAddTorsor\n (EuclideanSpace Real (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))))\n (EuclideanSpace Real (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))))\n (@PiLp.seminormedAddCommGroup\n (@OfNat.ofNat ENNReal (nat_lit 2)\n (@instOfNatAtLeastTwo ENNReal (nat_lit 2)\n (@AddMonoidWithOne.toNatCast ENNReal\n (@AddCommMonoidWithOne.toAddMonoidWithOne ENNReal instENNRealAddCommMonoidWithOne))\n EuclideanSpace.proof_1))\n (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))))\n (fun (x : Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) => Real)\n fact_one_le_two_ennreal (Fin.fintype (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))))\n fun (i : Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) =>\n @NonUnitalSeminormedRing.toSeminormedAddCommGroup Real\n (@NonUnitalSeminormedCommRing.toNonUnitalSeminormedRing Real\n (@SeminormedCommRing.toNonUnitalSeminormedCommRing Real\n (@NormedCommRing.toSeminormedCommRing Real Real.normedCommRing))))\n (@SeminormedAddCommGroup.toPseudoMetricSpace\n (EuclideanSpace Real (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))))\n (@PiLp.seminormedAddCommGroup\n (@OfNat.ofNat ENNReal (nat_lit 2)\n (@instOfNatAtLeastTwo ENNReal (nat_lit 2)\n (@AddMonoidWithOne.toNatCast ENNReal\n (@AddCommMonoidWithOne.toAddMonoidWithOne ENNReal instENNRealAddCommMonoidWithOne))\n EuclideanSpace.proof_1))\n (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))))\n (fun (x : Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) => Real)\n fact_one_le_two_ennreal (Fin.fintype (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))))\n fun (i : Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) =>\n @NonUnitalSeminormedRing.toSeminormedAddCommGroup Real\n (@NonUnitalSeminormedCommRing.toNonUnitalSeminormedRing Real\n (@SeminormedCommRing.toNonUnitalSeminormedCommRing Real\n (@NormedCommRing.toSeminormedCommRing Real Real.normedCommRing)))))\n (@SeminormedAddCommGroup.toNormedAddTorsor\n (EuclideanSpace Real (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))))\n (@PiLp.seminormedAddCommGroup\n (@OfNat.ofNat ENNReal (nat_lit 2)\n (@instOfNatAtLeastTwo ENNReal (nat_lit 2)\n (@AddMonoidWithOne.toNatCast ENNReal\n (@AddCommMonoidWithOne.toAddMonoidWithOne ENNReal instENNRealAddCommMonoidWithOne))\n EuclideanSpace.proof_1))\n (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))))\n (fun (x : Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) => Real)\n fact_one_le_two_ennreal (Fin.fintype (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))))\n fun (i : Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) =>\n @NonUnitalSeminormedRing.toSeminormedAddCommGroup Real\n (@NonUnitalSeminormedCommRing.toNonUnitalSeminormedRing Real\n (@SeminormedCommRing.toNonUnitalSeminormedCommRing Real\n (@NormedCommRing.toSeminormedCommRing Real Real.normedCommRing))))))\n O1_1 O2_1))\n (@OfNat.ofNat Real (nat_lit 1) (@One.toOfNat1 Real Real.instOne)))\n (@LE.le Real Real.instLE\n (@Dist.dist (EuclideanSpace Real (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))))\n (@PiLp.instDist\n (@OfNat.ofNat ENNReal (nat_lit 2)\n (@instOfNatAtLeastTwo ENNReal (nat_lit 2)\n (@AddMonoidWithOne.toNatCast ENNReal\n (@AddCommMonoidWithOne.toAddMonoidWithOne ENNReal instENNRealAddCommMonoidWithOne))\n EuclideanSpace.proof_1))\n (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))))\n (fun (x : Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) => Real)\n (Fin.fintype (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))))\n fun (i : Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) =>\n @PseudoMetricSpace.toDist Real Real.pseudoMetricSpace)\n p\n (@midpoint Real (EuclideanSpace Real (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))))\n (EuclideanSpace Real (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))))) Real.instRing\n (@invertibleTwo Real Real.instDivisionRing (@RCLike.charZero_rclike Real Real.instRCLike))\n (@WithLp.instAddCommGroup\n (@OfNat.ofNat ENNReal (nat_lit 2)\n (@instOfNatAtLeastTwo ENNReal (nat_lit 2)\n (@AddMonoidWithOne.toNatCast ENNReal\n (@AddCommMonoidWithOne.toAddMonoidWithOne ENNReal instENNRealAddCommMonoidWithOne))\n EuclideanSpace.proof_1))\n ((i : Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) →\n (fun (x : Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) => Real) i)\n (@Pi.addCommGroup (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))))\n (fun (x : Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) => Real)\n fun (i : Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) => Real.instAddCommGroup))\n (@WithLp.instModule\n (@OfNat.ofNat ENNReal (nat_lit 2)\n (@instOfNatAtLeastTwo ENNReal (nat_lit 2)\n (@AddMonoidWithOne.toNatCast ENNReal\n (@AddCommMonoidWithOne.toAddMonoidWithOne ENNReal instENNRealAddCommMonoidWithOne))\n EuclideanSpace.proof_1))\n Real\n ((i : Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) →\n (fun (x : Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) => Real) i)\n (@Ring.toSemiring Real Real.instRing)\n (@Pi.addCommGroup (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))))\n (fun (x : Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) => Real)\n fun (i : Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) => Real.instAddCommGroup)\n (@Pi.Function.module (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real Real\n (@Ring.toSemiring Real Real.instRing)\n (@NonUnitalNonAssocSemiring.toAddCommMonoid Real\n (@NonUnitalSemiring.toNonUnitalNonAssocSemiring Real\n (@Semiring.toNonUnitalSemiring Real (@Ring.toSemiring Real Real.instRing))))\n (@NormedSpace.toModule Real Real Real.normedField\n (@NonUnitalSeminormedRing.toSeminormedAddCommGroup Real\n (@NonUnitalSeminormedCommRing.toNonUnitalSeminormedRing Real\n (@SeminormedCommRing.toNonUnitalSeminormedCommRing Real\n (@NormedCommRing.toSeminormedCommRing Real Real.normedCommRing))))\n (@InnerProductSpace.toNormedSpace Real Real Real.instRCLike\n (@NonUnitalSeminormedRing.toSeminormedAddCommGroup Real\n (@NonUnitalSeminormedCommRing.toNonUnitalSeminormedRing Real\n (@SeminormedCommRing.toNonUnitalSeminormedCommRing Real\n (@NormedCommRing.toSeminormedCommRing Real Real.normedCommRing))))\n (@RCLike.toInnerProductSpaceReal Real Real.instRCLike)))))\n (@NormedAddTorsor.toAddTorsor\n (EuclideanSpace Real (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))))\n (EuclideanSpace Real (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))))\n (@PiLp.seminormedAddCommGroup\n (@OfNat.ofNat ENNReal (nat_lit 2)\n (@instOfNatAtLeastTwo ENNReal (nat_lit 2)\n (@AddMonoidWithOne.toNatCast ENNReal\n (@AddCommMonoidWithOne.toAddMonoidWithOne ENNReal instENNRealAddCommMonoidWithOne))\n EuclideanSpace.proof_1))\n (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))))\n (fun (x : Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) => Real)\n fact_one_le_two_ennreal (Fin.fintype (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))))\n fun (i : Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) =>\n @NonUnitalSeminormedRing.toSeminormedAddCommGroup Real\n (@NonUnitalSeminormedCommRing.toNonUnitalSeminormedRing Real\n (@SeminormedCommRing.toNonUnitalSeminormedCommRing Real\n (@NormedCommRing.toSeminormedCommRing Real Real.normedCommRing))))\n (@SeminormedAddCommGroup.toPseudoMetricSpace\n (EuclideanSpace Real (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))))\n (@PiLp.seminormedAddCommGroup\n (@OfNat.ofNat ENNReal (nat_lit 2)\n (@instOfNatAtLeastTwo ENNReal (nat_lit 2)\n (@AddMonoidWithOne.toNatCast ENNReal\n (@AddCommMonoidWithOne.toAddMonoidWithOne ENNReal instENNRealAddCommMonoidWithOne))\n EuclideanSpace.proof_1))\n (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))))\n (fun (x : Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) => Real)\n fact_one_le_two_ennreal (Fin.fintype (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))))\n fun (i : Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) =>\n @NonUnitalSeminormedRing.toSeminormedAddCommGroup Real\n (@NonUnitalSeminormedCommRing.toNonUnitalSeminormedRing Real\n (@SeminormedCommRing.toNonUnitalSeminormedCommRing Real\n (@NormedCommRing.toSeminormedCommRing Real Real.normedCommRing)))))\n (@SeminormedAddCommGroup.toNormedAddTorsor\n (EuclideanSpace Real (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))))\n (@PiLp.seminormedAddCommGroup\n (@OfNat.ofNat ENNReal (nat_lit 2)\n (@instOfNatAtLeastTwo ENNReal (nat_lit 2)\n (@AddMonoidWithOne.toNatCast ENNReal\n (@AddCommMonoidWithOne.toAddMonoidWithOne ENNReal instENNRealAddCommMonoidWithOne))\n EuclideanSpace.proof_1))\n (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))))\n (fun (x : Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) => Real)\n fact_one_le_two_ennreal (Fin.fintype (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))))\n fun (i : Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) =>\n @NonUnitalSeminormedRing.toSeminormedAddCommGroup Real\n (@NonUnitalSeminormedCommRing.toNonUnitalSeminormedRing Real\n (@SeminormedCommRing.toNonUnitalSeminormedCommRing Real\n (@NormedCommRing.toSeminormedCommRing Real Real.normedCommRing))))))\n O1_1 O2_1))\n (@OfNat.ofNat Real (nat_lit 2)\n (@instOfNatAtLeastTwo Real (nat_lit 2) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 0) (instOfNatNat (nat_lit 0)))))))", "formal_answer_type": "(EuclideanSpace ℝ (Fin 2)) → (EuclideanSpace ℝ (Fin 2)) → Set (EuclideanSpace ℝ (Fin 2))", "outros": [{"t": "EuclideanSpace ℝ (Fin 2)", "v": null, "name": "O1"}, {"t": "EuclideanSpace ℝ (Fin 2)", "v": null, "name": "O2"}, {"t": "Set (EuclideanSpace ℝ (Fin 2))", "v": null, "name": "C1"}, {"t": "Set (EuclideanSpace ℝ (Fin 2))", "v": null, "name": "C2"}, {"t": "C1 = Metric.sphere O1 1", "v": null, "name": "hC1"}, {"t": "C2 = Metric.sphere O2 3", "v": null, "name": "hC2"}, {"t": "dist O1 O2 = 10", "v": null, "name": "hO1O2"}, {"t": "{M : EuclideanSpace ℝ (Fin 2) | ∃ X Y, X ∈ C1 ∧ Y ∈ C2 ∧ M = midpoint ℝ X Y} = answer O1 O2", "v": null, "name": "h_answer"}]} -{"informal_problem": "Suppose that each of 20 students has made a choice of anywhere from 0 to 6 courses from a total of 6 courses offered. Prove or disprove: there are 5 students and 2 courses such that all 5 have chosen both courses or all 5 have chosen neither course.", "informal_answer": "False", "informal_solution": "Show that the solution is that the statement is false.", "header": null, "intros": [], "formal_answer": "@Eq Prop answer False", "formal_answer_type": "Prop", "outros": [{"t": "Fin 20 → Set (Fin 6)", "v": null, "name": "choices"}, {"t": "answer ↔ (∃ (students : Finset (Fin 20)) (courses : Finset (Fin 6)),\n students.card = 5 ∧\n courses.card = 2 ∧\n (↑courses ⊆ ⋂ s ∈ students, choices s ∨ ↑courses ⊆ ⋂ s ∈ students, (choices s)ᶜ))", "v": null, "name": "h_answer"}]} +{"informal_problem": "Suppose that each of 20 students has made a choice of anywhere from 0 to 6 courses from a total of 6 courses offered. Prove or disprove: there are 5 students and 2 courses such that all 5 have chosen both courses or all 5 have chosen neither course.", "informal_answer": "False", "informal_solution": "Show that the solution is that the statement is false.", "header": "open BigOperators Real Nat Topology", "intros": [], "formal_answer": "@Eq Prop answer False", "formal_answer_type": "Prop", "outros": [{"t": "Fin 20 → Set (Fin 6)", "v": null, "name": "choices"}, {"t": "answer ↔ (∃ (students : Finset (Fin 20)) (courses : Finset (Fin 6)),\n students.card = 5 ∧\n courses.card = 2 ∧\n (↑courses ⊆ ⋂ s ∈ students, choices s ∨ ↑courses ⊆ ⋂ s ∈ students, (choices s)ᶜ))", "v": null, "name": "h_answer"}]} {"informal_problem": "Let $c>0$ be a constant. Give a complete description, with proof, of the set of all continuous functions $f:\\mathbb{R} \\to \\mathbb{R}$ such that $f(x)=f(x^2+c)$ for all $x \\in \\mathbb{R}$.", "informal_answer": "the set of functions described by the condition", "informal_solution": "Show that if $c \\leq 1/4$ then $f$ must be constant, and if $c>1/4$ then $f$ can be defined on $[0,c]$ as any continuous function with equal values on the endpoints, then extended to $x>c$ by the relation $f(x)=f(x^2+c)$, then extended further to $x<0$ by the relation $f(x)=f(-x)$.", "header": "open Function", "intros": [], "formal_answer": "@Eq (Real → Set (Real → Real)) answer fun (c_1 : Real) =>\n @ite (Set (Real → Real))\n (@LE.le Real Real.instLE c_1\n (@HDiv.hDiv Real Real Real (@instHDiv Real (@DivInvMonoid.toDiv Real Real.instDivInvMonoid))\n (@OfNat.ofNat Real (nat_lit 1) (@One.toOfNat1 Real Real.instOne))\n (@OfNat.ofNat Real (nat_lit 4)\n (@instOfNatAtLeastTwo Real (nat_lit 4) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))))))))\n (Real.decidableLE c_1\n (@HDiv.hDiv Real Real Real (@instHDiv Real (@DivInvMonoid.toDiv Real Real.instDivInvMonoid))\n (@OfNat.ofNat Real (nat_lit 1) (@One.toOfNat1 Real Real.instOne))\n (@OfNat.ofNat Real (nat_lit 4)\n (@instOfNatAtLeastTwo Real (nat_lit 4) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))))))))\n (@setOf (Real → Real) fun (f_1 : Real → Real) => @Exists Real fun (d : Real) => ∀ (x : Real), @Eq Real (f_1 x) d)\n (@setOf (Real → Real) fun (f_1 : Real → Real) =>\n And\n (@ContinuousOn Real Real\n (@UniformSpace.toTopologicalSpace Real (@PseudoMetricSpace.toUniformSpace Real Real.pseudoMetricSpace))\n (@UniformSpace.toTopologicalSpace Real (@PseudoMetricSpace.toUniformSpace Real Real.pseudoMetricSpace)) f_1\n (@Set.Icc Real Real.instPreorder (@OfNat.ofNat Real (nat_lit 0) (@Zero.toOfNat0 Real Real.instZero)) c_1))\n (And (@Eq Real (f_1 (@OfNat.ofNat Real (nat_lit 0) (@Zero.toOfNat0 Real Real.instZero))) (f_1 c_1))\n (And\n (∀ (x : Real),\n @GT.gt Real Real.instLT x (@OfNat.ofNat Real (nat_lit 0) (@Zero.toOfNat0 Real Real.instZero)) →\n @Eq Real (f_1 x)\n (f_1\n (@HAdd.hAdd Real Real Real (@instHAdd Real Real.instAdd)\n (@HPow.hPow Real Nat Real (@instHPow Real Nat (@Monoid.toNatPow Real Real.instMonoid)) x\n (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))))\n c_1)))\n (∀ (x : Real),\n @LT.lt Real Real.instLT x (@OfNat.ofNat Real (nat_lit 0) (@Zero.toOfNat0 Real Real.instZero)) →\n @Eq Real (f_1 x) (f_1 (@Neg.neg Real Real.instNeg x))))))", "formal_answer_type": "ℝ → Set (ℝ → ℝ)", "outros": [{"t": "ℝ", "v": null, "name": "c"}, {"t": "ℝ → ℝ", "v": null, "name": "f"}, {"t": "c > 0", "v": null, "name": "cgt0"}, {"t": "(Continuous f ∧ ∀ x : ℝ, f x = f (x ^ 2 + c)) ↔ f ∈ answer c", "v": null, "name": "h_answer"}]} {"informal_problem": "Define a \\emph{selfish} set to be a set which has its own cardinality (number of elements) as an element. Find, with proof, the number of subsets of $\\{1,2,\\ldots,n\\}$ which are \\emph{minimal} selfish sets, that is, selfish sets none of whose proper subsets is selfish.", "informal_answer": "the nth Fibonacci number", "informal_solution": "Show that the number of subsets is $F_n$, the $n$th Fibonacci number.", "header": "open Function", "intros": [], "formal_answer": "@Eq (Nat → Nat) answer Nat.fib", "formal_answer_type": "ℕ → ℕ", "outros": [{"t": "Finset ℕ → Prop", "v": null, "name": "selfish"}, {"t": "ℕ", "v": null, "name": "n"}, {"t": "∀ s : Finset ℕ, selfish s = (s.card ∈ s)", "v": null, "name": "hselfish"}, {"t": "n ≥ 1", "v": null, "name": "npos"}, {"t": "{s : Finset ℕ | (s : Set ℕ) ⊆ Set.Icc 1 n ∧ selfish s ∧ (∀ ss : Finset ℕ, ss ⊂ s → ¬selfish ss)}.encard = answer n", "v": null, "name": "h_answer"}]} {"informal_problem": "Given that $\\{x_1,x_2,\\ldots,x_n\\}=\\{1,2,\\ldots,n\\}$, find, with proof, the largest possible value, as a function of $n$ (with $n \\geq 2$), of $x_1x_2+x_2x_3+\\cdots+x_{n-1}x_n+x_nx_1$.", "informal_answer": "$(2n^3 + 3n^2 - 11n + 18) / 6$", "informal_solution": "Show that the maximum is $(2n^3+3n^2-11n+18)/6$.", "header": "open Function", "intros": [], "formal_answer": "@Eq (Nat → Nat) answer fun (n_1 : Nat) =>\n @HDiv.hDiv Nat Nat Nat (@instHDiv Nat Nat.instDiv)\n (@HAdd.hAdd Nat Nat Nat (@instHAdd Nat instAddNat)\n (@HSub.hSub Nat Nat Nat (@instHSub Nat instSubNat)\n (@HAdd.hAdd Nat Nat Nat (@instHAdd Nat instAddNat)\n (@HMul.hMul Nat Nat Nat (@instHMul Nat instMulNat) (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))\n (@HPow.hPow Nat Nat Nat (@instHPow Nat Nat (@Monoid.toNatPow Nat Nat.instMonoid)) n_1\n (@OfNat.ofNat Nat (nat_lit 3) (instOfNatNat (nat_lit 3)))))\n (@HMul.hMul Nat Nat Nat (@instHMul Nat instMulNat) (@OfNat.ofNat Nat (nat_lit 3) (instOfNatNat (nat_lit 3)))\n (@HPow.hPow Nat Nat Nat (@instHPow Nat Nat (@Monoid.toNatPow Nat Nat.instMonoid)) n_1\n (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))))))\n (@HMul.hMul Nat Nat Nat (@instHMul Nat instMulNat) (@OfNat.ofNat Nat (nat_lit 11) (instOfNatNat (nat_lit 11)))\n n_1))\n (@OfNat.ofNat Nat (nat_lit 18) (instOfNatNat (nat_lit 18))))\n (@OfNat.ofNat Nat (nat_lit 6) (instOfNatNat (nat_lit 6)))", "formal_answer_type": "ℕ → ℕ", "outros": [{"t": "ℕ", "v": null, "name": "n"}, {"t": "n ≥ 2", "v": null, "name": "hn"}, {"t": "IsGreatest\n {k | ∃ x : ℕ → ℤ,\n (x '' (Finset.range n) = Set.Icc (1 : ℤ) n) ∧\n ∑ i : Fin n, x i * x ((i + 1) % n) = k}\n (answer n)", "v": null, "name": "h_answer"}]} @@ -171,12 +171,12 @@ {"informal_problem": "For a positive integer $n$ and any real number $c$, define $x_k$ recursively by $x_0=0$, $x_1=1$, and for $k\\geq 0$, \\[x_{k+2}=\\frac{cx_{k+1}-(n-k)x_k}{k+1}.\\] Fix $n$ and then take $c$ to be the largest value for which $x_{n+1}=0$. Find $x_k$ in terms of $n$ and $k$, $1\\leq k\\leq n$.", "informal_answer": "fun n k => Nat.choose (n.toNat-1) (k.toNat-1)", "informal_solution": "Show that the solution is that $x_k = {n - 1 \\choose k - 1}$.", "header": "open Filter Topology", "intros": [], "formal_answer": "@Eq (Int → Int → Real) answer fun (n_1 k : Int) =>\n @Nat.cast Real Real.instNatCast\n (Nat.choose\n (@HSub.hSub Nat Nat Nat (@instHSub Nat instSubNat) (Int.toNat n_1)\n (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1))))\n (@HSub.hSub Nat Nat Nat (@instHSub Nat instSubNat) (Int.toNat k)\n (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1)))))", "formal_answer_type": "ℤ → ℤ → ℝ", "outros": [{"t": "ℤ", "v": null, "name": "n"}, {"t": "n > 0", "v": null, "name": "hn"}, {"t": "ℝ → (ℤ → ℝ)", "v": null, "name": "x"}, {"t": "∀ c, x c 0 = 0", "v": null, "name": "hx0"}, {"t": "∀ c, x c 1 = 1", "v": null, "name": "hx1"}, {"t": "∀ c, ∀ k ≥ 0, x c (k + 2) = (c*(x c (k + 1)) - (n - k)*(x c k))/(k + 1)", "v": null, "name": "hxk"}, {"t": "Set ℝ", "v": null, "name": "S"}, {"t": "S = {c : ℝ | x c (n + 1) = 0}", "v": null, "name": "hS"}, {"t": "∀ k : Set.Icc 1 n, x (sSup S) k = answer n k", "v": null, "name": "h_answer"}]} {"informal_problem": "Let $\\{x\\}$ denote the distance between the real number $x$ and the nearest integer. For each positive integer $n$, evaluate \\[F_n=\\sum_{m=1}^{6n-1} \\min(\\{\\frac{m}{6n}\\},\\{\\frac{m}{3n}\\}).\\] (Here $\\min(a,b)$ denotes the minimum of $a$ and $b$.)", "informal_answer": "fun n => n", "informal_solution": "Show that the solution is $n$.", "header": "open Filter Topology", "intros": [{"t": "Real", "v": null, "name": "r"}], "formal_answer": "@Eq (Nat → Real) answer fun (n : Nat) => @Nat.cast Real Real.instNatCast n", "formal_answer_type": "ℕ → ℝ", "outros": [{"t": "ℝ → ℝ", "v": null, "name": "dist_to_int"}, {"t": "dist_to_int r = |r - round r|", "v": null, "name": "h_dist_to_int"}, {"t": "ℕ → ℝ", "v": null, "name": "F"}, {"t": "F = fun (n : ℕ) => ∑ m in Finset.Icc 1 (6 * n - 1), min (dist_to_int (m/(6*n)) ) (dist_to_int (m/(3*n)))", "v": null, "name": "hF"}, {"t": "∀ n, n > 0 → F n = answer n", "v": null, "name": "h_answer"}]} {"informal_problem": "For each positive integer $n$, write the sum $\\sum_{m=1}^n 1/m$ in the form $p_n/q_n$, where $p_n$ and $q_n$ are relatively prime positive integers. Determine all $n$ such that 5 does not divide $q_n$.", "informal_answer": "{n | (1 ≤ n ∧ n ≤ 4) ∨ (20 ≤ n ∧ n ≤ 24) ∨ (100 ≤ n ∧ n ≤ 104) ∨ (120 ≤ n ∧ n ≤ 124)}", "informal_solution": "Show that the solution is the set of natural numbers which are between $1$ and $4$, or between $20$ and $24$, or between $100$ and $104$, or between $120$ and $124$.", "header": "open Filter Topology Bornology Set", "intros": [], "formal_answer": "@Eq (Set Nat) answer\n (@setOf Nat fun (n_1 : Nat) =>\n Or\n (And (@LE.le Nat instLENat (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1))) n_1)\n (@LE.le Nat instLENat n_1 (@OfNat.ofNat Nat (nat_lit 4) (instOfNatNat (nat_lit 4)))))\n (Or\n (And (@LE.le Nat instLENat (@OfNat.ofNat Nat (nat_lit 20) (instOfNatNat (nat_lit 20))) n_1)\n (@LE.le Nat instLENat n_1 (@OfNat.ofNat Nat (nat_lit 24) (instOfNatNat (nat_lit 24)))))\n (Or\n (And (@LE.le Nat instLENat (@OfNat.ofNat Nat (nat_lit 100) (instOfNatNat (nat_lit 100))) n_1)\n (@LE.le Nat instLENat n_1 (@OfNat.ofNat Nat (nat_lit 104) (instOfNatNat (nat_lit 104)))))\n (And (@LE.le Nat instLENat (@OfNat.ofNat Nat (nat_lit 120) (instOfNatNat (nat_lit 120))) n_1)\n (@LE.le Nat instLENat n_1 (@OfNat.ofNat Nat (nat_lit 124) (instOfNatNat (nat_lit 124))))))))", "formal_answer_type": "Set ℕ", "outros": [{"t": "ℕ", "v": null, "name": "n"}, {"t": "n > 0", "v": null, "name": "hn"}, {"t": "n ∈ answer ↔ ¬5 ∣ (∑ m in Finset.Icc 1 n, 1/m : ℚ).den", "v": null, "name": "h_answer"}]} -{"informal_problem": "Let $A_1=0$ and $A_2=1$. For $n>2$, the number $A_n$ is defined by concatenating the decimal expansions of $A_{n-1}$ and $A_{n-2}$ from left to right. For example $A_3=A_2 A_1=10$, $A_4=A_3 A_2 = 101$, $A_5=A_4 A_3 = 10110$, and so forth. Determine all $n$ such that $11$ divides $A_n$.", "informal_answer": "all $n$ such that $n \\equiv 1 \\pmod{6}$", "informal_solution": "Show that the solution is those n for which n can be written as 6k+1 for some integer k.", "header": null, "intros": [], "formal_answer": "@Eq (Set Nat) answer\n (@setOf Nat fun (n : Nat) =>\n Nat.ModEq (@OfNat.ofNat Nat (nat_lit 6) (instOfNatNat (nat_lit 6))) n\n (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1))))", "formal_answer_type": "Set ℕ", "outros": [{"t": "ℕ → List ℕ", "v": null, "name": "A"}, {"t": "A 1 = [0]", "v": null, "name": "hA1"}, {"t": "A 2 = [1]", "v": null, "name": "hA2"}, {"t": "∀ n > 0, A (n + 2) = A (n + 1) ++ A n", "v": null, "name": "hA"}, {"t": "{n | 1 ≤ n ∧ 11 ∣ Nat.ofDigits 10 (A n).reverse} = answer", "v": null, "name": "h_answer"}]} +{"informal_problem": "Let $A_1=0$ and $A_2=1$. For $n>2$, the number $A_n$ is defined by concatenating the decimal expansions of $A_{n-1}$ and $A_{n-2}$ from left to right. For example $A_3=A_2 A_1=10$, $A_4=A_3 A_2 = 101$, $A_5=A_4 A_3 = 10110$, and so forth. Determine all $n$ such that $11$ divides $A_n$.", "informal_answer": "all $n$ such that $n \\equiv 1 \\pmod{6}$", "informal_solution": "Show that the solution is those n for which n can be written as 6k+1 for some integer k.", "header": "open BigOperators Real Nat Topology", "intros": [], "formal_answer": "@Eq (Set Nat) answer\n (@setOf Nat fun (n : Nat) =>\n Nat.ModEq (@OfNat.ofNat Nat (nat_lit 6) (instOfNatNat (nat_lit 6))) n\n (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1))))", "formal_answer_type": "Set ℕ", "outros": [{"t": "ℕ → List ℕ", "v": null, "name": "A"}, {"t": "A 1 = [0]", "v": null, "name": "hA1"}, {"t": "A 2 = [1]", "v": null, "name": "hA2"}, {"t": "∀ n > 0, A (n + 2) = A (n + 1) ++ A n", "v": null, "name": "hA"}, {"t": "{n | 1 ≤ n ∧ 11 ∣ Nat.ofDigits 10 (A n).reverse} = answer", "v": null, "name": "h_answer"}]} {"informal_problem": "Find the minimum value of \\[\\frac{(x+1/x)^6-(x^6+1/x^6)-2}{(x+1/x)^3+(x^3+1/x^3)}\\] for $x>0$.", "informal_answer": "6", "informal_solution": "Show that the minimum value is 6.", "header": "open Set Function Metric", "intros": [], "formal_answer": "@Eq Real answer\n (@OfNat.ofNat Real (nat_lit 6)\n (@instOfNatAtLeastTwo Real (nat_lit 6) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 4) (instOfNatNat (nat_lit 4))))))", "formal_answer_type": "ℝ", "outros": [{"t": "sInf {((x + 1/x)^6 - (x^6 + 1/x^6) - 2)/((x + 1/x)^3 + (x^3 + 1/x^3)) | x > (0 : ℝ)} = answer", "v": null, "name": "h_answer"}]} {"informal_problem": "Given a point $(a,b)$ with $0 b$, otherwise $0$", "informal_solution": "Show that the solution is $\\sqrt{2a^2 + 2b^2}.", "header": "open Set Function Metric", "intros": [], "formal_answer": "@Eq (Real → Real → Real) answer fun (a_1 b_1 : Real) =>\n @ite Real (@GT.gt Real Real.instLT a_1 b_1) (Real.decidableLT b_1 a_1)\n (Real.sqrt\n (@HAdd.hAdd Real Real Real (@instHAdd Real Real.instAdd)\n (@HMul.hMul Real Real Real (@instHMul Real Real.instMul)\n (@OfNat.ofNat Real (nat_lit 2)\n (@instOfNatAtLeastTwo Real (nat_lit 2) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 0) (instOfNatNat (nat_lit 0))))))\n (@HPow.hPow Real Nat Real (@instHPow Real Nat (@Monoid.toNatPow Real Real.instMonoid)) a_1\n (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))))\n (@HMul.hMul Real Real Real (@instHMul Real Real.instMul)\n (@OfNat.ofNat Real (nat_lit 2)\n (@instOfNatAtLeastTwo Real (nat_lit 2) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 0) (instOfNatNat (nat_lit 0))))))\n (@HPow.hPow Real Nat Real (@instHPow Real Nat (@Monoid.toNatPow Real Real.instMonoid)) b_1\n (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))))))\n (@OfNat.ofNat Real (nat_lit 0) (@Zero.toOfNat0 Real Real.instZero))", "formal_answer_type": "ℝ → ℝ → ℝ", "outros": [{"t": "ℝ", "v": null, "name": "a"}, {"t": "ℝ", "v": null, "name": "b"}, {"t": "0 < b ∧ b < a", "v": null, "name": "hab"}, {"t": "sInf {d : ℝ | ∃ (c : ℝ) (x : ℝ), d = Real.sqrt ((a - c)^2 + (b - 0)^2) + Real.sqrt ((c - x)^2 + (0 - x)^2) + Real.sqrt ((a - x)^2 + (b - x)^2) ∧\n Real.sqrt ((a - c)^2 + (b - 0)^2) + Real.sqrt ((c - x)^2 + (0 - x)^2) > Real.sqrt ((a - x)^2 + (b - x)^2) ∧\n Real.sqrt ((a - c)^2 + (b - 0)^2) + Real.sqrt ((a - x)^2 + (b - x)^2) > Real.sqrt ((c - x)^2 + (0 - x)^2) ∧\n Real.sqrt ((c - x)^2 + (0 - x)^2) + Real.sqrt ((a - x)^2 + (b - x)^2) > Real.sqrt ((a - c)^2 + (b - 0)^2)} = answer a b", "v": null, "name": "h_answer"}]} {"informal_problem": "Find necessary and sufficient conditions on positive integers $m$ and $n$ so that \\[\\sum_{i=0}^{mn-1} (-1)^{\\lfloor i/m \\rfloor +\\lfloor i/n\\rfloor}=0.\\]", "informal_answer": "{nm | let ⟨n,m⟩ := nm; multiplicity 2 n ≠ multiplicity 2 m}", "informal_solution": "Show that the sum is 0 if and only if the largest powers of $2$ dividing $m$ and $n$ are different.", "header": "open Set Function Metric", "intros": [], "formal_answer": "@Eq (Set (Prod Nat Nat)) answer\n (@setOf (Prod Nat Nat) fun (nm : Prod Nat Nat) =>\n _example.match_1 (fun (nm_1 : Prod Nat Nat) => Prop) nm fun (n_1 m_1 : Nat) =>\n @Ne Nat (@multiplicity Nat Nat.instMonoid (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))) n_1)\n (@multiplicity Nat Nat.instMonoid (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))) m_1))", "formal_answer_type": "Set (ℕ × ℕ)", "outros": [{"t": "ℕ → ℕ → ℤ", "v": null, "name": "quantity"}, {"t": "quantity = fun n m => ∑ i in Finset.range (m * n), (-1)^(i/m + i/n)", "v": null, "name": "hquantity"}, {"t": "ℕ", "v": null, "name": "n"}, {"t": "ℕ", "v": null, "name": "m"}, {"t": "n > 0 ∧ m > 0", "v": null, "name": "hnm"}, {"t": "quantity n m = 0 ↔ ⟨n, m⟩ ∈ answer", "v": null, "name": "h_answer"}]} {"informal_problem": "Let $N$ be the positive integer with 1998 decimal digits, all of them 1; that is, \\[N=1111\\cdots 11.\\] Find the thousandth digit after the decimal point of $\\sqrt N$.", "informal_answer": "1", "informal_solution": "Show that the thousandth digit is 1.", "header": "open Set Function Metric", "intros": [], "formal_answer": "@Eq Nat answer (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1)))", "formal_answer_type": "ℕ", "outros": [{"t": "ℕ", "v": null, "name": "N"}, {"t": "N = ∑ i in Finset.range 1998, 10^i", "v": null, "name": "hN"}, {"t": "answer = (Nat.floor (10^1000 * Real.sqrt N)) % 10", "v": null, "name": "h_answer"}]} -{"informal_problem": "Find polynomials $f(x)$,$g(x)$, and $h(x)$, if they exist, such that for all $x$, \\[|f(x)|-|g(x)|+h(x) = \\begin{cases} -1 & \\mbox{if $x<-1$} \\\\3x+2 & \\mbox{if $-1 \\leq x \\leq 0$} \\\\-2x+2 & \\mbox{if $x>0$.}\\end{cases}\\]?", "informal_answer": "True", "informal_solution": "Show that the answer is such functions do exist.", "header": null, "intros": [], "formal_answer": "@Eq Prop answer True", "formal_answer_type": "Prop", "outros": [{"t": "answer ↔ ∃ f g h : Polynomial ℝ, ∀ x : ℝ, |f.eval x| - |g.eval x| + h.eval x = if x < -1 then -1 else (if (x ≤ 0) then 3 * x + 2 else -2 * x + 2)", "v": null, "name": "h_answer"}]} +{"informal_problem": "Find polynomials $f(x)$,$g(x)$, and $h(x)$, if they exist, such that for all $x$, \\[|f(x)|-|g(x)|+h(x) = \\begin{cases} -1 & \\mbox{if $x<-1$} \\\\3x+2 & \\mbox{if $-1 \\leq x \\leq 0$} \\\\-2x+2 & \\mbox{if $x>0$.}\\end{cases}\\]?", "informal_answer": "True", "informal_solution": "Show that the answer is such functions do exist.", "header": "open BigOperators Real Nat Topology", "intros": [], "formal_answer": "@Eq Prop answer True", "formal_answer_type": "Prop", "outros": [{"t": "answer ↔ ∃ f g h : Polynomial ℝ, ∀ x : ℝ, |f.eval x| - |g.eval x| + h.eval x = if x < -1 then -1 else (if (x ≤ 0) then 3 * x + 2 else -2 * x + 2)", "v": null, "name": "h_answer"}]} {"informal_problem": "Sum the series \\[\\sum_{m=1}^\\infty \\sum_{n=1}^\\infty \\frac{m^2 n}{3^m(n3^m+m3^n)}.\\]", "informal_answer": "9/32", "informal_solution": "Show that the solution is 9/32.", "header": "open Filter Topology Metric", "intros": [], "formal_answer": "@Eq Real answer\n (@HDiv.hDiv Real Real Real (@instHDiv Real (@DivInvMonoid.toDiv Real Real.instDivInvMonoid))\n (@OfNat.ofNat Real (nat_lit 9)\n (@instOfNatAtLeastTwo Real (nat_lit 9) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 7) (instOfNatNat (nat_lit 7))))))\n (@OfNat.ofNat Real (nat_lit 32)\n (@instOfNatAtLeastTwo Real (nat_lit 32) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 30) (instOfNatNat (nat_lit 30)))))))", "formal_answer_type": "ℝ", "outros": [{"t": "Tendsto (fun i => ∑ m in Finset.range i, ∑' n : ℕ, (((m + 1)^2*(n+1))/(3^(m + 1) * ((n+1)*3^(m + 1) + (m + 1)*3^(n+1))) : ℝ)) atTop (𝓝 answer)", "v": null, "name": "h_answer"}]} {"informal_problem": "Let $A=\\{(x,y):0\\leq x,y<1\\}$. For $(x,y)\\in A$, let \\[S(x,y) = \\sum_{\\frac{1}{2}\\leq \\frac{m}{n}\\leq 2} x^m y^n,\\] where the sum ranges over all pairs $(m,n)$ of positive integers satisfying the indicated inequalities. Evaluate \\[\\lim_{(x,y)\\rightarrow (1,1), (x,y)\\in A} (1-xy^2)(1-x^2y)S(x,y).\\]", "informal_answer": "3", "informal_solution": "Show that the answer is 3.", "header": "open Filter Topology Metric", "intros": [], "formal_answer": "@Eq Real answer\n (@OfNat.ofNat Real (nat_lit 3)\n (@instOfNatAtLeastTwo Real (nat_lit 3) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1))))))", "formal_answer_type": "ℝ", "outros": [{"t": "Set (ℝ × ℝ)", "v": null, "name": "A"}, {"t": "A = {xy | 0 ≤ xy.1 ∧ xy.1 < 1 ∧ 0 ≤ xy.2 ∧ xy.2 < 1}", "v": null, "name": "hA"}, {"t": "ℝ → ℝ → ℝ", "v": null, "name": "S"}, {"t": "S = fun x y => ∑' m : ℕ, ∑' n : ℕ, if (m > 0 ∧ n > 0 ∧ 1/2 ≤ m/n ∧ m/n ≤ 2) then x^m * y^n else 0", "v": null, "name": "hS"}, {"t": "Tendsto (fun xy : (ℝ × ℝ) => (1 - xy.1 * xy.2^2) * (1 - xy.1^2 * xy.2) * (S xy.1 xy.2)) (𝓝[A] ⟨1,1⟩) (𝓝 answer)", "v": null, "name": "h_answer"}]} {"informal_problem": "For an integer $n\\geq 3$, let $\\theta=2\\pi/n$. Evaluate the determinant of the $n\\times n$ matrix $I+A$, where $I$ is the $n\\times n$ identity matrix and $A=(a_{jk})$ has entries $a_{jk}=\\cos(j\\theta+k\\theta)$ for all $j,k$.", "informal_answer": "fun n => 1 - n^2/4", "informal_solution": "Show that the answer is $(1 - n^2)/4$.", "header": "open Filter Topology Metric", "intros": [], "formal_answer": "@Eq (Nat → Real) answer fun (n_1 : Nat) =>\n @HSub.hSub Real Real Real (@instHSub Real Real.instSub)\n (@OfNat.ofNat Real (nat_lit 1) (@One.toOfNat1 Real Real.instOne))\n (@HDiv.hDiv Real Real Real (@instHDiv Real (@DivInvMonoid.toDiv Real Real.instDivInvMonoid))\n (@HPow.hPow Real Nat Real (@instHPow Real Nat (@Monoid.toNatPow Real Real.instMonoid))\n (@Nat.cast Real Real.instNatCast n_1) (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))))\n (@OfNat.ofNat Real (nat_lit 4)\n (@instOfNatAtLeastTwo Real (nat_lit 4) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))))))", "formal_answer_type": "ℕ → ℝ", "outros": [{"t": "ℕ", "v": null, "name": "n"}, {"t": "n ≥ 3", "v": null, "name": "hn"}, {"t": "ℝ", "v": null, "name": "theta"}, {"t": "theta = 2 * Real.pi / n", "v": null, "name": "htheta"}, {"t": "Matrix (Fin n) (Fin n) ℝ", "v": null, "name": "A"}, {"t": "A = fun j k => Real.cos ((j.1 + 1) * theta + (k.1 + 1) * theta)", "v": null, "name": "hA"}, {"t": "(1 + A).det = answer n", "v": null, "name": "h_answer"}]} @@ -199,15 +199,15 @@ {"informal_problem": "Find a nonzero polynomial $P(x,y)$ such that $P(\\lfloor a \\rfloor,\\lfloor 2a \\rfloor)=0$ for all real numbers $a$. (Note: $\\lfloor \\nu \\rfloor$ is the greatest integer less than or equal to $\\nu$.)", "informal_answer": "(y - 2x)(y - 2x - 1)", "informal_solution": "Show that $P(x,y)=(y-2x)(y-2x-1)$ works.", "header": "open Nat Set", "intros": [], "formal_answer": "@Eq (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real Real.instCommSemiring) answer\n (@HMul.hMul (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real Real.instCommSemiring)\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real Real.instCommSemiring)\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real Real.instCommSemiring)\n (@instHMul\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real Real.instCommSemiring)\n (@Distrib.toMul\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real Real.instCommSemiring)\n (@NonUnitalNonAssocSemiring.toDistrib\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real Real.instCommSemiring)\n (@NonUnitalNonAssocCommSemiring.toNonUnitalNonAssocSemiring\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real Real.instCommSemiring)\n (@NonUnitalNonAssocCommRing.toNonUnitalNonAssocCommSemiring\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real Real.instCommSemiring)\n (@NonUnitalCommRing.toNonUnitalNonAssocCommRing\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real\n Real.instCommSemiring)\n (@CommRing.toNonUnitalCommRing\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real\n Real.instCommSemiring)\n (@MvPolynomial.instCommRingMvPolynomial Real\n (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real.commRing))))))))\n (@HSub.hSub\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real Real.instCommSemiring)\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real Real.instCommSemiring)\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real Real.instCommSemiring)\n (@instHSub\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real Real.instCommSemiring)\n (@SubNegMonoid.toSub\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real Real.instCommSemiring)\n (@AddGroup.toSubNegMonoid\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real Real.instCommSemiring)\n (@AddGroupWithOne.toAddGroup\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real Real.instCommSemiring)\n (@Ring.toAddGroupWithOne\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real\n Real.instCommSemiring)\n (@CommRing.toRing\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real\n Real.instCommSemiring)\n (@MvPolynomial.instCommRingMvPolynomial Real\n (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real.commRing)))))))\n (@MvPolynomial.X Real (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real.instCommSemiring\n (@OfNat.ofNat (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) (nat_lit 1)\n (@Fin.instOfNat (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))\n (@Nat.instNeZeroSucc (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1)))) (nat_lit 1))))\n (@HMul.hMul\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real Real.instCommSemiring)\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real Real.instCommSemiring)\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real Real.instCommSemiring)\n (@instHMul\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real Real.instCommSemiring)\n (@Distrib.toMul\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real Real.instCommSemiring)\n (@NonUnitalNonAssocSemiring.toDistrib\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real Real.instCommSemiring)\n (@NonUnitalNonAssocCommSemiring.toNonUnitalNonAssocSemiring\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real\n Real.instCommSemiring)\n (@NonUnitalNonAssocCommRing.toNonUnitalNonAssocCommSemiring\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real\n Real.instCommSemiring)\n (@NonUnitalCommRing.toNonUnitalNonAssocCommRing\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real\n Real.instCommSemiring)\n (@CommRing.toNonUnitalCommRing\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real\n Real.instCommSemiring)\n (@MvPolynomial.instCommRingMvPolynomial Real\n (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real.commRing))))))))\n (@OfNat.ofNat\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real Real.instCommSemiring)\n (nat_lit 2)\n (@instOfNatAtLeastTwo\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real Real.instCommSemiring)\n (nat_lit 2)\n (@AddMonoidWithOne.toNatCast\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real Real.instCommSemiring)\n (@AddGroupWithOne.toAddMonoidWithOne\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real\n Real.instCommSemiring)\n (@Ring.toAddGroupWithOne\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real\n Real.instCommSemiring)\n (@CommRing.toRing\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real\n Real.instCommSemiring)\n (@MvPolynomial.instCommRingMvPolynomial Real\n (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real.commRing)))))\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 0) (instOfNatNat (nat_lit 0))))))\n (@MvPolynomial.X Real (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real.instCommSemiring\n (@OfNat.ofNat (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) (nat_lit 0)\n (@Fin.instOfNat (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))\n (@Nat.instNeZeroSucc (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1)))) (nat_lit 0))))))\n (@HSub.hSub\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real Real.instCommSemiring)\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real Real.instCommSemiring)\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real Real.instCommSemiring)\n (@instHSub\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real Real.instCommSemiring)\n (@SubNegMonoid.toSub\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real Real.instCommSemiring)\n (@AddGroup.toSubNegMonoid\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real Real.instCommSemiring)\n (@AddGroupWithOne.toAddGroup\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real Real.instCommSemiring)\n (@Ring.toAddGroupWithOne\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real\n Real.instCommSemiring)\n (@CommRing.toRing\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real\n Real.instCommSemiring)\n (@MvPolynomial.instCommRingMvPolynomial Real\n (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real.commRing)))))))\n (@HSub.hSub\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real Real.instCommSemiring)\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real Real.instCommSemiring)\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real Real.instCommSemiring)\n (@instHSub\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real Real.instCommSemiring)\n (@SubNegMonoid.toSub\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real Real.instCommSemiring)\n (@AddGroup.toSubNegMonoid\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real Real.instCommSemiring)\n (@AddGroupWithOne.toAddGroup\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real\n Real.instCommSemiring)\n (@Ring.toAddGroupWithOne\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real\n Real.instCommSemiring)\n (@CommRing.toRing\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real\n Real.instCommSemiring)\n (@MvPolynomial.instCommRingMvPolynomial Real\n (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real.commRing)))))))\n (@MvPolynomial.X Real (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real.instCommSemiring\n (@OfNat.ofNat (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) (nat_lit 1)\n (@Fin.instOfNat (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))\n (@Nat.instNeZeroSucc (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1)))) (nat_lit 1))))\n (@HMul.hMul\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real Real.instCommSemiring)\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real Real.instCommSemiring)\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real Real.instCommSemiring)\n (@instHMul\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real Real.instCommSemiring)\n (@Distrib.toMul\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real Real.instCommSemiring)\n (@NonUnitalNonAssocSemiring.toDistrib\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real\n Real.instCommSemiring)\n (@NonUnitalNonAssocCommSemiring.toNonUnitalNonAssocSemiring\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real\n Real.instCommSemiring)\n (@NonUnitalNonAssocCommRing.toNonUnitalNonAssocCommSemiring\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real\n Real.instCommSemiring)\n (@NonUnitalCommRing.toNonUnitalNonAssocCommRing\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real\n Real.instCommSemiring)\n (@CommRing.toNonUnitalCommRing\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real\n Real.instCommSemiring)\n (@MvPolynomial.instCommRingMvPolynomial Real\n (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real.commRing))))))))\n (@OfNat.ofNat\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real Real.instCommSemiring)\n (nat_lit 2)\n (@instOfNatAtLeastTwo\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real Real.instCommSemiring)\n (nat_lit 2)\n (@AddMonoidWithOne.toNatCast\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real\n Real.instCommSemiring)\n (@AddGroupWithOne.toAddMonoidWithOne\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real\n Real.instCommSemiring)\n (@Ring.toAddGroupWithOne\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real\n Real.instCommSemiring)\n (@CommRing.toRing\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real\n Real.instCommSemiring)\n (@MvPolynomial.instCommRingMvPolynomial Real\n (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real.commRing)))))\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 0) (instOfNatNat (nat_lit 0))))))\n (@MvPolynomial.X Real (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real.instCommSemiring\n (@OfNat.ofNat (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) (nat_lit 0)\n (@Fin.instOfNat (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))\n (@Nat.instNeZeroSucc (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1)))) (nat_lit 0))))))\n (@OfNat.ofNat\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real Real.instCommSemiring)\n (nat_lit 1)\n (@One.toOfNat1\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real Real.instCommSemiring)\n (@AddMonoidWithOne.toOne\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real Real.instCommSemiring)\n (@AddGroupWithOne.toAddMonoidWithOne\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real Real.instCommSemiring)\n (@Ring.toAddGroupWithOne\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real\n Real.instCommSemiring)\n (@CommRing.toRing\n (@MvPolynomial (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real\n Real.instCommSemiring)\n (@MvPolynomial.instCommRingMvPolynomial Real\n (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real.commRing)))))))))", "formal_answer_type": "MvPolynomial (Fin 2) ℝ", "outros": [{"t": "answer ≠ 0", "v": null, "name": "h_nonzero"}, {"t": "∀ a : ℝ, MvPolynomial.eval (fun n : Fin 2 => if (n = 0) then (Int.floor a : ℝ) else (Int.floor (2 * a))) answer = 0", "v": null, "name": "h_eval"}]} {"informal_problem": "Find all positive integers $n,k_1,\\dots,k_n$ such that $k_1+\\cdots+k_n=5n-4$ and $\\frac{1}{k_1}+\\cdots+\\frac{1}{k_n}=1$.", "informal_answer": "{(n, k) : ℕ × (ℕ → ℤ) | (n = 1 ∧ k 0 = 1) ∨ (n = 3 ∧ (k '' {0, 1, 2} = {2, 3, 6})) ∨ (n = 4 ∧ (∀ i : Fin 4, k i = 4))}", "informal_solution": "Show that the solutions are $n=1$ and $k_1=1$, $n=3$ and $(k_1,k_2,k_3)$ is a permutation of $(2,3,6)$, and $n=4$ and $(k_1,k_2,k_3,k_4)=(4,4,4,4)$.", "header": "open Nat Set", "intros": [], "formal_answer": "@Eq (Set (Prod Nat (Nat → Int))) answer\n (@setOf (Prod Nat (Nat → Int)) fun (x : Prod Nat (Nat → Int)) =>\n _example.match_1 (fun (x_1 : Prod Nat (Nat → Int)) => Prop) x fun (n : Nat) (k : Nat → Int) =>\n Or\n (And (@Eq Nat n (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1))))\n (@Eq Int (k (@OfNat.ofNat Nat (nat_lit 0) (instOfNatNat (nat_lit 0))))\n (@OfNat.ofNat Int (nat_lit 1) (@instOfNat (nat_lit 1)))))\n (Or\n (And (@Eq Nat n (@OfNat.ofNat Nat (nat_lit 3) (instOfNatNat (nat_lit 3))))\n (@Eq (Set Int)\n (@Set.image Nat Int k\n (@Insert.insert Nat (Set Nat) (@Set.instInsert Nat)\n (@OfNat.ofNat Nat (nat_lit 0) (instOfNatNat (nat_lit 0)))\n (@Insert.insert Nat (Set Nat) (@Set.instInsert Nat)\n (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1)))\n (@Singleton.singleton Nat (Set Nat) (@Set.instSingletonSet Nat)\n (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))))))\n (@Insert.insert Int (Set Int) (@Set.instInsert Int)\n (@OfNat.ofNat Int (nat_lit 2) (@instOfNat (nat_lit 2)))\n (@Insert.insert Int (Set Int) (@Set.instInsert Int)\n (@OfNat.ofNat Int (nat_lit 3) (@instOfNat (nat_lit 3)))\n (@Singleton.singleton Int (Set Int) (@Set.instSingletonSet Int)\n (@OfNat.ofNat Int (nat_lit 6) (@instOfNat (nat_lit 6))))))))\n (And (@Eq Nat n (@OfNat.ofNat Nat (nat_lit 4) (instOfNatNat (nat_lit 4))))\n (∀ (i : Fin (@OfNat.ofNat Nat (nat_lit 4) (instOfNatNat (nat_lit 4)))),\n @Eq Int (k (@Fin.val (@OfNat.ofNat Nat (nat_lit 4) (instOfNatNat (nat_lit 4))) i))\n (@OfNat.ofNat Int (nat_lit 4) (@instOfNat (nat_lit 4)))))))", "formal_answer_type": "Set (ℕ × (ℕ → ℤ))", "outros": [{"t": "{((n : ℕ), (k : ℕ → ℤ)) | (n > 0) ∧ (∀ i ∈ Finset.range n, k i > 0) ∧ (∑ i in Finset.range n, k i = 5 * n - 4) ∧ (∑ i : Finset.range n, (1 : ℝ) / (k i) = 1)} = answer", "v": null, "name": "h_answer"}]} {"informal_problem": "Find all differentiable functions $f:(0,\\infty) \\to (0,\\infty)$ for which there is a positive real number $a$ such that $f'(\\frac{a}{x})=\\frac{x}{f(x)}$ for all $x>0$.", "informal_answer": "the set of functions $f$ such that $f(x) = c x^d$ for some $c > 0$ and $d > 0$, with $d = 1$ implying $c = 1$", "informal_solution": "Show that the functions are precisely $f(x)=cx^d$ for $c,d>0$ arbitrary except that we must take $c=1$ in case $d=1$.", "header": "open Nat Set", "intros": [], "formal_answer": "@Eq (Set (Real → Real)) answer\n (@setOf (Real → Real) fun (f_1 : Real → Real) =>\n @Exists Real fun (c : Real) =>\n And (@GT.gt Real Real.instLT c (@OfNat.ofNat Real (nat_lit 0) (@Zero.toOfNat0 Real Real.instZero)))\n (@Exists Real fun (d : Real) =>\n And (@GT.gt Real Real.instLT d (@OfNat.ofNat Real (nat_lit 0) (@Zero.toOfNat0 Real Real.instZero)))\n (And\n (@Eq Real d (@OfNat.ofNat Real (nat_lit 1) (@One.toOfNat1 Real Real.instOne)) →\n @Eq Real c (@OfNat.ofNat Real (nat_lit 1) (@One.toOfNat1 Real Real.instOne)))\n (@Set.EqOn Real Real f_1\n (fun (x : Real) =>\n @HMul.hMul Real Real Real (@instHMul Real Real.instMul) c\n (@HPow.hPow Real Real Real (@instHPow Real Real Real.instPow) x d))\n (@Set.Ioi Real Real.instPreorder\n (@OfNat.ofNat Real (nat_lit 0) (@Zero.toOfNat0 Real Real.instZero)))))))", "formal_answer_type": "Set (ℝ → ℝ)", "outros": [{"t": "ℝ → ℝ", "v": null, "name": "f"}, {"t": "∀ x > 0, 0 < f x", "v": null, "name": "hf"}, {"t": "DifferentiableOn ℝ f (Ioi 0)", "v": null, "name": "hf'"}, {"t": "(∃ a > 0, ∀ x > 0, deriv f (a / x) = x / f x) ↔ f ∈ answer", "v": null, "name": "h_answer"}]} -{"informal_problem": "Find the volume of the region of points $(x,y,z)$ such that\n\\[\n(x^2 + y^2 + z^2 + 8)^2 \\leq 36(x^2 + y^2).\n\\]", "informal_answer": "6 * Real.pi ^ 2", "informal_solution": "Show that the volume is $6\\pi^2$.", "header": null, "intros": [], "formal_answer": "@Eq Real answer\n (@HMul.hMul Real Real Real (@instHMul Real Real.instMul)\n (@OfNat.ofNat Real (nat_lit 6)\n (@instOfNatAtLeastTwo Real (nat_lit 6) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 4) (instOfNatNat (nat_lit 4))))))\n (@HPow.hPow Real Nat Real (@instHPow Real Nat (@Monoid.toNatPow Real Real.instMonoid)) Real.pi\n (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))))", "formal_answer_type": "ℝ", "outros": [{"t": "(MeasureTheory.volume {a : ℝ × ℝ × ℝ | (a.1 ^ 2 + a.2.1 ^ 2 + a.2.2 ^ 2 + 8) ^ 2 ≤ 36 * (a.1 ^ 2 + a.2.1 ^ 2)}).toReal = answer", "v": null, "name": "h_answer"}]} -{"informal_problem": "Let $S=\\{1,2,\\dots,n\\}$ for some integer $n>1$. Say a permutation $\\pi$ of $S$ has a \\emph{local maximum} at $k \\in S$ if\n\\begin{enumerate}\n\\item[(i)] $\\pi(k)>\\pi(k+1)$ for $k=1$;\n\\item[(ii)] $\\pi(k-1)<\\pi(k)$ and $\\pi(k)>\\pi(k+1)$ for $1 (n + 1) / 3)", "informal_solution": "Show that the average number of local maxima is $\\frac{n+1}{3}$.", "header": null, "intros": [], "formal_answer": "@Eq (Nat → Real) answer fun (n_1 : Nat) =>\n @HDiv.hDiv Real Real Real (@instHDiv Real (@DivInvMonoid.toDiv Real Real.instDivInvMonoid))\n (@HAdd.hAdd Real Real Real (@instHAdd Real Real.instAdd) (@Nat.cast Real Real.instNatCast n_1)\n (@OfNat.ofNat Real (nat_lit 1) (@One.toOfNat1 Real Real.instOne)))\n (@OfNat.ofNat Real (nat_lit 3)\n (@instOfNatAtLeastTwo Real (nat_lit 3) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1))))))", "formal_answer_type": "ℕ → ℝ", "outros": [{"t": "ℕ", "v": null, "name": "n"}, {"t": "Equiv.Perm (Fin n) → (ℕ → ℕ)", "v": null, "name": "pnat"}, {"t": "Equiv.Perm (Fin n) → ℕ", "v": null, "name": "pcount"}, {"t": "n > 1", "v": null, "name": "ngt1"}, {"t": "∀ p : Equiv.Perm (Fin n), ∀ k : Fin n, (pnat p) k = p k", "v": null, "name": "hpnat"}, {"t": "∀ p : Equiv.Perm (Fin n), pcount p = {k : Fin n | (k.1 = 0 ∨ (pnat p) (k - 1) < (pnat p) k) ∧ (k = n - 1 ∨ (pnat p) k > (pnat p) (k + 1))}.encard", "v": null, "name": "hpcount"}, {"t": "(∑ p : Equiv.Perm (Fin n), pcount p) / {p : Equiv.Perm (Fin n) | true}.ncard = answer n", "v": null, "name": "h_answer"}]} -{"informal_problem": "Let $n$ be a positive odd integer and let $\\theta$ be a real number such that $\\theta/\\pi$ is irrational. Set $a_k=\\tan(\\theta+k\\pi/n)$, $k=1,2,\\dots,n$. Prove that $\\frac{a_1+a_2+\\cdots+a_n}{a_1a_2 \\cdots a_n}$ is an integer, and determine its value.", "informal_answer": "(fun n : ℕ => if (n ≡ 1 [MOD 4]) then n else -n)", "informal_solution": "Show that $\\frac{a_1+\\cdots+a_n}{a_1 \\cdots a_n}=\\begin{cases} n & n \\equiv 1 \\pmod{4} \\\\ -n & n \\equiv 3 \\pmod{4}. \\end{cases}$", "header": null, "intros": [], "formal_answer": "@Eq (Nat → Int) answer fun (n_1 : Nat) =>\n @ite Int\n (Nat.ModEq (@OfNat.ofNat Nat (nat_lit 4) (instOfNatNat (nat_lit 4))) n_1\n (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1))))\n (@Nat.instDecidableModEq (@OfNat.ofNat Nat (nat_lit 4) (instOfNatNat (nat_lit 4))) n_1\n (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1))))\n (@Nat.cast Int instNatCastInt n_1) (@Neg.neg Int Int.instNegInt (@Nat.cast Int instNatCastInt n_1))", "formal_answer_type": "ℕ → ℤ", "outros": [{"t": "ℕ", "v": null, "name": "n"}, {"t": "ℝ", "v": null, "name": "theta"}, {"t": "Set.Icc 1 n → ℝ", "v": null, "name": "a"}, {"t": "Odd n", "v": null, "name": "nodd"}, {"t": "Irrational (theta / Real.pi)", "v": null, "name": "thetairr"}, {"t": "∀ k : Set.Icc 1 n, a k = Real.tan (theta + (k * Real.pi) / n)", "v": null, "name": "ha"}, {"t": "(∑ k : Set.Icc 1 n, a k) / (∏ k : Set.Icc 1 n, a k) = answer n", "v": null, "name": "h_answer"}]} -{"informal_problem": "Show that the curve $x^3 + 3xy + y^3 = 1$ contains only one set of three distinct points, $A$, $B$, and $C$, which are vertices of an equilateral triangle, and find its area.", "informal_answer": "3 * Real.sqrt 3 / 2", "informal_solution": "Prove that the triangle has area $\\frac{3 \\sqrt 3}{2}$.", "header": null, "intros": [], "formal_answer": "@Eq Real answer\n (@HDiv.hDiv Real Real Real (@instHDiv Real (@DivInvMonoid.toDiv Real Real.instDivInvMonoid))\n (@HMul.hMul Real Real Real (@instHMul Real Real.instMul)\n (@OfNat.ofNat Real (nat_lit 3)\n (@instOfNatAtLeastTwo Real (nat_lit 3) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1))))))\n (Real.sqrt\n (@OfNat.ofNat Real (nat_lit 3)\n (@instOfNatAtLeastTwo Real (nat_lit 3) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1))))))))\n (@OfNat.ofNat Real (nat_lit 2)\n (@instOfNatAtLeastTwo Real (nat_lit 2) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 0) (instOfNatNat (nat_lit 0)))))))", "formal_answer_type": "ℝ", "outros": [{"t": "Set (ℝ × ℝ)", "v": null, "name": "curve"}, {"t": "curve = {c | c.1 ^ 3 + 3 * c.1 * c.2 + c.2 ^ 3 = 1}", "v": null, "name": "hcurve"}, {"t": "Set (ℝ × ℝ) → Prop", "v": null, "name": "equilateral"}, {"t": "∀ S, equilateral S ↔ S.encard = 3 ∧\n ∃ d : ℝ, ∀ P ∈ S, ∀ Q ∈ S, P ≠ Q →\n Real.sqrt ((P.1 - Q.1)^2 + (P.2 - Q.2)^2) = d", "v": null, "name": "hequilateral"}, {"t": "(∃! S : Set (ℝ × ℝ), S ⊆ curve ∧ equilateral S) ∧ (∃ S : Set (ℝ × ℝ), S ⊆ curve ∧ equilateral S ∧ (MeasureTheory.volume (convexHull ℝ S)).toReal = answer)", "v": null, "name": "h_answer"}]} -{"informal_problem": "Let $S$ be a finite set of points in the plane. A linear partition of $S$ is an unordered pair $\\{A,B\\}$ of subsets of $S$ such that $A \\cup B=S$, $A \\cap B=\\emptyset$, and $A$ and $B$ lie on opposite sides of some straight line disjoint from $S$ ($A$ or $B$ may be empty). Let $L_S$ be the number of linear partitions of $S$. For each positive integer $n$, find the maximum of $L_S$ over all sets $S$ of $n$ points.", "informal_answer": "$\\binom{n}{2} + 1$", "informal_solution": "Show that the maximum is $\\binom{n}{2}+1$.", "header": null, "intros": [], "formal_answer": "@Eq (Nat → Nat) answer fun (n_1 : Nat) =>\n @HAdd.hAdd Nat Nat Nat (@instHAdd Nat instAddNat)\n (Nat.choose n_1 (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))))\n (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1)))", "formal_answer_type": "ℕ → ℕ", "outros": [{"t": "Finset (Fin 2 → ℝ) → Finset (Finset (Fin 2 → ℝ)) → Prop", "v": null, "name": "IsLinearPartition"}, {"t": "∀ S AB, IsLinearPartition S AB ↔\n (AB.card = 2 ∧ ∃ A ∈ AB, ∃ B ∈ AB,\n A ≠ B ∧ (A ∪ B = S) ∧ (A ∩ B = ∅) ∧\n (∃ m b : ℝ,\n (∀ p ∈ A, p 1 > m * p 0 + b) ∧\n (∀ p ∈ B, p 1 < m * p 0 + b)))", "v": null, "name": "IsLinearPartition_def"}, {"t": "Finset (Fin 2 → ℝ) → ℕ", "v": null, "name": "L"}, {"t": "∀ S, L S = {AB | IsLinearPartition S AB}.encard", "v": null, "name": "hL"}, {"t": "ℕ", "v": null, "name": "n"}, {"t": "0 < n", "v": null, "name": "npos"}, {"t": "IsGreatest {L S | (S) (hS : S.card = n)} (answer n)", "v": null, "name": "h_answer"}]} -{"informal_problem": "Let $Z$ denote the set of points in $\\mathbb{R}^n$ whose coordinates are $0$ or $1$. (Thus $Z$ has $2^n$ elements, which are the vertices of a unit hypercube in $\\mathbb{R}^n$.) Given a vector subspace $V$ of $\\mathbb{R}^n$, let $Z(V)$ denote the number of members of $Z$ that lie in $V$. Let $k$ be given, $0 \\leq k \\leq n$. Find the maximum, over all vector subspaces $V \\subseteq \\mathbb{R}^n$ of dimension $k$, of the number of points in $V \\cap Z$.", "informal_answer": "$2^k$", "informal_solution": "Prove that the maximum is $2^k$.", "header": null, "intros": [], "formal_answer": "@Eq (Nat → Nat) answer fun (k_1 : Nat) =>\n @HPow.hPow Nat Nat Nat (@instHPow Nat Nat (@Monoid.toNatPow Nat Nat.instMonoid))\n (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))) k_1", "formal_answer_type": "ℕ → ℕ", "outros": [{"t": "ℕ", "v": null, "name": "n"}, {"t": "ℕ", "v": null, "name": "k"}, {"t": "n > 0", "v": null, "name": "npos"}, {"t": "k ≤ n", "v": null, "name": "hk"}, {"t": "Set (Fin n → ℝ)", "v": null, "name": "Z"}, {"t": "Z = {P : Fin n → ℝ | ∀ j : Fin n, P j = 0 ∨ P j = 1}", "v": null, "name": "hZ"}, {"t": "IsGreatest\n {y | ∃ V : Subspace ℝ (Fin n → ℝ), Module.rank ℝ V = k ∧ (Z ∩ V).ncard = y}\n (answer k)", "v": null, "name": "h_answer"}]} +{"informal_problem": "Find the volume of the region of points $(x,y,z)$ such that\n\\[\n(x^2 + y^2 + z^2 + 8)^2 \\leq 36(x^2 + y^2).\n\\]", "informal_answer": "6 * Real.pi ^ 2", "informal_solution": "Show that the volume is $6\\pi^2$.", "header": "open BigOperators Real Nat Topology", "intros": [], "formal_answer": "@Eq Real answer\n (@HMul.hMul Real Real Real (@instHMul Real Real.instMul)\n (@OfNat.ofNat Real (nat_lit 6)\n (@instOfNatAtLeastTwo Real (nat_lit 6) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 4) (instOfNatNat (nat_lit 4))))))\n (@HPow.hPow Real Nat Real (@instHPow Real Nat (@Monoid.toNatPow Real Real.instMonoid)) Real.pi\n (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))))", "formal_answer_type": "ℝ", "outros": [{"t": "(MeasureTheory.volume {a : ℝ × ℝ × ℝ | (a.1 ^ 2 + a.2.1 ^ 2 + a.2.2 ^ 2 + 8) ^ 2 ≤ 36 * (a.1 ^ 2 + a.2.1 ^ 2)}).toReal = answer", "v": null, "name": "h_answer"}]} +{"informal_problem": "Let $S=\\{1,2,\\dots,n\\}$ for some integer $n>1$. Say a permutation $\\pi$ of $S$ has a \\emph{local maximum} at $k \\in S$ if\n\\begin{enumerate}\n\\item[(i)] $\\pi(k)>\\pi(k+1)$ for $k=1$;\n\\item[(ii)] $\\pi(k-1)<\\pi(k)$ and $\\pi(k)>\\pi(k+1)$ for $1 (n + 1) / 3)", "informal_solution": "Show that the average number of local maxima is $\\frac{n+1}{3}$.", "header": "open BigOperators Real Nat Topology", "intros": [], "formal_answer": "@Eq (Nat → Real) answer fun (n_1 : Nat) =>\n @HDiv.hDiv Real Real Real (@instHDiv Real (@DivInvMonoid.toDiv Real Real.instDivInvMonoid))\n (@HAdd.hAdd Real Real Real (@instHAdd Real Real.instAdd) (@Nat.cast Real Real.instNatCast n_1)\n (@OfNat.ofNat Real (nat_lit 1) (@One.toOfNat1 Real Real.instOne)))\n (@OfNat.ofNat Real (nat_lit 3)\n (@instOfNatAtLeastTwo Real (nat_lit 3) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1))))))", "formal_answer_type": "ℕ → ℝ", "outros": [{"t": "ℕ", "v": null, "name": "n"}, {"t": "Equiv.Perm (Fin n) → (ℕ → ℕ)", "v": null, "name": "pnat"}, {"t": "Equiv.Perm (Fin n) → ℕ", "v": null, "name": "pcount"}, {"t": "n > 1", "v": null, "name": "ngt1"}, {"t": "∀ p : Equiv.Perm (Fin n), ∀ k : Fin n, (pnat p) k = p k", "v": null, "name": "hpnat"}, {"t": "∀ p : Equiv.Perm (Fin n), pcount p = {k : Fin n | (k.1 = 0 ∨ (pnat p) (k - 1) < (pnat p) k) ∧ (k = n - 1 ∨ (pnat p) k > (pnat p) (k + 1))}.encard", "v": null, "name": "hpcount"}, {"t": "(∑ p : Equiv.Perm (Fin n), pcount p) / {p : Equiv.Perm (Fin n) | true}.ncard = answer n", "v": null, "name": "h_answer"}]} +{"informal_problem": "Let $n$ be a positive odd integer and let $\\theta$ be a real number such that $\\theta/\\pi$ is irrational. Set $a_k=\\tan(\\theta+k\\pi/n)$, $k=1,2,\\dots,n$. Prove that $\\frac{a_1+a_2+\\cdots+a_n}{a_1a_2 \\cdots a_n}$ is an integer, and determine its value.", "informal_answer": "(fun n : ℕ => if (n ≡ 1 [MOD 4]) then n else -n)", "informal_solution": "Show that $\\frac{a_1+\\cdots+a_n}{a_1 \\cdots a_n}=\\begin{cases} n & n \\equiv 1 \\pmod{4} \\\\ -n & n \\equiv 3 \\pmod{4}. \\end{cases}$", "header": "open BigOperators Real Nat Topology", "intros": [], "formal_answer": "@Eq (Nat → Int) answer fun (n_1 : Nat) =>\n @ite Int\n (Nat.ModEq (@OfNat.ofNat Nat (nat_lit 4) (instOfNatNat (nat_lit 4))) n_1\n (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1))))\n (@Nat.instDecidableModEq (@OfNat.ofNat Nat (nat_lit 4) (instOfNatNat (nat_lit 4))) n_1\n (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1))))\n (@Nat.cast Int instNatCastInt n_1) (@Neg.neg Int Int.instNegInt (@Nat.cast Int instNatCastInt n_1))", "formal_answer_type": "ℕ → ℤ", "outros": [{"t": "ℕ", "v": null, "name": "n"}, {"t": "ℝ", "v": null, "name": "theta"}, {"t": "Set.Icc 1 n → ℝ", "v": null, "name": "a"}, {"t": "Odd n", "v": null, "name": "nodd"}, {"t": "Irrational (theta / Real.pi)", "v": null, "name": "thetairr"}, {"t": "∀ k : Set.Icc 1 n, a k = Real.tan (theta + (k * Real.pi) / n)", "v": null, "name": "ha"}, {"t": "(∑ k : Set.Icc 1 n, a k) / (∏ k : Set.Icc 1 n, a k) = answer n", "v": null, "name": "h_answer"}]} +{"informal_problem": "Show that the curve $x^3 + 3xy + y^3 = 1$ contains only one set of three distinct points, $A$, $B$, and $C$, which are vertices of an equilateral triangle, and find its area.", "informal_answer": "3 * Real.sqrt 3 / 2", "informal_solution": "Prove that the triangle has area $\\frac{3 \\sqrt 3}{2}$.", "header": "open BigOperators Real Nat Topology", "intros": [], "formal_answer": "@Eq Real answer\n (@HDiv.hDiv Real Real Real (@instHDiv Real (@DivInvMonoid.toDiv Real Real.instDivInvMonoid))\n (@HMul.hMul Real Real Real (@instHMul Real Real.instMul)\n (@OfNat.ofNat Real (nat_lit 3)\n (@instOfNatAtLeastTwo Real (nat_lit 3) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1))))))\n (Real.sqrt\n (@OfNat.ofNat Real (nat_lit 3)\n (@instOfNatAtLeastTwo Real (nat_lit 3) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1))))))))\n (@OfNat.ofNat Real (nat_lit 2)\n (@instOfNatAtLeastTwo Real (nat_lit 2) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 0) (instOfNatNat (nat_lit 0)))))))", "formal_answer_type": "ℝ", "outros": [{"t": "Set (ℝ × ℝ)", "v": null, "name": "curve"}, {"t": "curve = {c | c.1 ^ 3 + 3 * c.1 * c.2 + c.2 ^ 3 = 1}", "v": null, "name": "hcurve"}, {"t": "Set (ℝ × ℝ) → Prop", "v": null, "name": "equilateral"}, {"t": "∀ S, equilateral S ↔ S.encard = 3 ∧\n ∃ d : ℝ, ∀ P ∈ S, ∀ Q ∈ S, P ≠ Q →\n Real.sqrt ((P.1 - Q.1)^2 + (P.2 - Q.2)^2) = d", "v": null, "name": "hequilateral"}, {"t": "(∃! S : Set (ℝ × ℝ), S ⊆ curve ∧ equilateral S) ∧ (∃ S : Set (ℝ × ℝ), S ⊆ curve ∧ equilateral S ∧ (MeasureTheory.volume (convexHull ℝ S)).toReal = answer)", "v": null, "name": "h_answer"}]} +{"informal_problem": "Let $S$ be a finite set of points in the plane. A linear partition of $S$ is an unordered pair $\\{A,B\\}$ of subsets of $S$ such that $A \\cup B=S$, $A \\cap B=\\emptyset$, and $A$ and $B$ lie on opposite sides of some straight line disjoint from $S$ ($A$ or $B$ may be empty). Let $L_S$ be the number of linear partitions of $S$. For each positive integer $n$, find the maximum of $L_S$ over all sets $S$ of $n$ points.", "informal_answer": "$\\binom{n}{2} + 1$", "informal_solution": "Show that the maximum is $\\binom{n}{2}+1$.", "header": "open BigOperators Real Nat Topology", "intros": [], "formal_answer": "@Eq (Nat → Nat) answer fun (n_1 : Nat) =>\n @HAdd.hAdd Nat Nat Nat (@instHAdd Nat instAddNat)\n (Nat.choose n_1 (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))))\n (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1)))", "formal_answer_type": "ℕ → ℕ", "outros": [{"t": "Finset (Fin 2 → ℝ) → Finset (Finset (Fin 2 → ℝ)) → Prop", "v": null, "name": "IsLinearPartition"}, {"t": "∀ S AB, IsLinearPartition S AB ↔\n (AB.card = 2 ∧ ∃ A ∈ AB, ∃ B ∈ AB,\n A ≠ B ∧ (A ∪ B = S) ∧ (A ∩ B = ∅) ∧\n (∃ m b : ℝ,\n (∀ p ∈ A, p 1 > m * p 0 + b) ∧\n (∀ p ∈ B, p 1 < m * p 0 + b)))", "v": null, "name": "IsLinearPartition_def"}, {"t": "Finset (Fin 2 → ℝ) → ℕ", "v": null, "name": "L"}, {"t": "∀ S, L S = {AB | IsLinearPartition S AB}.encard", "v": null, "name": "hL"}, {"t": "ℕ", "v": null, "name": "n"}, {"t": "0 < n", "v": null, "name": "npos"}, {"t": "IsGreatest {L S | (S) (hS : S.card = n)} (answer n)", "v": null, "name": "h_answer"}]} +{"informal_problem": "Let $Z$ denote the set of points in $\\mathbb{R}^n$ whose coordinates are $0$ or $1$. (Thus $Z$ has $2^n$ elements, which are the vertices of a unit hypercube in $\\mathbb{R}^n$.) Given a vector subspace $V$ of $\\mathbb{R}^n$, let $Z(V)$ denote the number of members of $Z$ that lie in $V$. Let $k$ be given, $0 \\leq k \\leq n$. Find the maximum, over all vector subspaces $V \\subseteq \\mathbb{R}^n$ of dimension $k$, of the number of points in $V \\cap Z$.", "informal_answer": "$2^k$", "informal_solution": "Prove that the maximum is $2^k$.", "header": "open BigOperators Real Nat Topology", "intros": [], "formal_answer": "@Eq (Nat → Nat) answer fun (k_1 : Nat) =>\n @HPow.hPow Nat Nat Nat (@instHPow Nat Nat (@Monoid.toNatPow Nat Nat.instMonoid))\n (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))) k_1", "formal_answer_type": "ℕ → ℕ", "outros": [{"t": "ℕ", "v": null, "name": "n"}, {"t": "ℕ", "v": null, "name": "k"}, {"t": "n > 0", "v": null, "name": "npos"}, {"t": "k ≤ n", "v": null, "name": "hk"}, {"t": "Set (Fin n → ℝ)", "v": null, "name": "Z"}, {"t": "Z = {P : Fin n → ℝ | ∀ j : Fin n, P j = 0 ∨ P j = 1}", "v": null, "name": "hZ"}, {"t": "IsGreatest\n {y | ∃ V : Subspace ℝ (Fin n → ℝ), Module.rank ℝ V = k ∧ (Z ∩ V).ncard = y}\n (answer k)", "v": null, "name": "h_answer"}]} {"informal_problem": "For each continuous function $f: [0,1] \\to \\mathbb{R}$, let $I(f) = \\int_0^1 x^2 f(x)\\,dx$ and $J(x) = \\int_0^1 x \\left(f(x)\\right)^2\\,dx$. Find the maximum value of $I(f) - J(f)$ over all such functions $f$.", "informal_answer": "$\\frac{1}{16}$", "informal_solution": "Show that the answer is \\frac{1}{16}.", "header": "open Set", "intros": [], "formal_answer": "@Eq Real answer\n (@HDiv.hDiv Real Real Real (@instHDiv Real (@DivInvMonoid.toDiv Real Real.instDivInvMonoid))\n (@OfNat.ofNat Real (nat_lit 1) (@One.toOfNat1 Real Real.instOne))\n (@OfNat.ofNat Real (nat_lit 16)\n (@instOfNatAtLeastTwo Real (nat_lit 16) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 14) (instOfNatNat (nat_lit 14)))))))", "formal_answer_type": "ℝ", "outros": [{"t": "(ℝ → ℝ) → ℝ", "v": null, "name": "I"}, {"t": "(ℝ → ℝ) → ℝ", "v": null, "name": "J"}, {"t": "I = fun f ↦ ∫ x in (0)..1, x ^ 2 * (f x)", "v": null, "name": "hI"}, {"t": "J = fun f ↦ ∫ x in (0)..1, x * (f x) ^ 2", "v": null, "name": "hJ"}, {"t": "IsGreatest {y | ∃ f : ℝ → ℝ, ContinuousOn f (Icc 0 1) ∧ I f - J f = y} answer", "v": null, "name": "h_answer"}]} {"informal_problem": "Let $k$ be an integer greater than 1. Suppose $a_0 > 0$, and define \\[ a_{n+1} = a_n + \\frac{1}{\\sqrt[k]{a_n}} \\] for $n > 0$. Evaluate \\[\\lim_{n \\to \\infty} \\frac{a_n^{k+1}}{n^k}.\\]", "informal_answer": "fun k => ((k+1)/k)^k", "informal_solution": "Show that the solution is $(\\frac{k+1}{k})^k$.", "header": "open Set Topology Filter", "intros": [], "formal_answer": "@Eq (Nat → Real) answer fun (k_1 : Nat) =>\n @HPow.hPow Real Nat Real (@instHPow Real Nat (@Monoid.toNatPow Real Real.instMonoid))\n (@HDiv.hDiv Real Real Real (@instHDiv Real (@DivInvMonoid.toDiv Real Real.instDivInvMonoid))\n (@HAdd.hAdd Real Real Real (@instHAdd Real Real.instAdd) (@Nat.cast Real Real.instNatCast k_1)\n (@OfNat.ofNat Real (nat_lit 1) (@One.toOfNat1 Real Real.instOne)))\n (@Nat.cast Real Real.instNatCast k_1))\n k_1", "formal_answer_type": "ℕ → ℝ", "outros": [{"t": "ℕ", "v": null, "name": "k"}, {"t": "k > 1", "v": null, "name": "hk"}, {"t": "ℕ → ℝ", "v": null, "name": "a"}, {"t": "a 0 > 0", "v": null, "name": "ha0"}, {"t": "∀ n : ℕ, a (n + 1) = a n + 1/((a n)^((1 : ℝ)/k))", "v": null, "name": "ha"}, {"t": "Tendsto (fun n => (a n)^(k+1)/(n ^ k)) atTop (𝓝 (answer k))", "v": null, "name": "h_answer"}]} -{"informal_problem": "Find all values of $\\alpha$ for which the curves $y = \\alpha*x^2 + \\alpha*x + 1/24$ and $x = \\alpha*y^2 + \\alpha*y + 1/24$ are tangent to each other.", "informal_answer": "{2 / 3, 3 / 2, (13 + √601) / 12, (13 - √601) / 12}", "informal_solution": "Show that the solution is the set \\{2/3, 3/2, (13 + \\sqrt{601})/12, (13 - \\sqrt{601})/12}.", "header": null, "intros": [], "formal_answer": "@Eq (Set Real) answer\n (@Insert.insert Real (Set Real) (@Set.instInsert Real)\n (@HDiv.hDiv Real Real Real (@instHDiv Real (@DivInvMonoid.toDiv Real Real.instDivInvMonoid))\n (@OfNat.ofNat Real (nat_lit 2)\n (@instOfNatAtLeastTwo Real (nat_lit 2) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 0) (instOfNatNat (nat_lit 0))))))\n (@OfNat.ofNat Real (nat_lit 3)\n (@instOfNatAtLeastTwo Real (nat_lit 3) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1)))))))\n (@Insert.insert Real (Set Real) (@Set.instInsert Real)\n (@HDiv.hDiv Real Real Real (@instHDiv Real (@DivInvMonoid.toDiv Real Real.instDivInvMonoid))\n (@OfNat.ofNat Real (nat_lit 3)\n (@instOfNatAtLeastTwo Real (nat_lit 3) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1))))))\n (@OfNat.ofNat Real (nat_lit 2)\n (@instOfNatAtLeastTwo Real (nat_lit 2) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 0) (instOfNatNat (nat_lit 0)))))))\n (@Insert.insert Real (Set Real) (@Set.instInsert Real)\n (@HDiv.hDiv Real Real Real (@instHDiv Real (@DivInvMonoid.toDiv Real Real.instDivInvMonoid))\n (@HAdd.hAdd Real Real Real (@instHAdd Real Real.instAdd)\n (@OfNat.ofNat Real (nat_lit 13)\n (@instOfNatAtLeastTwo Real (nat_lit 13) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 11) (instOfNatNat (nat_lit 11))))))\n (Real.sqrt\n (@OfNat.ofNat Real (nat_lit 601)\n (@instOfNatAtLeastTwo Real (nat_lit 601) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 599) (instOfNatNat (nat_lit 599))))))))\n (@OfNat.ofNat Real (nat_lit 12)\n (@instOfNatAtLeastTwo Real (nat_lit 12) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 10) (instOfNatNat (nat_lit 10)))))))\n (@Singleton.singleton Real (Set Real) (@Set.instSingletonSet Real)\n (@HDiv.hDiv Real Real Real (@instHDiv Real (@DivInvMonoid.toDiv Real Real.instDivInvMonoid))\n (@HSub.hSub Real Real Real (@instHSub Real Real.instSub)\n (@OfNat.ofNat Real (nat_lit 13)\n (@instOfNatAtLeastTwo Real (nat_lit 13) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 11) (instOfNatNat (nat_lit 11))))))\n (Real.sqrt\n (@OfNat.ofNat Real (nat_lit 601)\n (@instOfNatAtLeastTwo Real (nat_lit 601) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 599) (instOfNatNat (nat_lit 599))))))))\n (@OfNat.ofNat Real (nat_lit 12)\n (@instOfNatAtLeastTwo Real (nat_lit 12) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 10) (instOfNatNat (nat_lit 10)))))))))))", "formal_answer_type": "Set ℝ", "outros": [{"t": "ℝ", "v": null, "name": "α"}, {"t": "(ℝ → ℝ) → Prop", "v": null, "name": "P"}, {"t": "∀ f, P f ↔ ∃ x y, f x = y ∧ f y = x ∧ deriv f x * deriv f y = 1", "v": null, "name": "P_def"}, {"t": "α ∈ answer", "v": null, "name": "h_answer"}]} +{"informal_problem": "Find all values of $\\alpha$ for which the curves $y = \\alpha*x^2 + \\alpha*x + 1/24$ and $x = \\alpha*y^2 + \\alpha*y + 1/24$ are tangent to each other.", "informal_answer": "{2 / 3, 3 / 2, (13 + √601) / 12, (13 - √601) / 12}", "informal_solution": "Show that the solution is the set \\{2/3, 3/2, (13 + \\sqrt{601})/12, (13 - \\sqrt{601})/12}.", "header": "open BigOperators Real Nat Topology", "intros": [], "formal_answer": "@Eq (Set Real) answer\n (@Insert.insert Real (Set Real) (@Set.instInsert Real)\n (@HDiv.hDiv Real Real Real (@instHDiv Real (@DivInvMonoid.toDiv Real Real.instDivInvMonoid))\n (@OfNat.ofNat Real (nat_lit 2)\n (@instOfNatAtLeastTwo Real (nat_lit 2) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 0) (instOfNatNat (nat_lit 0))))))\n (@OfNat.ofNat Real (nat_lit 3)\n (@instOfNatAtLeastTwo Real (nat_lit 3) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1)))))))\n (@Insert.insert Real (Set Real) (@Set.instInsert Real)\n (@HDiv.hDiv Real Real Real (@instHDiv Real (@DivInvMonoid.toDiv Real Real.instDivInvMonoid))\n (@OfNat.ofNat Real (nat_lit 3)\n (@instOfNatAtLeastTwo Real (nat_lit 3) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1))))))\n (@OfNat.ofNat Real (nat_lit 2)\n (@instOfNatAtLeastTwo Real (nat_lit 2) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 0) (instOfNatNat (nat_lit 0)))))))\n (@Insert.insert Real (Set Real) (@Set.instInsert Real)\n (@HDiv.hDiv Real Real Real (@instHDiv Real (@DivInvMonoid.toDiv Real Real.instDivInvMonoid))\n (@HAdd.hAdd Real Real Real (@instHAdd Real Real.instAdd)\n (@OfNat.ofNat Real (nat_lit 13)\n (@instOfNatAtLeastTwo Real (nat_lit 13) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 11) (instOfNatNat (nat_lit 11))))))\n (Real.sqrt\n (@OfNat.ofNat Real (nat_lit 601)\n (@instOfNatAtLeastTwo Real (nat_lit 601) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 599) (instOfNatNat (nat_lit 599))))))))\n (@OfNat.ofNat Real (nat_lit 12)\n (@instOfNatAtLeastTwo Real (nat_lit 12) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 10) (instOfNatNat (nat_lit 10)))))))\n (@Singleton.singleton Real (Set Real) (@Set.instSingletonSet Real)\n (@HDiv.hDiv Real Real Real (@instHDiv Real (@DivInvMonoid.toDiv Real Real.instDivInvMonoid))\n (@HSub.hSub Real Real Real (@instHSub Real Real.instSub)\n (@OfNat.ofNat Real (nat_lit 13)\n (@instOfNatAtLeastTwo Real (nat_lit 13) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 11) (instOfNatNat (nat_lit 11))))))\n (Real.sqrt\n (@OfNat.ofNat Real (nat_lit 601)\n (@instOfNatAtLeastTwo Real (nat_lit 601) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 599) (instOfNatNat (nat_lit 599))))))))\n (@OfNat.ofNat Real (nat_lit 12)\n (@instOfNatAtLeastTwo Real (nat_lit 12) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 10) (instOfNatNat (nat_lit 10)))))))))))", "formal_answer_type": "Set ℝ", "outros": [{"t": "ℝ", "v": null, "name": "α"}, {"t": "(ℝ → ℝ) → Prop", "v": null, "name": "P"}, {"t": "∀ f, P f ↔ ∃ x y, f x = y ∧ f y = x ∧ deriv f x * deriv f y = 1", "v": null, "name": "P_def"}, {"t": "α ∈ answer", "v": null, "name": "h_answer"}]} {"informal_problem": "Find the least possible area of a convex set in the plane that intersects both branches of the hyperbola $xy=1$ and both branches of the hyperbola $xy=-1$. (A set $S$ in the plane is called \\emph{convex} if for any two points in $S$ the line segment connecting them is contained in $S$.)", "informal_answer": "4", "informal_solution": "Show that the minimum is $4$.", "header": "open MeasureTheory", "intros": [], "formal_answer": "@Eq ENNReal answer\n (@OfNat.ofNat ENNReal (nat_lit 4)\n (@instOfNatAtLeastTwo ENNReal (nat_lit 4)\n (@AddMonoidWithOne.toNatCast ENNReal\n (@AddCommMonoidWithOne.toAddMonoidWithOne ENNReal instENNRealAddCommMonoidWithOne))\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))))))", "formal_answer_type": "ENNReal", "outros": [{"t": "Set (Fin 2 → ℝ)", "v": null, "name": "S"}, {"t": "Convex ℝ S", "v": null, "name": "h_convex"}, {"t": "∃ p ∈ S, p 0 > 0 ∧ p 1 > 0 ∧ p 0 * p 1 = 1", "v": null, "name": "h_hyperbola1"}, {"t": "∃ p ∈ S, p 0 < 0 ∧ p 1 < 0 ∧ p 0 * p 1 = 1", "v": null, "name": "h_hyperbola2"}, {"t": "∃ p ∈ S, p 0 < 0 ∧ p 1 > 0 ∧ p 0 * p 1 = -1", "v": null, "name": "h_hyperbola3"}, {"t": "∃ p ∈ S, p 0 > 0 ∧ p 1 < 0 ∧ p 0 * p 1 = -1", "v": null, "name": "h_hyperbola4"}, {"t": "volume S = answer", "v": null, "name": "h_area"}]} {"informal_problem": "Let $k$ be a positive integer. Suppose that the integers $1, 2, 3, \\dots, 3k+1$ are written down in random order. What is the probability that at no time during this process, the sum of the integers that have been written up to that time is a positive integer divisible by $3$? Your answer should be in closed form, but may include factorials.", "informal_answer": "fun k ↦ (k)! * (k + 1)! / ((3 * k + 1) * (2 * k)!)", "informal_solution": "Prove that the desired probability is $\\frac{k!(k+1)!}{(3k+1)(2k)!}$.", "header": "open Set Nat", "intros": [], "formal_answer": "@Eq (Nat → Rat) answer fun (k_1 : Nat) =>\n @HDiv.hDiv Rat Rat Rat (@instHDiv Rat Rat.instDiv)\n (@HMul.hMul Rat Rat Rat (@instHMul Rat Rat.instMul) (@Nat.cast Rat Rat.instNatCast (Nat.factorial k_1))\n (@Nat.cast Rat Rat.instNatCast\n (Nat.factorial\n (@HAdd.hAdd Nat Nat Nat (@instHAdd Nat instAddNat) k_1\n (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1)))))))\n (@HMul.hMul Rat Rat Rat (@instHMul Rat Rat.instMul)\n (@HAdd.hAdd Rat Rat Rat (@instHAdd Rat Rat.instAdd)\n (@HMul.hMul Rat Rat Rat (@instHMul Rat Rat.instMul) (@OfNat.ofNat Rat (nat_lit 3) (@Rat.instOfNat (nat_lit 3)))\n (@Nat.cast Rat Rat.instNatCast k_1))\n (@OfNat.ofNat Rat (nat_lit 1) (@Rat.instOfNat (nat_lit 1))))\n (@Nat.cast Rat Rat.instNatCast\n (Nat.factorial\n (@HMul.hMul Nat Nat Nat (@instHMul Nat instMulNat) (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))\n k_1))))", "formal_answer_type": "ℕ → ℚ", "outros": [{"t": "ℕ", "v": null, "name": "k"}, {"t": "k > 0", "v": null, "name": "kpos"}, {"t": "Set (Fin (3 * k + 1) → ℤ)", "v": null, "name": "perms"}, {"t": "Set (Fin (3 * k + 1) → ℤ)", "v": null, "name": "goodperms"}, {"t": "goodperms = {f ∈ perms | ¬∃ j : Fin (3 * k + 1), 3 ∣ ∑ i : Fin (3 * k + 1), ite (i ≤ j) (f i) 0}", "v": null, "name": "hgoodperms"}, {"t": "perms = {f : Fin (3 * k + 1) → ℤ | ∀ y ∈ Icc 1 (3 * k + 1), ∃! x : Fin (3 * k + 1), f x = y}", "v": null, "name": "hperms"}, {"t": "goodperms.ncard = perms.ncard * (answer k)", "v": null, "name": "h_answer"}]} {"informal_problem": "A \\emph{repunit} is a positive integer whose digits in base 10 are all ones. Find all polynomials $f$ with real coefficients such that if $n$ is a repunit, then so is $f(n)$.", "informal_answer": "the set of polynomials of the form $f(n) = \\frac{1}{9} \\left(10^c (9n + 1)^d - 1\\right)$ where $d \\in \\mathbb{N}$ and $c \\geq 1 - d$", "informal_solution": "Show that the desired polynomials $f$ are those of the form\n\\[\nf(n) = \\frac{1}{9}(10^c (9n+1)^d - 1)\n\\]\nfor integers $d \\geq 0$ and $c \\geq 1-d$.", "header": "open Set Nat", "intros": [], "formal_answer": "@Eq (Set (@Polynomial Real Real.semiring)) answer\n (@setOf (@Polynomial Real Real.semiring) fun (f : @Polynomial Real Real.semiring) =>\n @Exists Nat fun (d : Nat) =>\n @Exists Int fun (c : Int) =>\n And\n (@GE.ge Int Int.instLEInt c\n (@HSub.hSub Int Int Int (@instHSub Int Int.instSub) (@OfNat.ofNat Int (nat_lit 1) (@instOfNat (nat_lit 1)))\n (@Nat.cast Int instNatCastInt d)))\n (∀ (n : Real),\n @Eq Real (@Polynomial.eval Real Real.semiring n f)\n (@HMul.hMul Real Real Real (@instHMul Real Real.instMul)\n (@HDiv.hDiv Real Real Real (@instHDiv Real (@DivInvMonoid.toDiv Real Real.instDivInvMonoid))\n (@OfNat.ofNat Real (nat_lit 1) (@One.toOfNat1 Real Real.instOne))\n (@OfNat.ofNat Real (nat_lit 9)\n (@instOfNatAtLeastTwo Real (nat_lit 9) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 7) (instOfNatNat (nat_lit 7)))))))\n (@HSub.hSub Real Real Real (@instHSub Real Real.instSub)\n (@HMul.hMul Real Real Real (@instHMul Real Real.instMul)\n (@HPow.hPow Real Int Real (@instHPow Real Int (@DivInvMonoid.toZPow Real Real.instDivInvMonoid))\n (@OfNat.ofNat Real (nat_lit 10)\n (@instOfNatAtLeastTwo Real (nat_lit 10) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 8) (instOfNatNat (nat_lit 8))))))\n c)\n (@HPow.hPow Real Nat Real (@instHPow Real Nat (@Monoid.toNatPow Real Real.instMonoid))\n (@HAdd.hAdd Real Real Real (@instHAdd Real Real.instAdd)\n (@HMul.hMul Real Real Real (@instHMul Real Real.instMul)\n (@OfNat.ofNat Real (nat_lit 9)\n (@instOfNatAtLeastTwo Real (nat_lit 9) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 7) (instOfNatNat (nat_lit 7))))))\n n)\n (@OfNat.ofNat Real (nat_lit 1) (@One.toOfNat1 Real Real.instOne)))\n d))\n (@OfNat.ofNat Real (nat_lit 1) (@One.toOfNat1 Real Real.instOne))))))", "formal_answer_type": "Set (Polynomial ℝ)", "outros": [{"t": "Set (Polynomial ℝ)", "v": null, "name": "S"}, {"t": "ℝ → Prop", "v": null, "name": "repunit"}, {"t": "∀ x, repunit x ↔ x > 0 ∧ x = floor x ∧ ∀ d ∈ (digits 10 (floor x)), d = 1", "v": null, "name": "hrepunit"}, {"t": "∀ f, f ∈ S ↔ (∀ n : ℝ, repunit n → repunit (f.eval n))", "v": null, "name": "hS"}, {"t": "S = answer", "v": null, "name": "h_answer"}]} @@ -226,14 +226,14 @@ {"informal_problem": "A game involves jumping to the right on the real number line. If $a$ and $b$ are real numbers and $b > a$, the cost of jumping from $a$ to $b$ is $b^3-ab^2$. For what real numbers $c$ can one travel from $0$ to $1$ in a finite number of jumps with total cost exactly $c$?", "informal_answer": "the interval (1/3, 1]", "informal_solution": "Prove that the possible costs are $1/3 < c \\leq 1.$", "header": "open Topology MvPolynomial Filter Set", "intros": [], "formal_answer": "@Eq (Set Real) answer\n (@Set.Ioc Real Real.instPreorder\n (@HDiv.hDiv Real Real Real (@instHDiv Real (@DivInvMonoid.toDiv Real Real.instDivInvMonoid))\n (@OfNat.ofNat Real (nat_lit 1) (@One.toOfNat1 Real Real.instOne))\n (@OfNat.ofNat Real (nat_lit 3)\n (@instOfNatAtLeastTwo Real (nat_lit 3) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1)))))))\n (@OfNat.ofNat Real (nat_lit 1) (@One.toOfNat1 Real Real.instOne)))", "formal_answer_type": "Set ℝ", "outros": [{"t": "{c : ℝ | ∃ s : ℕ → ℝ, s 0 = 0 ∧ StrictMono s ∧ (∃ n : ℕ, s n = 1 ∧ ((∑ i in Finset.range n, ((s (i + 1)) ^ 3 - (s i) * (s (i + 1)) ^ 2)) = c))} = answer", "v": null, "name": "h_answer"}]} {"informal_problem": "Call a subset $S$ of $\\{1, 2, \\dots, n\\}$ \\emph{mediocre} if it has the following property: Whenever $a$ and $b$ are elements of $S$ whose average is an integer, that average is also an element of $S$. Let $A(n)$ be the number of mediocre subsets of $\\{1,2,\\dots,n\\}$. [For instance, every subset of $\\{1,2,3\\}$ except $\\{1,3\\}$ is mediocre, so $A(3) = 7$.] Find all positive integers $n$ such that $A(n+2) - 2A(n+1) + A(n) = 1$.", "informal_answer": "{n : ℤ | ∃ k ≥ 1, n = 2 ^ k - 1}", "informal_solution": "Show that the answer is $n = 2^k - 1$ for some integer $k$.", "header": "open Topology MvPolynomial Filter Set", "intros": [], "formal_answer": "@Eq (Set Int) answer\n (@setOf Int fun (n : Int) =>\n @Exists Nat fun (k : Nat) =>\n And (@GE.ge Nat instLENat k (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1))))\n (@Eq Int n\n (@HSub.hSub Int Int Int (@instHSub Int Int.instSub)\n (@HPow.hPow Int Nat Int (@instHPow Int Nat (@Monoid.toNatPow Int Int.instMonoid))\n (@OfNat.ofNat Int (nat_lit 2) (@instOfNat (nat_lit 2))) k)\n (@OfNat.ofNat Int (nat_lit 1) (@instOfNat (nat_lit 1))))))", "formal_answer_type": "Set ℤ", "outros": [{"t": "ℤ → Set ℤ → Prop", "v": null, "name": "mediocre"}, {"t": "∀ n S, mediocre n S ↔ (S ⊆ Icc 1 n) ∧ ∀ a ∈ S, ∀ b ∈ S, 2 ∣ a + b → (a + b) / 2 ∈ S", "v": null, "name": "hmediocre"}, {"t": "ℤ → ℤ", "v": null, "name": "A"}, {"t": "A = fun n ↦ ({S : Set ℤ | mediocre n S}.ncard : ℤ)", "v": null, "name": "hA"}, {"t": "{n : ℤ | n > 0 ∧ A (n + 2) - 2 * A (n + 1) + A n = 1} = answer", "v": null, "name": "h_answer"}]} {"informal_problem": "Say that a polynomial with real coefficients in two variables, $x,y$, is \\emph{balanced} if the average value of the polynomial on each circle centered at the origin is $0$. The balanced polynomials of degree at most $2009$ form a vector space $V$ over $\\mathbb{R}$. Find the dimension of $V$.", "informal_answer": "2020050", "informal_solution": "Prove that the dimension of $V$ is $2020050$.", "header": "open intervalIntegral MvPolynomial Real", "intros": [], "formal_answer": "@Eq Nat answer (@OfNat.ofNat Nat (nat_lit 2020050) (instOfNatNat (nat_lit 2020050)))", "formal_answer_type": "ℕ", "outros": [{"t": "MvPolynomial (Fin 2) ℝ → Prop", "v": null, "name": "IsBalanced"}, {"t": "∀ P, IsBalanced P ↔ ∀ r > 0,\n (∫ t in (0 : ℝ)..(2 * π), eval ![r * cos t, r * sin t] P) / (2 * π * r) = 0", "v": null, "name": "IsBalanced_def"}, {"t": "Submodule ℝ (MvPolynomial (Fin 2) ℝ)", "v": null, "name": "V"}, {"t": "∀ P, P ∈ V ↔ IsBalanced P ∧ P.totalDegree ≤ 2009", "v": null, "name": "V_def"}, {"t": "Module.rank ℝ V = answer", "v": null, "name": "h_answer"}]} -{"informal_problem": "Given a positive integer $n$, what is the largest $k$ such that the numbers $1,2,\\dots,n$ can be put into $k$ boxes so that the sum of the numbers in each box is the same? [When $n=8$, the example $\\{1,2,3,6\\},\\{4,8\\},\\{5,7\\}$ shows that the largest $k$ is \\emph{at least} $3$.]", "informal_answer": "the ceiling of n/2", "informal_solution": "Show that the largest such $k$ is $\\lceil \\frac{n}{2} \\rceil$.", "header": null, "intros": [], "formal_answer": "@Eq (Nat → Nat) answer fun (n_1 : Nat) =>\n @Nat.ceil Real Real.orderedSemiring (@FloorRing.toFloorSemiring Real Real.instLinearOrderedRing Real.instFloorRing)\n (@HDiv.hDiv Real Real Real (@instHDiv Real (@DivInvMonoid.toDiv Real Real.instDivInvMonoid))\n (@Nat.cast Real Real.instNatCast n_1)\n (@OfNat.ofNat Real (nat_lit 2)\n (@instOfNatAtLeastTwo Real (nat_lit 2) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 0) (instOfNatNat (nat_lit 0)))))))", "formal_answer_type": "ℕ → ℕ", "outros": [{"t": "ℕ", "v": null, "name": "n"}, {"t": "ℕ → Prop", "v": null, "name": "kboxes"}, {"t": "n > 0", "v": null, "name": "npos"}, {"t": "∀ k : ℕ, kboxes k =\n (∃ boxes : Finset.Icc 1 n → Fin k, ∀ i j : Fin k,\n ∑ x in Finset.univ.filter (boxes · = i), (x : ℕ) =\n ∑ x in Finset.univ.filter (boxes · = j), (x : ℕ))", "v": null, "name": "hkboxes"}, {"t": "IsGreatest kboxes (answer n)", "v": null, "name": "h_answer"}]} -{"informal_problem": "Find all differentiable functions $f:\\mathbb{R} \\to \\mathbb{R}$ such that\n\\[\nf'(x) = \\frac{f(x+n)-f(x)}{n}\n\\]\nfor all real numbers $x$ and all positive integers $n$.", "informal_answer": "{f : ℝ → ℝ | ∃ c d : ℝ, ∀ x : ℝ, f x = c*x + d}", "informal_solution": "The solution consists of all functions of the form $f(x) = cx+d$ for some real numbers $c,d$.", "header": null, "intros": [], "formal_answer": "@Eq (Set (Real → Real)) answer\n (@setOf (Real → Real) fun (f : Real → Real) =>\n @Exists Real fun (c : Real) =>\n @Exists Real fun (d : Real) =>\n ∀ (x : Real),\n @Eq Real (f x)\n (@HAdd.hAdd Real Real Real (@instHAdd Real Real.instAdd)\n (@HMul.hMul Real Real Real (@instHMul Real Real.instMul) c x) d))", "formal_answer_type": "Set (ℝ → ℝ)", "outros": [{"t": "{f : ℝ → ℝ | Differentiable ℝ f ∧\n∀ x : ℝ, ∀ n : ℤ, n > 0 → deriv f x = (f (x + n) - f x)/n} = answer", "v": null, "name": "h_answer"}]} +{"informal_problem": "Given a positive integer $n$, what is the largest $k$ such that the numbers $1,2,\\dots,n$ can be put into $k$ boxes so that the sum of the numbers in each box is the same? [When $n=8$, the example $\\{1,2,3,6\\},\\{4,8\\},\\{5,7\\}$ shows that the largest $k$ is \\emph{at least} $3$.]", "informal_answer": "the ceiling of n/2", "informal_solution": "Show that the largest such $k$ is $\\lceil \\frac{n}{2} \\rceil$.", "header": "open BigOperators Real Nat Topology", "intros": [], "formal_answer": "@Eq (Nat → Nat) answer fun (n_1 : Nat) =>\n @Nat.ceil Real Real.orderedSemiring (@FloorRing.toFloorSemiring Real Real.instLinearOrderedRing Real.instFloorRing)\n (@HDiv.hDiv Real Real Real (@instHDiv Real (@DivInvMonoid.toDiv Real Real.instDivInvMonoid))\n (@Nat.cast Real Real.instNatCast n_1)\n (@OfNat.ofNat Real (nat_lit 2)\n (@instOfNatAtLeastTwo Real (nat_lit 2) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 0) (instOfNatNat (nat_lit 0)))))))", "formal_answer_type": "ℕ → ℕ", "outros": [{"t": "ℕ", "v": null, "name": "n"}, {"t": "ℕ → Prop", "v": null, "name": "kboxes"}, {"t": "n > 0", "v": null, "name": "npos"}, {"t": "∀ k : ℕ, kboxes k =\n (∃ boxes : Finset.Icc 1 n → Fin k, ∀ i j : Fin k,\n ∑ x in Finset.univ.filter (boxes · = i), (x : ℕ) =\n ∑ x in Finset.univ.filter (boxes · = j), (x : ℕ))", "v": null, "name": "hkboxes"}, {"t": "IsGreatest kboxes (answer n)", "v": null, "name": "h_answer"}]} +{"informal_problem": "Find all differentiable functions $f:\\mathbb{R} \\to \\mathbb{R}$ such that\n\\[\nf'(x) = \\frac{f(x+n)-f(x)}{n}\n\\]\nfor all real numbers $x$ and all positive integers $n$.", "informal_answer": "{f : ℝ → ℝ | ∃ c d : ℝ, ∀ x : ℝ, f x = c*x + d}", "informal_solution": "The solution consists of all functions of the form $f(x) = cx+d$ for some real numbers $c,d$.", "header": "open BigOperators Real Nat Topology", "intros": [], "formal_answer": "@Eq (Set (Real → Real)) answer\n (@setOf (Real → Real) fun (f : Real → Real) =>\n @Exists Real fun (c : Real) =>\n @Exists Real fun (d : Real) =>\n ∀ (x : Real),\n @Eq Real (f x)\n (@HAdd.hAdd Real Real Real (@instHAdd Real Real.instAdd)\n (@HMul.hMul Real Real Real (@instHMul Real Real.instMul) c x) d))", "formal_answer_type": "Set (ℝ → ℝ)", "outros": [{"t": "{f : ℝ → ℝ | Differentiable ℝ f ∧\n∀ x : ℝ, ∀ n : ℤ, n > 0 → deriv f x = (f (x + n) - f x)/n} = answer", "v": null, "name": "h_answer"}]} {"informal_problem": "Is there an infinite sequence of real numbers $a_1, a_2, a_3, \\dots$ such that \\[ a_1^m + a_2^m + a_3^m + \\cdots = m \\] for every positive integer $m$?", "informal_answer": "False", "informal_solution": "Show that the solution is no such infinite sequence exists.", "header": "open Filter Topology Set", "intros": [], "formal_answer": "@Eq Prop answer False", "formal_answer_type": "Prop", "outros": [{"t": "answer = (∃ a : ℕ → ℝ, ∀ m : ℕ, m > 0 → ∑' i : ℕ, (a i)^m = m)", "v": null, "name": "h_answer"}]} {"informal_problem": "Given that $A$, $B$, and $C$ are noncollinear points in the plane with integer coordinates such that the distances $AB$, $AC$, and $BC$ are integers, what is the smallest possible value of $AB$?", "informal_answer": "3", "informal_solution": "Show that the smallest distance is $3$.", "header": "open Filter Topology Set", "intros": [], "formal_answer": "@Eq Nat answer (@OfNat.ofNat Nat (nat_lit 3) (instOfNatNat (nat_lit 3)))", "formal_answer_type": "ℕ", "outros": [{"t": "EuclideanSpace ℝ (Fin 2)", "v": null, "name": "A"}, {"t": "EuclideanSpace ℝ (Fin 2)", "v": null, "name": "B"}, {"t": "EuclideanSpace ℝ (Fin 2)", "v": null, "name": "C"}, {"t": "∀ i : Fin 2, A i = round (A i) ∧ B i = round (B i) ∧ C i = round (C i)", "v": null, "name": "hABCintcoords"}, {"t": "dist A B = round (dist A B) ∧ dist A C = round (dist A C) ∧ dist B C = round (dist B C)", "v": null, "name": "hABCintdists"}, {"t": "¬Collinear ℝ {A, B, C}", "v": null, "name": "hABCall"}, {"t": "answer = dist A B", "v": null, "name": "h_answer"}]} {"informal_problem": "There are $2010$ boxes labeled $B_1, B_2, \\dots, B_{2010}$, and $2010n$ balls have been distributed among them, for some positive integer $n$. You may redistribute the balls by a sequence of moves, each of which consists of choosing an $i$ and moving \\emph{exactly} $i$ balls from box $B_i$ into any one other box. For which values of $n$ is it possible to reach the distribution with exactly $n$ balls in each box, regardless of the initial distribution of balls?", "informal_answer": "{1005}", "informal_solution": "Prove that it is possible if and only if $n \\geq 1005$.", "header": "open Filter Topology Set", "intros": [], "formal_answer": "@Eq (Set Nat) answer\n (@Singleton.singleton Nat (Set Nat) (@Set.instSingletonSet Nat)\n (@OfNat.ofNat Nat (nat_lit 1005) (instOfNatNat (nat_lit 1005))))", "formal_answer_type": "Set ℕ", "outros": [{"t": "ℕ", "v": null, "name": "n"}, {"t": "n > 0", "v": null, "name": "hn"}, {"t": "(ℕ → Fin 2010 → ℕ) → ℕ → Prop", "v": null, "name": "trans"}, {"t": "∀ P T, trans P T ↔ ∀ t : ℕ, t < T → ∃ i j,\n i ≠ j ∧\n P t i ≥ i.1 + 1 ∧ P (t + 1) i = P t i - (i.1 + 1) ∧ P (t + 1) j = P t j + (i.1 + 1) ∧\n ∀ k : Fin 2010, k ≠ i → k ≠ j → P (t + 1) k = P t k", "v": null, "name": "htrans"}, {"t": "(∀ B, ∑ i, B i = 2010 * n → ∃ᵉ (P) (T), P 0 = B ∧ trans P T ∧ ∀ i, P T i = n) ↔ n ∈ answer", "v": null, "name": "h_answer"}]} {"informal_problem": "Find all pairs of polynomials $p(x)$ and $q(x)$ with real coefficients for which $p(x)q(x+1)-p(x+1)q(x)=1$.", "informal_answer": "{(p, q) : Polynomial ℝ × Polynomial ℝ | p.degree ≤ 1 ∧ q.degree ≤ 1 ∧ p.coeff 0 * q.coeff 1 - p.coeff 1 * q.coeff 0 = 1}", "informal_solution": "Show that the pairs $(p,q)$ satisfying the given equation are those of the form $p(x)=ax+b,q(x)=cx+d$ for $a,b,c,d \\in \\mathbb{R}$ such that $bc-ad=1$.", "header": "open Filter Topology Set", "intros": [], "formal_answer": "@Eq (Set (Prod (@Polynomial Real Real.semiring) (@Polynomial Real Real.semiring))) answer\n (@setOf (Prod (@Polynomial Real Real.semiring) (@Polynomial Real Real.semiring))\n fun (x : Prod (@Polynomial Real Real.semiring) (@Polynomial Real Real.semiring)) =>\n _example.match_1 (fun (x_1 : Prod (@Polynomial Real Real.semiring) (@Polynomial Real Real.semiring)) => Prop) x\n fun (p_1 q_1 : @Polynomial Real Real.semiring) =>\n And\n (@LE.le (WithBot Nat) (@Preorder.toLE (WithBot Nat) (@WithBot.preorder Nat Nat.instPreorder))\n (@Polynomial.degree Real Real.semiring p_1)\n (@OfNat.ofNat (WithBot Nat) (nat_lit 1)\n (@One.toOfNat1 (WithBot Nat) (@WithBot.one Nat (@AddMonoidWithOne.toOne Nat Nat.instAddMonoidWithOne)))))\n (And\n (@LE.le (WithBot Nat) (@Preorder.toLE (WithBot Nat) (@WithBot.preorder Nat Nat.instPreorder))\n (@Polynomial.degree Real Real.semiring q_1)\n (@OfNat.ofNat (WithBot Nat) (nat_lit 1)\n (@One.toOfNat1 (WithBot Nat) (@WithBot.one Nat (@AddMonoidWithOne.toOne Nat Nat.instAddMonoidWithOne)))))\n (@Eq Real\n (@HSub.hSub Real Real Real (@instHSub Real Real.instSub)\n (@HMul.hMul Real Real Real (@instHMul Real Real.instMul)\n (@Polynomial.coeff Real Real.semiring p_1 (@OfNat.ofNat Nat (nat_lit 0) (instOfNatNat (nat_lit 0))))\n (@Polynomial.coeff Real Real.semiring q_1 (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1)))))\n (@HMul.hMul Real Real Real (@instHMul Real Real.instMul)\n (@Polynomial.coeff Real Real.semiring p_1 (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1))))\n (@Polynomial.coeff Real Real.semiring q_1 (@OfNat.ofNat Nat (nat_lit 0) (instOfNatNat (nat_lit 0))))))\n (@OfNat.ofNat Real (nat_lit 1) (@One.toOfNat1 Real Real.instOne)))))", "formal_answer_type": "Set (Polynomial ℝ × Polynomial ℝ)", "outros": [{"t": "Polynomial ℝ", "v": null, "name": "p"}, {"t": "Polynomial ℝ", "v": null, "name": "q"}, {"t": "(∀ x : ℝ, p.eval x * q.eval (x + 1) - p.eval (x + 1) * q.eval x = 1) ↔ (p, q) ∈ answer", "v": null, "name": "h_answer"}]} {"informal_problem": "Is there a strictly increasing function $f: \\mathbb{R} \\to \\mathbb{R}$ such that $f'(x) = f(f(x))$ for all $x$?", "informal_answer": "False", "informal_solution": "Show that the solution is no such function exists.", "header": "open Filter Topology Set", "intros": [], "formal_answer": "@Eq Prop answer False", "formal_answer_type": "Prop", "outros": [{"t": "(∃ f : ℝ → ℝ, StrictMono f ∧ Differentiable ℝ f ∧ (∀ x : ℝ, deriv f x = f (f x))) ↔ answer", "v": null, "name": "h_answer"}]} -{"informal_problem": "Define a \\emph{growing spiral} in the plane to be a sequence of points with integer coordinates $P_0=(0,0),P_1,\\dots,P_n$ such that $n \\geq 2$ and:\n\\begin{itemize}\n\\item the directed line segments $P_0P_1,P_1P_2,\\dots,P_{n-1}P_n$ are in the successive coordinate directions east (for $P_0P_1$), north, west, south, east, etc.;\n\\item the lengths of these line segments are positive and strictly increasing.\n\\end{itemize}\nHow many of the points $(x,y)$ with integer coordinates $0 \\leq x \\leq 2011,0 \\leq y \\leq 2011$ \\emph{cannot} be the last point, $P_n$ of any growing spiral?", "informal_answer": "10053", "informal_solution": "Show that there are $10053$ excluded points.", "header": null, "intros": [], "formal_answer": "@Eq Nat answer (@OfNat.ofNat Nat (nat_lit 10053) (instOfNatNat (nat_lit 10053)))", "formal_answer_type": "ℕ", "outros": [{"t": "List (Fin 2 → ℤ) → Prop", "v": null, "name": "IsSpiral"}, {"t": "∀ P, IsSpiral P ↔ P.length ≥ 3 ∧ P[0]! = 0 ∧\n (∃ l : Fin (P.length - 1) → ℕ, l > 0 ∧ StrictMono l ∧ (∀ i : Fin (P.length - 1),\n (i.1 % 4 = 0 → (P[i] 0 + l i = P[i.1 + 1]! 0 ∧ P[i] 1 = P[i.1 + 1]! 1)) ∧\n (i.1 % 4 = 1 → (P[i] 0 = P[i.1 + 1]! 0 ∧ P[i] 1 + l i = P[i.1 + 1]! 1)) ∧\n (i.1 % 4 = 2 → (P[i] 0 - l i = P[i.1 + 1]! 0 ∧ P[i] 1 = P[i.1 + 1]! 1)) ∧\n (i.1 % 4 = 3 → (P[i] 0 = P[i.1 + 1]! 0 ∧ P[i] 1 - l i = P[i.1 + 1]! 1))))", "v": null, "name": "IsSpiral_def"}, {"t": "{p | 0 ≤ p 0 ∧ p 0 ≤ 2011 ∧ 0 ≤ p 1 ∧ p 1 ≤ 2011 ∧ ¬∃ spiral, IsSpiral spiral ∧ spiral.getLast! = p}.encard = answer", "v": null, "name": "h_answer"}]} +{"informal_problem": "Define a \\emph{growing spiral} in the plane to be a sequence of points with integer coordinates $P_0=(0,0),P_1,\\dots,P_n$ such that $n \\geq 2$ and:\n\\begin{itemize}\n\\item the directed line segments $P_0P_1,P_1P_2,\\dots,P_{n-1}P_n$ are in the successive coordinate directions east (for $P_0P_1$), north, west, south, east, etc.;\n\\item the lengths of these line segments are positive and strictly increasing.\n\\end{itemize}\nHow many of the points $(x,y)$ with integer coordinates $0 \\leq x \\leq 2011,0 \\leq y \\leq 2011$ \\emph{cannot} be the last point, $P_n$ of any growing spiral?", "informal_answer": "10053", "informal_solution": "Show that there are $10053$ excluded points.", "header": "open BigOperators Real Nat Topology", "intros": [], "formal_answer": "@Eq Nat answer (@OfNat.ofNat Nat (nat_lit 10053) (instOfNatNat (nat_lit 10053)))", "formal_answer_type": "ℕ", "outros": [{"t": "List (Fin 2 → ℤ) → Prop", "v": null, "name": "IsSpiral"}, {"t": "∀ P, IsSpiral P ↔ P.length ≥ 3 ∧ P[0]! = 0 ∧\n (∃ l : Fin (P.length - 1) → ℕ, l > 0 ∧ StrictMono l ∧ (∀ i : Fin (P.length - 1),\n (i.1 % 4 = 0 → (P[i] 0 + l i = P[i.1 + 1]! 0 ∧ P[i] 1 = P[i.1 + 1]! 1)) ∧\n (i.1 % 4 = 1 → (P[i] 0 = P[i.1 + 1]! 0 ∧ P[i] 1 + l i = P[i.1 + 1]! 1)) ∧\n (i.1 % 4 = 2 → (P[i] 0 - l i = P[i.1 + 1]! 0 ∧ P[i] 1 = P[i.1 + 1]! 1)) ∧\n (i.1 % 4 = 3 → (P[i] 0 = P[i.1 + 1]! 0 ∧ P[i] 1 - l i = P[i.1 + 1]! 1))))", "v": null, "name": "IsSpiral_def"}, {"t": "{p | 0 ≤ p 0 ∧ p 0 ≤ 2011 ∧ 0 ≤ p 1 ∧ p 1 ≤ 2011 ∧ ¬∃ spiral, IsSpiral spiral ∧ spiral.getLast! = p}.encard = answer", "v": null, "name": "h_answer"}]} {"informal_problem": "Let $a_1,a_2,\\dots$ and $b_1,b_2,\\dots$ be sequences of positive real numbers such that $a_1 = b_1 = 1$ and $b_n = b_{n-1} a_n - 2$ for$n=2,3,\\dots$. Assume that the sequence $(b_j)$ is bounded. Prove tha \\[ S = \\sum_{n=1}^\\infty \\frac{1}{a_1...a_n} \\] converges, and evaluate $S$.", "informal_answer": "3/2", "informal_solution": "Show that the solution is $S = 3/2$.", "header": "open Topology Filter", "intros": [], "formal_answer": "@Eq Real answer\n (@HDiv.hDiv Real Real Real (@instHDiv Real (@DivInvMonoid.toDiv Real Real.instDivInvMonoid))\n (@OfNat.ofNat Real (nat_lit 3)\n (@instOfNatAtLeastTwo Real (nat_lit 3) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1))))))\n (@OfNat.ofNat Real (nat_lit 2)\n (@instOfNatAtLeastTwo Real (nat_lit 2) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 0) (instOfNatNat (nat_lit 0)))))))", "formal_answer_type": "ℝ", "outros": [{"t": "ℕ → ℝ", "v": null, "name": "a"}, {"t": "ℕ → ℝ", "v": null, "name": "b"}, {"t": "∀ n : ℕ, a n > 0 ∧ b n > 0", "v": null, "name": "habn"}, {"t": "a 0 = 1 ∧ b 0 = 1", "v": null, "name": "hab1"}, {"t": "∀ n ≥ 1, b n = b (n-1) * a n - 2", "v": null, "name": "hb"}, {"t": "∃ B : ℝ, ∀ n : ℕ, |b n| ≤ B", "v": null, "name": "hbnd"}, {"t": "Tendsto (fun n => ∑ i : Fin n, 1/(∏ j : Fin (i + 1), (a j))) atTop (𝓝 answer)", "v": null, "name": "h_answer"}]} {"informal_problem": "Find a real number $c$ and a positive number $L$ for which $\\lim_{r \\to \\infty} \\frac{r^c \\int_0^{\\pi/2} x^r\\sin x\\,dx}{\\int_0^{\\pi/2} x^r\\cos x\\,dx}=L$.", "informal_answer": "(-1, 2 / π)", "informal_solution": "Show that $(c,L)=(-1,2/\\pi)$ works.", "header": "open Topology Filter", "intros": [], "formal_answer": "@Eq (Prod Real Real) answer\n (@Prod.mk Real Real (@Neg.neg Real Real.instNeg (@OfNat.ofNat Real (nat_lit 1) (@One.toOfNat1 Real Real.instOne)))\n (@HDiv.hDiv Real Real Real (@instHDiv Real (@DivInvMonoid.toDiv Real Real.instDivInvMonoid))\n (@OfNat.ofNat Real (nat_lit 2)\n (@instOfNatAtLeastTwo Real (nat_lit 2) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 0) (instOfNatNat (nat_lit 0))))))\n Real.pi))", "formal_answer_type": "ℝ × ℝ", "outros": [{"t": "ℝ", "v": null, "name": "c"}, {"t": "ℝ", "v": null, "name": "L"}, {"t": "answer = (c, L)", "v": null, "name": "h_answer"}, {"t": "L > 0", "v": null, "name": "h_L_pos"}, {"t": "Tendsto (fun r : ℝ => (r ^ c * ∫ x in Set.Ioo 0 (Real.pi / 2), x ^ r * Real.sin x) / (∫ x in Set.Ioo 0 (Real.pi / 2), x ^ r * Real.cos x)) atTop (𝓝 L)", "v": null, "name": "h_limit"}]} {"informal_problem": "For which positive integers $n$ is there an $n \\times n$ matrix with integer entries such that every dot product of a row with itself is even, while every dot product of two different rows is odd?", "informal_answer": "the set of odd positive integers", "informal_solution": "Show that the answer is $n$ odd.", "header": "open Topology Filter Matrix", "intros": [], "formal_answer": "@Eq (Set Nat) answer (@setOf Nat fun (n_1 : Nat) => @Odd Nat Nat.instSemiring n_1)", "formal_answer_type": "Set ℕ", "outros": [{"t": "ℕ → Prop", "v": null, "name": "nmat"}, {"t": "∀ n, nmat n ↔\n ∃ A : Matrix (Fin n) (Fin n) ℤ,\n (∀ r, Even ((A r) ⬝ᵥ (A r))) ∧\n Pairwise fun r1 r2 ↦ Odd ((A r1) ⬝ᵥ (A r2))", "v": null, "name": "hnmat"}, {"t": "ℕ", "v": null, "name": "n"}, {"t": "0 < n", "v": null, "name": "npos"}, {"t": "nmat n ↔ n ∈ answer", "v": null, "name": "h_answer"}]} @@ -252,12 +252,12 @@ {"informal_problem": "Let \\( n \\) be a positive integer. What is the largest \\( k \\) for which there exist \\( n \\times n \\) matrices \\( M_1, \\ldots, M_k \\) and \\( N_1, \\ldots, N_k \\) with real entries such that for all \\( i \\) and \\( j \\), the matrix product \\( M_i N_j \\) has a zero entry somewhere on its diagonal if and only if \\( i \\neq j \\)?", "informal_answer": "n^n", "informal_solution": "Show that the solution has the form k \\<= n ^ n.", "header": "open Topology Filter Nat", "intros": [], "formal_answer": "@Eq (Nat → Nat) answer fun (n_1 : Nat) =>\n @HPow.hPow Nat Nat Nat (@instHPow Nat Nat (@Monoid.toNatPow Nat Nat.instMonoid)) n_1 n_1", "formal_answer_type": "ℕ → ℕ", "outros": [{"t": "ℕ", "v": null, "name": "n"}, {"t": "ℕ → Prop", "v": null, "name": "kex"}, {"t": "n > 0", "v": null, "name": "npos"}, {"t": "∀ k ≥ 1, kex k = ∃ M N : Fin k → Matrix (Fin n) (Fin n) ℝ, ∀ i j : Fin k, ((∃ p : Fin n, (M i * N j) p p = 0) ↔ i ≠ j)", "v": null, "name": "hkex"}, {"t": "(answer n ≥ 1 ∧ kex (answer n)) ∧ (∀ k ≥ 1, kex k → k ≤ answer n)", "v": null, "name": "h_answer"}]} {"informal_problem": "A \\emph{base $10$ over-expansion} of a positive integer $N$ is an expression of the form\n\\[\nN = d_k 10^k + d_{k-1} 10^{k-1} + \\cdots + d_0 10^0\n\\]\nwith $d_k \\neq 0$ and $d_i \\in \\{0,1,2,\\dots,10\\}$ for all $i$. For instance, the integer $N = 10$ has two base $10$ over-expansions: $10 = 10 \\cdot 10^0$ and the usual base $10$ expansion $10 = 1 \\cdot 10^1 + 0 \\cdot 10^0$. Which positive integers have a unique base $10$ over-expansion?", "informal_answer": "the set of positive integers that do not contain the digit 0 in their base 10 representation", "informal_solution": "Prove that the answer is the integers with no $0$'s in their usual base $10$ expansion.", "header": "open Topology Filter Nat", "intros": [], "formal_answer": "@Eq (Set Nat) answer\n (@setOf Nat fun (n : Nat) =>\n And (@GT.gt Nat instLTNat n (@OfNat.ofNat Nat (nat_lit 0) (instOfNatNat (nat_lit 0))))\n (Not\n (@Exists Nat fun (a : Nat) =>\n And\n (@Membership.mem Nat (List Nat) (@List.instMembership Nat)\n (Nat.digits (@OfNat.ofNat Nat (nat_lit 10) (instOfNatNat (nat_lit 10))) n) a)\n (@Eq Nat a (@OfNat.ofNat Nat (nat_lit 0) (instOfNatNat (nat_lit 0)))))))", "formal_answer_type": "Set ℕ", "outros": [{"t": "ℕ → List ℕ → Prop", "v": null, "name": "overexpansion"}, {"t": "overexpansion = fun N d ↦ N = ∑ i : Fin d.length, (d.get i) * 10 ^ i.1 ∧ d.getLastI ≠ 0 ∧ ∀ a ∈ d, a ∈ Finset.range 11", "v": null, "name": "hoverexpansion"}, {"t": "Set ℕ", "v": null, "name": "S"}, {"t": "∀ N : ℕ, N ∈ S ↔ N > 0 ∧ ∃! d : List ℕ, overexpansion N d", "v": null, "name": "hS"}, {"t": "S = answer", "v": null, "name": "h_answer"}]} {"informal_problem": "Suppose that \\( f \\) is a function on the interval \\([1,3]\\) such that \\(-1 \\leq f(x) \\leq 1\\) for all \\( x \\) and \\( \\int_{1}^{3} f(x) \\, dx = 0 \\). How large can \\(\\int_{1}^{3} \\frac{f(x)}{x} \\, dx \\) be?", "informal_answer": "\\( \\log(4/3) \\)", "informal_solution": "Show that the solution is log (4 / 3).", "header": "open Topology Filter Nat", "intros": [], "formal_answer": "@Eq Real answer\n (Real.log\n (@HDiv.hDiv Real Real Real (@instHDiv Real (@DivInvMonoid.toDiv Real Real.instDivInvMonoid))\n (@OfNat.ofNat Real (nat_lit 4)\n (@instOfNatAtLeastTwo Real (nat_lit 4) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))))))\n (@OfNat.ofNat Real (nat_lit 3)\n (@instOfNatAtLeastTwo Real (nat_lit 3) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1))))))))", "formal_answer_type": "ℝ", "outros": [{"t": "ℝ → ℝ", "v": null, "name": "f"}, {"t": "∀ x : Set.Icc (1 : ℝ) 3, -1 ≤ f x ∧ f x ≤ 1", "v": null, "name": "h_bound"}, {"t": "∫ x in Set.Ioo 1 3, f x = 0", "v": null, "name": "h_integral_zero"}, {"t": "∫ x in Set.Ioo 1 3, (f x) / x = answer", "v": null, "name": "h_integral_x"}]} -{"informal_problem": "Let $a_0=1$, $a_1=2$, and $a_n=4a_{n-1}-a_{n-2}$ for $n \\geq 2$. Find an odd prime factor of $a_{2015}$.", "informal_answer": "181", "informal_solution": "Show that one possible answer is $181$.", "header": null, "intros": [], "formal_answer": "@Eq Nat answer (@OfNat.ofNat Nat (nat_lit 181) (instOfNatNat (nat_lit 181)))", "formal_answer_type": "ℕ", "outros": [{"t": "ℕ → ℤ", "v": null, "name": "a"}, {"t": "a 0 = 1 ∧ a 1 = 2", "v": null, "name": "abase"}, {"t": "∀ n ≥ 2, a n = 4 * a (n - 1) - a (n - 2)", "v": null, "name": "arec"}, {"t": "Odd answer ∧ answer.Prime ∧ ((answer : ℤ) ∣ a 2015)", "v": null, "name": "h_answer"}]} -{"informal_problem": "Compute $\\log_2 \\left( \\prod_{a=1}^{2015}\\prod_{b=1}^{2015}(1+e^{2\\pi iab/2015}) \\right)$. Here $i$ is the imaginary unit (that is, $i^2=-1$).", "informal_answer": "13725", "informal_solution": "Show that the answer is $13725$.", "header": null, "intros": [], "formal_answer": "@Eq Complex answer\n (@OfNat.ofNat Complex (nat_lit 13725)\n (@instOfNatAtLeastTwo Complex (nat_lit 13725)\n (@AddMonoidWithOne.toNatCast Complex (@AddGroupWithOne.toAddMonoidWithOne Complex Complex.addGroupWithOne))\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 13723) (instOfNatNat (nat_lit 13723))))))", "formal_answer_type": "ℂ", "outros": [{"t": "Complex.log (∏ a : Fin 2015, ∏ b : Fin 2015, (1 + Complex.exp (2 * Real.pi * Complex.I * (a.1 + 1) * (b.1 + 1) / 2015))) / Complex.log 2 = answer", "v": null, "name": "h_answer"}]} -{"informal_problem": "For each real number $x$, let\n\\[\nf(x) = \\sum_{n\\in S_x} \\frac{1}{2^n},\n\\]\nwhere $S_x$ is the set of positive integers $n$ for which $\\lfloor nx \\rfloor$ is even. What is the largest real number $L$ such that $f(x) \\geq L$ for all $x \\in [0,1)$? (As usual, $\\lfloor z \\rfloor$ denotes the greatest integer less than or equal to $z$.)", "informal_answer": "4/7", "informal_solution": "Prove that $L = \\frac{4}{7}$.", "header": null, "intros": [], "formal_answer": "@Eq Real answer\n (@HDiv.hDiv Real Real Real (@instHDiv Real (@DivInvMonoid.toDiv Real Real.instDivInvMonoid))\n (@OfNat.ofNat Real (nat_lit 4)\n (@instOfNatAtLeastTwo Real (nat_lit 4) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))))))\n (@OfNat.ofNat Real (nat_lit 7)\n (@instOfNatAtLeastTwo Real (nat_lit 7) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 5) (instOfNatNat (nat_lit 5)))))))", "formal_answer_type": "ℝ", "outros": [{"t": "ℝ → Set ℤ", "v": null, "name": "S"}, {"t": "ℝ → ℝ", "v": null, "name": "f"}, {"t": "S = fun (x : ℝ) ↦ {n : ℤ | n > 0 ∧ Even ⌊n * x⌋}", "v": null, "name": "hS"}, {"t": "f = fun (x : ℝ) ↦ ∑' n : S x, 1 / 2 ^ (n : ℤ)", "v": null, "name": "hf"}, {"t": "IsGreatest {l : ℝ | ∀ x ∈ Set.Ico 0 1, f x ≥ l} answer", "v": null, "name": "h_answer"}]} -{"informal_problem": "Given a list of the positive integers $1,2,3,4,\\dots$, take the first three numbers $1,2,3$ and their sum $6$ and cross all four numbers off the list. Repeat with the three smallest remaining numbers $4,5,7$ and their sum $16$. Continue in this way, crossing off the three smallest remaining numbers and their sum, and consider the sequence of sums produced: $6,16,27,36,\\dots$. Prove or disprove that there is some number in the sequence whose base $10$ representation ends with $2015$.", "informal_answer": "True", "informal_solution": "Show that such a number does exist.", "header": null, "intros": [], "formal_answer": "@Eq Prop answer True", "formal_answer_type": "Prop", "outros": [{"t": "ℕ → Set ℕ", "v": null, "name": "sets"}, {"t": "Set ℕ → (Fin 3 → ℕ)", "v": null, "name": "Smin3"}, {"t": "ℕ → ℕ", "v": null, "name": "sums"}, {"t": "sets 0 = Set.Ici 1", "v": null, "name": "hsets0"}, {"t": "∀ S : Set ℕ, S.encard ≥ 3 → ((Smin3 S) 0 = sInf S ∧ (Smin3 S) 1 = sInf (S \\ {(Smin3 S) 0}) ∧ (Smin3 S) 2 = sInf (S \\ {(Smin3 S) 0, (Smin3 S) 1}))", "v": null, "name": "hmin3"}, {"t": "∀ n : ℕ, sums n = (Smin3 (sets n)) 0 + (Smin3 (sets n)) 1 + (Smin3 (sets n)) 2", "v": null, "name": "hsums"}, {"t": "∀ n : ℕ, sets (n + 1) = sets n \\ {(Smin3 (sets n)) 0, (Smin3 (sets n)) 1, (Smin3 (sets n)) 2, sums n}", "v": null, "name": "hsetsn"}, {"t": "(∃ n : ℕ, List.IsPrefix [5, 1, 0, 2] (Nat.digits 10 (sums n))) ↔ answer", "v": null, "name": "h_answer"}]} -{"informal_problem": "Let $S$ be the set of all $2 \\times 2$ real matrices $M=\\begin{pmatrix} a & b \\\\ c & d \\end{pmatrix}$ whose entries $a,b,c,d$ (in that order) form an arithmetic progression. Find all matrices $M$ in $S$ for which there is some integer $k>1$ such that $M^k$ is also in $S$.", "informal_answer": "the set of all matrices of the form α * I or β * A, where I is the identity matrix and A is a specific matrix", "informal_solution": "Show that matrices of the form $\\alpha A$ or $\\beta B$, where $A=\\left(\\begin{smallmatrix} 1 & 1 \\\\ 1 & 1 \\end{smallmatrix}\\right)$, $B=\\left(\\begin{smallmatrix} -3 & -1 \\\\ 1 & 3 \\end{smallmatrix}\\right)$, and $\\alpha,\\beta \\in \\mathbb{R}$, are the only matrices in $S$ that satisfy the given condition.", "header": null, "intros": [], "formal_answer": "@Eq\n (Set\n (Matrix (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))))\n (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real))\n answer\n (@setOf\n (Matrix (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))))\n (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real)\n fun\n (A :\n Matrix (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))))\n (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real) =>\n Or\n (@Exists Real fun (α : Real) =>\n ∀ (i j : Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))),\n @Eq Real (A i j)\n (@HMul.hMul Real Real Real (@instHMul Real Real.instMul) α\n (@OfNat.ofNat Real (nat_lit 1) (@One.toOfNat1 Real Real.instOne))))\n (@Exists Real fun (β : Real) =>\n And\n (@Eq Real\n (A\n (@OfNat.ofNat (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) (nat_lit 0)\n (@Fin.instOfNat (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))\n (@Nat.instNeZeroSucc (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1)))) (nat_lit 0)))\n (@OfNat.ofNat (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) (nat_lit 0)\n (@Fin.instOfNat (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))\n (@Nat.instNeZeroSucc (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1)))) (nat_lit 0))))\n (@HMul.hMul Real Real Real (@instHMul Real Real.instMul) β\n (@Neg.neg Real Real.instNeg\n (@OfNat.ofNat Real (nat_lit 3)\n (@instOfNatAtLeastTwo Real (nat_lit 3) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1)))))))))\n (And\n (@Eq Real\n (A\n (@OfNat.ofNat (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) (nat_lit 0)\n (@Fin.instOfNat (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))\n (@Nat.instNeZeroSucc (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1)))) (nat_lit 0)))\n (@OfNat.ofNat (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) (nat_lit 1)\n (@Fin.instOfNat (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))\n (@Nat.instNeZeroSucc (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1)))) (nat_lit 1))))\n (@HMul.hMul Real Real Real (@instHMul Real Real.instMul) β\n (@Neg.neg Real Real.instNeg (@OfNat.ofNat Real (nat_lit 1) (@One.toOfNat1 Real Real.instOne)))))\n (And\n (@Eq Real\n (A\n (@OfNat.ofNat (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) (nat_lit 1)\n (@Fin.instOfNat (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))\n (@Nat.instNeZeroSucc (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1)))) (nat_lit 1)))\n (@OfNat.ofNat (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) (nat_lit 0)\n (@Fin.instOfNat (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))\n (@Nat.instNeZeroSucc (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1)))) (nat_lit 0))))\n (@HMul.hMul Real Real Real (@instHMul Real Real.instMul) β\n (@OfNat.ofNat Real (nat_lit 1) (@One.toOfNat1 Real Real.instOne))))\n (@Eq Real\n (A\n (@OfNat.ofNat (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) (nat_lit 1)\n (@Fin.instOfNat (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))\n (@Nat.instNeZeroSucc (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1)))) (nat_lit 1)))\n (@OfNat.ofNat (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) (nat_lit 1)\n (@Fin.instOfNat (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))\n (@Nat.instNeZeroSucc (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1)))) (nat_lit 1))))\n (@HMul.hMul Real Real Real (@instHMul Real Real.instMul) β\n (@OfNat.ofNat Real (nat_lit 3)\n (@instOfNatAtLeastTwo Real (nat_lit 3) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1))))))))))))", "formal_answer_type": "Set (Matrix (Fin 2) (Fin 2) ℝ)", "outros": [{"t": "Matrix (Fin 2) (Fin 2) ℝ", "v": null, "name": "M"}, {"t": "Set (Matrix (Fin 2) (Fin 2) ℝ)", "v": null, "name": "S"}, {"t": "S = {M' | (M' 0 1 - M' 0 0 = M' 1 0 - M' 0 1) ∧ (M' 1 0 - M' 0 1 = M' 1 1 - M' 1 0)}", "v": null, "name": "hS"}, {"t": "M ∈ S ∧ (∃ k > 1, M ^ k ∈ S) ↔ M ∈ answer", "v": null, "name": "h_answer"}]} -{"informal_problem": "Let $T$ be the set of all triples $(a,b,c)$ of positive integers for which there exist triangles with side lengths $a,b,c$. Express\n\\[\n\\sum_{(a,b,c) \\in T} \\frac{2^a}{3^b 5^c}\n\\]\nas a rational number in lowest terms.", "informal_answer": "(17, 21)", "informal_solution": "The answer is $17/21$.", "header": null, "intros": [], "formal_answer": "@Eq (Prod Int Nat) answer\n (@Prod.mk Int Nat (@OfNat.ofNat Int (nat_lit 17) (@instOfNat (nat_lit 17)))\n (@OfNat.ofNat Nat (nat_lit 21) (instOfNatNat (nat_lit 21))))", "formal_answer_type": "ℤ × ℕ", "outros": [{"t": "ℚ → (ℤ × ℕ)", "v": null, "name": "quotientof"}, {"t": "∀ q : ℚ, quotientof q = (q.num, q.den)", "v": null, "name": "hquotientof"}, {"t": "quotientof (∑' t : (Fin 3 → ℤ), if (∀ n : Fin 3, t n > 0) ∧ t 0 < t 1 + t 2 ∧ t 1 < t 2 + t 0 ∧ t 2 < t 0 + t 1\n then 2^(t 0)/(3^(t 1)*5^(t 2)) else 0) = answer", "v": null, "name": "h_answer"}]} +{"informal_problem": "Let $a_0=1$, $a_1=2$, and $a_n=4a_{n-1}-a_{n-2}$ for $n \\geq 2$. Find an odd prime factor of $a_{2015}$.", "informal_answer": "181", "informal_solution": "Show that one possible answer is $181$.", "header": "open BigOperators Real Nat Topology", "intros": [], "formal_answer": "@Eq Nat answer (@OfNat.ofNat Nat (nat_lit 181) (instOfNatNat (nat_lit 181)))", "formal_answer_type": "ℕ", "outros": [{"t": "ℕ → ℤ", "v": null, "name": "a"}, {"t": "a 0 = 1 ∧ a 1 = 2", "v": null, "name": "abase"}, {"t": "∀ n ≥ 2, a n = 4 * a (n - 1) - a (n - 2)", "v": null, "name": "arec"}, {"t": "Odd answer ∧ answer.Prime ∧ ((answer : ℤ) ∣ a 2015)", "v": null, "name": "h_answer"}]} +{"informal_problem": "Compute $\\log_2 \\left( \\prod_{a=1}^{2015}\\prod_{b=1}^{2015}(1+e^{2\\pi iab/2015}) \\right)$. Here $i$ is the imaginary unit (that is, $i^2=-1$).", "informal_answer": "13725", "informal_solution": "Show that the answer is $13725$.", "header": "open BigOperators Real Nat Topology", "intros": [], "formal_answer": "@Eq Complex answer\n (@OfNat.ofNat Complex (nat_lit 13725)\n (@instOfNatAtLeastTwo Complex (nat_lit 13725)\n (@AddMonoidWithOne.toNatCast Complex (@AddGroupWithOne.toAddMonoidWithOne Complex Complex.addGroupWithOne))\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 13723) (instOfNatNat (nat_lit 13723))))))", "formal_answer_type": "ℂ", "outros": [{"t": "Complex.log (∏ a : Fin 2015, ∏ b : Fin 2015, (1 + Complex.exp (2 * Real.pi * Complex.I * (a.1 + 1) * (b.1 + 1) / 2015))) / Complex.log 2 = answer", "v": null, "name": "h_answer"}]} +{"informal_problem": "For each real number $x$, let\n\\[\nf(x) = \\sum_{n\\in S_x} \\frac{1}{2^n},\n\\]\nwhere $S_x$ is the set of positive integers $n$ for which $\\lfloor nx \\rfloor$ is even. What is the largest real number $L$ such that $f(x) \\geq L$ for all $x \\in [0,1)$? (As usual, $\\lfloor z \\rfloor$ denotes the greatest integer less than or equal to $z$.)", "informal_answer": "4/7", "informal_solution": "Prove that $L = \\frac{4}{7}$.", "header": "open BigOperators Real Nat Topology", "intros": [], "formal_answer": "@Eq Real answer\n (@HDiv.hDiv Real Real Real (@instHDiv Real (@DivInvMonoid.toDiv Real Real.instDivInvMonoid))\n (@OfNat.ofNat Real (nat_lit 4)\n (@instOfNatAtLeastTwo Real (nat_lit 4) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))))))\n (@OfNat.ofNat Real (nat_lit 7)\n (@instOfNatAtLeastTwo Real (nat_lit 7) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 5) (instOfNatNat (nat_lit 5)))))))", "formal_answer_type": "ℝ", "outros": [{"t": "ℝ → Set ℤ", "v": null, "name": "S"}, {"t": "ℝ → ℝ", "v": null, "name": "f"}, {"t": "S = fun (x : ℝ) ↦ {n : ℤ | n > 0 ∧ Even ⌊n * x⌋}", "v": null, "name": "hS"}, {"t": "f = fun (x : ℝ) ↦ ∑' n : S x, 1 / 2 ^ (n : ℤ)", "v": null, "name": "hf"}, {"t": "IsGreatest {l : ℝ | ∀ x ∈ Set.Ico 0 1, f x ≥ l} answer", "v": null, "name": "h_answer"}]} +{"informal_problem": "Given a list of the positive integers $1,2,3,4,\\dots$, take the first three numbers $1,2,3$ and their sum $6$ and cross all four numbers off the list. Repeat with the three smallest remaining numbers $4,5,7$ and their sum $16$. Continue in this way, crossing off the three smallest remaining numbers and their sum, and consider the sequence of sums produced: $6,16,27,36,\\dots$. Prove or disprove that there is some number in the sequence whose base $10$ representation ends with $2015$.", "informal_answer": "True", "informal_solution": "Show that such a number does exist.", "header": "open BigOperators Real Nat Topology", "intros": [], "formal_answer": "@Eq Prop answer True", "formal_answer_type": "Prop", "outros": [{"t": "ℕ → Set ℕ", "v": null, "name": "sets"}, {"t": "Set ℕ → (Fin 3 → ℕ)", "v": null, "name": "Smin3"}, {"t": "ℕ → ℕ", "v": null, "name": "sums"}, {"t": "sets 0 = Set.Ici 1", "v": null, "name": "hsets0"}, {"t": "∀ S : Set ℕ, S.encard ≥ 3 → ((Smin3 S) 0 = sInf S ∧ (Smin3 S) 1 = sInf (S \\ {(Smin3 S) 0}) ∧ (Smin3 S) 2 = sInf (S \\ {(Smin3 S) 0, (Smin3 S) 1}))", "v": null, "name": "hmin3"}, {"t": "∀ n : ℕ, sums n = (Smin3 (sets n)) 0 + (Smin3 (sets n)) 1 + (Smin3 (sets n)) 2", "v": null, "name": "hsums"}, {"t": "∀ n : ℕ, sets (n + 1) = sets n \\ {(Smin3 (sets n)) 0, (Smin3 (sets n)) 1, (Smin3 (sets n)) 2, sums n}", "v": null, "name": "hsetsn"}, {"t": "(∃ n : ℕ, List.IsPrefix [5, 1, 0, 2] (Nat.digits 10 (sums n))) ↔ answer", "v": null, "name": "h_answer"}]} +{"informal_problem": "Let $S$ be the set of all $2 \\times 2$ real matrices $M=\\begin{pmatrix} a & b \\\\ c & d \\end{pmatrix}$ whose entries $a,b,c,d$ (in that order) form an arithmetic progression. Find all matrices $M$ in $S$ for which there is some integer $k>1$ such that $M^k$ is also in $S$.", "informal_answer": "the set of all matrices of the form α * I or β * A, where I is the identity matrix and A is a specific matrix", "informal_solution": "Show that matrices of the form $\\alpha A$ or $\\beta B$, where $A=\\left(\\begin{smallmatrix} 1 & 1 \\\\ 1 & 1 \\end{smallmatrix}\\right)$, $B=\\left(\\begin{smallmatrix} -3 & -1 \\\\ 1 & 3 \\end{smallmatrix}\\right)$, and $\\alpha,\\beta \\in \\mathbb{R}$, are the only matrices in $S$ that satisfy the given condition.", "header": "open BigOperators Real Nat Topology", "intros": [], "formal_answer": "@Eq\n (Set\n (Matrix (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))))\n (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real))\n answer\n (@setOf\n (Matrix (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))))\n (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real)\n fun\n (A :\n Matrix (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))))\n (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) Real) =>\n Or\n (@Exists Real fun (α : Real) =>\n ∀ (i j : Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))),\n @Eq Real (A i j)\n (@HMul.hMul Real Real Real (@instHMul Real Real.instMul) α\n (@OfNat.ofNat Real (nat_lit 1) (@One.toOfNat1 Real Real.instOne))))\n (@Exists Real fun (β : Real) =>\n And\n (@Eq Real\n (A\n (@OfNat.ofNat (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) (nat_lit 0)\n (@Fin.instOfNat (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))\n (@Nat.instNeZeroSucc (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1)))) (nat_lit 0)))\n (@OfNat.ofNat (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) (nat_lit 0)\n (@Fin.instOfNat (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))\n (@Nat.instNeZeroSucc (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1)))) (nat_lit 0))))\n (@HMul.hMul Real Real Real (@instHMul Real Real.instMul) β\n (@Neg.neg Real Real.instNeg\n (@OfNat.ofNat Real (nat_lit 3)\n (@instOfNatAtLeastTwo Real (nat_lit 3) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1)))))))))\n (And\n (@Eq Real\n (A\n (@OfNat.ofNat (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) (nat_lit 0)\n (@Fin.instOfNat (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))\n (@Nat.instNeZeroSucc (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1)))) (nat_lit 0)))\n (@OfNat.ofNat (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) (nat_lit 1)\n (@Fin.instOfNat (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))\n (@Nat.instNeZeroSucc (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1)))) (nat_lit 1))))\n (@HMul.hMul Real Real Real (@instHMul Real Real.instMul) β\n (@Neg.neg Real Real.instNeg (@OfNat.ofNat Real (nat_lit 1) (@One.toOfNat1 Real Real.instOne)))))\n (And\n (@Eq Real\n (A\n (@OfNat.ofNat (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) (nat_lit 1)\n (@Fin.instOfNat (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))\n (@Nat.instNeZeroSucc (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1)))) (nat_lit 1)))\n (@OfNat.ofNat (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) (nat_lit 0)\n (@Fin.instOfNat (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))\n (@Nat.instNeZeroSucc (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1)))) (nat_lit 0))))\n (@HMul.hMul Real Real Real (@instHMul Real Real.instMul) β\n (@OfNat.ofNat Real (nat_lit 1) (@One.toOfNat1 Real Real.instOne))))\n (@Eq Real\n (A\n (@OfNat.ofNat (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) (nat_lit 1)\n (@Fin.instOfNat (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))\n (@Nat.instNeZeroSucc (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1)))) (nat_lit 1)))\n (@OfNat.ofNat (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))) (nat_lit 1)\n (@Fin.instOfNat (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))\n (@Nat.instNeZeroSucc (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1)))) (nat_lit 1))))\n (@HMul.hMul Real Real Real (@instHMul Real Real.instMul) β\n (@OfNat.ofNat Real (nat_lit 3)\n (@instOfNatAtLeastTwo Real (nat_lit 3) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1))))))))))))", "formal_answer_type": "Set (Matrix (Fin 2) (Fin 2) ℝ)", "outros": [{"t": "Matrix (Fin 2) (Fin 2) ℝ", "v": null, "name": "M"}, {"t": "Set (Matrix (Fin 2) (Fin 2) ℝ)", "v": null, "name": "S"}, {"t": "S = {M' | (M' 0 1 - M' 0 0 = M' 1 0 - M' 0 1) ∧ (M' 1 0 - M' 0 1 = M' 1 1 - M' 1 0)}", "v": null, "name": "hS"}, {"t": "M ∈ S ∧ (∃ k > 1, M ^ k ∈ S) ↔ M ∈ answer", "v": null, "name": "h_answer"}]} +{"informal_problem": "Let $T$ be the set of all triples $(a,b,c)$ of positive integers for which there exist triangles with side lengths $a,b,c$. Express\n\\[\n\\sum_{(a,b,c) \\in T} \\frac{2^a}{3^b 5^c}\n\\]\nas a rational number in lowest terms.", "informal_answer": "(17, 21)", "informal_solution": "The answer is $17/21$.", "header": "open BigOperators Real Nat Topology", "intros": [], "formal_answer": "@Eq (Prod Int Nat) answer\n (@Prod.mk Int Nat (@OfNat.ofNat Int (nat_lit 17) (@instOfNat (nat_lit 17)))\n (@OfNat.ofNat Nat (nat_lit 21) (instOfNatNat (nat_lit 21))))", "formal_answer_type": "ℤ × ℕ", "outros": [{"t": "ℚ → (ℤ × ℕ)", "v": null, "name": "quotientof"}, {"t": "∀ q : ℚ, quotientof q = (q.num, q.den)", "v": null, "name": "hquotientof"}, {"t": "quotientof (∑' t : (Fin 3 → ℤ), if (∀ n : Fin 3, t n > 0) ∧ t 0 < t 1 + t 2 ∧ t 1 < t 2 + t 0 ∧ t 2 < t 0 + t 1\n then 2^(t 0)/(3^(t 1)*5^(t 2)) else 0) = answer", "v": null, "name": "h_answer"}]} {"informal_problem": "Let $P_n$ be the number of permutations $\\pi$ of $\\{1,2,\\dots,n\\}$ such that\n\\[\n|i-j| = 1 \\mbox{ implies } |\\pi(i) -\\pi(j)| \\leq 2\n\\]\nfor all $i,j$ in $\\{1,2,\\dots,n\\}$. Show that for $n \\geq 2$, the quantity\n\\[\nP_{n+5} - P_{n+4} - P_{n+3} + P_n\n\\]\ndoes not depend on $n$, and find its value.", "informal_answer": "4", "informal_solution": "Prove that answer is $4$.", "header": "open Function", "intros": [], "formal_answer": "@Eq Nat answer (@OfNat.ofNat Nat (nat_lit 4) (instOfNatNat (nat_lit 4)))", "formal_answer_type": "ℕ", "outros": [{"t": "ℕ → ℕ", "v": null, "name": "P"}, {"t": "P = fun n ↦ {pi : Finset.Icc 1 n → Finset.Icc 1 n | Bijective pi ∧ ∀ i j : Finset.Icc 1 n, Nat.dist i j = 1 → Nat.dist (pi i) (pi j) ≤ 2}.ncard", "v": null, "name": "hP"}, {"t": "∀ n : ℕ, n ≥ 2 → (P (n + 5) : ℤ) - (P (n + 4) : ℤ) - (P (n + 3) : ℤ) + (P n : ℤ) = answer", "v": null, "name": "h_answer"}]} {"informal_problem": "For each positive integer $k$, let $A(k)$ be the number of odd divisors of $k$ in the interval $[1,\\sqrt{2k})$. Evaluate $\\sum_{k=1}^\\infty (-1)^{k-1}\\frac{A(k)}{k}$.", "informal_answer": "π² / 16", "informal_solution": "Show that the sum converges to $\\pi^2/16$.", "header": "open Filter Topology", "intros": [], "formal_answer": "@Eq Real answer\n (@HDiv.hDiv Real Real Real (@instHDiv Real (@DivInvMonoid.toDiv Real Real.instDivInvMonoid))\n (@HPow.hPow Real Nat Real (@instHPow Real Nat (@Monoid.toNatPow Real Real.instMonoid)) Real.pi\n (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))))\n (@OfNat.ofNat Real (nat_lit 16)\n (@instOfNatAtLeastTwo Real (nat_lit 16) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 14) (instOfNatNat (nat_lit 14)))))))", "formal_answer_type": "ℝ", "outros": [{"t": "ℕ → ℕ", "v": null, "name": "A"}, {"t": "∀ k > 0, A k = {j : ℕ | Odd j ∧ j ∣ k ∧ j < Real.sqrt (2 * k)}.encard", "v": null, "name": "hA"}, {"t": "Tendsto (fun K : ℕ ↦ ∑ k in Finset.Icc 1 K, (-1 : ℝ) ^ ((k : ℝ) - 1) * (A k / (k : ℝ))) atTop (𝓝 answer)", "v": null, "name": "h_answer"}]} {"informal_problem": "Find the smallest positive integer $j$ such that for every polynomial $p(x)$ with integer coefficients and for every integer $k$, the integer \\[ p^{(j)}(k) = \\left. \\frac{d^j}{dx^j} p(x) \\right|_{x=k} \\] (the $j$-th derivative of $p(x)$ at $k$) is divisible by 2016.", "informal_answer": "8", "informal_solution": "Show that the solution is $8$.", "header": "open Polynomial Filter Topology Real Set Nat", "intros": [], "formal_answer": "@Eq Nat answer (@OfNat.ofNat Nat (nat_lit 8) (instOfNatNat (nat_lit 8)))", "formal_answer_type": "ℕ", "outros": [{"t": "IsLeast {j : ℕ | 0 < j ∧ ∀ P : ℤ[X], ∀ k : ℤ, 2016 ∣ (derivative^[j] P).eval k} answer", "v": null, "name": "h_answer"}]} @@ -269,15 +269,15 @@ {"informal_problem": "Let $A$ be a $2n \\times 2n$ matrix, with entries chosen independently at random. Every entry is chosen to be $0$ or $1$, each with probability $1/2$. Find the expected value of $\\det(A-A^t)$ (as a function of $n$), where $A^t$ is the transpose of $A$.", "informal_answer": "(fun n : ℕ => (2 * n)! / (4 ^ n * (n)!))", "informal_solution": "Show that the expected value equals $\\frac{(2n)!}{4^nn!}$.", "header": "open Real Set Nat", "intros": [], "formal_answer": "@Eq (Nat → Real) answer fun (n_1 : Nat) =>\n @HDiv.hDiv Real Real Real (@instHDiv Real (@DivInvMonoid.toDiv Real Real.instDivInvMonoid))\n (@Nat.cast Real Real.instNatCast\n (Nat.factorial\n (@HMul.hMul Nat Nat Nat (@instHMul Nat instMulNat) (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))\n n_1)))\n (@HMul.hMul Real Real Real (@instHMul Real Real.instMul)\n (@HPow.hPow Real Nat Real (@instHPow Real Nat (@Monoid.toNatPow Real Real.instMonoid))\n (@OfNat.ofNat Real (nat_lit 4)\n (@instOfNatAtLeastTwo Real (nat_lit 4) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))))))\n n_1)\n (@Nat.cast Real Real.instNatCast (Nat.factorial n_1)))", "formal_answer_type": "ℕ → ℝ", "outros": [{"t": "ℕ", "v": null, "name": "n"}, {"t": "n ≥ 1", "v": null, "name": "npos"}, {"t": "Set (Matrix (Fin (2 * n)) (Fin (2 * n)) ℝ)", "v": null, "name": "mats01"}, {"t": "mats01 = {A | ∀ i j : Fin (2 * n), A i j = 0 ∨ A i j = 1}", "v": null, "name": "hmats01"}, {"t": "(∑' A : mats01, (A.1 - (Matrix.transpose A)).det) / mats01.ncard = answer n", "v": null, "name": "h_answer"}]} {"informal_problem": "Find all functions $f$ from the interval $(1,\\infty)$ to $(1,\\infty)$ with the following property: if $x,y \\in (1,\\infty)$ and $x^2 \\leq y \\leq x^3$, then $(f(x))^2 \\leq f(y) \\leq (f(x))^3$.", "informal_answer": "the set of all functions of the form f(x) = x^c for some c > 0", "informal_solution": "Show that the only such functions are the functions $f(x)=x^c$ for some $c>0$.", "header": "open Polynomial Filter Topology Real Set Nat List", "intros": [], "formal_answer": "@Eq\n (Set\n (@Set.Elem Real\n (@Set.Ioi Real Real.instPreorder (@OfNat.ofNat Real (nat_lit 1) (@One.toOfNat1 Real Real.instOne))) →\n @Set.Elem Real\n (@Set.Ioi Real Real.instPreorder (@OfNat.ofNat Real (nat_lit 1) (@One.toOfNat1 Real Real.instOne)))))\n answer\n (@setOf\n (@Set.Elem Real\n (@Set.Ioi Real Real.instPreorder (@OfNat.ofNat Real (nat_lit 1) (@One.toOfNat1 Real Real.instOne))) →\n @Set.Elem Real\n (@Set.Ioi Real Real.instPreorder (@OfNat.ofNat Real (nat_lit 1) (@One.toOfNat1 Real Real.instOne))))\n fun\n (f_1 :\n @Set.Elem Real\n (@Set.Ioi Real Real.instPreorder (@OfNat.ofNat Real (nat_lit 1) (@One.toOfNat1 Real Real.instOne))) →\n @Set.Elem Real\n (@Set.Ioi Real Real.instPreorder (@OfNat.ofNat Real (nat_lit 1) (@One.toOfNat1 Real Real.instOne)))) =>\n @Exists Real fun (c : Real) =>\n And (@GT.gt Real Real.instLT c (@OfNat.ofNat Real (nat_lit 0) (@Zero.toOfNat0 Real Real.instZero)))\n (∀\n (x :\n @Set.Elem Real\n (@Set.Ioi Real Real.instPreorder (@OfNat.ofNat Real (nat_lit 1) (@One.toOfNat1 Real Real.instOne)))),\n @Eq Real\n (@Subtype.val Real\n (fun (x_1 : Real) =>\n @Membership.mem Real (Set Real) (@Set.instMembership Real)\n (@Set.Ioi Real Real.instPreorder (@OfNat.ofNat Real (nat_lit 1) (@One.toOfNat1 Real Real.instOne)))\n x_1)\n (f_1 x))\n (@HPow.hPow Real Real Real (@instHPow Real Real Real.instPow)\n (@Subtype.val Real\n (fun (x_1 : Real) =>\n @Membership.mem Real (Set Real) (@Set.instMembership Real)\n (@Set.Ioi Real Real.instPreorder (@OfNat.ofNat Real (nat_lit 1) (@One.toOfNat1 Real Real.instOne)))\n x_1)\n x)\n c)))", "formal_answer_type": "Set (Set.Ioi (1 : ℝ) → Set.Ioi (1 : ℝ))", "outros": [{"t": "Set.Ioi (1 : ℝ) → Set.Ioi (1 : ℝ)", "v": null, "name": "f"}, {"t": "f ∈ answer ↔\n (∀ x y : Set.Ioi (1 : ℝ), ((x : ℝ) ^ 2 ≤ y ∧ y ≤ (x : ℝ) ^ 3) → ((f x : ℝ) ^ 2 ≤ f y ∧ f y ≤ (f x : ℝ) ^ 3))", "v": null, "name": "h_answer"}]} {"informal_problem": "Evaluate $\\sum_{k=1}^\\infty \\frac{(-1)^{k-1}}{k} \\sum_{n=0}^\\infty \\frac{1}{k2^n+1}$.", "informal_answer": "1", "informal_solution": "Show that the desired sum equals $1$.", "header": "open Polynomial Filter Topology Real Set Nat List", "intros": [], "formal_answer": "@Eq Real answer (@OfNat.ofNat Real (nat_lit 1) (@One.toOfNat1 Real Real.instOne))", "formal_answer_type": "ℝ", "outros": [{"t": "∑' k : ℕ, ((-1 : ℝ) ^ ((k + 1 : ℤ) - 1) / (k + 1 : ℝ)) * ∑' n : ℕ, (1 : ℝ) / ((k + 1) * (2 ^ n) + 1) = answer", "v": null, "name": "h_answer"}]} -{"informal_problem": "Let $S$ be the smallest set of positive integers such that (a) $2$ is in $S$, (b) $n$ is in $S$ whenever $n^2$ is in $S$, and (c) $(n+5)^2$ is in $S$ whenever $n$ is in $S$. Which positive integers are not in $S$?.", "informal_answer": "{x : ℤ | x > 0 ∧ (x = 1 ∨ 5 ∣ x)}", "informal_solution": "Show that all solutions are in the set $\\{x \\in \\mathbb{Z}\\, |\\, x > 0 \\land (x = 1 \\lor 5 \\mid x)\\}", "header": null, "intros": [], "formal_answer": "@Eq (Set Int) answer\n (@setOf Int fun (x : Int) =>\n And (@GT.gt Int Int.instLTInt x (@OfNat.ofNat Int (nat_lit 0) (@instOfNat (nat_lit 0))))\n (Or (@Eq Int x (@OfNat.ofNat Int (nat_lit 1) (@instOfNat (nat_lit 1))))\n (@Dvd.dvd Int Int.instDvd (@OfNat.ofNat Int (nat_lit 5) (@instOfNat (nat_lit 5))) x)))", "formal_answer_type": "Set ℤ", "outros": [{"t": "Set ℤ → Prop", "v": null, "name": "IsQualifying"}, {"t": "∀ S, IsQualifying S ↔\n (∀ n ∈ S, 0 < n) ∧\n 2 ∈ S ∧\n (∀ n > 0, n ^ 2 ∈ S → n ∈ S) ∧\n (∀ n ∈ S, (n + 5) ^ 2 ∈ S)", "v": null, "name": "IsQualifying_def"}, {"t": "Set ℤ", "v": null, "name": "S"}, {"t": "IsLeast IsQualifying S", "v": null, "name": "hS"}, {"t": "Sᶜ ∩ {n | 0 < n} = answer", "v": null, "name": "h_answer"}]} +{"informal_problem": "Let $S$ be the smallest set of positive integers such that (a) $2$ is in $S$, (b) $n$ is in $S$ whenever $n^2$ is in $S$, and (c) $(n+5)^2$ is in $S$ whenever $n$ is in $S$. Which positive integers are not in $S$?.", "informal_answer": "{x : ℤ | x > 0 ∧ (x = 1 ∨ 5 ∣ x)}", "informal_solution": "Show that all solutions are in the set $\\{x \\in \\mathbb{Z}\\, |\\, x > 0 \\land (x = 1 \\lor 5 \\mid x)\\}", "header": "open BigOperators Real Nat Topology", "intros": [], "formal_answer": "@Eq (Set Int) answer\n (@setOf Int fun (x : Int) =>\n And (@GT.gt Int Int.instLTInt x (@OfNat.ofNat Int (nat_lit 0) (@instOfNat (nat_lit 0))))\n (Or (@Eq Int x (@OfNat.ofNat Int (nat_lit 1) (@instOfNat (nat_lit 1))))\n (@Dvd.dvd Int Int.instDvd (@OfNat.ofNat Int (nat_lit 5) (@instOfNat (nat_lit 5))) x)))", "formal_answer_type": "Set ℤ", "outros": [{"t": "Set ℤ → Prop", "v": null, "name": "IsQualifying"}, {"t": "∀ S, IsQualifying S ↔\n (∀ n ∈ S, 0 < n) ∧\n 2 ∈ S ∧\n (∀ n > 0, n ^ 2 ∈ S → n ∈ S) ∧\n (∀ n ∈ S, (n + 5) ^ 2 ∈ S)", "v": null, "name": "IsQualifying_def"}, {"t": "Set ℤ", "v": null, "name": "S"}, {"t": "IsLeast IsQualifying S", "v": null, "name": "hS"}, {"t": "Sᶜ ∩ {n | 0 < n} = answer", "v": null, "name": "h_answer"}]} {"informal_problem": "Suppose that a positive integer $N$ can be expressed as the sum of $k$ consecutive positive integers\n\\[\nN = a + (a+1) +(a+2) + \\cdots + (a+k-1)\n\\]\nfor $k=2017$ but for no other values of $k>1$. Considering all positive integers $N$ with this property, what is the smallest positive integer $a$ that occurs in any of these expressions?", "informal_answer": "16", "informal_solution": "Prove that the smallest value of $a$ is $16$.", "header": "open Topology Filter", "intros": [], "formal_answer": "@Eq Nat answer (@OfNat.ofNat Nat (nat_lit 16) (instOfNatNat (nat_lit 16)))", "formal_answer_type": "ℕ", "outros": [{"t": "ℤ → ℕ → ℤ", "v": null, "name": "S"}, {"t": "ℤ → ℕ → Prop", "v": null, "name": "p"}, {"t": "ℤ → Prop", "v": null, "name": "q"}, {"t": "S = fun (a : ℤ) k ↦ ∑ i in Finset.range k, (a + i)", "v": null, "name": "hS"}, {"t": "∀ N k, p N k ↔ ∃ a > 0, S a k = N", "v": null, "name": "hp"}, {"t": "∀ N, q N ↔ p N 2017 ∧ ∀ k : ℕ, k > 1 → k ≠ 2017 → ¬p N k", "v": null, "name": "hq"}, {"t": "IsLeast {a : ℤ | q (S a 2017)} answer", "v": null, "name": "h_answer"}]} {"informal_problem": "Evaluate the sum \\begin{gather*} \\sum_{k=0}^\\infty \\left( 3 \\cdot \\frac{\\ln(4k+2)}{4k+2} - \\frac{\\ln(4k+3)}{4k+3} - \\frac{\\ln(4k+4)}{4k+4} - \\frac{\\ln(4k+5)}{4k+5} \\right) \\ = 3 \\cdot \\frac{\\ln 2}{2} - \\frac{\\ln 3}{3} - \\frac{\\ln 4}{4} - \\frac{\\ln 5}{5} + 3 \\cdot \\frac{\\ln 6}{6} - \\frac{\\ln 7}{7} \\ - \\frac{\\ln 8}{8} - \\frac{\\ln 9}{9} + 3 \\cdot \\frac{\\ln 10}{10} - \\cdots . \\end{gather*} (As usual, $\\ln x$ denotes the natural logarithm of $x$.)", "informal_answer": "(log 2) ^ 2", "informal_solution": "Prove that the sum equals $(\\ln 2)^2$.", "header": "open Topology Filter Real", "intros": [], "formal_answer": "@Eq Real answer\n (@HPow.hPow Real Nat Real (@instHPow Real Nat (@Monoid.toNatPow Real Real.instMonoid))\n (Real.log\n (@OfNat.ofNat Real (nat_lit 2)\n (@instOfNatAtLeastTwo Real (nat_lit 2) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 0) (instOfNatNat (nat_lit 0)))))))\n (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))))", "formal_answer_type": "ℝ", "outros": [{"t": "(∑' k : ℕ, (3 * Real.log (4 * k + 2) / (4 * k + 2) - Real.log (4 * k + 3) / (4 * k + 3) - Real.log (4 * k + 4) / (4 * k + 4) - Real.log (4 * k + 5) / (4 * k + 5)) = answer)", "v": null, "name": "h_answer"}]} {"informal_problem": "Find the number of ordered $64$-tuples $(x_0,x_1,\\dots,x_{63})$ such that $x_0,x_1,\\dots,x_{63}$ are distinct elements of $\\{1,2,\\dots,2017\\}$ and\n\\[\nx_0 + x_1 + 2x_2 + 3x_3 + \\cdots + 63 x_{63}\n\\]\nis divisible by 2017.", "informal_answer": "2016! / 1953! - 63! * 2016", "informal_solution": "Prove that the answer is $\\frac{2016!}{1953!} - 63! \\cdot 2016$", "header": "open Topology Filter Real Function Nat", "intros": [], "formal_answer": "@Eq Nat answer\n (@HSub.hSub Nat Nat Nat (@instHSub Nat instSubNat)\n (@HDiv.hDiv Nat Nat Nat (@instHDiv Nat Nat.instDiv)\n (Nat.factorial (@OfNat.ofNat Nat (nat_lit 2016) (instOfNatNat (nat_lit 2016))))\n (Nat.factorial (@OfNat.ofNat Nat (nat_lit 1953) (instOfNatNat (nat_lit 1953)))))\n (@HMul.hMul Nat Nat Nat (@instHMul Nat instMulNat)\n (Nat.factorial (@OfNat.ofNat Nat (nat_lit 63) (instOfNatNat (nat_lit 63))))\n (@OfNat.ofNat Nat (nat_lit 2016) (instOfNatNat (nat_lit 2016)))))", "formal_answer_type": "ℕ", "outros": [{"t": "Finset (Finset.range 64 → Finset.Icc 1 2017)", "v": null, "name": "S"}, {"t": "∀ x, x ∈ S ↔ (Injective x ∧ (2017 ∣ (∑ i : Finset.range 64, if i ≤ (⟨1, by norm_num⟩ : Finset.range 64) then (x i : ℤ) else i * (x i : ℤ))))", "v": null, "name": "hs"}, {"t": "S.card = answer", "v": null, "name": "h_answer"}]} -{"informal_problem": "Find all ordered pairs $(a,b)$ of positive integers for which $\\frac{1}{a} + \\frac{1}{b} = \\frac{3}{2018}$.", "informal_answer": "{⟨673, 1358114⟩, ⟨674, 340033⟩, ⟨1009, 2018⟩, ⟨2018, 1009⟩, ⟨340033, 674⟩, ⟨1358114, 673⟩}", "informal_solution": "Show that all solutions are in the set of ${(673,1358114), (674,340033), (1009,2018), (2018,1009), (340033,674), (1358114,673)}$.", "header": null, "intros": [], "formal_answer": "@Eq (Set (Prod Int Int)) answer\n (@Insert.insert (Prod Int Int) (Set (Prod Int Int)) (@Set.instInsert (Prod Int Int))\n (@Prod.mk Int Int (@OfNat.ofNat Int (nat_lit 673) (@instOfNat (nat_lit 673)))\n (@OfNat.ofNat Int (nat_lit 1358114) (@instOfNat (nat_lit 1358114))))\n (@Insert.insert (Prod Int Int) (Set (Prod Int Int)) (@Set.instInsert (Prod Int Int))\n (@Prod.mk Int Int (@OfNat.ofNat Int (nat_lit 674) (@instOfNat (nat_lit 674)))\n (@OfNat.ofNat Int (nat_lit 340033) (@instOfNat (nat_lit 340033))))\n (@Insert.insert (Prod Int Int) (Set (Prod Int Int)) (@Set.instInsert (Prod Int Int))\n (@Prod.mk Int Int (@OfNat.ofNat Int (nat_lit 1009) (@instOfNat (nat_lit 1009)))\n (@OfNat.ofNat Int (nat_lit 2018) (@instOfNat (nat_lit 2018))))\n (@Insert.insert (Prod Int Int) (Set (Prod Int Int)) (@Set.instInsert (Prod Int Int))\n (@Prod.mk Int Int (@OfNat.ofNat Int (nat_lit 2018) (@instOfNat (nat_lit 2018)))\n (@OfNat.ofNat Int (nat_lit 1009) (@instOfNat (nat_lit 1009))))\n (@Insert.insert (Prod Int Int) (Set (Prod Int Int)) (@Set.instInsert (Prod Int Int))\n (@Prod.mk Int Int (@OfNat.ofNat Int (nat_lit 340033) (@instOfNat (nat_lit 340033)))\n (@OfNat.ofNat Int (nat_lit 674) (@instOfNat (nat_lit 674))))\n (@Singleton.singleton (Prod Int Int) (Set (Prod Int Int)) (@Set.instSingletonSet (Prod Int Int))\n (@Prod.mk Int Int (@OfNat.ofNat Int (nat_lit 1358114) (@instOfNat (nat_lit 1358114)))\n (@OfNat.ofNat Int (nat_lit 673) (@instOfNat (nat_lit 673))))))))))", "formal_answer_type": "Set (ℤ × ℤ)", "outros": [{"t": "ℤ", "v": null, "name": "a"}, {"t": "ℤ", "v": null, "name": "b"}, {"t": "0 < a ∧ 0 < b", "v": null, "name": "h"}, {"t": "((1 : ℚ) / a + (1 : ℚ) / b = (3 : ℚ) / 2018) ↔ (⟨a, b⟩ ∈ answer)", "v": null, "name": "h_answer"}]} -{"informal_problem": "Let \\( S_1, S_2, \\ldots, S_{2^n-1} \\) be the nonempty subsets of \\( \\{1, 2, \\ldots, n\\} \\) in some order, and let \\( M \\) be the \\( (2^n - 1) \\times (2^n - 1) \\) matrix whose \\((i, j)\\) entry is $m_{ij} = \\begin{cases} 0 & \\text{if } S_i \\cap S_j = \\emptyset; \\\\ 1 & \\text{otherwise}. \\end{cases} $ Calculate the determinant of \\( M \\).", "informal_answer": "1 if n = 1, otherwise -1", "informal_solution": "Show that the solution is 1 if n = 1, and otherwise -1.", "header": null, "intros": [], "formal_answer": "@Eq (Nat → Real) answer fun (n_1 : Nat) =>\n @ite Real (@Eq Nat n_1 (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1))))\n (instDecidableEqNat n_1 (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1))))\n (@OfNat.ofNat Real (nat_lit 1) (@One.toOfNat1 Real Real.instOne))\n (@Neg.neg Real Real.instNeg (@OfNat.ofNat Real (nat_lit 1) (@One.toOfNat1 Real Real.instOne)))", "formal_answer_type": "ℕ → ℝ", "outros": [{"t": "ℕ", "v": null, "name": "n"}, {"t": "Fin (2 ^ n - 1) → Set ℕ", "v": null, "name": "S"}, {"t": "Matrix (Fin (2 ^ n - 1)) (Fin (2 ^ n - 1)) ℝ", "v": null, "name": "M"}, {"t": "n ≥ 1", "v": null, "name": "npos"}, {"t": "Set.range S = (Set.Icc 1 n).powerset \\ {∅}", "v": null, "name": "hS"}, {"t": "∀ i j, M i j = if (S i ∩ S j = ∅) = True then 0 else 1", "v": null, "name": "hM"}, {"t": "M.det = answer n", "v": null, "name": "h_answer"}]} -{"informal_problem": "Determine the greatest possible value of $\\sum_{i=1}^{10} \\cos(3x_i)$ for real numbers $x_1, x_2, \\ldots, x_{10}$ satisfying $\\sum_{i=1}^{10} \\cos(x_i) = 0$.", "informal_answer": "480/49", "informal_solution": "Show that the solution is $\\frac{480}{49}$", "header": null, "intros": [], "formal_answer": "@Eq Real answer\n (@HDiv.hDiv Real Real Real (@instHDiv Real (@DivInvMonoid.toDiv Real Real.instDivInvMonoid))\n (@OfNat.ofNat Real (nat_lit 480)\n (@instOfNatAtLeastTwo Real (nat_lit 480) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 478) (instOfNatNat (nat_lit 478))))))\n (@OfNat.ofNat Real (nat_lit 49)\n (@instOfNatAtLeastTwo Real (nat_lit 49) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 47) (instOfNatNat (nat_lit 47)))))))", "formal_answer_type": "ℝ", "outros": [{"t": "IsGreatest\n {∑ i, Real.cos (3 * x i) | (x : Fin 10 → ℝ) (hx : ∑ i, Real.cos (x i) = 0)}\n answer", "v": null, "name": "h_answer"}]} -{"informal_problem": "Let $\\mathcal{P}$ be the set of vectors defined by $\\mathcal{P}=\\left\\{\\left.\\begin{pmatrix} a \\\\ b \\end{pmatrix}\\right| 0 \\leq a \\leq 2, 0 \\leq b \\leq 100,\\text{ and }a,b \\in \\mathbb{Z}\\right\\}$. Find all $\\mathbf{v} \\in \\mathcal{P}$ such that the set $\\mathcal{P} \\setminus \\{\\mathbf{v}\\}$ obtained by omitting vector $\\mathbf{v}$ from $\\mathcal{P}$ can be partitioned into two sets of equal size and equal sum.", "informal_answer": "{v : Mathlib.Vector ℤ 2 | ∃ b : ℤ, 0 ≤ b ∧ b ≤ 100 ∧ Even b ∧ v.toList = [1, b]}", "informal_solution": "Show that the answer is the collection of vectors $\\begin{pmatrix} 1 \\\\ b \\end{pmatrix}$ where $0 \\leq b \\leq 100$ and $b$ is even.", "header": null, "intros": [], "formal_answer": "@Eq (Set (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))) → Int)) answer\n (@setOf (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))) → Int)\n fun (v_1 : Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))) → Int) =>\n @Exists Int fun (b : Int) =>\n And (@LE.le Int Int.instLEInt (@OfNat.ofNat Int (nat_lit 0) (@instOfNat (nat_lit 0))) b)\n (And (@LE.le Int Int.instLEInt b (@OfNat.ofNat Int (nat_lit 100) (@instOfNat (nat_lit 100))))\n (And (@Even Int Int.instAdd b)\n (@Eq (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))) → Int) v_1\n (@Matrix.vecCons Int (Nat.succ (@OfNat.ofNat Nat (nat_lit 0) (instOfNatNat (nat_lit 0))))\n (@OfNat.ofNat Int (nat_lit 1) (@instOfNat (nat_lit 1)))\n (@Matrix.vecCons Int (@OfNat.ofNat Nat (nat_lit 0) (instOfNatNat (nat_lit 0))) b\n (@Matrix.vecEmpty Int)))))))", "formal_answer_type": "Set (Fin 2 → ℤ)", "outros": [{"t": "Finset (Fin 2 → ℤ)", "v": null, "name": "P"}, {"t": "Finset (Fin 2 → ℤ)", "v": null, "name": "Pvdiff"}, {"t": "Fin 2 → ℤ", "v": null, "name": "v"}, {"t": "P = {v' : Fin 2 → ℤ | 0 ≤ v' 0 ∧ v' 0 ≤ 2 ∧ 0 ≤ v' 1 ∧ v' 1 ≤ 100}", "v": null, "name": "hP"}, {"t": "Pvdiff = P \\ ({v} : Finset (Fin 2 → ℤ))", "v": null, "name": "hPvdiff"}, {"t": "(v ∈ P ∧ (∃ Q R : Finset (Fin 2 → ℤ),\n (Q ∪ R = Pvdiff) ∧ (Q ∩ R = ∅) ∧ (Q.card = R.card) ∧\n (∑ q in Q, q 0 = ∑ r in R, r 0) ∧ (∑ q in Q, q 1 = ∑ r in R, r 1)))\n ↔ v ∈ answer", "v": null, "name": "h_answer"}]} -{"informal_problem": "Find all positive integers $n < 10^{100}$ for which simultaneously $n$ divides $2^n$, $n-1$ divides $2^n-1$, and $n-2$ divides $2^n - 2$.", "informal_answer": "{2^2, 2^4, 2^16, 2^256}", "informal_solution": "Show that the solution is the set $\\{2^2, 2^4, 2^8, 2^16\\}$.", "header": null, "intros": [], "formal_answer": "@Eq (Set Nat) answer\n (@Insert.insert Nat (Set Nat) (@Set.instInsert Nat)\n (@HPow.hPow Nat Nat Nat (@instHPow Nat Nat (@Monoid.toNatPow Nat Nat.instMonoid))\n (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))\n (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))))\n (@Insert.insert Nat (Set Nat) (@Set.instInsert Nat)\n (@HPow.hPow Nat Nat Nat (@instHPow Nat Nat (@Monoid.toNatPow Nat Nat.instMonoid))\n (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))\n (@OfNat.ofNat Nat (nat_lit 4) (instOfNatNat (nat_lit 4))))\n (@Insert.insert Nat (Set Nat) (@Set.instInsert Nat)\n (@HPow.hPow Nat Nat Nat (@instHPow Nat Nat (@Monoid.toNatPow Nat Nat.instMonoid))\n (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))\n (@OfNat.ofNat Nat (nat_lit 16) (instOfNatNat (nat_lit 16))))\n (@Singleton.singleton Nat (Set Nat) (@Set.instSingletonSet Nat)\n (@HPow.hPow Nat Nat Nat (@instHPow Nat Nat (@Monoid.toNatPow Nat Nat.instMonoid))\n (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))\n (@OfNat.ofNat Nat (nat_lit 256) (instOfNatNat (nat_lit 256))))))))", "formal_answer_type": "Set ℕ", "outros": [{"t": "ℕ", "v": null, "name": "n"}, {"t": "0 < n", "v": null, "name": "hn"}, {"t": "(n < 10^100 ∧ ((n : ℤ) ∣ (2^n : ℤ) ∧ (n - 1 : ℤ) ∣ (2^n - 1 : ℤ) ∧ (n - 2 : ℤ) ∣ (2^n - 2 : ℤ))) ↔ n ∈ answer", "v": null, "name": "h_answer"}]} +{"informal_problem": "Find all ordered pairs $(a,b)$ of positive integers for which $\\frac{1}{a} + \\frac{1}{b} = \\frac{3}{2018}$.", "informal_answer": "{⟨673, 1358114⟩, ⟨674, 340033⟩, ⟨1009, 2018⟩, ⟨2018, 1009⟩, ⟨340033, 674⟩, ⟨1358114, 673⟩}", "informal_solution": "Show that all solutions are in the set of ${(673,1358114), (674,340033), (1009,2018), (2018,1009), (340033,674), (1358114,673)}$.", "header": "open BigOperators Real Nat Topology", "intros": [], "formal_answer": "@Eq (Set (Prod Int Int)) answer\n (@Insert.insert (Prod Int Int) (Set (Prod Int Int)) (@Set.instInsert (Prod Int Int))\n (@Prod.mk Int Int (@OfNat.ofNat Int (nat_lit 673) (@instOfNat (nat_lit 673)))\n (@OfNat.ofNat Int (nat_lit 1358114) (@instOfNat (nat_lit 1358114))))\n (@Insert.insert (Prod Int Int) (Set (Prod Int Int)) (@Set.instInsert (Prod Int Int))\n (@Prod.mk Int Int (@OfNat.ofNat Int (nat_lit 674) (@instOfNat (nat_lit 674)))\n (@OfNat.ofNat Int (nat_lit 340033) (@instOfNat (nat_lit 340033))))\n (@Insert.insert (Prod Int Int) (Set (Prod Int Int)) (@Set.instInsert (Prod Int Int))\n (@Prod.mk Int Int (@OfNat.ofNat Int (nat_lit 1009) (@instOfNat (nat_lit 1009)))\n (@OfNat.ofNat Int (nat_lit 2018) (@instOfNat (nat_lit 2018))))\n (@Insert.insert (Prod Int Int) (Set (Prod Int Int)) (@Set.instInsert (Prod Int Int))\n (@Prod.mk Int Int (@OfNat.ofNat Int (nat_lit 2018) (@instOfNat (nat_lit 2018)))\n (@OfNat.ofNat Int (nat_lit 1009) (@instOfNat (nat_lit 1009))))\n (@Insert.insert (Prod Int Int) (Set (Prod Int Int)) (@Set.instInsert (Prod Int Int))\n (@Prod.mk Int Int (@OfNat.ofNat Int (nat_lit 340033) (@instOfNat (nat_lit 340033)))\n (@OfNat.ofNat Int (nat_lit 674) (@instOfNat (nat_lit 674))))\n (@Singleton.singleton (Prod Int Int) (Set (Prod Int Int)) (@Set.instSingletonSet (Prod Int Int))\n (@Prod.mk Int Int (@OfNat.ofNat Int (nat_lit 1358114) (@instOfNat (nat_lit 1358114)))\n (@OfNat.ofNat Int (nat_lit 673) (@instOfNat (nat_lit 673))))))))))", "formal_answer_type": "Set (ℤ × ℤ)", "outros": [{"t": "ℤ", "v": null, "name": "a"}, {"t": "ℤ", "v": null, "name": "b"}, {"t": "0 < a ∧ 0 < b", "v": null, "name": "h"}, {"t": "((1 : ℚ) / a + (1 : ℚ) / b = (3 : ℚ) / 2018) ↔ (⟨a, b⟩ ∈ answer)", "v": null, "name": "h_answer"}]} +{"informal_problem": "Let \\( S_1, S_2, \\ldots, S_{2^n-1} \\) be the nonempty subsets of \\( \\{1, 2, \\ldots, n\\} \\) in some order, and let \\( M \\) be the \\( (2^n - 1) \\times (2^n - 1) \\) matrix whose \\((i, j)\\) entry is $m_{ij} = \\begin{cases} 0 & \\text{if } S_i \\cap S_j = \\emptyset; \\\\ 1 & \\text{otherwise}. \\end{cases} $ Calculate the determinant of \\( M \\).", "informal_answer": "1 if n = 1, otherwise -1", "informal_solution": "Show that the solution is 1 if n = 1, and otherwise -1.", "header": "open BigOperators Real Nat Topology", "intros": [], "formal_answer": "@Eq (Nat → Real) answer fun (n_1 : Nat) =>\n @ite Real (@Eq Nat n_1 (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1))))\n (instDecidableEqNat n_1 (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1))))\n (@OfNat.ofNat Real (nat_lit 1) (@One.toOfNat1 Real Real.instOne))\n (@Neg.neg Real Real.instNeg (@OfNat.ofNat Real (nat_lit 1) (@One.toOfNat1 Real Real.instOne)))", "formal_answer_type": "ℕ → ℝ", "outros": [{"t": "ℕ", "v": null, "name": "n"}, {"t": "Fin (2 ^ n - 1) → Set ℕ", "v": null, "name": "S"}, {"t": "Matrix (Fin (2 ^ n - 1)) (Fin (2 ^ n - 1)) ℝ", "v": null, "name": "M"}, {"t": "n ≥ 1", "v": null, "name": "npos"}, {"t": "Set.range S = (Set.Icc 1 n).powerset \\ {∅}", "v": null, "name": "hS"}, {"t": "∀ i j, M i j = if (S i ∩ S j = ∅) = True then 0 else 1", "v": null, "name": "hM"}, {"t": "M.det = answer n", "v": null, "name": "h_answer"}]} +{"informal_problem": "Determine the greatest possible value of $\\sum_{i=1}^{10} \\cos(3x_i)$ for real numbers $x_1, x_2, \\ldots, x_{10}$ satisfying $\\sum_{i=1}^{10} \\cos(x_i) = 0$.", "informal_answer": "480/49", "informal_solution": "Show that the solution is $\\frac{480}{49}$", "header": "open BigOperators Real Nat Topology", "intros": [], "formal_answer": "@Eq Real answer\n (@HDiv.hDiv Real Real Real (@instHDiv Real (@DivInvMonoid.toDiv Real Real.instDivInvMonoid))\n (@OfNat.ofNat Real (nat_lit 480)\n (@instOfNatAtLeastTwo Real (nat_lit 480) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 478) (instOfNatNat (nat_lit 478))))))\n (@OfNat.ofNat Real (nat_lit 49)\n (@instOfNatAtLeastTwo Real (nat_lit 49) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 47) (instOfNatNat (nat_lit 47)))))))", "formal_answer_type": "ℝ", "outros": [{"t": "IsGreatest\n {∑ i, Real.cos (3 * x i) | (x : Fin 10 → ℝ) (hx : ∑ i, Real.cos (x i) = 0)}\n answer", "v": null, "name": "h_answer"}]} +{"informal_problem": "Let $\\mathcal{P}$ be the set of vectors defined by $\\mathcal{P}=\\left\\{\\left.\\begin{pmatrix} a \\\\ b \\end{pmatrix}\\right| 0 \\leq a \\leq 2, 0 \\leq b \\leq 100,\\text{ and }a,b \\in \\mathbb{Z}\\right\\}$. Find all $\\mathbf{v} \\in \\mathcal{P}$ such that the set $\\mathcal{P} \\setminus \\{\\mathbf{v}\\}$ obtained by omitting vector $\\mathbf{v}$ from $\\mathcal{P}$ can be partitioned into two sets of equal size and equal sum.", "informal_answer": "{v : Mathlib.Vector ℤ 2 | ∃ b : ℤ, 0 ≤ b ∧ b ≤ 100 ∧ Even b ∧ v.toList = [1, b]}", "informal_solution": "Show that the answer is the collection of vectors $\\begin{pmatrix} 1 \\\\ b \\end{pmatrix}$ where $0 \\leq b \\leq 100$ and $b$ is even.", "header": "open BigOperators Real Nat Topology", "intros": [], "formal_answer": "@Eq (Set (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))) → Int)) answer\n (@setOf (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))) → Int)\n fun (v_1 : Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))) → Int) =>\n @Exists Int fun (b : Int) =>\n And (@LE.le Int Int.instLEInt (@OfNat.ofNat Int (nat_lit 0) (@instOfNat (nat_lit 0))) b)\n (And (@LE.le Int Int.instLEInt b (@OfNat.ofNat Int (nat_lit 100) (@instOfNat (nat_lit 100))))\n (And (@Even Int Int.instAdd b)\n (@Eq (Fin (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))) → Int) v_1\n (@Matrix.vecCons Int (Nat.succ (@OfNat.ofNat Nat (nat_lit 0) (instOfNatNat (nat_lit 0))))\n (@OfNat.ofNat Int (nat_lit 1) (@instOfNat (nat_lit 1)))\n (@Matrix.vecCons Int (@OfNat.ofNat Nat (nat_lit 0) (instOfNatNat (nat_lit 0))) b\n (@Matrix.vecEmpty Int)))))))", "formal_answer_type": "Set (Fin 2 → ℤ)", "outros": [{"t": "Finset (Fin 2 → ℤ)", "v": null, "name": "P"}, {"t": "Finset (Fin 2 → ℤ)", "v": null, "name": "Pvdiff"}, {"t": "Fin 2 → ℤ", "v": null, "name": "v"}, {"t": "P = {v' : Fin 2 → ℤ | 0 ≤ v' 0 ∧ v' 0 ≤ 2 ∧ 0 ≤ v' 1 ∧ v' 1 ≤ 100}", "v": null, "name": "hP"}, {"t": "Pvdiff = P \\ ({v} : Finset (Fin 2 → ℤ))", "v": null, "name": "hPvdiff"}, {"t": "(v ∈ P ∧ (∃ Q R : Finset (Fin 2 → ℤ),\n (Q ∪ R = Pvdiff) ∧ (Q ∩ R = ∅) ∧ (Q.card = R.card) ∧\n (∑ q in Q, q 0 = ∑ r in R, r 0) ∧ (∑ q in Q, q 1 = ∑ r in R, r 1)))\n ↔ v ∈ answer", "v": null, "name": "h_answer"}]} +{"informal_problem": "Find all positive integers $n < 10^{100}$ for which simultaneously $n$ divides $2^n$, $n-1$ divides $2^n-1$, and $n-2$ divides $2^n - 2$.", "informal_answer": "{2^2, 2^4, 2^16, 2^256}", "informal_solution": "Show that the solution is the set $\\{2^2, 2^4, 2^8, 2^16\\}$.", "header": "open BigOperators Real Nat Topology", "intros": [], "formal_answer": "@Eq (Set Nat) answer\n (@Insert.insert Nat (Set Nat) (@Set.instInsert Nat)\n (@HPow.hPow Nat Nat Nat (@instHPow Nat Nat (@Monoid.toNatPow Nat Nat.instMonoid))\n (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))\n (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))))\n (@Insert.insert Nat (Set Nat) (@Set.instInsert Nat)\n (@HPow.hPow Nat Nat Nat (@instHPow Nat Nat (@Monoid.toNatPow Nat Nat.instMonoid))\n (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))\n (@OfNat.ofNat Nat (nat_lit 4) (instOfNatNat (nat_lit 4))))\n (@Insert.insert Nat (Set Nat) (@Set.instInsert Nat)\n (@HPow.hPow Nat Nat Nat (@instHPow Nat Nat (@Monoid.toNatPow Nat Nat.instMonoid))\n (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))\n (@OfNat.ofNat Nat (nat_lit 16) (instOfNatNat (nat_lit 16))))\n (@Singleton.singleton Nat (Set Nat) (@Set.instSingletonSet Nat)\n (@HPow.hPow Nat Nat Nat (@instHPow Nat Nat (@Monoid.toNatPow Nat Nat.instMonoid))\n (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))\n (@OfNat.ofNat Nat (nat_lit 256) (instOfNatNat (nat_lit 256))))))))", "formal_answer_type": "Set ℕ", "outros": [{"t": "ℕ", "v": null, "name": "n"}, {"t": "0 < n", "v": null, "name": "hn"}, {"t": "(n < 10^100 ∧ ((n : ℤ) ∣ (2^n : ℤ) ∧ (n - 1 : ℤ) ∣ (2^n - 1 : ℤ) ∧ (n - 2 : ℤ) ∣ (2^n - 2 : ℤ))) ↔ n ∈ answer", "v": null, "name": "h_answer"}]} {"informal_problem": "Determine all possible values of the expression\n\\[\nA^3+B^3+C^3-3ABC\n\\]\nwhere $A, B$, and $C$ are nonnegative integers.", "informal_answer": "the set of nonnegative integers not congruent to 3 or 6 modulo 9", "informal_solution": "The answer is all nonnegative integers not congruent to $3$ or $6 \\pmod{9}$.", "header": "open Topology Filter", "intros": [], "formal_answer": "@Eq (Set Int) answer\n (@setOf Int fun (n : Int) =>\n And (@GE.ge Int Int.instLEInt n (@OfNat.ofNat Int (nat_lit 0) (@instOfNat (nat_lit 0))))\n (And\n (Not\n (Int.ModEq (@OfNat.ofNat Int (nat_lit 9) (@instOfNat (nat_lit 9))) n\n (@OfNat.ofNat Int (nat_lit 3) (@instOfNat (nat_lit 3)))))\n (Not\n (Int.ModEq (@OfNat.ofNat Int (nat_lit 9) (@instOfNat (nat_lit 9))) n\n (@OfNat.ofNat Int (nat_lit 6) (@instOfNat (nat_lit 6)))))))", "formal_answer_type": "Set ℤ", "outros": [{"t": "{n : ℤ | ∃ A B C : ℤ, A ≥ 0 ∧ B ≥ 0 ∧ C ≥ 0 ∧ A^3 + B^3 + C^3 - 3*A*B*C = n} = answer", "v": null, "name": "h_answer"}]} {"informal_problem": "Given real numbers $b_0, b_1, \\dots, b_{2019}$ with $b_{2019} \\neq 0$, let $z_1,z_2,\\dots,z_{2019}$ be\nthe roots in the complex plane of the polynomial\n\\[\nP(z) = \\sum_{k=0}^{2019} b_k z^k.\n\\]\nLet $\\mu = (|z_1| + \\cdots + |z_{2019}|)/2019$ be the average of the distances from $z_1,z_2,\\dots,z_{2019}$ to the origin. Determine the largest constant $M$ such that $\\mu \\geq M$ for all choices of $b_0,b_1,\\dots, b_{2019}$ that satisfy\n\\[\n1 \\leq b_0 < b_1 < b_2 < \\cdots < b_{2019} \\leq 2019.\n\\]", "informal_answer": "2019^(-(1:ℝ)/2019)", "informal_solution": "The answer is $M = 2019^{-1/2019}$.", "header": "open Topology Filter", "intros": [], "formal_answer": "@Eq Real answer\n (@HPow.hPow Real Real Real (@instHPow Real Real Real.instPow)\n (@OfNat.ofNat Real (nat_lit 2019)\n (@instOfNatAtLeastTwo Real (nat_lit 2019) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 2017) (instOfNatNat (nat_lit 2017))))))\n (@HDiv.hDiv Real Real Real (@instHDiv Real (@DivInvMonoid.toDiv Real Real.instDivInvMonoid))\n (@Neg.neg Real Real.instNeg (@OfNat.ofNat Real (nat_lit 1) (@One.toOfNat1 Real Real.instOne)))\n (@OfNat.ofNat Real (nat_lit 2019)\n (@instOfNatAtLeastTwo Real (nat_lit 2019) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 2017) (instOfNatNat (nat_lit 2017))))))))", "formal_answer_type": "ℝ", "outros": [{"t": "Polynomial ℂ → Prop", "v": null, "name": "v"}, {"t": "v = fun b => b.degree = 2019 ∧ 1 ≤ (b.coeff 0).re ∧ (b.coeff 2019).re ≤ 2019 ∧\n (∀ i : Fin 2020, (b.coeff i).im = 0) ∧ (∀ i : Fin 2019, (b.coeff i).re < (b.coeff (i + 1)).re)", "v": null, "name": "hv"}, {"t": "Polynomial ℂ → ℝ", "v": null, "name": "μ"}, {"t": "μ = fun b => (Multiset.map (fun ω : ℂ => ‖ω‖) (Polynomial.roots b)).sum/2019", "v": null, "name": "hμ"}, {"t": "IsGreatest {M : ℝ | ∀ b, v b → μ b ≥ M} answer", "v": null, "name": "h_answer"}]} {"informal_problem": "Let $f$ be a continuous real-valued function on $\\mathbb{R}^3$. Suppose that for every sphere $S$ of radius $1$, the integral of $f(x,y,z)$ over the surface of $S$ equals $0$. Must $f(x,y,z)$ be identically 0?", "informal_answer": "False", "informal_solution": "Show that the answer is no.", "header": "open MeasureTheory Metric Topology Filter", "intros": [], "formal_answer": "@Eq Prop answer False", "formal_answer_type": "Prop", "outros": [{"t": "(EuclideanSpace ℝ (Fin 3) → ℝ) → Prop", "v": null, "name": "P"}, {"t": "∀ f, P f ↔ ∀ C, ∫ x in sphere C 1, f x ∂μH[2] = 0", "v": null, "name": "P_def"}, {"t": "(∀ f, Continuous f → P f → f = 0) ↔ answer", "v": null, "name": "h_answer"}]} @@ -287,8 +287,8 @@ {"informal_problem": "Let $\\mathcal{F}$ be the set of functions $f(x,y)$ that are twice continuously differentiable for $x \\geq 1,y \\geq 1$ and that satisfy the following two equations (where subscripts denote partial derivatives):\n\\begin{gather*}\nxf_x+yf_y=xy\\ln(xy), \\\\\nx^2f_{xx}+y^2f_{yy}=xy.\n\\end{gather*}\nFor each $f \\in \\mathcal{F}$, let $m(f)=\\min_{s \\geq 1} (f(s+1,s+1)-f(s+1,s)-f(s,s+1)+f(s,s))$. Determine $m(f)$, and show that it is independent of the choice of $f$.", "informal_answer": "$2 \\ln 2 - \\frac{1}{2}$", "informal_solution": "Show that $m(f)=2\\ln 2-\\frac{1}{2}$.", "header": "open Topology Filter Set Matrix", "intros": [], "formal_answer": "@Eq Real answer\n (@HSub.hSub Real Real Real (@instHSub Real Real.instSub)\n (@HMul.hMul Real Real Real (@instHMul Real Real.instMul)\n (@OfNat.ofNat Real (nat_lit 2)\n (@instOfNatAtLeastTwo Real (nat_lit 2) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 0) (instOfNatNat (nat_lit 0))))))\n (Real.log\n (@OfNat.ofNat Real (nat_lit 2)\n (@instOfNatAtLeastTwo Real (nat_lit 2) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 0) (instOfNatNat (nat_lit 0))))))))\n (@HDiv.hDiv Real Real Real (@instHDiv Real (@DivInvMonoid.toDiv Real Real.instDivInvMonoid))\n (@OfNat.ofNat Real (nat_lit 1) (@One.toOfNat1 Real Real.instOne))\n (@OfNat.ofNat Real (nat_lit 2)\n (@instOfNatAtLeastTwo Real (nat_lit 2) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 0) (instOfNatNat (nat_lit 0))))))))", "formal_answer_type": "ℝ", "outros": [{"t": "(Fin 2 → ℝ) → ℝ", "v": null, "name": "f"}, {"t": "ℝ → ℝ → (Fin 2 → ℝ)", "v": null, "name": "vec"}, {"t": "ContDiff ℝ 2 f", "v": null, "name": "fdiff"}, {"t": "∀ x y : ℝ, (vec x y) 0 = x ∧ (vec x y 1) = y", "v": null, "name": "hvec"}, {"t": "∀ x ≥ 1, ∀ y ≥ 1, x * deriv (fun x' : ℝ => f (vec x' y)) x + y * deriv (fun y' : ℝ => f (vec x y')) y = x * y * Real.log (x * y)", "v": null, "name": "feq1"}, {"t": "∀ x ≥ 1, ∀ y ≥ 1, x ^ 2 * iteratedDeriv 2 (fun x' : ℝ => f (vec x' y)) x + y ^ 2 * iteratedDeriv 2 (fun y' : ℝ => f (vec x y')) y = x * y", "v": null, "name": "feq2"}, {"t": "sInf {f (vec (s + 1) (s + 1)) - f (vec (s + 1) s) - f (vec s (s + 1)) + f (vec s s) | s ≥ 1} = answer", "v": null, "name": "h_answer"}]} {"informal_problem": "Let $F_m$ be the $m$th Fibonacci number, defined by $F_1 = F_2 = 1$ and $F_m = F_{m-1} + F_{m-2}$ for all $m \\geq 3$. Let $p(x)$ be the polynomial of degree $1008$ such that $p(2n + 1) = F_{2n+1}$ for $n = 0,1,2,\\ldots,1008$. Find integers $j$ and $k$ such that $p(2019) = F_j - F_k$.", "informal_answer": "⟨2019, 1010⟩", "informal_solution": "Show that the solution takes the form of $(j, k) = (2019, 1010)$.", "header": "open Topology Filter Set Matrix", "intros": [], "formal_answer": "@Eq (Prod Nat Nat) answer\n (@Prod.mk Nat Nat (@OfNat.ofNat Nat (nat_lit 2019) (instOfNatNat (nat_lit 2019)))\n (@OfNat.ofNat Nat (nat_lit 1010) (instOfNatNat (nat_lit 1010))))", "formal_answer_type": "ℕ × ℕ", "outros": [{"t": "ℕ → ℤ", "v": null, "name": "F"}, {"t": "Polynomial ℝ", "v": null, "name": "P"}, {"t": "∀ x, x ≥ 1 → F (x + 2) = F (x + 1) + F x", "v": null, "name": "hF"}, {"t": "F 1 = 1 ∧ F 2 = 1", "v": null, "name": "F12"}, {"t": "Polynomial.degree P = 1008", "v": null, "name": "Pdeg"}, {"t": "∀ n : ℕ, (n ≤ 1008) → P.eval (2 * n + 1 : ℝ) = F (2 * n + 1)", "v": null, "name": "hp"}, {"t": "∀ j k : ℕ, (P.eval 2019 = F j - F k) ↔ ⟨j, k⟩ = answer", "v": null, "name": "h_answer"}]} {"informal_problem": "Let \\( \\mathbb{Z}^n \\) be the integer lattice in \\( \\mathbb{R}^n \\). Two points in \\( \\mathbb{Z}^n \\) are called neighbors if they differ by exactly 1 in one coordinate and are equal in all other coordinates. For which integers \\( n \\geq 1 \\) does there exist a set of points \\( S \\subset \\mathbb{Z}^n \\) satisfying the following two conditions? \\begin{enumerate} \\item If \\( p \\) is in \\( S \\), then none of the neighbors of \\( p \\) is in \\( S \\). \\item If \\( p \\in \\mathbb{Z}^n \\) is not in \\( S \\), then exactly one of the neighbors of \\( p \\) is in \\( S \\). \\end{enumerate}", "informal_answer": "the set of all integers n ≥ 1", "informal_solution": "Show that the statement is true for every \\(n \\geq 1\\)", "header": "open Topology Filter Set Matrix", "intros": [], "formal_answer": "@Eq (Set Nat) answer (@Set.Ici Nat Nat.instPreorder (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1))))", "formal_answer_type": "Set ℕ", "outros": [{"t": "ℕ", "v": null, "name": "n"}, {"t": "(Fin n → ℤ) → (Fin n → ℤ) → Prop", "v": null, "name": "neighbors"}, {"t": "∀ p q, neighbors p q ↔ (∃ i : Fin n, abs (p i - q i) = 1 ∧ ∀ j ≠ i, p j = q j)", "v": null, "name": "neighbors_def"}, {"t": "(1 ≤ n ∧ ∃ S : Set (Fin n → ℤ),\n (∀ p ∈ S, ∀ q, neighbors p q → q ∉ S) ∧ (∀ p ∉ S, {q ∈ S | neighbors p q}.encard = 1)) ↔ n ∈ answer", "v": null, "name": "h_answer"}]} -{"informal_problem": "Find the number of positive integers $N$ satisfying: (i) $N$ is divisible by $2020$, (ii) $N$ has at most $2020$ decimal digits, (iii) The decimal digits of $N$ are a string of consecutive ones followed by a string of consecutive zeros.", "informal_answer": "508536", "informal_solution": "Show that the solution is $508536$.", "header": null, "intros": [], "formal_answer": "@Eq Nat answer (@OfNat.ofNat Nat (nat_lit 508536) (instOfNatNat (nat_lit 508536)))", "formal_answer_type": "ℕ", "outros": [{"t": "ℕ", "v": null, "name": "N"}, {"t": "2020 ∣ N", "v": null, "name": "h_div"}, {"t": "Nat.log 10 N + 1 ≤ 2020", "v": null, "name": "h_digits"}, {"t": "∃ k l, k ≥ l ∧ N = ∑ i in Finset.range (k - l + 1), 10 ^ (i + l)", "v": null, "name": "h_pattern"}, {"t": "Set.ncard {x : ℕ | (2020 ∣ x) ∧ (Nat.log 10 x) + 1 ≤ 2020 ∧ (∃ k l, k ≥ l ∧ x = ∑ i in Finset.range (k - l + 1), 10 ^ (i + l))} = answer", "v": null, "name": "h_answer"}]} -{"informal_problem": "Let $k$ be a nonnegative integer. Evaluate\n\\[\n\\sum_{j=0}^k 2^{k-j} \\binom{k+j}{j}.\n\\]\n", "informal_answer": "4^k", "informal_solution": "Show that the answer is $4^k$.", "header": null, "intros": [], "formal_answer": "@Eq (Nat → Nat) answer fun (k_1 : Nat) =>\n @HPow.hPow Nat Nat Nat (@instHPow Nat Nat (@Monoid.toNatPow Nat Nat.instMonoid))\n (@OfNat.ofNat Nat (nat_lit 4) (instOfNatNat (nat_lit 4))) k_1", "formal_answer_type": "ℕ → ℕ", "outros": [{"t": "ℕ", "v": null, "name": "k"}, {"t": "(∑ j in Finset.Icc 0 k, 2 ^ (k - j) * Nat.choose (k + j) j) = answer k", "v": null, "name": "h_answer"}]} +{"informal_problem": "Find the number of positive integers $N$ satisfying: (i) $N$ is divisible by $2020$, (ii) $N$ has at most $2020$ decimal digits, (iii) The decimal digits of $N$ are a string of consecutive ones followed by a string of consecutive zeros.", "informal_answer": "508536", "informal_solution": "Show that the solution is $508536$.", "header": "open BigOperators Real Nat Topology", "intros": [], "formal_answer": "@Eq Nat answer (@OfNat.ofNat Nat (nat_lit 508536) (instOfNatNat (nat_lit 508536)))", "formal_answer_type": "ℕ", "outros": [{"t": "ℕ", "v": null, "name": "N"}, {"t": "2020 ∣ N", "v": null, "name": "h_div"}, {"t": "Nat.log 10 N + 1 ≤ 2020", "v": null, "name": "h_digits"}, {"t": "∃ k l, k ≥ l ∧ N = ∑ i in Finset.range (k - l + 1), 10 ^ (i + l)", "v": null, "name": "h_pattern"}, {"t": "Set.ncard {x : ℕ | (2020 ∣ x) ∧ (Nat.log 10 x) + 1 ≤ 2020 ∧ (∃ k l, k ≥ l ∧ x = ∑ i in Finset.range (k - l + 1), 10 ^ (i + l))} = answer", "v": null, "name": "h_answer"}]} +{"informal_problem": "Let $k$ be a nonnegative integer. Evaluate\n\\[\n\\sum_{j=0}^k 2^{k-j} \\binom{k+j}{j}.\n\\]\n", "informal_answer": "4^k", "informal_solution": "Show that the answer is $4^k$.", "header": "open BigOperators Real Nat Topology", "intros": [], "formal_answer": "@Eq (Nat → Nat) answer fun (k_1 : Nat) =>\n @HPow.hPow Nat Nat Nat (@instHPow Nat Nat (@Monoid.toNatPow Nat Nat.instMonoid))\n (@OfNat.ofNat Nat (nat_lit 4) (instOfNatNat (nat_lit 4))) k_1", "formal_answer_type": "ℕ → ℕ", "outros": [{"t": "ℕ", "v": null, "name": "k"}, {"t": "(∑ j in Finset.Icc 0 k, 2 ^ (k - j) * Nat.choose (k + j) j) = answer k", "v": null, "name": "h_answer"}]} {"informal_problem": "Let $a_0 = \\pi/2$, and let $a_n = \\sin(a_{n-1})$ for $n \\geq 1$. Determine whether\n\\[\n\\sum_{n=1}^\\infty a_n^2\n\\]\nconverges.", "informal_answer": "False", "informal_solution": "The series diverges.", "header": "open Filter Topology Set", "intros": [], "formal_answer": "@Eq Prop answer False", "formal_answer_type": "Prop", "outros": [{"t": "ℕ → ℝ", "v": null, "name": "a"}, {"t": "a 0 = Real.pi / 2", "v": null, "name": "ha0"}, {"t": "∀ n, a (n+1) = Real.sin (a n)", "v": null, "name": "ha"}, {"t": "(∃ L, Tendsto (fun m : ℕ => ∑ n in Finset.Icc 1 m, (a n)^2) atTop (𝓝 L)) ↔ answer", "v": null, "name": "h_answer"}]} {"informal_problem": "Let $a_n$ be the number of sets $S$ of positive integers for which\n\\[\n\\sum_{k \\in S} F_k = n,\n\\]\nwhere the Fibonacci sequence $(F_k)_{k \\geq 1}$ satisfies $F_{k+2} = F_{k+1} + F_k$ and begins $F_1 = 1, F_2 = 1, F_3 = 2, F_4 = 3$. Find the largest integer $n$ such that $a_n = 2020$.", "informal_answer": "(Nat.fib 4040) - 1", "informal_solution": "The answer is $n=F_{4040}-1$.", "header": "open Filter Topology Set", "intros": [], "formal_answer": "@Eq Int answer\n (@HSub.hSub Int Int Int (@instHSub Int Int.instSub)\n (@Nat.cast Int instNatCastInt (Nat.fib (@OfNat.ofNat Nat (nat_lit 4040) (instOfNatNat (nat_lit 4040)))))\n (@OfNat.ofNat Int (nat_lit 1) (@instOfNat (nat_lit 1))))", "formal_answer_type": "ℤ", "outros": [{"t": "ℤ → ℕ", "v": null, "name": "a"}, {"t": "a = fun n : ℤ => {S : Finset ℕ | (∀ k ∈ S, k > 0) ∧ ∑ k : S, Nat.fib k = n}.ncard", "v": null, "name": "ha"}, {"t": "IsGreatest {n | a n = 2020} answer", "v": null, "name": "h_answer"}]} {"informal_problem": "For a positive integer $N$, let $f_N$ be the function defined by\n\\[\nf_N(x) = \\sum_{n=0}^N \\frac{N+1/2-n}{(N+1)(2n+1)} \\sin((2n+1)x).\n\\]\nDetermine the smallest constant $M$ such that $f_N(x) \\leq M$ for all $N$ and all real $x$.", "informal_answer": "π/4", "informal_solution": "The smallest constant $M$ is $\\pi/4$.", "header": "open Filter Topology Set", "intros": [], "formal_answer": "@Eq Real answer\n (@HDiv.hDiv Real Real Real (@instHDiv Real (@DivInvMonoid.toDiv Real Real.instDivInvMonoid)) Real.pi\n (@OfNat.ofNat Real (nat_lit 4)\n (@instOfNatAtLeastTwo Real (nat_lit 4) Real.instNatCast\n (@instNatAtLeastTwo (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))))))", "formal_answer_type": "ℝ", "outros": [{"t": "ℤ → (ℝ → ℝ)", "v": null, "name": "f"}, {"t": "f = fun N : ℤ => fun x : ℝ =>\n ∑ n in Finset.Icc 0 N, (N + 1/2 - n)/((N + 1)*(2*n + 1)) * Real.sin ((2*n + 1)*x)", "v": null, "name": "hf"}, {"t": "answer = sSup {y | ∃ᵉ (N > 0) (x : ℝ), y = f N x}", "v": null, "name": "h_answer"}]} @@ -304,7 +304,7 @@ {"informal_problem": "Let $h(x,y)$ be a real-valued function that is twice continuously differentiable throughout $\\mathbb{R}^2$, and define $\\rho(x,y)=yh_x-xh_y$. Prove or disprove: For any positive constants $d$ and $r$ with $d>r$, there is a circle $\\mathcal{S}$ of radius $r$ whose center is a distance $d$ away from the origin such that the integral of $\\rho$ over the interior of $\\mathcal{S}$ is zero.", "informal_answer": "True", "informal_solution": "Show that the given statement is true.", "header": "open Filter Topology Metric", "intros": [], "formal_answer": "@Eq Prop answer True", "formal_answer_type": "Prop", "outros": [{"t": "((EuclideanSpace ℝ (Fin 2)) → ℝ) → (EuclideanSpace ℝ (Fin 2)) → ℝ", "v": null, "name": "rho"}, {"t": "∀ (h : (EuclideanSpace ℝ (Fin 2)) → ℝ) (p : EuclideanSpace ℝ (Fin 2)),\n rho h p = (p 1) *\n deriv (fun x' : ℝ => h ((WithLp.equiv 2 (EuclideanSpace ℝ (Fin 2))).symm ![x', p 1])) (p 0)\n - (p 0) * deriv (fun y' : ℝ => h ((WithLp.equiv 2 (EuclideanSpace ℝ (Fin 2))).symm ![p 0, y'])) (p 1)", "v": null, "name": "rho_def"}, {"t": "(∀ h : (EuclideanSpace ℝ (Fin 2)) → ℝ, ContDiff ℝ 2 h →\n (∀ d > 0, ∀ r > 0, d > r → (∃ c : EuclideanSpace ℝ (Fin 2), dist c 0 = d ∧ (∫ p in (ball c r), rho h p) = 0))) ↔ answer", "v": null, "name": "h_answer"}]} {"informal_problem": "Determine all ordered pairs of real numbers $(a,b)$ such that the line $y = ax+b$ intersects the curve $y = \\ln(1+x^2)$ in exactly one point.", "informal_answer": "{(a, b) | (a = 0 ∧ b = 0) ∨ 1 ≤ |a| ∨ (0 < |a| ∧ |a| < 1 ∧ letI rm := (1 - √(1 - a ^ 2)) / a; letI rp := (1 + √(1 - a ^ 2)) / a; (b < Real.log (1 + rm ^ 2) - a * rm ∨ b > Real.log (1 + rp ^ 2) - a * rp))}", "informal_solution": "Show that the solution is the set of ordered pairs $(a,b)$ which satisfy at least one of (1) $a = b = 0$, (2) $|a| \\geq 1$, and (3) $0 < |a| < 1$ and $b < \\log(1 + r_{-}^2) - ar_{-}$ or $b > \\log(1 + r_{+}^2) - ar_{+}$ where $r_{\\pm} = \\frac{1 \\pm \\sqrt{1 - a^2}}{a}$.", "header": "open Polynomial", "intros": [], "formal_answer": "@Eq (Set (Prod Real Real)) answer\n (@setOf (Prod Real Real) fun (x : Prod Real Real) =>\n _example.match_1 (fun (x_1 : Prod Real Real) => Prop) x fun (a b : Real) =>\n Or\n (And (@Eq Real a (@OfNat.ofNat Real (nat_lit 0) (@Zero.toOfNat0 Real Real.instZero)))\n (@Eq Real b (@OfNat.ofNat Real (nat_lit 0) (@Zero.toOfNat0 Real Real.instZero))))\n (Or\n (@LE.le Real Real.instLE (@OfNat.ofNat Real (nat_lit 1) (@One.toOfNat1 Real Real.instOne))\n (@abs Real Real.lattice Real.instAddGroup a))\n (And\n (@LT.lt Real Real.instLT (@OfNat.ofNat Real (nat_lit 0) (@Zero.toOfNat0 Real Real.instZero))\n (@abs Real Real.lattice Real.instAddGroup a))\n (And\n (@LT.lt Real Real.instLT (@abs Real Real.lattice Real.instAddGroup a)\n (@OfNat.ofNat Real (nat_lit 1) (@One.toOfNat1 Real Real.instOne)))\n (Or\n (@LT.lt Real Real.instLT b\n (@HSub.hSub Real Real Real (@instHSub Real Real.instSub)\n (Real.log\n (@HAdd.hAdd Real Real Real (@instHAdd Real Real.instAdd)\n (@OfNat.ofNat Real (nat_lit 1) (@One.toOfNat1 Real Real.instOne))\n (@HPow.hPow Real Nat Real (@instHPow Real Nat (@Monoid.toNatPow Real Real.instMonoid))\n (@HDiv.hDiv Real Real Real (@instHDiv Real (@DivInvMonoid.toDiv Real Real.instDivInvMonoid))\n (@HSub.hSub Real Real Real (@instHSub Real Real.instSub)\n (@OfNat.ofNat Real (nat_lit 1) (@One.toOfNat1 Real Real.instOne))\n (Real.sqrt\n (@HSub.hSub Real Real Real (@instHSub Real Real.instSub)\n (@OfNat.ofNat Real (nat_lit 1) (@One.toOfNat1 Real Real.instOne))\n (@HPow.hPow Real Nat Real (@instHPow Real Nat (@Monoid.toNatPow Real Real.instMonoid))\n a (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))))))\n a)\n (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))))))\n (@HMul.hMul Real Real Real (@instHMul Real Real.instMul) a\n (@HDiv.hDiv Real Real Real (@instHDiv Real (@DivInvMonoid.toDiv Real Real.instDivInvMonoid))\n (@HSub.hSub Real Real Real (@instHSub Real Real.instSub)\n (@OfNat.ofNat Real (nat_lit 1) (@One.toOfNat1 Real Real.instOne))\n (Real.sqrt\n (@HSub.hSub Real Real Real (@instHSub Real Real.instSub)\n (@OfNat.ofNat Real (nat_lit 1) (@One.toOfNat1 Real Real.instOne))\n (@HPow.hPow Real Nat Real (@instHPow Real Nat (@Monoid.toNatPow Real Real.instMonoid)) a\n (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))))))\n a))))\n (@GT.gt Real Real.instLT b\n (@HSub.hSub Real Real Real (@instHSub Real Real.instSub)\n (Real.log\n (@HAdd.hAdd Real Real Real (@instHAdd Real Real.instAdd)\n (@OfNat.ofNat Real (nat_lit 1) (@One.toOfNat1 Real Real.instOne))\n (@HPow.hPow Real Nat Real (@instHPow Real Nat (@Monoid.toNatPow Real Real.instMonoid))\n (@HDiv.hDiv Real Real Real (@instHDiv Real (@DivInvMonoid.toDiv Real Real.instDivInvMonoid))\n (@HAdd.hAdd Real Real Real (@instHAdd Real Real.instAdd)\n (@OfNat.ofNat Real (nat_lit 1) (@One.toOfNat1 Real Real.instOne))\n (Real.sqrt\n (@HSub.hSub Real Real Real (@instHSub Real Real.instSub)\n (@OfNat.ofNat Real (nat_lit 1) (@One.toOfNat1 Real Real.instOne))\n (@HPow.hPow Real Nat Real (@instHPow Real Nat (@Monoid.toNatPow Real Real.instMonoid))\n a (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))))))\n a)\n (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))))))\n (@HMul.hMul Real Real Real (@instHMul Real Real.instMul) a\n (@HDiv.hDiv Real Real Real (@instHDiv Real (@DivInvMonoid.toDiv Real Real.instDivInvMonoid))\n (@HAdd.hAdd Real Real Real (@instHAdd Real Real.instAdd)\n (@OfNat.ofNat Real (nat_lit 1) (@One.toOfNat1 Real Real.instOne))\n (Real.sqrt\n (@HSub.hSub Real Real Real (@instHSub Real Real.instSub)\n (@OfNat.ofNat Real (nat_lit 1) (@One.toOfNat1 Real Real.instOne))\n (@HPow.hPow Real Nat Real (@instHPow Real Nat (@Monoid.toNatPow Real Real.instMonoid)) a\n (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))))))\n a)))))))))", "formal_answer_type": "Set (ℝ × ℝ)", "outros": [{"t": "{a : (ℝ × ℝ) | ∃! x : ℝ, a.1 * x + a.2 = Real.log (1 + x^2)} = answer", "v": null, "name": "h_answer"}]} {"informal_problem": "Let $n$ be an integer with $n \\geq 2$. Over all real polynomials $p(x)$ of degree $n$, what is the largest possible number of negative coefficients of $p(x)^2$?", "informal_answer": "$2n - 2$", "informal_solution": "Show that the solution is $2n - 2$.", "header": "open Polynomial", "intros": [], "formal_answer": "@Eq (Nat → Nat) answer fun (n_1 : Nat) =>\n @HSub.hSub Nat Nat Nat (@instHSub Nat instSubNat)\n (@HMul.hMul Nat Nat Nat (@instHMul Nat instMulNat) (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2))) n_1)\n (@OfNat.ofNat Nat (nat_lit 2) (instOfNatNat (nat_lit 2)))", "formal_answer_type": "ℕ → ℕ", "outros": [{"t": "ℕ", "v": null, "name": "n"}, {"t": "n ≥ 2", "v": null, "name": "hn"}, {"t": "Set ℝ[X]", "v": null, "name": "S"}, {"t": "S = {P | natDegree P = n}", "v": null, "name": "hS"}, {"t": "ℝ[X] → ℕ", "v": null, "name": "negs"}, {"t": "∀ P : ℝ[X], negs P = ∑ i in Finset.range (P.natDegree + 1), if P.coeff i < 0 then 1 else 0", "v": null, "name": "hnegs"}, {"t": "sSup {negs (P^2) | P ∈ S} = answer n", "v": null, "name": "h_answer"}]} -{"informal_problem": "Alice and Bob play a game on a board consisting of one row of 2022 consecutive squares. They take turns placing tiles that cover two adjacent squares, with Alice going first. By rule, a tile must not cover a square that is already covered by another tile. The game ends when no tile can be placed according to this rule. Alice's goal is to maximize the number of uncovered squares when the game ends; Bob's goal is to minimize it. What is the greatest number of uncovered squares that Alice can ensure at the end of the game, no matter how Bob plays?", "informal_answer": "290", "informal_solution": "Show that the solution is 290.", "header": null, "intros": [], "formal_answer": "@Eq Nat answer (@OfNat.ofNat Nat (nat_lit 290) (instOfNatNat (nat_lit 290)))", "formal_answer_type": "ℕ", "outros": [{"t": "Set (Fin 2022) → Set (Fin 2022) → Prop", "v": null, "name": "IsValidMove"}, {"t": "∀ x y, IsValidMove x y ↔\n (x = y ∧ ∀ i < 2021, i ∉ x → i + 1 ∈ x) ∨\n ∃ i < 2021, i ∉ x ∧ i + 1 ∉ x ∧ y = x ∪ {i, i + 1}", "v": null, "name": "IsValidMove_def"}, {"t": "List (Set (Fin 2022)) → Prop", "v": null, "name": "IsValidGame"}, {"t": "∀ g, IsValidGame g ↔ (∃ gt, g = ∅ :: gt) ∧ g.Chain' IsValidMove", "v": null, "name": "IsValidGame_def"}, {"t": "List (Set (Fin 2022)) → (Set (Fin 2022) → Set (Fin 2022)) → Prop", "v": null, "name": "ConformsToStrategy"}, {"t": "∀ g s, ConformsToStrategy g s ↔\n ∀ (i) (h : i + 1 < g.length), Even i → g[i + 1] = s g[i]", "v": null, "name": "ConformsToStrategy_def"}, {"t": "IsGreatest\n {n | ∃ s, (∀ x, IsValidMove x (s x)) ∧ ∀ g,\n IsValidGame g → ConformsToStrategy g s → ∃ gh x, g = gh ++ [x] ∧ n ≤ xᶜ.ncard}\n answer", "v": null, "name": "h_answer"}]} +{"informal_problem": "Alice and Bob play a game on a board consisting of one row of 2022 consecutive squares. They take turns placing tiles that cover two adjacent squares, with Alice going first. By rule, a tile must not cover a square that is already covered by another tile. The game ends when no tile can be placed according to this rule. Alice's goal is to maximize the number of uncovered squares when the game ends; Bob's goal is to minimize it. What is the greatest number of uncovered squares that Alice can ensure at the end of the game, no matter how Bob plays?", "informal_answer": "290", "informal_solution": "Show that the solution is 290.", "header": "open BigOperators Real Nat Topology", "intros": [], "formal_answer": "@Eq Nat answer (@OfNat.ofNat Nat (nat_lit 290) (instOfNatNat (nat_lit 290)))", "formal_answer_type": "ℕ", "outros": [{"t": "Set (Fin 2022) → Set (Fin 2022) → Prop", "v": null, "name": "IsValidMove"}, {"t": "∀ x y, IsValidMove x y ↔\n (x = y ∧ ∀ i < 2021, i ∉ x → i + 1 ∈ x) ∨\n ∃ i < 2021, i ∉ x ∧ i + 1 ∉ x ∧ y = x ∪ {i, i + 1}", "v": null, "name": "IsValidMove_def"}, {"t": "List (Set (Fin 2022)) → Prop", "v": null, "name": "IsValidGame"}, {"t": "∀ g, IsValidGame g ↔ (∃ gt, g = ∅ :: gt) ∧ g.Chain' IsValidMove", "v": null, "name": "IsValidGame_def"}, {"t": "List (Set (Fin 2022)) → (Set (Fin 2022) → Set (Fin 2022)) → Prop", "v": null, "name": "ConformsToStrategy"}, {"t": "∀ g s, ConformsToStrategy g s ↔\n ∀ (i) (h : i + 1 < g.length), Even i → g[i + 1] = s g[i]", "v": null, "name": "ConformsToStrategy_def"}, {"t": "IsGreatest\n {n | ∃ s, (∀ x, IsValidMove x (s x)) ∧ ∀ g,\n IsValidGame g → ConformsToStrategy g s → ∃ gh x, g = gh ++ [x] ∧ n ≤ xᶜ.ncard}\n answer", "v": null, "name": "h_answer"}]} {"informal_problem": "Let $n$ be a positive integer. Determine, in terms of $n$, the largest integer $m$ with the following property: There exist real numbers $x_1,\\dots,x_{2n}$ with $-1 n)", "informal_solution": "Show that the largest such $m$ is $n$.", "header": "open Set", "intros": [], "formal_answer": "@Eq (Nat → Nat) answer fun (n_1 : Nat) => n_1", "formal_answer_type": "ℕ → ℕ", "outros": [{"t": "ℕ", "v": null, "name": "n"}, {"t": "0 < n", "v": null, "name": "hn"}, {"t": "IsGreatest\n {m : ℕ | ∃ x : ℕ → ℝ,\n StrictMono x ∧ -1 < x 1 ∧ x (2 * n) < 1 ∧\n ∀ k ∈ Icc 1 m, ∑ i in Icc 1 n, ((x (2 * i) : ℝ) ^ (2 * k - 1) - (x (2 * i - 1)) ^ (2 * k - 1)) = 1}\n (answer n)", "v": null, "name": "h_answer"}]} {"informal_problem": "Let $\\times$ represent the cross product in $\\mathbb{R}^3$. For what positive integers $n$ does there exist a set $S \\subset \\mathbb{R}^3$ with exactly $n$ elements such that $S=\\{v \\times w:v,w \\in S\\}$?", "informal_answer": "{1, 7}", "informal_solution": "Show that the possible values of $n$ are $1$ and $7$.", "header": "open Polynomial", "intros": [], "formal_answer": "@Eq (Set Nat) answer\n (@Insert.insert Nat (Set Nat) (@Set.instInsert Nat) (@OfNat.ofNat Nat (nat_lit 1) (instOfNatNat (nat_lit 1)))\n (@Singleton.singleton Nat (Set Nat) (@Set.instSingletonSet Nat)\n (@OfNat.ofNat Nat (nat_lit 7) (instOfNatNat (nat_lit 7)))))", "formal_answer_type": "Set ℕ", "outros": [{"t": "ℕ", "v": null, "name": "n"}, {"t": "Finset (Fin 3 → ℝ) → Prop", "v": null, "name": "P"}, {"t": "∀ S : Finset (Fin 3 → ℝ), P S ↔ (S = {u : Fin 3 → ℝ | ∃ v w : S, u = crossProduct v w})", "v": null, "name": "P_def"}, {"t": "(0 < n ∧ ∃ S : Finset (Fin 3 → ℝ), S.card = n ∧ P S) ↔ n ∈ answer", "v": null, "name": "h_answer"}]} {"informal_problem": "Assign to each positive real number a color, either red or blue. Let $D$ be the set of all distances $d>0$ such that there are two points of the same color at distance $d$ apart. Recolor the positive reals so that the numbers in $D$ are red and the numbers not in $D$ are blue. If we iterate this recoloring process, will we always end up with all the numbers red after a finite number of steps?", "informal_answer": "True", "informal_solution": "Show that the answer is yes.", "header": "open Polynomial", "intros": [], "formal_answer": "@Eq Prop answer True", "formal_answer_type": "Prop", "outros": [{"t": "(ℝ → Prop) → (ℝ → Prop)", "v": null, "name": "recolor"}, {"t": "∀ isred d, recolor isred d ↔ ∃ p q : ℝ, p > 0 ∧ q > 0 ∧ p < q ∧ isred p = isred q ∧ q - p = d", "v": null, "name": "hrecolor"}, {"t": "(∀ isred, (∃ k, ∀ p > 0, (recolor^[k] isred) p)) ↔ answer", "v": null, "name": "h_answer"}]}