diff -r 3b3089863eda -r 3a1b2d8c89aa src/Doc/Datatypes/Datatypes.thy --- a/src/Doc/Datatypes/Datatypes.thy Sun Apr 07 12:44:37 2019 +0200 +++ b/src/Doc/Datatypes/Datatypes.thy Sun Apr 07 08:26:57 2019 +0200 @@ -13,12 +13,16 @@ imports Setup "HOL-Library.BNF_Axiomatization" - "HOL-Library.Cardinal_Notations" "HOL-Library.Countable" "HOL-Library.FSet" "HOL-Library.Simps_Case_Conv" begin + +(*<*) +unbundle cardinal_syntax +(*>*) + section \Introduction \label{sec:introduction}\ @@ -2761,8 +2765,8 @@ text \ The example below shows how to register a type as a BNF using the @{command bnf} -command. Some of the proof obligations are best viewed with the theory -\<^file>\~~/src/HOL/Library/Cardinal_Notations.thy\ imported. +command. Some of the proof obligations are best viewed with the bundle +"cardinal_syntax" included. The type is simply a copy of the function space \<^typ>\'d \ 'a\, where \<^typ>\'a\ is live and \<^typ>\'d\ is dead. We introduce it together with its map function,