src/HOL/Nonstandard_Analysis/HyperDef.thy
changeset 67399 eab6ce8368fa
parent 64438 f91cae6c1d74
child 67613 ce654b0e6d69
--- a/src/HOL/Nonstandard_Analysis/HyperDef.thy	Wed Jan 10 15:21:49 2018 +0100
+++ b/src/HOL/Nonstandard_Analysis/HyperDef.thy	Wed Jan 10 15:25:09 2018 +0100
@@ -375,7 +375,7 @@
 
 text \<open>Hypernatural powers of hyperreals.\<close>
 definition pow :: "'a::power star \<Rightarrow> nat star \<Rightarrow> 'a star"  (infixr "pow" 80)
-  where hyperpow_def [transfer_unfold]: "R pow N = ( *f2* op ^) R N"
+  where hyperpow_def [transfer_unfold]: "R pow N = ( *f2* (^)) R N"
 
 lemma Standard_hyperpow [simp]: "r \<in> Standard \<Longrightarrow> n \<in> Standard \<Longrightarrow> r pow n \<in> Standard"
   by (simp add: hyperpow_def)