SlideShare a Scribd company logo
1 of 18
Download to read offline
580 Optimization Approach to Nash Equilibria
with Applications to Interchangeability
Yosuke YASUDA
Osaka University, Department of Economics
(visiting ISEG, University of Lisbon)
yasuda@econ.osaka-u.ac.jp
July, 2021
1 / 18
Summary
What is Optimization Approach? (1st Part)
The set of Nash equilibria, if it is nonempty, is identical to the
set of minimizers of real-valued function.
Connect equilibrium problem to optimization problem.
→ Similar characterizations are known in the literature.
Is it Useful? Any application? (2nd Part)
Existing results on interchangeability can be derived, in a
unified fashion, by lattice structure of optimal solutions.
→ NEW contribution! (looking for ompletely new results...)
Main Messages
Please use/apply/extend our characterization of NE!
2 / 18
Traditional Formulations of NE
Strategy profile x∗ ∈ X is called Nash equilibrium if and only if,
1 Inequality (Incentive) Constraints
ui(x∗
i , x∗
−i) ≥ ui(xi, x∗
−i) for all xi ∈ Xi and for all i ∈ N.
2 Solution to Multivariate Function
ui(x∗
i , x∗
−i) = max
xi∈Xi
ui(xi, x∗
−i) for all i ∈ N.
3 Fixed Point of BR Correspondence
x∗
∈ BR(x∗
),
where BRi(x−i) = arg max
x0
i∈Xi
ui(x0
i, x−i).
3 / 18
Alternative: Optimization Approach
Define f : X → R, which aggregates maximum deviation gains
(from a fixed action profile x ∈ X) across players.
f(x) =
X
i∈N

max
x0
i∈Xi
ui(x0
i, x−i) − ui(xi, x−i)

. (1)
Theorem 1
A strategy profile x∗ is a Nash equilibrium iff f(x∗) = 0.
Theorem 2
If there exists an NE, the set of Nash equilibria E∗ is identical to
the set of minimum solutions to f, i.e., arg minx∈X f(x).
4 / 18
Example: Prisoner’s Dilemma
Table: Payoff Matrix
C D
C 3, 3 0, 4
D 4, 0 1, 1
Table: Values of f
C D
C 2 (= (4 − 3) + (4 − 3)) 1 (= (1 − 0) + 0)
D 1 (= 0 + (1 − 0)) 0 (= 0 + 0)
5 / 18
Extensions
Let g(x) = −f(x). The set of Nash equilibria, if it is
nonempty, is identical to the set of maximum solutions to g.
arg max
x∈X
g(x).
f can be replaced by ˜
f : X → R, using a sign-preserving
function ψi : R+ → R+ such that ψi(x) = 0 iff x = 0.
˜
f(x) =
X
i∈N
ψi

max
x0
i∈Xi
ui(x0
i, x−i) − ui(xi, x−i)

.
Let t be a parameter contained in a parameter set T. Then,
(1) can be rewritten to incorporate this parameterization.
f(x, t) =
X
i∈N

max
x0
i∈Xi
ui(x0
i, x−i; t) − ui(xi, x−i; t)

.
6 / 18
From “Sum” to “Product”
The parallel characterization can be available when the objective
function is replaced with the product of deviation gains.
f(x) = Πi∈N

1 + max
x0
i∈Xi
ui(x0
i, x−i) − ui(xi, x−i)

. (2)
Note by construction that f(x) ≥ 1 holds for any x ∈ X.
Lemma 3
A strategy profile x∗ is an NE iff f(x∗) = 1. If there is an NE, E∗
is identical to the set of minimum solutions to f, arg minx∈X f(x).
1 can be replaced with any ε  0. (Then, f(x∗) = εn)
As ε goes to 0, (2) converges to the product of players’ payoff
differences, which may look similar to the Nash product.
7 / 18
Interchangeability for Two-Person Games
Let x = (x1, x2) and x0 = (x0
1, x0
2) be two distinct NE.
Definition 4
A pair of Nash equilibia x and x0 is called interchangeable if
(x1, x0
2) and (x0
1, x2) constitute NE of the same game.
Our approach can explain the following existing results on
interchangeability, independently derived in the literature:
1 for a zero-sum game any pairs of its mixed strategy Nash
equilibria are interchangeable (Luce and Raiffa, 1957).
2 for a supermodular game where each player’s strategy space
is totally ordered, any unordered pairs of the pure strategy
Nash equilibria are interchangeable (Echenique, 2003).
3 equilibrium set of a strictly supermodular game with totally
ordered strategy spaces, is totally ordered (Vives, 1985).
8 / 18
Introduction to Lattice (1)
Let = be a binary relation on a non-empty set S.
Definition 5
The pair (S, =) is a partially ordered set if, for x, y, z in S, = is
reflexive: x = x.
transitive: x = y and y = z implies x = z.
antisymmetric: x = y and y = x implies x = y.
A partially ordered set (S, =) is
totally ordered if for x and y in S either x = y or y = x is
satisfied, and is called chain.
called lattice if any two elements have a least upper bound
(join, ∨) and a greatest lower bound (meet, ∧) in the set.
A subset S∗(⊂ S) is called sublattice if x0 ∧ x00 ∈ S∗ and
x0 ∨ x00 ∈ S∗ hold for any x0, x00 ∈ S∗.
9 / 18
Introduction to Lattice (2)
Definition 6
A real-valued function h defined over a lattice S is called a
submodular function if, for any x0, x00 ∈ S, h satisfies
h(x0
∧ x00
) + h(x0
∨ x00
) − {h(x0
) + h(x00
)} ≤ 0. (3)
(3) trivially holds with equality whenever x0 and x00 are
ordered, i.e., x0 = x00 or x0 5 x00.
If ≤ in (3) is replaced with ≥, h is called supermodular.
h : S → R becomes a strictly submodular function if, for any
unordered pair x0, x00 ∈ S, i.e., x0  x00 and x0  x00, h satisfies
h(x0
∧ x00
) + h(x0
∨ x00
) − {h(x0
) + h(x00
)}  0. (4)
If  in (4) is replaced with , h is strictly supermodular.
10 / 18
Results by Topkis (1978)
Fact 7 (Topkis, 1978)
If h is a submodular function on a lattice S, then the set S∗ of
points at which h attains its minimum on S is a sublattice of S.
Fact 8 (Topkis, 1978)
If h is st. submodular on a lattice S, then the set S∗ of points at
which h attains its minimum on S is a chain.
Assume X is a lattice. The above facts imply the following.
Lemma 9
Suppose that f is defined by (1) and E∗ is nonempty. Then,
(i) If f is submodular on X, then E∗ is a sublattice of X.
(ii) If f is st. submodular on X, then E∗ is a chain.
11 / 18
Supermodular Game
Let us define u as the sum of the payoff functions.
u(x) = u1(x) + u2(x) for all x ∈ X.
Lemma 10
For any two-person game with totally ordered strategy space for
each player,
(i) f is submodular iff u is supermodular.
(ii) f is st. submodular iff u is st. supermodular.
Lemma 11
u (= u1 + u2) is supermodular (resp. strictly supermodular) for
any two-person supermodular (resp. strictly supermodular) games.
Supermodularity is preserved under addition.
The converse is not true, e.g., zero-sum game.
12 / 18
Proof of Lemma 10 (1)
Recall that f is a submodular function if, for any x0, x00 ∈ X,
f(x0
∧ x00
) + f(x0
∨ x00
) − {f(x0
) + f(x00
)} ≤ 0. (5)
If the above inequality is strict for any unordered pairs, f is a st.
submodular function. Since we consider two-person games,
f(x) = max
x1∈X1
u1(x1, x2) − u1(x1, x2)
+ max
x2∈X2
u2(x1, x2) − u2(x1, x2).
Now consider a pair of unordered strategy profiles, x0 = (x0
1, x0
2)
and x00 = (x00
1, x00
2). W.o.l.g, assume x0
1 =1 x00
1 and x0
2 52 x00
2.
Join: x0 ∧ x00 = (x00
1, x0
2)
Meet: x0 ∨ x00 = (x0
1, x00
2)
13 / 18
Proof of Lemma 10 (2)
The corresponding values of f are expressed by
f(x0
∧ x00
) = max
x1∈X1
u1(x1, x0
2) − u1(x00
1, x0
2)
+ max
x2∈X2
u2(x00
1, x2) − u2(x00
1, x0
2).
f(x0
∨ x00
) = max
x1∈X1
u1(x1, x00
2) − u1(x0
1, x00
2)
+ max
x2∈X2
u2(x00
1, x2) − u2(x0
1, x00
2).
Substituting them into (5), max ui parts will be canceled out.
The next equality illustrates that the (st.) submodularity of f
is completely characterized by the (st.) supermodularity of u.
14 / 18
Proof of Lemma 10 (3)
f(x0
∧ x00
) + f(x0
∨ x00
) − {f(x0
) + f(x00
)}
= − { u1(x00
1, x0
2) + u2(x00
1, x0
2) + u1(x0
1, x00
2) + u2(x0
1, x00
2)}
+

