(* * Copyright 2020, Data61, CSIRO (ABN 41 687 119 230) * Copyright (c) 2023 Apple Inc. All rights reserved. * * SPDX-License-Identifier: BSD-2-Clause *) (* License: BSD, terms see file ./LICENSE *) theory HeapRawState imports CTypes begin type_synonym typ_base = bool datatype s_heap_index = SIndexVal | SIndexTyp nat