Theory Datatypes
theory Datatypes
imports
Setup
"HOL-Library.BNF_Axiomatization"
"HOL-Library.Countable"
"HOL-Library.FSet"
"HOL-Library.Simps_Case_Conv"
begin
unbundle cardinal_syntax
section ‹Introduction
\label{sec:introduction}›
text ‹
The 2013 edition of Isabelle introduced a definitional package for freely
generated datatypes and codatatypes. This package replaces the earlier
implementation due to Berghofer and Wenzel @{cite "Berghofer-Wenzel:1999:TPHOL"}.
Perhaps the main advantage of the new package is that it supports recursion
through a large class of non-datatypes, such as finite sets:
›