Documentation

FraudProof.Games.FromBtoMTree

structure ComputationTree (α : Type) :
  • computation : BTree α
  • res :
Instances For
    def dac_leaf_winning_condition {α : Type} [BEq ] [o : Hash α ] (hc : ) (a : α) (h : ) :
    Equations
    Instances For
      def dac_node_winning_condition { : Type} [BEq ] [m : HashMagma ] (top hl hr : ) :
      Equations
      Instances For
        def data_challenge_game {α : Type} [BEq ] [o : Hash α ] [m : HashMagma ] (da : ComputationTree ) (reveler : ABTree (Option α) (Option ( × ))) (chooser : ABTree Unit ( × × Option ChooserMoves)) :
        Equations
        • One or more equations did not get rendered due to their size.
        Instances For
          theorem dac_winning_gen_chooser {α : Type} [hash : Hash α ] [HashMagma ] [BEq ] [LawfulBEq ] (pub_data : ABTree Unit) (revealer : ABTree (Option α) (Option ( × ))) (rev_res : ) (chooser : ABTree (Option α) (Option ( × ))) (ch_res : ) (good_chooser : winning_condition_player (fun (hc : ) (a : α) (h : ) => dac_leaf_winning_condition hc a h = true) (fun (x : Unit) (x : × ) (res : ) => match x with | (l, r) => dac_node_winning_condition res l r = true) (fun (x : ) => id) { data := pub_data, res := ch_res } chooser) (hneq : ¬rev_res = ch_res) :
          data_challenge_game { computation := pub_data, res := rev_res } revealer (ABTree.map (fun (x : Option α) => ()) gen_chooser_opt chooser) = Player.Chooser
          def treeArbitrationGame {α : Type} [BEq ] [o : Hash α ] [m : HashMagma ] (da : ComputationTree ) (reveler : ABTree (Option α) (Option ( × ))) (chooser : ABTree Unit ( × × Option ChooserMoves)) :
          Equations
          • One or more equations did not get rendered due to their size.
          Instances For
            def arbitrationTree {α : Type} [BEq ] [o : Hash α ] [m : HashMagma ] (arena : ABTree Unit Unit) (res : ) (reveler : ABTree (Option α) (Option ( × ))) (chooser : ABTree Unit ( × × Option ChooserMoves)) :
            Equations
            • One or more equations did not get rendered due to their size.
            Instances For