src/Doc/Implementation/Base.thy
author wenzelm
Sat, 21 Oct 2023 00:13:12 +0200
changeset 78806 aca84704d46f
parent 69605 a96320074298
permissions -rw-r--r--
more standard simproc_setup using ML antiquotation;

(*:maxLineLen=78:*)

theory Base
imports Main
begin

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

end