src/Doc/Datatypes/Setup.thy
author wenzelm
Tue, 16 Nov 2021 21:21:15 +0100
changeset 74798 507f50dbeb79
parent 69605 a96320074298
permissions -rw-r--r--
just one Presentation.State for all sessions: avoid duplication of already presented theories (very slow) and cached theory export (not very slow);
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
52822
ae938ac9a721 more (co)datatype docs
blanchet
parents:
diff changeset
     1
theory Setup
55073
9b96fb4c8cfd reduced dependencies + updated docs
blanchet
parents: 52824
diff changeset
     2
imports Main
52822
ae938ac9a721 more (co)datatype docs
blanchet
parents:
diff changeset
     3
begin
ae938ac9a721 more (co)datatype docs
blanchet
parents:
diff changeset
     4
69605
a96320074298 isabelle update -u path_cartouches;
wenzelm
parents: 56059
diff changeset
     5
ML_file \<open>../antiquote_setup.ML\<close>
52822
ae938ac9a721 more (co)datatype docs
blanchet
parents:
diff changeset
     6
ae938ac9a721 more (co)datatype docs
blanchet
parents:
diff changeset
     7
end