src/HOL/BNF_Examples/Stream.thy
changeset 57983 6edc3529bb4e
parent 57206 d9be905d6283
child 57986 0d60b9e58487
--- a/src/HOL/BNF_Examples/Stream.thy	Mon Aug 18 15:03:25 2014 +0200
+++ b/src/HOL/BNF_Examples/Stream.thy	Mon Aug 18 17:19:58 2014 +0200
@@ -49,9 +49,9 @@
   with Step prems show "P a s" by simp
 qed
 
-lemmas smap_simps[simp] = stream.sel_map
-lemmas shd_sset = stream.sel_set(1)
-lemmas stl_sset = stream.sel_set(2)
+lemmas smap_simps[simp] = stream.map_sel
+lemmas shd_sset = stream.set_sel(1)
+lemmas stl_sset = stream.set_sel(2)
 
 (* only for the non-mutual case: *)
 theorem sset_induct1[consumes 1, case_names shd stl, induct set: "sset"]: