src/Doc/Codegen/Setup.thy
author haftmann
Thu, 26 Jun 2025 17:25:29 +0200
changeset 82774 2865a6618cba
parent 81136 2b949a3bfaac
permissions -rw-r--r--
append (rather than prepend) code equations: the order within a theory is maintained in the resulting code

theory Setup
imports
  Complex_Main
  "HOL-Library.Dlist"
  "HOL-Library.RBT"
  "HOL-Library.Mapping"
  "HOL-Library.IArray"
begin

ML_file \<open>../antiquote_setup.ML\<close>
ML_file \<open>../more_antiquote.ML\<close>

unbundle constrain_space_syntax

declare [[default_code_width = 74]]

declare [[names_unique = false]]

end