Theory Update
section ‹Bisping's Updates›
theory Update
imports Energy_Order
begin
text ‹
In this theory we define a superset of Bisping's updates and their application. Further, we introduce Bisping's ``inversion''
of updates and relate the two.
›
subsection ‹Bisping's Updates›
text ‹
Bisping allows three ways of updating a component of an energy: ‹zero› does not change the respective entry,
‹minus_one› subtracts one and ‹min_set› $A$ for some set $A$ replaces the entry by the
minimum of entries whose index is contained in $A$. We further add ‹plus_one› to add one and omit the assumption that the a minimum has to consider the component it replaces.
Updates are vectors where each entry contains the information, how the update changes the respective
component of energies. We now introduce a datatype such that updates can be represented as lists of ‹update_component›s.
›