diff -r 46f59511b7bb -r d97fdabd9e2b src/HOL/Induct/Comb.thy --- a/src/HOL/Induct/Comb.thy Fri Sep 20 19:07:10 2024 +0200 +++ b/src/HOL/Induct/Comb.thy Fri Sep 20 19:51:08 2024 +0200 @@ -20,14 +20,14 @@ datatype comb = K | S - | Ap comb comb (infixl "\" 90) + | Ap comb comb (infixl \\\ 90) text \ Inductive definition of contractions, \\\<^sup>1\ and (multi-step) reductions, \\\. \ -inductive contract1 :: "[comb,comb] \ bool" (infixl "\\<^sup>1" 50) +inductive contract1 :: "[comb,comb] \ bool" (infixl \\\<^sup>1\ 50) where K: "K\x\y \\<^sup>1 x" | S: "S\x\y\z \\<^sup>1 (x\z)\(y\z)" @@ -35,7 +35,7 @@ | Ap2: "x \\<^sup>1 y \ z\x \\<^sup>1 z\y" abbreviation - contract :: "[comb,comb] \ bool" (infixl "\" 50) where + contract :: "[comb,comb] \ bool" (infixl \\\ 50) where "contract \ contract1\<^sup>*\<^sup>*" text \ @@ -43,7 +43,7 @@ (multi-step) parallel reductions, \\\. \ -inductive parcontract1 :: "[comb,comb] \ bool" (infixl "\\<^sup>1" 50) +inductive parcontract1 :: "[comb,comb] \ bool" (infixl \\\<^sup>1\ 50) where refl: "x \\<^sup>1 x" | K: "K\x\y \\<^sup>1 x" @@ -51,7 +51,7 @@ | Ap: "\x \\<^sup>1 y; z \\<^sup>1 w\ \ x\z \\<^sup>1 y\w" abbreviation - parcontract :: "[comb,comb] \ bool" (infixl "\" 50) where + parcontract :: "[comb,comb] \ bool" (infixl \\\ 50) where "parcontract \ parcontract1\<^sup>*\<^sup>*" text \