src/Doc/Datatypes/Setup.thy
author nipkow
Thu, 03 Jul 2025 13:53:14 +0200
changeset 82802 547335b41005
parent 69605 a96320074298
permissions -rw-r--r--
removed duplicate lemma; added the notion of the kernel of a function
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