diff -r 46f59511b7bb -r d97fdabd9e2b src/HOL/MicroJava/BV/BVExample.thy --- a/src/HOL/MicroJava/BV/BVExample.thy Fri Sep 20 19:07:10 2024 +0200 +++ b/src/HOL/MicroJava/BV/BVExample.thy Fri Sep 20 19:51:08 2024 +0200 @@ -163,7 +163,7 @@ @{prop [display] "P n"} \ -definition intervall :: "nat \ nat \ nat \ bool" ("_ \ [_, _')") where +definition intervall :: "nat \ nat \ nat \ bool" (\_ \ [_, _')\) where "x \ [a, b) \ a \ x \ x < b" lemma pc_0: "x < n \ (x \ [0, n) \ P x) \ P x" @@ -233,7 +233,7 @@ lemmas eff_simps [simp] = eff_def norm_eff_def xcpt_eff_def declare appInvoke [simp del] -definition phi_append :: method_type ("\\<^sub>a") where +definition phi_append :: method_type (\\\<^sub>a\) where "\\<^sub>a \ map (\(x,y). Some (x, map OK y)) [ ( [], [Class list_name, Class list_name]), ( [Class list_name], [Class list_name, Class list_name]), @@ -295,7 +295,7 @@ abbreviation Ctest :: ty where "Ctest == Class test_name" -definition phi_makelist :: method_type ("\\<^sub>m") where +definition phi_makelist :: method_type (\\\<^sub>m\) where "\\<^sub>m \ map (\(x,y). Some (x, y)) [ ( [], [OK Ctest, Err , Err ]), ( [Clist], [OK Ctest, Err , Err ]), @@ -369,7 +369,7 @@ done text \The whole program is welltyped:\ -definition Phi :: prog_type ("\") where +definition Phi :: prog_type (\\\) where "\ C sg \ if C = test_name \ sg = (makelist_name, []) then \\<^sub>m else if C = list_name \ sg = (append_name, [Class list_name]) then \\<^sub>a else []"