adapted example
authorblanchet
Mon, 03 Mar 2014 12:48:20 +0100
changeset 55873 aa50d903e0a7
parent 55872 75907f171d4c
child 55874 7eff011e2b36
adapted example
src/HOL/BNF_Comp.thy
src/HOL/BNF_Examples/Stream.thy
--- a/src/HOL/BNF_Comp.thy	Mon Mar 03 12:48:20 2014 +0100
+++ b/src/HOL/BNF_Comp.thy	Mon Mar 03 12:48:20 2014 +0100
@@ -147,7 +147,7 @@
 ML_file "Tools/BNF/bnf_comp_tactics.ML"
 ML_file "Tools/BNF/bnf_comp.ML"
 
-hide_const id_bnf_comp
-hide_fact id_bnf_comp_def type_definition_id_bnf_comp_UNIV
+hide_const (open) id_bnf_comp
+hide_fact (open) id_bnf_comp_def type_definition_id_bnf_comp_UNIV
 
 end
--- a/src/HOL/BNF_Examples/Stream.thy	Mon Mar 03 12:48:20 2014 +0100
+++ b/src/HOL/BNF_Examples/Stream.thy	Mon Mar 03 12:48:20 2014 +0100
@@ -33,16 +33,16 @@
   assume "a \<in> set1_pre_stream (dtor_stream s)"
   then have "a = shd s"
     by (cases "dtor_stream s")
-      (auto simp: shd_def fsts_def set1_pre_stream_def stream.dtor_ctor SCons_def
-        Abs_stream_pre_stream_inverse Abs_stream_pre_stream_inject split: stream.splits)
+      (auto simp: BNF_Comp.id_bnf_comp_def shd_def fsts_def set1_pre_stream_def stream.dtor_ctor SCons_def
+        split: stream.splits)
   with Base show "P a s" by simp
 next
   fix a :: 'a and s' :: "'a stream"  and s :: "'a stream"
   assume "s' \<in> set2_pre_stream (dtor_stream s)" and prems: "a \<in> sset s'" "P a s'"
   then have "s' = stl s"
     by (cases "dtor_stream s")
-      (auto simp: stl_def snds_def set2_pre_stream_def stream.dtor_ctor SCons_def
-        Abs_stream_pre_stream_inverse Abs_stream_pre_stream_inject split: stream.splits)
+      (auto simp: BNF_Comp.id_bnf_comp_def stl_def snds_def set2_pre_stream_def stream.dtor_ctor SCons_def
+        split: stream.splits)
   with Step prems show "P a s" by simp
 qed