u1(x0
1, x0
2) + u2(x0
1, x0
2) + u1(x00
1, x00
2) + u2(x00
1, x00
2)
	
= − { u1(x0
∧ x00
) + u2(x0
∧ x00
) + u1(x0
∨ x00
) + u2(x0
∨ x00
)}
+

u1(x0
) + u2(x0
) + u1(x00
) + u2(x00
)
	
= u(x0
) + u(x00
) − {u(x0
∧ x00
) + u(x0
∨ x00
)}.
Since u = u1 + u2 is constant for a zero-sum game, we obtain:
Lemma 12
For any two-person zero-sum game, f is submodular over mixed
strategy profiles with any order of strategy space for each player.
15 / 18
Main Result: Zero-Sum Game
Theorem 13
For a zero-sum game, any pairs of its (mixed strategy) Nash
equilibria are interchangeable.
Proof.
E∗ is nonempty.
Existence of NE by Nash (1950)
Existence of minimax solution by Neumann (1928).
Suppose that x = (x1, x2) and x0 = (x0
1, x0
2) are two distinct NE.
We can always construct an order that satisfies
x1 =1 x0
1 and x2 52 x0
2.
By Lemma 9 (i), E∗ is sublattice.
⇒ x ∧ x0 = (x0
1, x2) and x ∨ x0 = (x1, x0
2) are both NE.
16 / 18
Main Result: Supermodular Game
Since the existence of (pure strategy) NE for supermodular games
is guaranteed by Topkis (1979), we obtain the next theorem.
Theorem 14
Assume strategy space for each player is totally ordered. Then,
(i) For a two-person supermodular game, any unordered pairs of
its pure strategy NE are interchangeable.
(ii) For a two-person st. supermodular game, all pure strategy NE
are totally ordered.
The above results also hold for log-supermodular games.
If ui is log-supermodular, then ˆ
f must be submodular.
(Note f = 0 iff ˆ
f = 0)
ˆ
f(x) =
X
i∈N

max
x0
i∈Xi
ln ui(x0
i, x−i) − ln ui(xi, x−i)

.
17 / 18
Conclusion
Summary: Provide a functional formulation of NE.
Enables us to analyze Nash equilibrium as a solution to an
optimization problem without any constraints.
May connect non-cooperative game theory with other related
fields such as OR and CS.
Natural Reaction: So what? Is it really useful?
→ New insight on interchangeability of NE.
Existing results on two person (i) zero-sum games and (ii)
supermodular games can be derived, in a unified fashion:
The set of minimizers of submodular function is sublattice.
Applications to symmetric, potential, cooperative games (via
Nash implementation), etc? → Future research!
18 / 18

More Related Content

What's hot

Fuzzy random variables and Kolomogrov’s important results
Fuzzy random variables and Kolomogrov’s important resultsFuzzy random variables and Kolomogrov’s important results
Fuzzy random variables and Kolomogrov’s important resultsinventionjournals
 
Lesson 23: Antiderivatives (slides)
Lesson 23: Antiderivatives (slides)Lesson 23: Antiderivatives (slides)
Lesson 23: Antiderivatives (slides)Matthew Leingang
 
Lesson 21: Curve Sketching (slides)
Lesson 21: Curve Sketching (slides)Lesson 21: Curve Sketching (slides)
Lesson 21: Curve Sketching (slides)Matthew Leingang
 
Polya recurrence
Polya recurrencePolya recurrence
Polya recurrenceBrian Burns
 
11.fixed point theorem of discontinuity and weak compatibility in non complet...
11.fixed point theorem of discontinuity and weak compatibility in non complet...11.fixed point theorem of discontinuity and weak compatibility in non complet...
11.fixed point theorem of discontinuity and weak compatibility in non complet...Alexander Decker
 
Fixed point theorem of discontinuity and weak compatibility in non complete n...
Fixed point theorem of discontinuity and weak compatibility in non complete n...Fixed point theorem of discontinuity and weak compatibility in non complete n...
Fixed point theorem of discontinuity and weak compatibility in non complete n...Alexander Decker
 
Lesson 14: Derivatives of Logarithmic and Exponential Functions (slides)
Lesson 14: Derivatives of Logarithmic and Exponential Functions (slides)Lesson 14: Derivatives of Logarithmic and Exponential Functions (slides)
Lesson 14: Derivatives of Logarithmic and Exponential Functions (slides)Matthew Leingang
 
Classical optimization theory Unconstrained Problem
Classical optimization theory Unconstrained ProblemClassical optimization theory Unconstrained Problem
Classical optimization theory Unconstrained ProblemSurya Teja
 
Introduction to the theory of optimization
Introduction to the theory of optimizationIntroduction to the theory of optimization
Introduction to the theory of optimizationDelta Pi Systems
 
Lesson 26: The Fundamental Theorem of Calculus (slides)
Lesson 26: The Fundamental Theorem of Calculus (slides)Lesson 26: The Fundamental Theorem of Calculus (slides)
Lesson 26: The Fundamental Theorem of Calculus (slides)Matthew Leingang
 
Notes on Intersection theory
Notes on Intersection theoryNotes on Intersection theory
Notes on Intersection theoryHeinrich Hartmann
 
Paper finance hosseinkhan_remy
Paper finance hosseinkhan_remyPaper finance hosseinkhan_remy
Paper finance hosseinkhan_remyRémy Hosseinkhan
 
