* HOL/List: new function list_update written xs[i:=v] that updates the i-th
list position. May also be iterated as in xs[i:=a,j:=b,...].
(*Dummy theory to document dependencies *)
Datatype = "constructor" + "inductive" + "coinductive" + Univ + QUniv
(*this must be capital to avoid conflicts with ML's "datatype" *)