src/HOL/Analysis/Lipschitz.thy
changeset 81116 0fb1e2dd4122
parent 81106 849efff7de15
child 81142 6ad2c917dd2e
--- a/src/HOL/Analysis/Lipschitz.thy	Fri Oct 04 23:38:04 2024 +0200
+++ b/src/HOL/Analysis/Lipschitz.thy	Sat Oct 05 14:58:36 2024 +0200
@@ -17,11 +17,6 @@
 notation\<^marker>\<open>tag important\<close> lipschitz_on (\<open>_-lipschitz'_on\<close> [1000])
 end
 
-bundle no_lipschitz_syntax
-begin
-no_notation lipschitz_on (\<open>_-lipschitz'_on\<close> [1000])
-end
-
 lemma lipschitz_onI: "L-lipschitz_on X f"
   if "\<And>x y. x \<in> X \<Longrightarrow> y \<in> X \<Longrightarrow> dist (f x) (f y) \<le> L * dist x y" "0 \<le> L"
   using that by (auto simp: lipschitz_on_def)