Machine learning (1)
Machine learning (1)Machine learning (1)
Machine learning (1)NYversity
 
tensor-decomposition
tensor-decompositiontensor-decomposition
tensor-decompositionKenta Oono
 

What's hot (20)

Fuzzy random variables and Kolomogrov’s important results
Fuzzy random variables and Kolomogrov’s important resultsFuzzy random variables and Kolomogrov’s important results
Fuzzy random variables and Kolomogrov’s important results
 
Lesson 23: Antiderivatives (slides)
Lesson 23: Antiderivatives (slides)Lesson 23: Antiderivatives (slides)
Lesson 23: Antiderivatives (slides)
 
FUZZY LOGIC
FUZZY LOGICFUZZY LOGIC
FUZZY LOGIC
 
Lesson 21: Curve Sketching (slides)
Lesson 21: Curve Sketching (slides)Lesson 21: Curve Sketching (slides)
Lesson 21: Curve Sketching (slides)
 
Polya recurrence
Polya recurrencePolya recurrence
Polya recurrence
 
Ch02 fuzzyrelation
Ch02 fuzzyrelationCh02 fuzzyrelation
Ch02 fuzzyrelation
 
Nokton theory-en
Nokton theory-enNokton theory-en
Nokton theory-en
 
11.fixed point theorem of discontinuity and weak compatibility in non complet...
11.fixed point theorem of discontinuity and weak compatibility in non complet...11.fixed point theorem of discontinuity and weak compatibility in non complet...
11.fixed point theorem of discontinuity and weak compatibility in non complet...
 
Fixed point theorem of discontinuity and weak compatibility in non complete n...
Fixed point theorem of discontinuity and weak compatibility in non complete n...Fixed point theorem of discontinuity and weak compatibility in non complete n...
Fixed point theorem of discontinuity and weak compatibility in non complete n...
 
Lesson 14: Derivatives of Logarithmic and Exponential Functions (slides)
Lesson 14: Derivatives of Logarithmic and Exponential Functions (slides)Lesson 14: Derivatives of Logarithmic and Exponential Functions (slides)
Lesson 14: Derivatives of Logarithmic and Exponential Functions (slides)
 
Ch7
Ch7Ch7
Ch7
 
Universal algebra (1)
Universal algebra (1)Universal algebra (1)
Universal algebra (1)
 
Classical optimization theory Unconstrained Problem
Classical optimization theory Unconstrained ProblemClassical optimization theory Unconstrained Problem
Classical optimization theory Unconstrained Problem
 
Introduction to the theory of optimization
Introduction to the theory of optimizationIntroduction to the theory of optimization
Introduction to the theory of optimization
 
Lesson 26: The Fundamental Theorem of Calculus (slides)
Lesson 26: The Fundamental Theorem of Calculus (slides)Lesson 26: The Fundamental Theorem of Calculus (slides)
Lesson 26: The Fundamental Theorem of Calculus (slides)
 
Notes on Intersection theory
Notes on Intersection theoryNotes on Intersection theory
Notes on Intersection theory
 
Paper finance hosseinkhan_remy
Paper finance hosseinkhan_remyPaper finance hosseinkhan_remy
Paper finance hosseinkhan_remy
 
Polyadic integer numbers and finite (m,n) fields
Polyadic integer numbers and finite (m,n) fieldsPolyadic integer numbers and finite (m,n) fields
Polyadic integer numbers and finite (m,n) fields
 
Machine learning (1)
Machine learning (1)Machine learning (1)
Machine learning (1)
 
tensor-decomposition
tensor-decompositiontensor-decomposition
tensor-decomposition
 

Similar to Optimization Approach to Nash Euilibria with Applications to Interchangeability

APPLICATION OF PARTIAL DIFFERENTIATION
APPLICATION OF PARTIAL DIFFERENTIATIONAPPLICATION OF PARTIAL DIFFERENTIATION
APPLICATION OF PARTIAL DIFFERENTIATIONDhrupal Patel
 
Unique fixed point theorems for generalized weakly contractive condition in o...
Unique fixed point theorems for generalized weakly contractive condition in o...Unique fixed point theorems for generalized weakly contractive condition in o...
Unique fixed point theorems for generalized weakly contractive condition in o...Alexander Decker
 
B043007014
B043007014B043007014
B043007014inventy
 
B043007014
B043007014B043007014
B043007014inventy
 
B043007014
B043007014B043007014
B043007014inventy
 
UMAP - Mathematics and implementational details
UMAP - Mathematics and implementational detailsUMAP - Mathematics and implementational details
UMAP - Mathematics and implementational detailsUmberto Lupo
 
5.3 Basic functions. Dynamic slides.
5.3 Basic functions. Dynamic slides.5.3 Basic functions. Dynamic slides.
5.3 Basic functions. Dynamic slides.Jan Plaza
 
α -ANTI FUZZY NEW IDEAL OF PUALGEBRA
α -ANTI FUZZY NEW IDEAL OF PUALGEBRAα -ANTI FUZZY NEW IDEAL OF PUALGEBRA
α -ANTI FUZZY NEW IDEAL OF PUALGEBRAWireilla
 
a - ANTI FUZZY NEW IDEAL OF PUALGEBRA
a - ANTI FUZZY NEW IDEAL OF PUALGEBRAa - ANTI FUZZY NEW IDEAL OF PUALGEBRA
a - ANTI FUZZY NEW IDEAL OF PUALGEBRAijfls
 
FUZZY IDEALS AND FUZZY DOT IDEALS ON BH-ALGEBRAS
FUZZY IDEALS AND FUZZY DOT IDEALS ON BH-ALGEBRASFUZZY IDEALS AND FUZZY DOT IDEALS ON BH-ALGEBRAS
FUZZY IDEALS AND FUZZY DOT IDEALS ON BH-ALGEBRASIAEME Publication
 
FUZZY IDEALS AND FUZZY DOT IDEALS ON BH-ALGEBRAS
FUZZY IDEALS AND FUZZY DOT IDEALS ON BH-ALGEBRASFUZZY IDEALS AND FUZZY DOT IDEALS ON BH-ALGEBRAS
FUZZY IDEALS AND FUZZY DOT IDEALS ON BH-ALGEBRASIAEME Publication
 
MA500-2 Topological Structures 2016Aisling McCluskey, Dar.docx
MA500-2 Topological Structures 2016Aisling McCluskey, Dar.docxMA500-2 Topological Structures 2016Aisling McCluskey, Dar.docx
MA500-2 Topological Structures 2016Aisling McCluskey, Dar.docxsmile790243
 
On Frechet Derivatives with Application to the Inverse Function Theorem of Or...
On Frechet Derivatives with Application to the Inverse Function Theorem of Or...On Frechet Derivatives with Application to the Inverse Function Theorem of Or...
On Frechet Derivatives with Application to the Inverse Function Theorem of Or...BRNSS Publication Hub
 
Common Fixed Point Theorems in Compatible Mappings of Type (P*) of Generalize...
Common Fixed Point Theorems in Compatible Mappings of Type (P*) of Generalize...Common Fixed Point Theorems in Compatible Mappings of Type (P*) of Generalize...
Common Fixed Point Theorems in Compatible Mappings of Type (P*) of Generalize...mathsjournal
 
