Theory CombinatorialAuctionExamples
section ‹VCG auction: three simple examples evaluating the VCG allocation algorithm
vcgaAlg and the price determination algorithm vcgpAlg in Isabelle›
theory CombinatorialAuctionExamples
imports
CombinatorialAuction
begin
definition "r1 = 0"
definition "N1 = {1,2,3::integer}"
definition "Ω1 = [11, 12]"
definition "b1 = {((1::integer, {11::integer, 12}), 2::nat),
((2, {11}), 2),
((2, {12}), 2),
((3, {11}), 2),
((3, {12}), 2)}"
definition "vcga1 = vcgaAlg N1 Ω1 (b1 Elsee 0) r1"
value "vcga1"
value [nbe] "vcgpAlg N1 Ω1 (b1 Elsee 0) r1 1 vcga1"
value [nbe] "vcgpAlg N1 Ω1 (b1 Elsee 0) r1 2 vcga1"
value [nbe] "vcgpAlg N1 Ω1 (b1 Elsee 0) r1 3 vcga1"
definition "r2 = 1"
definition "N2 = {1,2,3::integer}"
definition "Ω2 = [11, 12]"
definition "b2 = {((1::integer, {11::integer, 12}), 5::nat),
((2, {11}), 3),
((2, {12}), 3),
((3, {11}), 2),
((3, {12}), 4)}"
definition "vcga2 = vcgaAlg N2 Ω2 (b2 Elsee 0) r2"
value "vcga2"
value [nbe] "vcgpAlg N2 Ω2 (b2 Elsee 0) r2 1 vcga2"
value [nbe] "vcgpAlg N2 Ω2 (b2 Elsee 0) r2 2 vcga2"
value [nbe] "vcgpAlg N2 Ω2 (b2 Elsee 0) r2 3 vcga2"
definition "r3 = 0"
definition "N3 = {1,2,3::integer}"
definition "Ω3 = [11, 12, 13]"
definition "b3 = {((1::integer, {11::integer, 12, 13}), 20::nat),
((1, {11,12}), 18),
((2, {11}), 10),
((2, {12}), 15),
((2, {13}), 15),
((2, {12,13}), 18),
((3, {11}), 2),
((3, {11,12}), 12),
((3, {11,13}), 17),
((3, {12,13}), 18),
((3, {11,12,13}), 19)}"
definition "vcga3 = vcgaAlg N3 Ω3 (b3 Elsee 0) r3"
value "vcga3"
value [nbe] "vcgpAlg N3 Ω3 (b3 Elsee 0) r3 1 vcga3"
value [nbe] "vcgpAlg N3 Ω3 (b3 Elsee 0) r3 2 vcga3"
value [nbe] "vcgpAlg N3 Ω3 (b3 Elsee 0) r3 3 vcga3"
end