Equations
instance
instDecidableIsExpertOfDecidableRelFin
{n : ℕ}
{s : GossipState n}
[DecidableRel s]
{i : Fin n}
:
instance
instDecidableRelFinMakeCall
{n : ℕ}
{s : GossipState n}
[DecidableRel s]
{c : Call n}
:
DecidableRel (makeCall s c)
Equations
- instDecidableRelFinMakeCall x✝¹ x✝ = if h : x✝¹ = i then decidable_of_iff (s i x✝ ∨ s j x✝) ⋯ else if h' : x✝¹ = j then decidable_of_iff (s j x✝ ∨ s i x✝) ⋯ else decidable_of_iff (s x✝¹ x✝) ⋯
Equations
- makeCalls s cs = List.foldl makeCall s cs
Instances For
instance
instDecidableRelFinMakeCalls
{n : ℕ}
{s : GossipState n}
[DecidableRel s]
{cs : List (Call n)}
:
DecidableRel (makeCalls s cs)
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- moreGossip s1 s2 = ∀ (a b : Fin n), s1 a b → s2 a b
Instances For
Equations
Instances For
Equations
- stateEquivalence s1 s2 = ∀ (a b : Fin n), s1 a b ↔ s2 a b
Instances For
theorem
makeCall_increases_gossip
{n : ℕ}
(s1 s2 : GossipState n)
(c : Call n)
:
moreGossip s1 s2 → moreGossip (makeCall s1 c) (makeCall s2 c)
theorem
makeCallsIncreasesGossip
{n : ℕ}
(s1 s2 : GossipState n)
(cs : List (Call n))
:
moreGossip s1 s2 → moreGossip (makeCalls s1 cs) (makeCalls s2 cs)
theorem
callsIncreaseGossip
{n : ℕ}
(s : GossipState n)
(cs : List (Call n))
:
moreGossip s (makeCalls s cs)