merged
authornipkow
Sun, 16 Feb 2025 17:06:09 +0100
changeset 82190 17e900a4a438
parent 82188 fa2c960fb232 (current diff)
parent 82189 4de658eaa94f (diff)
child 82191 3c88bec13e60
merged
--- a/src/HOL/Nat.thy	Sun Feb 16 11:57:41 2025 +0000
+++ b/src/HOL/Nat.thy	Sun Feb 16 17:06:09 2025 +0100
@@ -1625,7 +1625,7 @@
 qed
 
 lemma mono_pow: "mono f \<Longrightarrow> mono (f ^^ n)"
-  for f :: "'a \<Rightarrow> 'a::complete_lattice"
+  for f :: "'a \<Rightarrow> 'a::order"
   by (induct n) (auto simp: mono_def)
 
 lemma lfp_funpow:
@@ -2375,23 +2375,23 @@
 subsection \<open>Monotonicity of \<open>funpow\<close>\<close>
 
 lemma funpow_increasing: "m \<le> n \<Longrightarrow> mono f \<Longrightarrow> (f ^^ n) \<top> \<le> (f ^^ m) \<top>"
-  for f :: "'a::{lattice,order_top} \<Rightarrow> 'a"
+  for f :: "'a::order_top \<Rightarrow> 'a"
   by (induct rule: inc_induct)
     (auto simp del: funpow.simps(2) simp add: funpow_Suc_right
       intro: order_trans[OF _ funpow_mono])
 
 lemma funpow_decreasing: "m \<le> n \<Longrightarrow> mono f \<Longrightarrow> (f ^^ m) \<bottom> \<le> (f ^^ n) \<bottom>"
-  for f :: "'a::{lattice,order_bot} \<Rightarrow> 'a"
+  for f :: "'a::order_bot \<Rightarrow> 'a"
   by (induct rule: dec_induct)
     (auto simp del: funpow.simps(2) simp add: funpow_Suc_right
       intro: order_trans[OF _ funpow_mono])
 
 lemma mono_funpow: "mono Q \<Longrightarrow> mono (\<lambda>i. (Q ^^ i) \<bottom>)"
-  for Q :: "'a::{lattice,order_bot} \<Rightarrow> 'a"
+  for Q :: "'a::order_bot \<Rightarrow> 'a"
   by (auto intro!: funpow_decreasing simp: mono_def)
 
 lemma antimono_funpow: "mono Q \<Longrightarrow> antimono (\<lambda>i. (Q ^^ i) \<top>)"
-  for Q :: "'a::{lattice,order_top} \<Rightarrow> 'a"
+  for Q :: "'a::order_top \<Rightarrow> 'a"
   by (auto intro!: funpow_increasing simp: antimono_def)