diff -r fae6233c5f37 -r 8ffc4d0e652d src/HOL/HOLCF/Algebraic.thy --- a/src/HOL/HOLCF/Algebraic.thy Wed Jan 13 23:02:28 2016 +0100 +++ b/src/HOL/HOLCF/Algebraic.thy Wed Jan 13 23:07:06 2016 +0100 @@ -2,7 +2,7 @@ Author: Brian Huffman *) -section {* Algebraic deflations *} +section \Algebraic deflations\ theory Algebraic imports Universal Map_Functions @@ -10,7 +10,7 @@ default_sort bifinite -subsection {* Type constructor for finite deflations *} +subsection \Type constructor for finite deflations\ typedef 'a fin_defl = "{d::'a \ 'a. finite_deflation d}" by (fast intro: finite_deflation_bottom) @@ -72,7 +72,7 @@ using finite_deflation_Rep_fin_defl by (rule finite_deflation_imp_compact) -subsection {* Defining algebraic deflations by ideal completion *} +subsection \Defining algebraic deflations by ideal completion\ typedef 'a defl = "{S::'a fin_defl set. below.ideal S}" by (rule below.ex_ideal) @@ -132,7 +132,7 @@ using defl_principal_def fin_defl_countable by (rule below.typedef_ideal_completion) -text {* Algebraic deflations are pointed *} +text \Algebraic deflations are pointed\ lemma defl_minimal: "defl_principal (Abs_fin_defl \) \ x" apply (induct x rule: defl.principal_induct, simp) @@ -147,7 +147,7 @@ lemma inst_defl_pcpo: "\ = defl_principal (Abs_fin_defl \)" by (rule defl_minimal [THEN bottomI, symmetric]) -subsection {* Applying algebraic deflations *} +subsection \Applying algebraic deflations\ definition cast :: "'a defl \ 'a \ 'a" @@ -215,7 +215,7 @@ lemma cast_strict2 [simp]: "cast\A\\ = \" by (rule cast.below [THEN bottomI]) -subsection {* Deflation combinators *} +subsection \Deflation combinators\ definition "defl_fun1 e p f =