src/HOL/Lazy_Sequence.thy
changeset 55416 dd7992d4a61a
parent 55413 a8e96847523c
child 55466 786edc984c98
--- a/src/HOL/Lazy_Sequence.thy	Wed Feb 12 08:35:57 2014 +0100
+++ b/src/HOL/Lazy_Sequence.thy	Wed Feb 12 08:35:57 2014 +0100
@@ -35,12 +35,12 @@
   "size (xq :: 'a lazy_sequence) = 0"
   by (cases xq) simp
 
-lemma lazy_sequence_case [simp]:
-  "lazy_sequence_case f xq = f (list_of_lazy_sequence xq)"
+lemma case_lazy_sequence [simp]:
+  "case_lazy_sequence f xq = f (list_of_lazy_sequence xq)"
   by (cases xq) auto
 
-lemma lazy_sequence_rec [simp]:
-  "lazy_sequence_rec f xq = f (list_of_lazy_sequence xq)"
+lemma rec_lazy_sequence [simp]:
+  "rec_lazy_sequence f xq = f (list_of_lazy_sequence xq)"
   by (cases xq) auto
 
 definition Lazy_Sequence :: "(unit \<Rightarrow> ('a \<times> 'a lazy_sequence) option) \<Rightarrow> 'a lazy_sequence"
@@ -346,4 +346,3 @@
   if_seq_def those_def not_seq_def product_def 
 
 end
-