diff -r b9331caf92c3 -r 5399dfe9141c src/HOL/ex/Rewrite_Examples.thy --- a/src/HOL/ex/Rewrite_Examples.thy Wed Sep 29 11:55:09 2021 +0200 +++ b/src/HOL/ex/Rewrite_Examples.thy Wed Sep 29 18:21:22 2021 +0200 @@ -222,9 +222,9 @@ val (x, ctxt) = yield_singleton Variable.add_fixes "x" \<^context> (* Note that the pattern order is reversed *) val pat = [ - Rewrite.For [(x, SOME \<^typ>\nat\)], + Rewrite.For [(x, SOME \<^Type>\nat\)], Rewrite.In, - Rewrite.Term (@{const plus(nat)} $ Free (x, \<^typ>\nat\) $ \<^term>\1 :: nat\, [])] + Rewrite.Term (\<^Const>\plus \<^Type>\nat\ for \Free (x, \<^Type>\nat\)\ \<^term>\1 :: nat\\, [])] val to = NONE in CCONVERSION (Rewrite.rewrite_conv ctxt (pat, to) @{thms add.commute}) 1 end \) @@ -240,10 +240,10 @@ val pat = [ Rewrite.Concl, Rewrite.In, - Rewrite.Term (Free ("Q", (\<^typ>\int\ --> TVar (("'b",0), [])) --> \<^typ>\bool\) - $ Abs ("x", \<^typ>\int\, Rewrite.mk_hole 1 (\<^typ>\int\ --> TVar (("'b",0), [])) $ Bound 0), [(x, \<^typ>\int\)]), + Rewrite.Term (Free ("Q", (\<^Type>\int\ --> TVar (("'b",0), [])) --> \<^Type>\bool\) + $ Abs ("x", \<^Type>\int\, Rewrite.mk_hole 1 (\<^Type>\int\ --> TVar (("'b",0), [])) $ Bound 0), [(x, \<^Type>\int\)]), Rewrite.In, - Rewrite.Term (@{const plus(int)} $ Free (x, \<^typ>\int\) $ Var (("c", 0), \<^typ>\int\), []) + Rewrite.Term (\<^Const>\plus \<^Type>\int\ for \Free (x, \<^Type>\int\)\ \Var (("c", 0), \<^Type>\int\)\\, []) ] val to = NONE in CCONVERSION (Rewrite.rewrite_conv ctxt (pat, to) @{thms add.commute}) 1 end @@ -261,7 +261,7 @@ Rewrite.Term (Free ("Q", (\<^typ>\int\ --> TVar (("'b",0), [])) --> \<^typ>\bool\) $ Abs ("x", \<^typ>\int\, Rewrite.mk_hole 1 (\<^typ>\int\ --> TVar (("'b",0), [])) $ Bound 0), [(x, \<^typ>\int\)]), Rewrite.In, - Rewrite.Term (@{const plus(int)} $ Free (x, \<^typ>\int\) $ Var (("c", 0), \<^typ>\int\), []) + Rewrite.Term (\<^Const>\plus \<^Type>\int\ for \Free (x, \<^Type>\int\)\ \Var (("c", 0), \<^Type>\int\)\\, []) ] val to = NONE val th = Rewrite.rewrite_conv ctxt (pat, to) @{thms add.commute} ct @@ -274,7 +274,7 @@ val (x, ctxt) = yield_singleton Variable.add_fixes "x" \<^context> val pat = [ Rewrite.In, - Rewrite.Term (@{const plus(int)} $ Var (("c", 0), \<^typ>\int\) $ Var (("c", 0), \<^typ>\int\), []) + Rewrite.Term (\<^Const>\plus \<^Type>\int\ for \Var (("c", 0), \<^Type>\int\)\ \Var (("c", 0), \<^Type>\int\)\\, []) ] val to = NONE val _ =