Experimento numérico
El siguiente experimento numérico arroja, como veremos más adelante, los supuestos correctos para obtener un buen candidato al óptimo. La convexidad nos ayudará a demostrar que este candidato es efectivamente el óptimo.
Trazamos el conjunto activo del óptimo de una discretización:
Este es el resultado del siguiente código: activeset[k_] := Module[{h, constraints, vars, objective, optresult, result, pts}, h = 1/(2 k - 2); constraints = Flatten[Table[ Table[x[i] x[j] >= (2 k - i - j) h, {j, i, k}], {i, 1, k}]]; constraints = Join[constraints, Table[x[i] >= 0, {i, 1, k}]]; vars = Table[x[i], {i, 1, k}]; objective = Sum[x[i], {i, 1, k}] + Sum[x[i], {i, 2, k - 1}]; optresult = FindMinimum[{objective, constraints}, vars, Method -> "InteriorPoint"]; result = Table[{(i - 1) h, x[i]}, {i, 1, k}] /. optresult[[2]]; pts = Select[Flatten[Table[{i, j}, {i, 1, k}, {j, 1, k}], 1], Abs[x[#[[1]]] x[#[[2]]] - (2 k - #[[1]] - #[[2]]) h] < 10^(-5) /. optresult[[2]] &]; ListPlot[(pts - 1)/(k - 1), AspectRatio -> 1, PlotStyle -> Red, PlotTheme -> "Detailed"] ]; activeset[71]
Solución completa
Set $S:=\{(x,y) \in [0,1]^2 : x+y \leq 1\}$ . Definimos los mapas \begin{alignat*}{2} &J : C[0,1] \rightarrow \mathbb{R},\quad &&J(u) := \int_0^1 \! \exp(u(x)) \, \mathrm{d}x, \\[1em] &I : C[0,1] \rightarrow C(S),\quad &&I(u)(x,y) := u(x)+u(y)-\log(2-x-y). \end{alignat*} Estudiaremos los problemas de optimización \begin{align} & \text{minimize} && J(u) \nonumber\\ & \text{subject to} && I(u) \geq 0, \tag{1} \\[1em] \text{and}\nonumber \\[1em] & \text{minimize} && \int_0^1 \! f(x) \, \mathrm{d}x \nonumber\\ & \text{subject to} && f \in C[0,1], \tag{2}\\ &&& f \geq 0, \nonumber\\ &&& f(x)f(y) \geq |x-y| \text{ for all } x,y \in [0,1]. \nonumber \end{align}
Lo demostraremos:
La solución única $\bar{u}$ de $(1)$ viene dada por \begin{align*} \exp(\bar{u}(x)) &= \sqrt{2 \left(1+\sqrt{2}\right)}-\sqrt{2 x+\sqrt{2}-1}, \\[1em] J(\bar{u}) &= \frac{2}{3}\sqrt{1+\sqrt{2}}. \end{align*} La solución única $\bar{f}$ de $(2)$ viene dada por \begin{align*} \bar{f}(x) &= \begin{cases} \dfrac{\exp(\bar{u}(2x))}{\sqrt{2}}&\text{if}\quad 0 \leq x \leq \frac{1}{2},\\ \dfrac{\exp(\bar{u}(2(1-x)))}{\sqrt{2}}&\text{if}\quad \frac{1}{2} < x \leq 1, \end{cases} \N-[1em] \N-int_0^1 \N-. \bar{f}(x) \mathrm{d}x &= \frac{1}{3} \sqrt{2 \left(1+\sqrt{2}\right)}\quad (\approx 0.732456) \fin{align*} donde $\bar{u}$ es la única solución de $(1)$ .
Teorema 1 (Teorema de Kuhn-Tucker generalizado).
Dejemos que $X$ sea un espacio normado y $Y$ un espacio normado que tiene un cono positivo $P$ . Supongamos que $P$ contiene un punto interior.
Dejemos que $J$ sea una función de valor real diferenciable de Fréchet sobre $X$ y $I$ una cartografía diferenciable de Fréchet desde $X$ en $Y$ . Supongamos que $\bar{u}$ minimiza $J$ con sujeción a $I(\bar{u}) \geq 0$ y que $\bar{u}$ es un punto regular de la desigualdad $I(\bar{u}) \geq 0$ es decir, existe un $h \in X$ tal que $I(\bar{u}) + I'(\bar{u})(h) > 0$ . Entonces hay un funcional positivo $\psi \in Y^*$ tal que \begin{align} J'(\bar{u}) &= \psi \circ I'(\bar{u}), \tag{3} \\\psi(I(\bar{u})) &= 0. \tag{4} \end{align}
Prueba . Véase [Luenberger, David G, Optimization by vector space methods, Wiley, Nueva York, 1969, p. 249]. $$\tag*{$ \N - Caja $}$$
Nota: La siguiente suposición (iii) se inspira en nuestra experimento numérico .
Reclamación 1. Si
(i) $\bar{u}$ es la solución de $(1)$
(ii) $\bar{u} \in C[0,1]$
(iii) existe $g \in C^1[0,1]$ tal que $$A:=\{(x,g(x)) : x \in [0,1]\} = \left\{(x,y) \in S : I(\bar{u})(x,y) = 0\right\},$$
entonces $g$ es una involución y $$\exp(\bar{u}(x)) = -g'(x)\exp(\bar{u}(g(x)))$$ para todos $x \in [0,1]$ .
Prueba. Por (iii) tenemos $I(\bar{u})(x,g(x)) = 0$ para todos $x \in [0,1]$ .
Desde $I(\bar{u})(x,y) = I(\bar{u})(y,x)$ para todos $x,y \in [0,1]$ tenemos $I(\bar{u})(g(x),x) = 0$ y por lo tanto $g(g(x)) = x$ por (iii) para todo $x \in [0,1]$ . Por lo tanto, $g$ es una involución.
Ahora aplicaremos el Teorema 1. El punto $\bar{u}$ es regular, ya que $I'(\bar{u})(\mathbf{1}_{[0,1]}) = 2\cdot \mathbf{1}_S.$
Por lo tanto, existe un funcional positivo $\psi \in C(S)^*$ tal que $(3)$ y $(4)$ se satisfacen. Dado que $S$ es compacto, existe una única medida regular de Borel $\nu$ en $\mathcal{B}(S)$ por el teorema de representación de Riesz-Markov-Kakutani tal que $$\psi(v) = \int_S v(x,y) \, \mathrm{d}\nu(x,y)$$ para todos $v \in C(S)$ . Definimos una medida sobre $\mathcal{B}(S)$ al establecer $$\mu(E) := \lambda\left(\{x \in [0,1] : (x,g(x)) \in E\}\right)$$ para todos $E \in \mathcal{B}(S)$ , donde $\lambda$ es la medida de Lebesgue en $[0,1]$ . Demostraremos que $\nu \ll \mu$ es decir, que $\nu$ es absolutamente continua con respecto a $\mu$ . Sea $N \in \mathcal{B}(S)$ tal que $\mu(N)=0$ . Por $(4)$ tenemos $\psi(I(\bar{u})) = 0$ . Por lo tanto, $$\int_{S} I(\bar{u})(x,y) \, \mathrm{d}\nu(x,y) = 0,$$ y como $I(\bar{u}) \geq 0$ tenemos $\nu(S\setminus A)=0$ y $\nu(N \cap (S\setminus A))=0$ . Por $(3)$ tenemos $$\int_0^1 \exp(\bar{u}(x)) h(x) \, \mathrm{d}x = \int_S h(x) + h(y) \, \mathrm{d}\nu(x,y)$$ para todos $h \in C[0,1]$ . Establecer $N' = \{x \in [0,1] : (x,g(x)) \in N\}$ . Por definición de $\mu$ tenemos $\lambda(N') = 0$ . Sea $\epsilon > 0$ . Entonces existe $\bar{h} \in C[0,1]$ tal que $\bar{h}(x) = 1$ para todos $x \in N'$ , $\bar{h}\geq 0$ y $\int_0^1 \exp(\bar{u}(x)) \bar{h}(x) \, \mathrm{d}x<\epsilon$ . Ahora tenemos \begin{align*} \nu(N \cap A) &= \int_S \mathbf{1}_{N \cap A}(x,y) \, \mathrm{d}\nu(x,y) \\[1em] &= \int_S \mathbf{1}_{N'}(x) \, \mathrm{d}\nu(x,y) \\[1em] &\leq \int_S \bar{h}(x) + \bar{h}(y) \, \mathrm{d}\nu(x,y) \\[1em] &= \int_0^1 \exp(\bar{u}(x)) \bar{h}(x) \, \mathrm{d}x<\epsilon. \end{align*} Por lo tanto, $\nu(N \cap A) = 0$ Por lo tanto $\nu(N) = 0$ y $\nu \ll \mu$ . Por el teorema de Radon-Nikodym existe una función medible $w : S \rightarrow [0,\infty)$ tal que $$\psi(v) = \int_S v(x,y)\, \mathrm{d}\nu(x,y) = \int_S v(x,y)\,w(x,y) \, \mathrm{d}\mu(x,y)$$ para todos $v \in C(S)$ . Desde $\mu$ es la medida pushforward bajo $x \mapsto (x,g(x))$ tenemos $$\psi(v) = \int_0^1 v(x,g(x))\,w(x,g(x)) \, \mathrm{d}x$$ para todos $v \in C(S)$ . Por $(4)$ ahora tenemos $$\int_0^1 \exp(\bar{u}(x)) h(x) \, \mathrm{d}x = \int_0^1 (h(x) + h(g(x)))\,w(x,g(x)) \, \mathrm{d}x$$ para todos $h \in C[0,1]$ . Desde $g$ es un $C^1$ -involución en $[0,1]$ podemos sustituir $g(x)$ para $x$ en $\int_0^1 h(g(x))\,w(x,g(x)) \, \mathrm{d}x$ . Obtenemos $$\int_0^1 \exp(\bar{u}(x)) h(x) \, \mathrm{d}x = \int_0^1 h(x) (w(x,g(x))-w(g(x),x)g'(x)) \, \mathrm{d}x$$ para todos $h \in C[0,1]$ . Por lo tanto, $$\exp(\bar{u}(x)) = w(x,g(x))-w(g(x),x)g'(x)$$ para casi todos los $x \in [0,1]$ . Desde $g$ es una involución, tenemos \begin{align*} \exp(\bar{u}(g(x))) &= w(g(x),g(g(x)))-w(g(g(x)),g(x))g'(g(x)) \\[1em] &= w(g(x),x)-w(x,g(x)) \frac{1}{g'(x)} \\[1em] &= -\frac{1}{g'(x)}(w(x,g(x))-w(g(x),x)g'(x)) \\[1em] &= -\frac{1}{g'(x)}\exp(\bar{u}(x)) \end{align*} para casi todos los $x \in [0,1]$ . Desde $g$ , $g'$ y $\bar{u}$ son continuos tenemos \begin{align} \exp(\bar{u}(x)) = -g'(x)\exp(\bar{u}(g(x))) \tag{5} \end{align} para todos $x \in [0,1]$ . $$\tag*{$ \N - Caja $}$$
Reclamación 2. Si
(i) $\bar{u}$ es la solución de $(1)$
(ii) $\bar{u} \in C^1[0,1]$
(iii) existe $g \in C^2[0,1]$ tal que $$\{(x,g(x)) : x \in [0,1]\} = \left\{(x,y) \in S : I(\bar{u})(x,y) = 0\right\}$$ y $$\{(x,g(x)) : x \in (0,1)\} \subseteq \operatorname{int}(S),$$ entonces $$g(x) = 1+\sqrt{2}+x-\sqrt{4 \left(1+\sqrt{2}\right) x+2},$$ y $$\exp(\bar{u}(x)) = \sqrt{2 \left(1+\sqrt{2}\right)}-\sqrt{2 x+\sqrt{2}-1}.$$
Prueba. Dejemos que $x \in (0,1)$ . Tenemos $I(\bar{u})(x,g(x)) = 0$ . Desde $I(\bar{u}) \geq 0$ tenemos que $(x,g(x))$ es un punto mínimo de $I(\bar{u})$ . Desde $I(\bar{u})$ es un $C^1$ -función por $(ii)$ tenemos que $I(\bar{u})'(x,g(x)) = 0$ . Por lo tanto, \begin{align} \bar{u}'(x) = -\frac{1}{2-x-g(x)}. \tag{6} \end{align} Según la afirmación 1, tenemos $(5)$ . Veremos que $(5)$ y $(6)$ determinar $g$ y $\bar{u}$ de forma única. Los siguientes cálculos son válidos para todos los $x \in [0,1]$ .
Desde $I(\bar{u})(x,g(x)) = 0$ tenemos \begin{align*} \bar{u}(g(x)) = \log(2-x-g(x)) - \bar{u}(x), \end{align*} y por lo tanto con $(5)$ tenemos \begin{align} \bar{u}(x) = \frac{1}{2}\left(\log(-g'(x)) + \log(2-x-g(x))\right), \tag{7} \end{align} y por lo tanto \begin{align} \bar{u}'(x) = \frac{1}{2}\left(\frac{g''(x)}{g'(x)} + \frac{-1-g'(x)}{2-x-g(x)}\right). \tag{8} \end{align} Poniendo $(6)$ y $(8)$ en conjunto da como resultado $$g''(x)(2-x-g(x)) -g'(x)^2 +g'(x) = 0.$$ Por lo tanto, \begin{align} g'(x)(2-x-g(x)) +2g(x) = a. \tag{9} \end{align} para algunos $a \in \mathbb{R}$ . En particular, tenemos \begin{align} g'(0)(2-g(0)) +2g(0)= g'(1)(1-g(1)) +2g(1). \tag{10} \end{align} Desde $g$ es una involución tenemos $g(0) = 1$ , $g(1) = 0$ , $1 = g'(g(0))g'(0)= g'(1)g'(0)$ y $g' < 0$ . Lo ponemos en $(10)$ y obtener $a = 1-\sqrt{2}$ . Así, \begin{align} g'(x) = \frac{1-\sqrt{2}-2g(x)}{2-x-g(x)}. \tag{11} \end{align} Ahora sustituimos $x$ con $g(x)$ en $(9)$ y luego usar $g'(g(x)) = \frac{1}{g'(x)}$ . Obtenemos \begin{align} g'(x) = \frac{2-x-g(x)}{1-\sqrt{2}-2x}. \tag{12} \end{align} Poniendo $(11)$ y $(12)$ se obtiene una ecuación cuadrática para $g(x)$ . Sólo la solución \begin{align} g(x) = 1+\sqrt{2}+x-\sqrt{4 \left(1+\sqrt{2}\right) x+2} \tag{13} \end{align} satisface $g(0)=1$ . También tenemos \begin{align*} \exp(\bar{u}(g(x)))^2 &\underset{\hphantom{(12)}}{=} \frac{2-x-g(x)}{\exp(\bar{u}(x))}\exp(\bar{u}(g(x))) \\[1em] &\underset{(5)\hphantom{0}}{=} -\frac{2-x-g(x)}{g'(x)} \\[1em] &\underset{(12)}{=} 2 x+\sqrt{2}-1, \end{align*} y por lo tanto \begin{align*} \exp(\bar{u}(x)) &\underset{\hphantom{(12)}}{=} \frac{2-x-g(x)}{\sqrt{2 x+\sqrt{2}-1}} \\[1em] &\underset{(13)}{=} \frac{1-2x-\sqrt{2}+\sqrt{4 \left(1+\sqrt{2}\right) x+2}}{\sqrt{2 x+\sqrt{2}-1}} \\[1em] &\underset{\hphantom{(12)}}{=} -\sqrt{2 x+\sqrt{2}-1}+\frac{\sqrt{4 \left(1+\sqrt{2}\right) x+2}}{\sqrt{2 x+\sqrt{2}-1}} \\[1em] &\underset{\hphantom{(12)}}{=} -\sqrt{2 x+\sqrt{2}-1}+\sqrt{2 \left(1+\sqrt{2}\right)}. \end{align*} $$\tag*{$ \N - Caja $}$$
Definimos \begin{align*} \bar{u} : [0,1] \rightarrow \mathbb{R}, \quad \bar{u}(x) &:= \log\left(\sqrt{2 \left(1+\sqrt{2}\right)}-\sqrt{2 x+\sqrt{2}-1}\right), \\[1em]g : [0,1] \rightarrow [0,1], \quad g(x) &:= 1+\sqrt{2}+x-\sqrt{4 \left(1+\sqrt{2}\right) x+2}. \end{align*}
Reclamación 3. $g$ es una involución. Tenemos \begin{align*} I(\bar{u})(x,g(x)) &= 0, \\[0.5em] \exp(\bar{u}(x) + \bar{u}(y)) &\geq 2-x-y \end{align*} para todos $x,y \in [0,1]^2$ y por lo tanto $I(\bar{u}) \geq 0$ .
Prueba. Resolvemos $g(x)=y$ para $x$ y ver que $x=g(y)$ . Así, $g(g(x))=x$ y $g$ es una involución en $[0,1]$ . Definimos $$F : [0,1]^2 \rightarrow \mathbb{R}, \quad F(x,y) := \exp(\bar{u}(x)+\bar{u}(y)) - (2-x-y).$$ Para todos $x \in [0,1]$ tenemos $x + g(x) \leq 1$ y por lo tanto $(x,g(x)) \in S$ . Vemos que $\exp(\bar{u}(x))^2 = 2 g(x)+\sqrt{2}-1$ Por lo tanto $\exp(\bar{u}(g(x)))^2 = 2 x+\sqrt{2}-1$ y poniendo esto en $F(x,g(x))$ obtenemos $F(x,g(x)) = 0$ y $I(\bar{u})(x,g(x)) = 0$ . Para todos los $y \in [0,1]$ tenemos
\begin{align*} (\partial_{y y} F)(x,y) &= \exp(\bar{u}(x))\, \partial_{y y} \exp(\bar{u}(y)) \\ &= \exp(\bar{u}(x))\, \frac{1}{\left(2 y+\sqrt{2}-1\right)^{3/2}} \\ &> 0. \end{align*} Por lo tanto, $y \mapsto F(x,y)$ es convexo y como $(\partial_y F)(x,g(x))= 0$ tenemos que $(x,g(x))$ es el minimizador global de $y \mapsto F(x,y)$ . Desde $F(x,g(x)) = 0$ tenemos $F \geq 0$ y por lo tanto $I(\bar{u}) \geq 0$ . $$\tag*{$ \N - Caja $}$$
Reclamación 4. $\bar{u}$ es la única solución de $(1)$ .
Prueba. Definimos \begin{alignat*}{2} &w : [0,1] \rightarrow [0,\infty), \quad &&w(x) := \frac{\exp(\bar{u}(x))}{1-g'(x)}, \\[1em] &\psi : C(S) \rightarrow \mathbb{R}, \quad &&\psi(v) := \int_0^1 v(x,g(x)) \, w(x) \, \mathrm{d}x, \\[1em] &L : C[0,1] \rightarrow \mathbb{R}, \quad &&L(u) := J(u) - \psi(I(u)). \end{alignat*} $w$ está bien definido ya que $g$ al ser una involución y no la identidad implica $g'\leq0$ .
$\psi$ está bien definido ya que $(x,g(x)) \in S$ para todos $x \in [0,1]$ . Tenemos $w(g(x))=w(x)$ y por lo tanto \begin{align*} L'(\bar{u})(h) &= J'(\bar{u})(h) - \psi'(I(\bar{u}))(I'(h)) \\[1em] &= J'(\bar{u})(h) - \psi(I'(h)) \\[1em] &= \int_0^1 \exp(\bar{u}(x))\, h(x) \, \mathrm{d}x - \int_0^1 (h(x)+h(g(x))) \, w(x) \, \mathrm{d}x \\[1em] \text{by substitution:} \\[0.5em] &= \int_0^1 \exp(\bar{u}(x))\, h(x) \, \mathrm{d}x - \int_0^1 h(x) \, (1-g'(x)) \,w(x)\, \mathrm{d}x \\[1em] &= \int_0^1 \exp(\bar{u}(x))\, h(x) \, \mathrm{d}x - \int_0^1 \exp(\bar{u}(x)) \, h(x) \, \mathrm{d}x \\[1em] &= 0. \end{align*} para todos $h \in C[0,1]$ . Desde $J$ y $-(\psi \circ I)$ son convexos, $L$ es convexo. Tenemos $L'(\bar{u})=0$ y por lo tanto $\bar{u}$ es un minimizador global de $L$ . Desde $\psi$ es un funcional positivo, tenemos $L(u) \leq J(u)$ para todos $u \in C[0,1]$ con $I(u) \geq 0$ . Pero $\psi(I(\bar{u}))= 0$ desde $I(\bar{u})(x,g(x))=0$ por la reivindicación 3 para todos los $x \in [0,1]$ . Por lo tanto, $L(\bar{u})=J(\bar{u})$ y por lo tanto $J(\bar{u}) \leq J(u)$ para todos $u \in C[0,1]$ con $I(u) \geq 0$ . Por la afirmación 3 tenemos $I(\bar{u}) \geq 0$ . Por lo tanto, $\bar{u}$ es una solución de $(1)$ .
Supongamos que hay un $\tilde{u} \in C[0,1]$ tal que $I(\tilde{u}) \geq 0$ y $J(\tilde{u}) \leq J(\bar{u})$ . Establecemos $$\widehat{u} := \frac{\tilde{u} + \bar{u}}{2}.$$ Tenemos $I(\widehat{u})\geq 0$ . Desde $J$ es estrictamente convexo, $\bar{u} = \widehat{u} = \tilde{u}$ . Por lo tanto, $\bar{u}$ es la única solución de $(1)$ . $$\tag*{$ \N - Caja $}$$
Reclamación 5. La solución única de $(2)$ viene dada por $$\bar{f}(x)= \begin{cases} \dfrac{\exp(\bar{u}(2x))}{\sqrt{2}}&\text{if}\quad 0 \leq x \leq \frac{1}{2},\\ \dfrac{\exp(\bar{u}(2(1-x)))}{\sqrt{2}}&\text{if}\quad \frac{1}{2} < x \leq 1. \end{cases}$$
Prueba. Desde $\exp > 0$ tenemos $\bar{f} > 0$ . Sea $x,y \in[0,1]$ tal que $x \leq y$ .
Si $x \leq \frac{1}{2} \leq y$ entonces \begin{align} \bar{f}(x)\bar{f}(y)&=\frac{1}{2}\exp\left(\bar{u}(2x)+\bar{u}(2(1-y))\right) \nonumber \\ &\geq \frac{1}{2}(2- 2x - 2(1-y)) \qquad \text{(by Claim 3)} \nonumber \\ &=y-x \tag{14} \\ &= |x-y|. \nonumber \end{align} Si $x \leq y \leq \frac{1}{2}$ entonces $$\bar{f}(x)\bar{f}(y)=\bar{f}(x)\bar{f}(1-y) \underset{(14)}{\geq} 1-y-x \geq y-x = |x-y|.$$ Si $\frac{1}{2} \leq x \leq y$ entonces $$\bar{f}(x)\bar{f}(y)=\bar{f}(1-x)\bar{f}(y) \underset{(14)}{\geq} y-(1-x) \geq y-x = |x-y|.$$ Así, $\bar{f}(x)\bar{f}(y) \geq |x-y|$ para todos $x,y \in [0,1]$ .
Supongamos que existe $\tilde{f}$ tal que $\tilde{f}$ satisface las restricciones de (2) y $$\int_0^1 \tilde{f} \, \mathrm{d}x \leq \int_0^1 \bar{f} \, \mathrm{d}x.$$ Hemos establecido $$\widehat{f}(x):= \left(\tilde{f}(x)\tilde{f}(1-x)\bar{f}(x)^2\right)^\frac{1}{4}.$$ $\widehat{f}$ satisface las restricciones de (2) y \begin{align} \int_0^1 \widehat{f}(x) \, \mathrm{d}x &= \int_0^1 \left(\tilde{f}(x)\tilde{f}(1-x)\bar{f}(x)^2\right)^\frac{1}{4} \, \mathrm{d}x \nonumber \\[1em] &\leq \int_0^1 \frac{\tilde{f}(x)+\tilde{f}(1-x)+2\bar{f}(1-x)}{4} \, \mathrm{d}x \tag{15} \\[1em] &= \int_0^1 \frac{\tilde{f}(x)+\bar{f}(x)}{2} \, \mathrm{d}x \nonumber \\[1em] &\leq \int_0^1 \bar{f}(x) \, \mathrm{d}x. \nonumber \end{align} Desde $\widehat{f}(x) = \widehat{f}(1-x)$ y $\bar{f}(x) = \bar{f}(1-x)$ para todos $x \in [0,1]$ Así pues, tenemos \begin{align} \int_0^{\frac{1}{2}} \widehat{f}(x) \, \mathrm{d}x \leq \int_0^{\frac{1}{2}} \bar{f}(x) \, \mathrm{d}x. \tag{16} \end{align} Hemos establecido $$\widehat{u}(x) := \log\left(\sqrt{2}\, \widehat{f}\left(\frac{x}{2}\right)\right),$$ y por $(16)$ tenemos $J(\widehat{u}) \leq J(\bar{u})$ . También tenemos $I(\widehat{u}) \geq 0$ desde \begin{align*} \exp(\widehat{u}(x)+\widehat{u}(y)) &= 2\widehat{f}\left(\frac{x}{2}\right)\widehat{f}\left(\frac{y}{2}\right) \\[1em] &= 2\widehat{f}\left(\frac{x}{2}\right)\widehat{f}\left(1-\frac{y}{2}\right) \\[1em] &\geq 2\left|1-\frac{x}{2}-\frac{y}{2}\right| \\[1em] &= 2-x-y \end{align*} para todos $x,y \in [0,1]$ . Por la reivindicación 4, $\widehat{u} = \bar{u}$ . Desde $$\widehat{f}(x)=\frac{\exp(\widehat{u}(2x))}{\sqrt{2}}$$ para todos $x \in [0,\frac{1}{2}]$ por definición de $\widehat{u}$ tenemos $\widehat{f} = \bar{f}$ . La desigualdad en $(15)$ debe ser una igualdad y por lo tanto $\tilde{f} = \widehat{f} = \bar{f}$ . Por lo tanto, $\bar{f}$ es la única solución de $(2)$ . $$\tag*{$ \N - Caja $}$$
0 votos
¿Tiene un ejemplo de una función $f \in E$ ?
1 votos
@usuario159517 $f(x) > \sup_{x,y} |x-y| = 1$ lo hará.
0 votos
@CalvinKhor ah, por supuesto. Eso también demuestra que $E$ no está acotado, por lo que no es compacto, lo que dificulta la existencia de un elemento minimizador.