diff -r 46f59511b7bb -r d97fdabd9e2b src/HOL/IMP/Small_Step.thy --- a/src/HOL/IMP/Small_Step.thy Fri Sep 20 19:07:10 2024 +0200 +++ b/src/HOL/IMP/Small_Step.thy Fri Sep 20 19:51:08 2024 +0200 @@ -5,7 +5,7 @@ subsection "The transition relation" inductive - small_step :: "com * state \ com * state \ bool" (infix "\" 55) + small_step :: "com * state \ com * state \ bool" (infix \\\ 55) where Assign: "(x ::= a, s) \ (SKIP, s(x := aval a s))" | @@ -20,7 +20,7 @@ abbreviation - small_steps :: "com * state \ com * state \ bool" (infix "\*" 55) + small_steps :: "com * state \ com * state \ bool" (infix \\*\ 55) where "x \* y == star small_step x y" subsection\Executability\