5.4 Saddle-point interpretation, 5.5 Optimality conditions, 5.6 Perturbation ...
5.4 Saddle-point interpretation, 5.5 Optimality conditions, 5.6 Perturbation ...5.4 Saddle-point interpretation, 5.5 Optimality conditions, 5.6 Perturbation ...
5.4 Saddle-point interpretation, 5.5 Optimality conditions, 5.6 Perturbation ...RyotaroTsukada
 
Interval valued intuitionistic fuzzy homomorphism of bf algebras
Interval valued intuitionistic fuzzy homomorphism of bf algebrasInterval valued intuitionistic fuzzy homomorphism of bf algebras
Interval valued intuitionistic fuzzy homomorphism of bf algebrasAlexander Decker
 
590-Article Text.pdf
590-Article Text.pdf590-Article Text.pdf
590-Article Text.pdfBenoitValea
 
590-Article Text.pdf
590-Article Text.pdf590-Article Text.pdf
590-Article Text.pdfBenoitValea
 
Fourier 3
Fourier 3Fourier 3
Fourier 3nugon
 

Similar to Optimization Approach to Nash Euilibria with Applications to Interchangeability (20)

APPLICATION OF PARTIAL DIFFERENTIATION
APPLICATION OF PARTIAL DIFFERENTIATIONAPPLICATION OF PARTIAL DIFFERENTIATION
APPLICATION OF PARTIAL DIFFERENTIATION
 
Unique fixed point theorems for generalized weakly contractive condition in o...
Unique fixed point theorems for generalized weakly contractive condition in o...Unique fixed point theorems for generalized weakly contractive condition in o...
Unique fixed point theorems for generalized weakly contractive condition in o...
 
B043007014
B043007014B043007014
B043007014
 
B043007014
B043007014B043007014
B043007014
 
B043007014
B043007014B043007014
B043007014
 
UMAP - Mathematics and implementational details
UMAP - Mathematics and implementational detailsUMAP - Mathematics and implementational details
UMAP - Mathematics and implementational details
 
5.3 Basic functions. Dynamic slides.
5.3 Basic functions. Dynamic slides.5.3 Basic functions. Dynamic slides.
5.3 Basic functions. Dynamic slides.
 
α -ANTI FUZZY NEW IDEAL OF PUALGEBRA
α -ANTI FUZZY NEW IDEAL OF PUALGEBRAα -ANTI FUZZY NEW IDEAL OF PUALGEBRA
α -ANTI FUZZY NEW IDEAL OF PUALGEBRA
 
a - ANTI FUZZY NEW IDEAL OF PUALGEBRA
a - ANTI FUZZY NEW IDEAL OF PUALGEBRAa - ANTI FUZZY NEW IDEAL OF PUALGEBRA
a - ANTI FUZZY NEW IDEAL OF PUALGEBRA
 
FUZZY IDEALS AND FUZZY DOT IDEALS ON BH-ALGEBRAS
FUZZY IDEALS AND FUZZY DOT IDEALS ON BH-ALGEBRASFUZZY IDEALS AND FUZZY DOT IDEALS ON BH-ALGEBRAS
FUZZY IDEALS AND FUZZY DOT IDEALS ON BH-ALGEBRAS
 
FUZZY IDEALS AND FUZZY DOT IDEALS ON BH-ALGEBRAS
FUZZY IDEALS AND FUZZY DOT IDEALS ON BH-ALGEBRASFUZZY IDEALS AND FUZZY DOT IDEALS ON BH-ALGEBRAS
FUZZY IDEALS AND FUZZY DOT IDEALS ON BH-ALGEBRAS
 
MA500-2 Topological Structures 2016Aisling McCluskey, Dar.docx
MA500-2 Topological Structures 2016Aisling McCluskey, Dar.docxMA500-2 Topological Structures 2016Aisling McCluskey, Dar.docx
MA500-2 Topological Structures 2016Aisling McCluskey, Dar.docx
 
On Frechet Derivatives with Application to the Inverse Function Theorem of Or...
On Frechet Derivatives with Application to the Inverse Function Theorem of Or...On Frechet Derivatives with Application to the Inverse Function Theorem of Or...
On Frechet Derivatives with Application to the Inverse Function Theorem of Or...
 
Common Fixed Point Theorems in Compatible Mappings of Type (P*) of Generalize...
Common Fixed Point Theorems in Compatible Mappings of Type (P*) of Generalize...Common Fixed Point Theorems in Compatible Mappings of Type (P*) of Generalize...
Common Fixed Point Theorems in Compatible Mappings of Type (P*) of Generalize...
 
5.4 Saddle-point interpretation, 5.5 Optimality conditions, 5.6 Perturbation ...
5.4 Saddle-point interpretation, 5.5 Optimality conditions, 5.6 Perturbation ...5.4 Saddle-point interpretation, 5.5 Optimality conditions, 5.6 Perturbation ...
5.4 Saddle-point interpretation, 5.5 Optimality conditions, 5.6 Perturbation ...
 
Interval valued intuitionistic fuzzy homomorphism of bf algebras
Interval valued intuitionistic fuzzy homomorphism of bf algebrasInterval valued intuitionistic fuzzy homomorphism of bf algebras
Interval valued intuitionistic fuzzy homomorphism of bf algebras
 
590-Article Text.pdf
590-Article Text.pdf590-Article Text.pdf
590-Article Text.pdf
 
590-Article Text.pdf
590-Article Text.pdf590-Article Text.pdf
590-Article Text.pdf
 
1_AJMS_229_19[Review].pdf
1_AJMS_229_19[Review].pdf1_AJMS_229_19[Review].pdf
1_AJMS_229_19[Review].pdf
 
Fourier 3
Fourier 3Fourier 3
Fourier 3
 

More from Yosuke YASUDA

社会的共通資本と資本主義
社会的共通資本と資本主義社会的共通資本と資本主義
社会的共通資本と資本主義Yosuke YASUDA
 
「戦略的思考」で読み解くビジネスと社会
「戦略的思考」で読み解くビジネスと社会「戦略的思考」で読み解くビジネスと社会
「戦略的思考」で読み解くビジネスと社会Yosuke YASUDA
 
「立命館西園寺塾2021・2回目」資料
「立命館西園寺塾2021・2回目」資料「立命館西園寺塾2021・2回目」資料
「立命館西園寺塾2021・2回目」資料Yosuke YASUDA
 
「立命館西園寺塾2021」資料
「立命館西園寺塾2021」資料「立命館西園寺塾2021」資料
「立命館西園寺塾2021」資料Yosuke YASUDA
 
資本主義と金融 2021
資本主義と金融 2021資本主義と金融 2021
資本主義と金融 2021Yosuke YASUDA
 
目からウロコのモラルハザード解決法
目からウロコのモラルハザード解決法目からウロコのモラルハザード解決法
目からウロコのモラルハザード解決法Yosuke YASUDA
 
「戦略的思考」で世の中の見方を変えよう!
「戦略的思考」で世の中の見方を変えよう!「戦略的思考」で世の中の見方を変えよう!
「戦略的思考」で世の中の見方を変えよう!Yosuke YASUDA
 
