(* * Copyright 2020, Data61, CSIRO (ABN 41 687 119 230) * * SPDX-License-Identifier: BSD-2-Clause *) (* * Regression for VER-320 and other array-related bugs. * Here we prove that writing a pointer that points into an array * will update the array. *) theory array_indirect_update imports "AutoCorres2_Main.AutoCorres_Main" begin