src/HOL/Deriv.thy
changeset 67149 e61557884799
parent 64272 f76b6dda2e56
child 67399 eab6ce8368fa
--- a/src/HOL/Deriv.thy	Wed Dec 06 19:34:59 2017 +0100
+++ b/src/HOL/Deriv.thy	Wed Dec 06 20:43:09 2017 +0100
@@ -51,7 +51,7 @@
     fun eq_rule thm = get_first (try (fn eq_thm => eq_thm OF [thm])) eq_thms
   in
     Global_Theory.add_thms_dynamic
-      (@{binding derivative_eq_intros},
+      (\<^binding>\<open>derivative_eq_intros\<close>,
         fn context =>
           Named_Theorems.get (Context.proof_of context) @{named_theorems derivative_intros}
           |> map_filter eq_rule)