宇沢弘文を読む
宇沢弘文を読む宇沢弘文を読む
宇沢弘文を読むYosuke YASUDA
 
オークションの仕組み
オークションの仕組みオークションの仕組み
オークションの仕組みYosuke YASUDA
 
宇沢弘文没後5年追悼シンポジウム
宇沢弘文没後5年追悼シンポジウム宇沢弘文没後5年追悼シンポジウム
宇沢弘文没後5年追悼シンポジウムYosuke YASUDA
 
資本主義とお金の未来
資本主義とお金の未来資本主義とお金の未来
資本主義とお金の未来Yosuke YASUDA
 
令和時代における産業のあり方と行うべき人材投資
令和時代における産業のあり方と行うべき人材投資令和時代における産業のあり方と行うべき人材投資
令和時代における産業のあり方と行うべき人材投資Yosuke YASUDA
 
グローバル経済の動きから読み解く日本企業の課題とチャンス
グローバル経済の動きから読み解く日本企業の課題とチャンスグローバル経済の動きから読み解く日本企業の課題とチャンス
グローバル経済の動きから読み解く日本企業の課題とチャンスYosuke YASUDA
 
経済学で読み解く「働き方」と「イノベーション」2.0
経済学で読み解く「働き方」と「イノベーション」2.0経済学で読み解く「働き方」と「イノベーション」2.0
経済学で読み解く「働き方」と「イノベーション」2.0Yosuke YASUDA
 
人材・組織を生かすコミュニティ戦略
人材・組織を生かすコミュニティ戦略人材・組織を生かすコミュニティ戦略
人材・組織を生かすコミュニティ戦略Yosuke YASUDA
 
資本主義と金融 2019
資本主義と金融 2019資本主義と金融 2019
資本主義と金融 2019Yosuke YASUDA
 
人材・組織を生かすマッチング戦略
人材・組織を生かすマッチング戦略人材・組織を生かすマッチング戦略
人材・組織を生かすマッチング戦略Yosuke YASUDA
 
マッチングの仕組み
マッチングの仕組みマッチングの仕組み
マッチングの仕組みYosuke YASUDA
 

More from Yosuke YASUDA (20)

社会的共通資本と資本主義
社会的共通資本と資本主義社会的共通資本と資本主義
社会的共通資本と資本主義
 
「戦略的思考」で読み解くビジネスと社会
「戦略的思考」で読み解くビジネスと社会「戦略的思考」で読み解くビジネスと社会
「戦略的思考」で読み解くビジネスと社会
 
「立命館西園寺塾2021・2回目」資料
「立命館西園寺塾2021・2回目」資料「立命館西園寺塾2021・2回目」資料
「立命館西園寺塾2021・2回目」資料
 
「立命館西園寺塾2021」資料
「立命館西園寺塾2021」資料「立命館西園寺塾2021」資料
「立命館西園寺塾2021」資料
 
資本主義と金融 2021
資本主義と金融 2021資本主義と金融 2021
資本主義と金融 2021
 
[ICF2020]資料
[ICF2020]資料[ICF2020]資料
[ICF2020]資料
 
目からウロコのモラルハザード解決法
目からウロコのモラルハザード解決法目からウロコのモラルハザード解決法
目からウロコのモラルハザード解決法
 
Economics Design
Economics DesignEconomics Design
Economics Design
 
「戦略的思考」で世の中の見方を変えよう!
「戦略的思考」で世の中の見方を変えよう!「戦略的思考」で世の中の見方を変えよう!
「戦略的思考」で世の中の見方を変えよう!
 
宇沢弘文を読む
宇沢弘文を読む宇沢弘文を読む
宇沢弘文を読む
 
オークションの仕組み
オークションの仕組みオークションの仕組み
オークションの仕組み
 
宇沢弘文没後5年追悼シンポジウム
宇沢弘文没後5年追悼シンポジウム宇沢弘文没後5年追悼シンポジウム
宇沢弘文没後5年追悼シンポジウム
 
資本主義とお金の未来
資本主義とお金の未来資本主義とお金の未来
資本主義とお金の未来
 
令和時代における産業のあり方と行うべき人材投資
令和時代における産業のあり方と行うべき人材投資令和時代における産業のあり方と行うべき人材投資
令和時代における産業のあり方と行うべき人材投資
 
グローバル経済の動きから読み解く日本企業の課題とチャンス
グローバル経済の動きから読み解く日本企業の課題とチャンスグローバル経済の動きから読み解く日本企業の課題とチャンス
グローバル経済の動きから読み解く日本企業の課題とチャンス
 
経済学で読み解く「働き方」と「イノベーション」2.0
経済学で読み解く「働き方」と「イノベーション」2.0経済学で読み解く「働き方」と「イノベーション」2.0
経済学で読み解く「働き方」と「イノベーション」2.0
 
人材・組織を生かすコミュニティ戦略
人材・組織を生かすコミュニティ戦略人材・組織を生かすコミュニティ戦略
人材・組織を生かすコミュニティ戦略
 
資本主義と金融 2019
資本主義と金融 2019資本主義と金融 2019
資本主義と金融 2019
 
人材・組織を生かすマッチング戦略
人材・組織を生かすマッチング戦略人材・組織を生かすマッチング戦略
人材・組織を生かすマッチング戦略
 
マッチングの仕組み
マッチングの仕組みマッチングの仕組み
マッチングの仕組み
 

Recently uploaded

Speech, hearing, noise, intelligibility.pptx
Speech, hearing, noise, intelligibility.pptxSpeech, hearing, noise, intelligibility.pptx
Speech, hearing, noise, intelligibility.pptxpriyankatabhane
 
Pests of castor_Binomics_Identification_Dr.UPR.pdf
Pests of castor_Binomics_Identification_Dr.UPR.pdfPests of castor_Binomics_Identification_Dr.UPR.pdf
Pests of castor_Binomics_Identification_Dr.UPR.pdfPirithiRaju
 
ALL ABOUT MIXTURES IN GRADE 7 CLASS PPTX
ALL ABOUT MIXTURES IN GRADE 7 CLASS PPTXALL ABOUT MIXTURES IN GRADE 7 CLASS PPTX
ALL ABOUT MIXTURES IN GRADE 7 CLASS PPTXDole Philippines School
 
User Guide: Pulsar™ Weather Station (Columbia Weather Systems)
User Guide: Pulsar™ Weather Station (Columbia Weather Systems)User Guide: Pulsar™ Weather Station (Columbia Weather Systems)
User Guide: Pulsar™ Weather Station (Columbia Weather Systems)Columbia Weather Systems
 
Radiation physics in Dental Radiology...
Radiation physics in Dental Radiology...Radiation physics in Dental Radiology...
Radiation physics in Dental Radiology...navyadasi1992
 
Harmful and Useful Microorganisms Presentation
Harmful and Useful Microorganisms PresentationHarmful and Useful Microorganisms Presentation
Harmful and Useful Microorganisms Presentationtahreemzahra82
 
GenBio2 - Lesson 1 - Introduction to Genetics.pptx
GenBio2 - Lesson 1 - Introduction to Genetics.pptxGenBio2 - Lesson 1 - Introduction to Genetics.pptx
GenBio2 - Lesson 1 - Introduction to Genetics.pptxBerniceCayabyab1
 
