src/HOL/BNF_Composition.thy
changeset 60918 4ceef1592e8c
parent 60758 d8d85a8172b5
child 61032 b57df8eecad6
--- a/src/HOL/BNF_Composition.thy	Wed Aug 12 13:56:46 2015 +0200
+++ b/src/HOL/BNF_Composition.thy	Wed Aug 12 20:46:33 2015 +0200
@@ -10,8 +10,14 @@
 
 theory BNF_Composition
 imports BNF_Def
+keywords
+  "copy_bnf" :: thy_decl and
+  "lift_bnf" :: thy_goal
 begin
 
+lemma ssubst_mem: "\<lbrakk>t = s; s \<in> X\<rbrakk> \<Longrightarrow> t \<in> X"
+  by simp
+
 lemma empty_natural: "(\<lambda>_. {}) o f = image g o (\<lambda>_. {})"
   by (rule ext) simp
 
@@ -168,6 +174,7 @@
 
 ML_file "Tools/BNF/bnf_comp_tactics.ML"
 ML_file "Tools/BNF/bnf_comp.ML"
+ML_file "Tools/BNF/bnf_lift.ML"
 
 hide_fact
   DEADID.inj_map DEADID.inj_map_strong DEADID.map_comp DEADID.map_cong DEADID.map_cong0