src/HOL/Lazy_Sequence.thy
changeset 34957 3b1957113753
parent 34948 2d5f2a9f7601
child 36020 3ee4c29ead7f
--- a/src/HOL/Lazy_Sequence.thy	Thu Jan 21 14:13:21 2010 +0100
+++ b/src/HOL/Lazy_Sequence.thy	Fri Jan 22 11:42:28 2010 +0100
@@ -153,6 +153,6 @@
 
 hide (open) type lazy_sequence
 hide (open) const Empty Insert Lazy_Sequence yield yieldn empty single append flat map bind if_seq not_seq
-hide (open) fact yield.simps yieldn.simps empty_def single_def append.simps flat.simps map.simps bind_def if_seq_def not_seq_def
+hide fact yield.simps yieldn.simps empty_def single_def append.simps flat.simps map.simps bind_def if_seq_def not_seq_def
 
 end