BIOETHICS IN RECOMBINANT DNA TECHNOLOGY.
BIOETHICS IN RECOMBINANT DNA TECHNOLOGY.BIOETHICS IN RECOMBINANT DNA TECHNOLOGY.
BIOETHICS IN RECOMBINANT DNA TECHNOLOGY.PraveenaKalaiselvan1
 
Environmental Biotechnology Topic:- Microbial Biosensor
Environmental Biotechnology Topic:- Microbial BiosensorEnvironmental Biotechnology Topic:- Microbial Biosensor
Environmental Biotechnology Topic:- Microbial Biosensorsonawaneprad
 
User Guide: Magellan MX™ Weather Station
User Guide: Magellan MX™ Weather StationUser Guide: Magellan MX™ Weather Station
User Guide: Magellan MX™ Weather StationColumbia Weather Systems
 
Pests of soyabean_Binomics_IdentificationDr.UPR.pdf
Pests of soyabean_Binomics_IdentificationDr.UPR.pdfPests of soyabean_Binomics_IdentificationDr.UPR.pdf
Pests of soyabean_Binomics_IdentificationDr.UPR.pdfPirithiRaju
 
Microphone- characteristics,carbon microphone, dynamic microphone.pptx
Microphone- characteristics,carbon microphone, dynamic microphone.pptxMicrophone- characteristics,carbon microphone, dynamic microphone.pptx
Microphone- characteristics,carbon microphone, dynamic microphone.pptxpriyankatabhane
 
Pests of Blackgram, greengram, cowpea_Dr.UPR.pdf
Pests of Blackgram, greengram, cowpea_Dr.UPR.pdfPests of Blackgram, greengram, cowpea_Dr.UPR.pdf
Pests of Blackgram, greengram, cowpea_Dr.UPR.pdfPirithiRaju
 
CHROMATOGRAPHY PALLAVI RAWAT.pptx
CHROMATOGRAPHY  PALLAVI RAWAT.pptxCHROMATOGRAPHY  PALLAVI RAWAT.pptx
CHROMATOGRAPHY PALLAVI RAWAT.pptxpallavirawat456
 
《Queensland毕业文凭-昆士兰大学毕业证成绩单》
《Queensland毕业文凭-昆士兰大学毕业证成绩单》《Queensland毕业文凭-昆士兰大学毕业证成绩单》
《Queensland毕业文凭-昆士兰大学毕业证成绩单》rnrncn29
 
GENERAL PHYSICS 2 REFRACTION OF LIGHT SENIOR HIGH SCHOOL GENPHYS2.pptx
GENERAL PHYSICS 2 REFRACTION OF LIGHT SENIOR HIGH SCHOOL GENPHYS2.pptxGENERAL PHYSICS 2 REFRACTION OF LIGHT SENIOR HIGH SCHOOL GENPHYS2.pptx
GENERAL PHYSICS 2 REFRACTION OF LIGHT SENIOR HIGH SCHOOL GENPHYS2.pptxRitchAndruAgustin
 
Vision and reflection on Mining Software Repositories research in 2024
Vision and reflection on Mining Software Repositories research in 2024Vision and reflection on Mining Software Repositories research in 2024
Vision and reflection on Mining Software Repositories research in 2024AyushiRastogi48
 
The dark energy paradox leads to a new structure of spacetime.pptx
The dark energy paradox leads to a new structure of spacetime.pptxThe dark energy paradox leads to a new structure of spacetime.pptx
The dark energy paradox leads to a new structure of spacetime.pptxEran Akiva Sinbar
 
Best Call Girls In Sector 29 Gurgaon❤️8860477959 EscorTs Service In 24/7 Delh...
Best Call Girls In Sector 29 Gurgaon❤️8860477959 EscorTs Service In 24/7 Delh...Best Call Girls In Sector 29 Gurgaon❤️8860477959 EscorTs Service In 24/7 Delh...
Best Call Girls In Sector 29 Gurgaon❤️8860477959 EscorTs Service In 24/7 Delh...lizamodels9
 
basic entomology with insect anatomy and taxonomy
basic entomology with insect anatomy and taxonomybasic entomology with insect anatomy and taxonomy
basic entomology with insect anatomy and taxonomyDrAnita Sharma
 

Recently uploaded (20)

Speech, hearing, noise, intelligibility.pptx
Speech, hearing, noise, intelligibility.pptxSpeech, hearing, noise, intelligibility.pptx
Speech, hearing, noise, intelligibility.pptx
 
Pests of castor_Binomics_Identification_Dr.UPR.pdf
Pests of castor_Binomics_Identification_Dr.UPR.pdfPests of castor_Binomics_Identification_Dr.UPR.pdf
Pests of castor_Binomics_Identification_Dr.UPR.pdf
 
ALL ABOUT MIXTURES IN GRADE 7 CLASS PPTX
ALL ABOUT MIXTURES IN GRADE 7 CLASS PPTXALL ABOUT MIXTURES IN GRADE 7 CLASS PPTX
ALL ABOUT MIXTURES IN GRADE 7 CLASS PPTX
 
User Guide: Pulsar™ Weather Station (Columbia Weather Systems)
User Guide: Pulsar™ Weather Station (Columbia Weather Systems)User Guide: Pulsar™ Weather Station (Columbia Weather Systems)
User Guide: Pulsar™ Weather Station (Columbia Weather Systems)
 
Radiation physics in Dental Radiology...
Radiation physics in Dental Radiology...Radiation physics in Dental Radiology...
Radiation physics in Dental Radiology...
 
Harmful and Useful Microorganisms Presentation
Harmful and Useful Microorganisms PresentationHarmful and Useful Microorganisms Presentation
Harmful and Useful Microorganisms Presentation
 
GenBio2 - Lesson 1 - Introduction to Genetics.pptx
GenBio2 - Lesson 1 - Introduction to Genetics.pptxGenBio2 - Lesson 1 - Introduction to Genetics.pptx
GenBio2 - Lesson 1 - Introduction to Genetics.pptx
 
BIOETHICS IN RECOMBINANT DNA TECHNOLOGY.
BIOETHICS IN RECOMBINANT DNA TECHNOLOGY.BIOETHICS IN RECOMBINANT DNA TECHNOLOGY.
BIOETHICS IN RECOMBINANT DNA TECHNOLOGY.
 
Environmental Biotechnology Topic:- Microbial Biosensor
Environmental Biotechnology Topic:- Microbial BiosensorEnvironmental Biotechnology Topic:- Microbial Biosensor
Environmental Biotechnology Topic:- Microbial Biosensor
 
User Guide: Magellan MX™ Weather Station
User Guide: Magellan MX™ Weather StationUser Guide: Magellan MX™ Weather Station
User Guide: Magellan MX™ Weather Station
 
Pests of soyabean_Binomics_IdentificationDr.UPR.pdf
Pests of soyabean_Binomics_IdentificationDr.UPR.pdfPests of soyabean_Binomics_IdentificationDr.UPR.pdf
Pests of soyabean_Binomics_IdentificationDr.UPR.pdf
 
