src/HOL/BNF/Examples/Stream.thy
changeset 53806 de4653037e0d
parent 53805 4163160853fd
child 53808 b3e2022530e3
--- a/src/HOL/BNF/Examples/Stream.thy	Mon Sep 23 17:43:23 2013 +0200
+++ b/src/HOL/BNF/Examples/Stream.thy	Mon Sep 23 18:40:02 2013 +0200
@@ -17,19 +17,7 @@
 
 declaration {*
   Nitpick_HOL.register_codatatype
-    @{typ "'stream_element_type stream"} @{const_name stream_case} [dest_Const @{term Stream}]
-    (*FIXME: long type variable name required to reduce the probability of
-        a name clash of Nitpick in context. E.g.:
-        context
-        fixes x :: 'stream_element_type
-        begin
-
-        lemma "sset s = {}"
-        nitpick
-        oops
-
-        end
-    *)
+    @{typ "'a stream"} @{const_name stream_case} [dest_Const @{term Stream}]
 *}
 
 code_datatype Stream