# HG changeset patch # User wenzelm # Date 1451507018 -3600 # Node ID b66d2ca1f907d1337e3429c9f91a46d582aadd1c # Parent 4d9518c3d031cff68adb1aa7fbd6c99acd7ec874 clarified print modes; diff -r 4d9518c3d031 -r b66d2ca1f907 src/HOL/HOLCF/Cfun.thy --- a/src/HOL/HOLCF/Cfun.thy Wed Dec 30 21:10:19 2015 +0100 +++ b/src/HOL/HOLCF/Cfun.thy Wed Dec 30 21:23:38 2015 +0100 @@ -15,16 +15,16 @@ definition "cfun = {f::'a => 'b. cont f}" -cpodef ('a, 'b) cfun (infixr "->" 0) = "cfun :: ('a => 'b) set" +cpodef ('a, 'b) cfun ("(_ \/ _)" [1, 0] 0) = "cfun :: ('a => 'b) set" unfolding cfun_def by (auto intro: cont_const adm_cont) -type_notation (xsymbols) - cfun ("(_ \/ _)" [1, 0] 0) +type_notation (ASCII) + cfun (infixr "->" 0) + +notation (ASCII) + Rep_cfun ("(_$/_)" [999,1000] 999) notation - Rep_cfun ("(_$/_)" [999,1000] 999) - -notation (xsymbols) Rep_cfun ("(_\/_)" [999,1000] 999) @@ -45,10 +45,10 @@ text {* Syntax for nested abstractions *} -syntax +syntax (ASCII) "_Lambda" :: "[cargs, logic] \ logic" ("(3LAM _./ _)" [1000, 10] 10) -syntax (xsymbols) +syntax "_Lambda" :: "[cargs, logic] \ logic" ("(3\ _./ _)" [1000, 10] 10) parse_ast_translation {* diff -r 4d9518c3d031 -r b66d2ca1f907 src/HOL/HOLCF/ConvexPD.thy --- a/src/HOL/HOLCF/ConvexPD.thy Wed Dec 30 21:10:19 2015 +0100 +++ b/src/HOL/HOLCF/ConvexPD.thy Wed Dec 30 21:23:38 2015 +0100 @@ -119,12 +119,10 @@ subsection {* Type definition *} -typedef 'a convex_pd = +typedef 'a convex_pd ("('(_')\)") = "{S::'a pd_basis set. convex_le.ideal S}" by (rule convex_le.ex_ideal) -type_notation (xsymbols) convex_pd ("('(_')\)") - instantiation convex_pd :: (bifinite) below begin diff -r 4d9518c3d031 -r b66d2ca1f907 src/HOL/HOLCF/FOCUS/Fstream.thy --- a/src/HOL/HOLCF/FOCUS/Fstream.thy Wed Dec 30 21:10:19 2015 +0100 +++ b/src/HOL/HOLCF/FOCUS/Fstream.thy Wed Dec 30 21:23:38 2015 +0100 @@ -29,16 +29,16 @@ "<> == \" abbreviation - fscons' :: "'a \ 'a fstream \ 'a fstream" ("(_~>_)" [66,65] 65) where - "a~>s == fscons a\s" + fscons' :: "'a \ 'a fstream \ 'a fstream" ("(_\_)" [66,65] 65) where + "a\s == fscons a\s" abbreviation - fsfilter' :: "'a set \ 'a fstream \ 'a fstream" ("(_'(C')_)" [64,63] 63) where - "A(C)s == fsfilter A\s" + fsfilter' :: "'a set \ 'a fstream \ 'a fstream" ("(_\_)" [64,63] 63) where + "A\s == fsfilter A\s" -notation (xsymbols) - fscons' ("(_\_)" [66,65] 65) and - fsfilter' ("(_\_)" [64,63] 63) +notation (ASCII) + fscons' ("(_~>_)" [66,65] 65) and + fsfilter' ("(_'(C')_)" [64,63] 63) lemma Def_maximal: "a = Def d \ a\b \ b = Def d" diff -r 4d9518c3d031 -r b66d2ca1f907 src/HOL/HOLCF/FOCUS/Fstreams.thy --- a/src/HOL/HOLCF/FOCUS/Fstreams.thy Wed Dec 30 21:10:19 2015 +0100 +++ b/src/HOL/HOLCF/FOCUS/Fstreams.thy Wed Dec 30 21:23:38 2015 +0100 @@ -44,11 +44,11 @@ "<> == \" abbreviation - fsfilter' :: "'a set \ 'a fstream \ 'a fstream" ("(_'(C')_)" [64,63] 63) where - "A(C)s == fsfilter A\s" + fsfilter' :: "'a set \ 'a fstream \ 'a fstream" ("(_\_)" [64,63] 63) where + "A\s == fsfilter A\s" -notation (xsymbols) - fsfilter' ("(_\_)" [64,63] 63) +notation (ASCII) + fsfilter' ("(_'(C')_)" [64,63] 63) lemma ft_fsingleton[simp]: "ft$() = Def a" diff -r 4d9518c3d031 -r b66d2ca1f907 src/HOL/HOLCF/Fix.thy --- a/src/HOL/HOLCF/Fix.thy Wed Dec 30 21:10:19 2015 +0100 +++ b/src/HOL/HOLCF/Fix.thy Wed Dec 30 21:23:38 2015 +0100 @@ -49,11 +49,11 @@ text {* Binder syntax for @{term fix} *} abbreviation - fix_syn :: "('a \ 'a) \ 'a" (binder "FIX " 10) where + fix_syn :: "('a \ 'a) \ 'a" (binder "\ " 10) where "fix_syn (\x. f x) \ fix\(\ x. f x)" -notation (xsymbols) - fix_syn (binder "\ " 10) +notation (ASCII) + fix_syn (binder "FIX " 10) text {* Properties of @{term fix} *} diff -r 4d9518c3d031 -r b66d2ca1f907 src/HOL/HOLCF/LowerPD.thy --- a/src/HOL/HOLCF/LowerPD.thy Wed Dec 30 21:10:19 2015 +0100 +++ b/src/HOL/HOLCF/LowerPD.thy Wed Dec 30 21:23:38 2015 +0100 @@ -74,12 +74,10 @@ subsection {* Type definition *} -typedef 'a lower_pd = +typedef 'a lower_pd ("('(_')\)") = "{S::'a pd_basis set. lower_le.ideal S}" by (rule lower_le.ex_ideal) -type_notation (xsymbols) lower_pd ("('(_')\)") - instantiation lower_pd :: (bifinite) below begin diff -r 4d9518c3d031 -r b66d2ca1f907 src/HOL/HOLCF/Pcpo.thy --- a/src/HOL/HOLCF/Pcpo.thy Wed Dec 30 21:10:19 2015 +0100 +++ b/src/HOL/HOLCF/Pcpo.thy Wed Dec 30 21:23:38 2015 +0100 @@ -143,12 +143,9 @@ assumes least: "\x. \y. x \ y" begin -definition bottom :: "'a" +definition bottom :: "'a" ("\") where "bottom = (THE x. \y. x \ y)" -notation (xsymbols) - bottom ("\") - lemma minimal [iff]: "\ \ x" unfolding bottom_def apply (rule the1I2) diff -r 4d9518c3d031 -r b66d2ca1f907 src/HOL/HOLCF/Porder.thy --- a/src/HOL/HOLCF/Porder.thy Wed Dec 30 21:10:19 2015 +0100 +++ b/src/HOL/HOLCF/Porder.thy Wed Dec 30 21:23:38 2015 +0100 @@ -17,18 +17,18 @@ fixes below :: "'a \ 'a \ bool" begin -notation +notation (ASCII) below (infix "<<" 50) -notation (xsymbols) +notation below (infix "\" 50) abbreviation - not_below :: "'a \ 'a \ bool" (infix "~<<" 50) + not_below :: "'a \ 'a \ bool" (infix "\" 50) where "not_below x y \ \ below x y" -notation (xsymbols) - not_below (infix "\" 50) +notation (ASCII) + not_below (infix "~<<" 50) lemma below_eq_trans: "\a \ b; b = c\ \ a \ c" by (rule subst) @@ -112,10 +112,10 @@ end -syntax +syntax (ASCII) "_BLub" :: "[pttrn, 'a set, 'b] \ 'b" ("(3LUB _:_./ _)" [0,0, 10] 10) -syntax (xsymbols) +syntax "_BLub" :: "[pttrn, 'a set, 'b] \ 'b" ("(3\_\_./ _)" [0,0, 10] 10) translations @@ -125,11 +125,11 @@ begin abbreviation - Lub (binder "LUB " 10) where - "LUB n. t n == lub (range t)" + Lub (binder "\" 10) where + "\n. t n == lub (range t)" -notation (xsymbols) - Lub (binder "\" 10) +notation (ASCII) + Lub (binder "LUB " 10) text {* access to some definition as inference rule *} diff -r 4d9518c3d031 -r b66d2ca1f907 src/HOL/HOLCF/Sfun.thy --- a/src/HOL/HOLCF/Sfun.thy Wed Dec 30 21:10:19 2015 +0100 +++ b/src/HOL/HOLCF/Sfun.thy Wed Dec 30 21:23:38 2015 +0100 @@ -8,12 +8,12 @@ imports Cfun begin -pcpodef ('a, 'b) sfun (infixr "->!" 0) +pcpodef ('a, 'b) sfun (infixr "\!" 0) = "{f :: 'a \ 'b. f\\ = \}" by simp_all -type_notation (xsymbols) - sfun (infixr "\!" 0) +type_notation (ASCII) + sfun (infixr "->!" 0) text {* TODO: Define nice syntax for abstraction, application. *} diff -r 4d9518c3d031 -r b66d2ca1f907 src/HOL/HOLCF/Sprod.thy --- a/src/HOL/HOLCF/Sprod.thy Wed Dec 30 21:10:19 2015 +0100 +++ b/src/HOL/HOLCF/Sprod.thy Wed Dec 30 21:23:38 2015 +0100 @@ -15,14 +15,14 @@ definition "sprod = {p::'a \ 'b. p = \ \ (fst p \ \ \ snd p \ \)}" -pcpodef ('a, 'b) sprod (infixr "**" 20) = "sprod :: ('a \ 'b) set" +pcpodef ('a, 'b) sprod ("(_ \/ _)" [21,20] 20) = "sprod :: ('a \ 'b) set" unfolding sprod_def by simp_all instance sprod :: ("{chfin,pcpo}", "{chfin,pcpo}") chfin by (rule typedef_chfin [OF type_definition_sprod below_sprod_def]) -type_notation (xsymbols) - sprod ("(_ \/ _)" [21,20] 20) +type_notation (ASCII) + sprod (infixr "**" 20) subsection {* Definitions of constants *} diff -r 4d9518c3d031 -r b66d2ca1f907 src/HOL/HOLCF/Ssum.thy --- a/src/HOL/HOLCF/Ssum.thy Wed Dec 30 21:10:19 2015 +0100 +++ b/src/HOL/HOLCF/Ssum.thy Wed Dec 30 21:23:38 2015 +0100 @@ -19,14 +19,14 @@ (fst p = TT \ fst (snd p) \ \ \ snd (snd p) = \) \ (fst p = FF \ fst (snd p) = \ \ snd (snd p) \ \)}" -pcpodef ('a, 'b) ssum (infixr "++" 10) = "ssum :: (tr \ 'a \ 'b) set" +pcpodef ('a, 'b) ssum ("(_ \/ _)" [21, 20] 20) = "ssum :: (tr \ 'a \ 'b) set" unfolding ssum_def by simp_all instance ssum :: ("{chfin,pcpo}", "{chfin,pcpo}") chfin by (rule typedef_chfin [OF type_definition_ssum below_ssum_def]) -type_notation (xsymbols) - ssum ("(_ \/ _)" [21, 20] 20) +type_notation (ASCII) + ssum (infixr "++" 10) subsection {* Definitions of constructors *} diff -r 4d9518c3d031 -r b66d2ca1f907 src/HOL/HOLCF/Up.thy --- a/src/HOL/HOLCF/Up.thy Wed Dec 30 21:10:19 2015 +0100 +++ b/src/HOL/HOLCF/Up.thy Wed Dec 30 21:23:38 2015 +0100 @@ -13,10 +13,7 @@ subsection {* Definition of new type for lifting *} -datatype 'a u = Ibottom | Iup 'a - -type_notation (xsymbols) - u ("(_\<^sub>\)" [1000] 999) +datatype 'a u ("(_\<^sub>\)" [1000] 999) = Ibottom | Iup 'a primrec Ifup :: "('a \ 'b::pcpo) \ 'a u \ 'b" where "Ifup f Ibottom = \" diff -r 4d9518c3d031 -r b66d2ca1f907 src/HOL/HOLCF/UpperPD.thy --- a/src/HOL/HOLCF/UpperPD.thy Wed Dec 30 21:10:19 2015 +0100 +++ b/src/HOL/HOLCF/UpperPD.thy Wed Dec 30 21:23:38 2015 +0100 @@ -72,12 +72,10 @@ subsection {* Type definition *} -typedef 'a upper_pd = +typedef 'a upper_pd ("('(_')\)") = "{S::'a pd_basis set. upper_le.ideal S}" by (rule upper_le.ex_ideal) -type_notation (xsymbols) upper_pd ("('(_')\)") - instantiation upper_pd :: (bifinite) below begin diff -r 4d9518c3d031 -r b66d2ca1f907 src/HOL/HOLCF/ex/Pattern_Match.thy --- a/src/HOL/HOLCF/ex/Pattern_Match.thy Wed Dec 30 21:10:19 2015 +0100 +++ b/src/HOL/HOLCF/ex/Pattern_Match.thy Wed Dec 30 21:23:38 2015 +0100 @@ -104,13 +104,13 @@ syntax "_Case_syntax":: "['a, Cases_syn] => 'b" ("(Case _ of/ _)" 10) - "_Case1" :: "[Case_pat, 'b] => Case_syn" ("(2_ =>/ _)" 10) + "_Case1" :: "[Case_pat, 'b] => Case_syn" ("(2_ \/ _)" 10) "" :: "Case_syn => Cases_syn" ("_") "_Case2" :: "[Case_syn, Cases_syn] => Cases_syn" ("_/ | _") "_strip_positions" :: "'a => Case_pat" ("_") -syntax (xsymbols) - "_Case1" :: "[Case_pat, 'b] => Case_syn" ("(2_ \/ _)" 10) +syntax (ASCII) + "_Case1" :: "[Case_pat, 'b] => Case_syn" ("(2_ =>/ _)" 10) translations "_Case_syntax x ms" == "CONST cases\(ms\x)"