src/HOL/Power.thy
changeset 61076 bdc1e2f0a86a
parent 60974 6a6f15d8fbc4
child 61378 3e04c9ca001a
--- a/src/HOL/Power.thy	Tue Sep 01 17:25:36 2015 +0200
+++ b/src/HOL/Power.thy	Tue Sep 01 22:32:58 2015 +0200
@@ -800,7 +800,7 @@
 Premises cannot be weakened: consider the case where @{term "i=0"},
 @{term "m=1"} and @{term "n=0"}.\<close>
 lemma nat_power_less_imp_less:
-  assumes nonneg: "0 < (i\<Colon>nat)"
+  assumes nonneg: "0 < (i::nat)"
   assumes less: "i ^ m < i ^ n"
   shows "m < n"
 proof (cases "i = 1")