Microphone- characteristics,carbon microphone, dynamic microphone.pptx
Microphone- characteristics,carbon microphone, dynamic microphone.pptxMicrophone- characteristics,carbon microphone, dynamic microphone.pptx
Microphone- characteristics,carbon microphone, dynamic microphone.pptx
 
Pests of Blackgram, greengram, cowpea_Dr.UPR.pdf
Pests of Blackgram, greengram, cowpea_Dr.UPR.pdfPests of Blackgram, greengram, cowpea_Dr.UPR.pdf
Pests of Blackgram, greengram, cowpea_Dr.UPR.pdf
 
CHROMATOGRAPHY PALLAVI RAWAT.pptx
CHROMATOGRAPHY  PALLAVI RAWAT.pptxCHROMATOGRAPHY  PALLAVI RAWAT.pptx
CHROMATOGRAPHY PALLAVI RAWAT.pptx
 
《Queensland毕业文凭-昆士兰大学毕业证成绩单》
《Queensland毕业文凭-昆士兰大学毕业证成绩单》《Queensland毕业文凭-昆士兰大学毕业证成绩单》
《Queensland毕业文凭-昆士兰大学毕业证成绩单》
 
GENERAL PHYSICS 2 REFRACTION OF LIGHT SENIOR HIGH SCHOOL GENPHYS2.pptx
GENERAL PHYSICS 2 REFRACTION OF LIGHT SENIOR HIGH SCHOOL GENPHYS2.pptxGENERAL PHYSICS 2 REFRACTION OF LIGHT SENIOR HIGH SCHOOL GENPHYS2.pptx
GENERAL PHYSICS 2 REFRACTION OF LIGHT SENIOR HIGH SCHOOL GENPHYS2.pptx
 
Vision and reflection on Mining Software Repositories research in 2024
Vision and reflection on Mining Software Repositories research in 2024Vision and reflection on Mining Software Repositories research in 2024
Vision and reflection on Mining Software Repositories research in 2024
 
The dark energy paradox leads to a new structure of spacetime.pptx
The dark energy paradox leads to a new structure of spacetime.pptxThe dark energy paradox leads to a new structure of spacetime.pptx
The dark energy paradox leads to a new structure of spacetime.pptx
 
Best Call Girls In Sector 29 Gurgaon❤️8860477959 EscorTs Service In 24/7 Delh...
Best Call Girls In Sector 29 Gurgaon❤️8860477959 EscorTs Service In 24/7 Delh...Best Call Girls In Sector 29 Gurgaon❤️8860477959 EscorTs Service In 24/7 Delh...
Best Call Girls In Sector 29 Gurgaon❤️8860477959 EscorTs Service In 24/7 Delh...
 
basic entomology with insect anatomy and taxonomy
basic entomology with insect anatomy and taxonomybasic entomology with insect anatomy and taxonomy
basic entomology with insect anatomy and taxonomy
 

