(* * Copyright (c) 2022 Apple Inc. All rights reserved. * * SPDX-License-Identifier: BSD-2-Clause *) (* * Tests for handling Spec constructs emitted by the C parser. *) theory mmio_assume imports "AutoCorres2_Main.AutoCorres_Main" begin text ‹A variant of theory ‹mmio›, but assuming (instead of specifying) hardware behaviour.› declare [[c_parser_assume_fnspec]] text ‹Some placeholders for a 'hardware-step' relation.› consts abs_step:: "word32 ⇒ word32 ⇒ bool" consts abs_step2:: "(word32 × word32) ⇒ (word32 × word32) ⇒ bool" declare [[c_parser_feedback_level=2]] include_C_file "mmio.c" for "mmio_assume.c"