lh-l4v/proof/invariant-abstract/RISCV64/ArchCrunchSetup_AI.thy

20 lines
316 B
Plaintext

(*
* Copyright 2020, Data61, CSIRO (ABN 41 687 119 230)
*
* SPDX-License-Identifier: GPL-2.0-only
*)
theory ArchCrunchSetup_AI
imports
"ASpec.Syscall_A"
"Lib.Crunch_Instances_NonDet"
begin
context Arch begin global_naming RISCV64
crunch_ignore (add: debugPrint clearMemory pt_lookup_from_level)
end
end