src/HOL/Library/Extended_Nonnegative_Real.thy
changeset 64425 b17acc1834e3
parent 64320 ba194424b895
child 65680 378a2f11bec9
--- a/src/HOL/Library/Extended_Nonnegative_Real.thy	Fri Oct 28 16:59:25 2016 +0200
+++ b/src/HOL/Library/Extended_Nonnegative_Real.thy	Fri Oct 28 19:54:41 2016 +0200
@@ -1354,7 +1354,7 @@
   fixes f :: "'a::topological_space \<Rightarrow> ennreal"
   shows "continuous_on A f \<Longrightarrow> continuous_on A (\<lambda>x. inverse (f x))"
 proof (transfer fixing: A)
-  show "pred_fun (\<lambda>_. True)  (op \<le> 0) f \<Longrightarrow> continuous_on A (\<lambda>x. inverse (f x))" if "continuous_on A f"
+  show "pred_fun top  (op \<le> 0) f \<Longrightarrow> continuous_on A (\<lambda>x. inverse (f x))" if "continuous_on A f"
     for f :: "'a \<Rightarrow> ereal"
     using continuous_on_compose2[OF continuous_on_inverse_ereal that] by (auto simp: subset_eq)
 qed