src/HOL/Library/Fun_Lexorder.thy
changeset 63040 eb4ddd18d635
parent 60500 903bb1495239
child 63060 293ede07b775
--- a/src/HOL/Library/Fun_Lexorder.thy	Sun Apr 24 21:31:14 2016 +0200
+++ b/src/HOL/Library/Fun_Lexorder.thy	Mon Apr 25 16:09:26 2016 +0200
@@ -76,12 +76,12 @@
   assumes "finite {k. f k \<noteq> g k}"
   shows "less_fun f g \<or> f = g \<or> less_fun g f"
 proof -
-  { def K \<equiv> "{k. f k \<noteq> g k}"
+  { define K where "K = {k. f k \<noteq> g k}"
     assume "f \<noteq> g"
     then obtain k' where "f k' \<noteq> g k'" by auto
     then have [simp]: "K \<noteq> {}" by (auto simp add: K_def)
     with assms have [simp]: "finite K" by (simp add: K_def)
-    def q \<equiv> "Min K"
+    define q where "q = Min K"
     then have "q \<in> K" and "\<And>k. k \<in> K \<Longrightarrow> k \<ge> q" by auto
     then have "\<And>k. \<not> k \<ge> q \<Longrightarrow> k \<notin> K" by blast
     then have *: "\<And>k. k < q \<Longrightarrow> f k = g k" by (simp add: K_def)