src/HOL/Quickcheck_Narrowing.thy
changeset 67399 eab6ce8368fa
parent 67091 1393c2340eec
child 68484 59793df7f853
--- a/src/HOL/Quickcheck_Narrowing.thy	Wed Jan 10 15:21:49 2018 +0100
+++ b/src/HOL/Quickcheck_Narrowing.thy	Wed Jan 10 15:25:09 2018 +0100
@@ -33,7 +33,7 @@
     fun print _ = Code_Haskell.print_numeral "Prelude.Int";
   in
     Numeral.add_code @{const_name Code_Numeral.Pos} I print target
-    #> Numeral.add_code @{const_name Code_Numeral.Neg} (op ~) print target
+    #> Numeral.add_code @{const_name Code_Numeral.Neg} (~) print target
   end
 \<close>