Documentation

FraudProof.Games.Simultaneous

inductive SimWinner :
Instances For
    def leaf_game {α : Type} [DecidableEq ] [o : Hash α ] (a : α) (p commit : ) :
    Equations
    Instances For
      def node_game { : Type} [DecidableEq ] [mag : HashMagma ] (lp rp : × ) (commit : ) (recl recr : SimWinner) :
      Equations
      Instances For
        def simultaneous_game {α : Type} [o : Hash α ] [mag : HashMagma ] [DecidableEq ] (public_data : ABTree Unit) (lplayer : ABTree (Option α) (Option ( × ))) (lplayer_commit : ) (rplayer : ABTree Unit (Option ( × ))) :
        Equations
        Instances For
          def gen_to_chooser { : Type} [DecidableEq ] (md : Option ( × )) (a : × × ) :
          Equations
          • One or more equations did not get rendered due to their size.
          Instances For
            theorem eq_sim_games {α : Type} [o : Hash α ] [mag : HashMagma ] [DecidableEq ] (pub : ABTree Unit) (lplayer : ABTree (Option α) (Option ( × ))) (lplayer_commit : ) (rplayer : ABTree Unit (Option ( × ))) :
            treeArbitrationGame { computation := pub, res := lplayer_commit } lplayer (ABTree.map id gen_to_chooser rplayer) = Player.Proposer simultaneous_game pub lplayer lplayer_commit rplayer = SimWinner.Left
            def simultaneous_elemenin_game {α : Type} [o : Hash α ] [mag : HashMagma ] [DecidableEq ] (public_data : ABTree SkElem Unit) (lplayer : ABTree (Option α) (Option )) (lplayer_commit : × ) (rplayer : ABTree Unit (Option )) :
            Equations
            Instances For