Optimization Approach to Nash Euilibria with Applications to Interchangeability

  • 1. 580 Optimization Approach to Nash Equilibria with Applications to Interchangeability Yosuke YASUDA Osaka University, Department of Economics (visiting ISEG, University of Lisbon) yasuda@econ.osaka-u.ac.jp July, 2021 1 / 18
  • 2. Summary What is Optimization Approach? (1st Part) The set of Nash equilibria, if it is nonempty, is identical to the set of minimizers of real-valued function. Connect equilibrium problem to optimization problem. → Similar characterizations are known in the literature. Is it Useful? Any application? (2nd Part) Existing results on interchangeability can be derived, in a unified fashion, by lattice structure of optimal solutions. → NEW contribution! (looking for ompletely new results...) Main Messages Please use/apply/extend our characterization of NE! 2 / 18
  • 3. Traditional Formulations of NE Strategy profile x∗ ∈ X is called Nash equilibrium if and only if, 1 Inequality (Incentive) Constraints ui(x∗ i , x∗ −i) ≥ ui(xi, x∗ −i) for all xi ∈ Xi and for all i ∈ N. 2 Solution to Multivariate Function ui(x∗ i , x∗ −i) = max xi∈Xi ui(xi, x∗ −i) for all i ∈ N. 3 Fixed Point of BR Correspondence x∗ ∈ BR(x∗ ), where BRi(x−i) = arg max x0 i∈Xi ui(x0 i, x−i). 3 / 18
  • 4. Alternative: Optimization Approach Define f : X → R, which aggregates maximum deviation gains (from a fixed action profile x ∈ X) across players. f(x) = X i∈N max x0 i∈Xi ui(x0 i, x−i) − ui(xi, x−i) . (1) Theorem 1 A strategy profile x∗ is a Nash equilibrium iff f(x∗) = 0. Theorem 2 If there exists an NE, the set of Nash equilibria E∗ is identical to the set of minimum solutions to f, i.e., arg minx∈X f(x). 4 / 18
  • 5. Example: Prisoner’s Dilemma Table: Payoff Matrix C D C 3, 3 0, 4 D 4, 0 1, 1 Table: Values of f C D C 2 (= (4 − 3) + (4 − 3)) 1 (= (1 − 0) + 0) D 1 (= 0 + (1 − 0)) 0 (= 0 + 0) 5 / 18
  • 6. Extensions Let g(x) = −f(x). The set of Nash equilibria, if it is nonempty, is identical to the set of maximum solutions to g. arg max x∈X g(x). f can be replaced by ˜ f : X → R, using a sign-preserving function ψi : R+ → R+ such that ψi(x) = 0 iff x = 0. ˜ f(x) = X i∈N ψi max x0 i∈Xi ui(x0 i, x−i) − ui(xi, x−i) . Let t be a parameter contained in a parameter set T. Then, (1) can be rewritten to incorporate this parameterization. f(x, t) = X i∈N max x0 i∈Xi ui(x0 i, x−i; t) − ui(xi, x−i; t) . 6 / 18
  • 7. From “Sum” to “Product” The parallel characterization can be available when the objective function is replaced with the product of deviation gains. f(x) = Πi∈N 1 + max x0 i∈Xi ui(x0 i, x−i) − ui(xi, x−i) . (2) Note by construction that f(x) ≥ 1 holds for any x ∈ X. Lemma 3 A strategy profile x∗ is an NE iff f(x∗) = 1. If there is an NE, E∗ is identical to the set of minimum solutions to f, arg minx∈X f(x). 1 can be replaced with any ε 0. (Then, f(x∗) = εn) As ε goes to 0, (2) converges to the product of players’ payoff differences, which may look similar to the Nash product. 7 / 18
  • 8. Interchangeability for Two-Person Games Let x = (x1, x2) and x0 = (x0 1, x0 2) be two distinct NE. Definition 4 A pair of Nash equilibia x and x0 is called interchangeable if (x1, x0 2) and (x0 1, x2) constitute NE of the same game. Our approach can explain the following existing results on interchangeability, independently derived in the literature: 1 for a zero-sum game any pairs of its mixed strategy Nash equilibria are interchangeable (Luce and Raiffa, 1957). 2 for a supermodular game where each player’s strategy space is totally ordered, any unordered pairs of the pure strategy Nash equilibria are interchangeable (Echenique, 2003). 3 equilibrium set of a strictly supermodular game with totally ordered strategy spaces, is totally ordered (Vives, 1985). 8 / 18
  • 9. Introduction to Lattice (1) Let = be a binary relation on a non-empty set S. Definition 5 The pair (S, =) is a partially ordered set if, for x, y, z in S, = is reflexive: x = x. transitive: x = y and y = z implies x = z. antisymmetric: x = y and y = x implies x = y. A partially ordered set (S, =) is totally ordered if for x and y in S either x = y or y = x is satisfied, and is called chain. called lattice if any two elements have a least upper bound (join, ∨) and a greatest lower bound (meet, ∧) in the set. A subset S∗(⊂ S) is called sublattice if x0 ∧ x00 ∈ S∗ and x0 ∨ x00 ∈ S∗ hold for any x0, x00 ∈ S∗. 9 / 18
  • 10. Introduction to Lattice (2) Definition 6 A real-valued function h defined over a lattice S is called a submodular function if, for any x0, x00 ∈ S, h satisfies h(x0 ∧ x00 ) + h(x0 ∨ x00 ) − {h(x0 ) + h(x00 )} ≤ 0. (3) (3) trivially holds with equality whenever x0 and x00 are ordered, i.e., x0 = x00 or x0 5 x00. If ≤ in (3) is replaced with ≥, h is called supermodular. h : S → R becomes a strictly submodular function if, for any unordered pair x0, x00 ∈ S, i.e., x0 x00 and x0 x00, h satisfies h(x0 ∧ x00 ) + h(x0 ∨ x00 ) − {h(x0 ) + h(x00 )} 0. (4) If in (4) is replaced with , h is strictly supermodular. 10 / 18
  • 11. Results by Topkis (1978) Fact 7 (Topkis, 1978) If h is a submodular function on a lattice S, then the set S∗ of points at which h attains its minimum on S is a sublattice of S. Fact 8 (Topkis, 1978) If h is st. submodular on a lattice S, then the set S∗ of points at which h attains its minimum on S is a chain. Assume X is a lattice. The above facts imply the following. Lemma 9 Suppose that f is defined by (1) and E∗ is nonempty. Then, (i) If f is submodular on X, then E∗ is a sublattice of X. (ii) If f is st. submodular on X, then E∗ is a chain. 11 / 18
  • 12. Supermodular Game Let us define u as the sum of the payoff functions. u(x) = u1(x) + u2(x) for all x ∈ X. Lemma 10 For any two-person game with totally ordered strategy space for each player, (i) f is submodular iff u is supermodular. (ii) f is st. submodular iff u is st. supermodular. Lemma 11 u (= u1 + u2) is supermodular (resp. strictly supermodular) for any two-person supermodular (resp. strictly supermodular) games. Supermodularity is preserved under addition. The converse is not true, e.g., zero-sum game. 12 / 18
  • 13. Proof of Lemma 10 (1) Recall that f is a submodular function if, for any x0, x00 ∈ X, f(x0 ∧ x00 ) + f(x0 ∨ x00 ) − {f(x0 ) + f(x00 )} ≤ 0. (5) If the above inequality is strict for any unordered pairs, f is a st. submodular function. Since we consider two-person games, f(x) = max x1∈X1 u1(x1, x2) − u1(x1, x2) + max x2∈X2 u2(x1, x2) − u2(x1, x2). Now consider a pair of unordered strategy profiles, x0 = (x0 1, x0 2) and x00 = (x00 1, x00 2). W.o.l.g, assume x0 1 =1 x00 1 and x0 2 52 x00 2. Join: x0 ∧ x00 = (x00 1, x0 2) Meet: x0 ∨ x00 = (x0 1, x00 2) 13 / 18
  • 14. Proof of Lemma 10 (2) The corresponding values of f are expressed by f(x0 ∧ x00 ) = max x1∈X1 u1(x1, x0 2) − u1(x00 1, x0 2) + max x2∈X2 u2(x00 1, x2) − u2(x00 1, x0 2). f(x0 ∨ x00 ) = max x1∈X1 u1(x1, x00 2) − u1(x0 1, x00 2) + max x2∈X2 u2(x00 1, x2) − u2(x0 1, x00 2). Substituting them into (5), max ui parts will be canceled out. The next equality illustrates that the (st.) submodularity of f is completely characterized by the (st.) supermodularity of u. 14 / 18
  • 15. Proof of Lemma 10 (3) f(x0 ∧ x00 ) + f(x0 ∨ x00 ) − {f(x0 ) + f(x00 )} = − { u1(x00 1, x0 2) + u2(x00 1, x0 2) + u1(x0 1, x00 2) + u2(x0 1, x00 2)} + u1(x0 1, x0 2) + u2(x0 1, x0 2) + u1(x00 1, x00 2) + u2(x00 1, x00 2) = − { u1(x0 ∧ x00 ) + u2(x0 ∧ x00 ) + u1(x0 ∨ x00 ) + u2(x0 ∨ x00 )} + u1(x0 ) + u2(x0 ) + u1(x00 ) + u2(x00 ) = u(x0 ) + u(x00 ) − {u(x0 ∧ x00 ) + u(x0 ∨ x00 )}. Since u = u1 + u2 is constant for a zero-sum game, we obtain: Lemma 12 For any two-person zero-sum game, f is submodular over mixed strategy profiles with any order of strategy space for each player. 15 / 18
  • 16. Main Result: Zero-Sum Game Theorem 13 For a zero-sum game, any pairs of its (mixed strategy) Nash equilibria are interchangeable. Proof. E∗ is nonempty. Existence of NE by Nash (1950) Existence of minimax solution by Neumann (1928). Suppose that x = (x1, x2) and x0 = (x0 1, x0 2) are two distinct NE. We can always construct an order that satisfies x1 =1 x0 1 and x2 52 x0 2. By Lemma 9 (i), E∗ is sublattice. ⇒ x ∧ x0 = (x0 1, x2) and x ∨ x0 = (x1, x0 2) are both NE. 16 / 18
  • 17. Main Result: Supermodular Game Since the existence of (pure strategy) NE for supermodular games is guaranteed by Topkis (1979), we obtain the next theorem. Theorem 14 Assume strategy space for each player is totally ordered. Then, (i) For a two-person supermodular game, any unordered pairs of its pure strategy NE are interchangeable. (ii) For a two-person st. supermodular game, all pure strategy NE are totally ordered. The above results also hold for log-supermodular games. If ui is log-supermodular, then ˆ f must be submodular. (Note f = 0 iff ˆ f = 0) ˆ f(x) = X i∈N max x0 i∈Xi ln ui(x0 i, x−i) − ln ui(xi, x−i) . 17 / 18
  • 18. Conclusion Summary: Provide a functional formulation of NE. Enables us to analyze Nash equilibrium as a solution to an optimization problem without any constraints. May connect non-cooperative game theory with other related fields such as OR and CS. Natural Reaction: So what? Is it really useful? → New insight on interchangeability of NE. Existing results on two person (i) zero-sum games and (ii) supermodular games can be derived, in a unified fashion: The set of minimizers of submodular function is sublattice. Applications to symmetric, potential, cooperative games (via Nash implementation), etc? → Future research! 18 / 18