src/HOL/Library/Type_Length.thy
changeset 71759 816e52bbfa60
parent 71195 d50a718ccf35
child 72281 beeadb35e357
--- a/src/HOL/Library/Type_Length.thy	Thu Apr 16 08:09:30 2020 +0200
+++ b/src/HOL/Library/Type_Length.thy	Thu Apr 16 08:09:31 2020 +0200
@@ -107,4 +107,14 @@
   \<open>\<not> 2 \<le> LENGTH('a::len) \<longleftrightarrow> LENGTH('a) = 1\<close>
   by (auto simp add: not_le dest: less_2_cases)
 
+context linordered_idom
+begin
+
+lemma two_less_eq_exp_length [simp]:
+  \<open>2 \<le> 2 ^ LENGTH('b::len)\<close>
+  using mult_left_mono [of 1 \<open>2 ^ (LENGTH('b::len) - 1)\<close> 2]
+		  by (cases \<open>LENGTH('b::len)\<close>) simp_all
+
 end
+
+end