reduced dependencies + updated docs
authorblanchet
Mon, 20 Jan 2014 18:24:56 +0100
changeset 55073 9b96fb4c8cfd
parent 55072 8488fdc4ddc0
child 55074 2b0b6f69b148
reduced dependencies + updated docs
src/Doc/Datatypes/Datatypes.thy
src/Doc/Datatypes/Setup.thy
src/Doc/ROOT
src/HOL/BNF/README.html
--- a/src/Doc/Datatypes/Datatypes.thy	Mon Jan 20 18:24:56 2014 +0100
+++ b/src/Doc/Datatypes/Datatypes.thy	Mon Jan 20 18:24:56 2014 +0100
@@ -8,7 +8,11 @@
 *)
 
 theory Datatypes
-imports Setup "~~/src/HOL/Library/Simps_Case_Conv"
+imports
+  Setup
+  "~~/src/HOL/BNF/BNF_Decl"
+  "~~/src/HOL/BNF/More_BNFs"
+  "~~/src/HOL/Library/Simps_Case_Conv"
 begin
 
 section {* Introduction
@@ -74,20 +78,10 @@
 finitely many direct subtrees, whereas those of the second and fourth may have
 infinite branching.
 
-To use the package, it is necessary to import the @{theory BNF} theory, which
-can be precompiled into the \texttt{HOL-BNF} image. The following commands show
-how to launch jEdit/PIDE with the image loaded and how to build the image
-without launching jEdit:
-*}
-
-text {*
-\noindent
-\ \ \ \ \texttt{isabelle jedit -l HOL-BNF} \\
-\noindent
-\hbox{}\ \ \ \ \texttt{isabelle build -b HOL-BNF}
-*}
-
-text {*
+The package is part of @{theory Main}. Additional functionality is provided by
+the theories @{theory BNF_Decl} and @{theory More_BNFs}, located in the
+@{text "~~/src/HOL/BNF"} directory.
+
 The package, like its predecessor, fully adheres to the LCF philosophy
 \cite{mgordon79}: The characteristic theorems associated with the specified
 (co)datatypes are derived rather than introduced axiomatically.%
@@ -2512,7 +2506,7 @@
 Tobias Nipkow and Makarius Wenzel encouraged us to implement the new
 (co)datatype package. Andreas Lochbihler provided lots of comments on earlier
 versions of the package, especially for the coinductive part. Brian Huffman
-suggested major simplifications to the internal constructions, much of which has
+suggested major simplifications to the internal constructions, many of which has
 yet to be implemented. Florian Haftmann and Christian Urban provided general
 advice on Isabelle and package writing. Stefan Milius and Lutz Schr\"oder
 found an elegant proof to eliminate one of the BNF assumptions. Andreas
--- a/src/Doc/Datatypes/Setup.thy	Mon Jan 20 18:24:56 2014 +0100
+++ b/src/Doc/Datatypes/Setup.thy	Mon Jan 20 18:24:56 2014 +0100
@@ -1,5 +1,5 @@
 theory Setup
-imports BNF
+imports Main
 begin
 
 ML_file "../antiquote_setup.ML"
--- a/src/Doc/ROOT	Mon Jan 20 18:24:56 2014 +0100
+++ b/src/Doc/ROOT	Mon Jan 20 18:24:56 2014 +0100
@@ -37,7 +37,7 @@
     "document/root.tex"
     "document/style.sty"
 
-session Datatypes (doc) in "Datatypes" = "HOL-BNF" +
+session Datatypes (doc) in "Datatypes" = HOL +
   options [document_variants = "datatypes"]
   theories [document = false] Setup
   theories Datatypes
--- a/src/HOL/BNF/README.html	Mon Jan 20 18:24:56 2014 +0100
+++ /dev/null	Thu Jan 01 00:00:00 1970 +0000
@@ -1,49 +0,0 @@
-<!DOCTYPE HTML PUBLIC "-//W3C//DTD HTML 4.01 Transitional//EN" "http://www.w3.org/TR/html4/loose.dtd">
-
-<html>
-
-<head>
-  <meta http-equiv="Content-Type" content="text/html; charset=iso-8859-1">
-  <title>BNF Package</title>
-</head>
-
-<body>
-
-<h3><i>BNF</i>: A (co)datatype package based on bounded natural functors
-(BNFs)</h3>
-
-<p>
-The <i>BNF</i> package provides a fully modular framework for constructing
-inductive and coinductive datatypes in HOL, with support for mixed mutual and
-nested (co)recursion. Mixed (co)recursion enables type definitions involving
-both datatypes and codatatypes, such as the type of finitely branching trees of
-possibly infinite depth. The framework draws heavily from category theory.
-
-<p>
-The package is described in <tt>isabelle doc datatypes</tt> and in the following
-paper:
-
-<ul>
-  <li><a href="http://www21.in.tum.de/~traytel/papers/lics12-codatatypes/index.html">Foundational, Compositional (Co)datatypes for Higher-Order Logic&mdash;Category Theory Applied to Theorem Proving</a>, <br>
-  Dmitriy Traytel, Andrei Popescu, and Jasmin Christian Blanchette.<br>
-  <i>Logic in Computer Science (LICS 2012)</i>, 2012.
-</ul>
-
-<p>
-Most of the package is loaded as part of <tt>Main.thy</tt>. Additional
-functionality is provided by <tt>BNF.thy</tt>. The <tt>Examples</tt> directory
-contains various examples of (co)datatypes, including the examples from the
-paper.
-
-<p>
-The key notion underlying the package is that of a <i>bounded natural functor</i>
-(<i>BNF</i>)&mdash;an enriched type constructor satisfying specific properties
-preserved by interesting categorical operations (composition, least fixed point,
-and greatest fixed point). The <tt>Basic_BNFs.thy</tt>, <tt>More_BNFs.thy</tt>,
-and <tt>Countable_Set_Type.thy</tt> files register various basic types, notably
-for sums, products, function spaces, finite sets, multisets, and countable sets.
-Custom BNFs can be registered as well.
-
-</body>
-
-</html>