src/HOL/Lazy_Sequence.thy
changeset 42163 392fd6c4669c
parent 40056 0bee30e3a4ad
child 45214 66ba67adafab
--- a/src/HOL/Lazy_Sequence.thy	Wed Mar 30 11:32:51 2011 +0200
+++ b/src/HOL/Lazy_Sequence.thy	Wed Mar 30 11:32:52 2011 +0200
@@ -208,7 +208,7 @@
 subsection {* With Hit Bound Value *}
 text {* assuming in negative context *}
 
-types 'a hit_bound_lazy_sequence = "'a option lazy_sequence"
+type_synonym 'a hit_bound_lazy_sequence = "'a option lazy_sequence"
 
 definition hit_bound :: "'a hit_bound_lazy_sequence"
 where