src/Doc/Implementation/Base.thy
author wenzelm
Sat, 05 Oct 2024 14:58:36 +0200
changeset 81116 0fb1e2dd4122
parent 69605 a96320074298
permissions -rw-r--r--
first-class support for "unbundle no foobar_syntax" -- avoid redundant "bundle no_foobar_syntax" definitions;

(*:maxLineLen=78:*)

theory Base
imports Main
begin

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

end