src/HOL/BNF/BNF_FP_Base.thy
author blanchet
Thu, 19 Sep 2013 02:30:45 +0200
changeset 54866 b9d727a767ea
parent 54835 e1b039dada7b
child 55005 c25acff63bfe
permissions -rw-r--r--
added helper function for code equations in primcorec
     1 (*  Title:      HOL/BNF/BNF_FP_Base.thy
     2     Author:     Lorenz Panny, TU Muenchen
     3     Author:     Dmitriy Traytel, TU Muenchen
     4     Author:     Jasmin Blanchette, TU Muenchen
     5     Copyright   2012, 2013
     6 
     7 Shared fixed point operations on bounded natural functors, including
     8 *)
     9 
    10 header {* Shared Fixed Point Operations on Bounded Natural Functors *}
    11 
    12 theory BNF_FP_Base
    13 imports BNF_Comp BNF_Ctr_Sugar
    14 begin
    15 
    16 lemma mp_conj: "(P \<longrightarrow> Q) \<and> R \<Longrightarrow> P \<Longrightarrow> R \<and> Q"
    17 by auto
    18 
    19 lemma eq_sym_Unity_conv: "(x = (() = ())) = x"
    20 by blast
    21 
    22 lemma unit_case_Unity: "(case u of () => f) = f"
    23 by (cases u) (hypsubst, rule unit.cases)
    24 
    25 lemma prod_case_Pair_iden: "(case p of (x, y) \<Rightarrow> (x, y)) = p"
    26 by simp
    27 
    28 lemma unit_all_impI: "(P () \<Longrightarrow> Q ()) \<Longrightarrow> \<forall>x. P x \<longrightarrow> Q x"
    29 by simp
    30 
    31 lemma prod_all_impI: "(\<And>x y. P (x, y) \<Longrightarrow> Q (x, y)) \<Longrightarrow> \<forall>x. P x \<longrightarrow> Q x"
    32 by clarify
    33 
    34 lemma prod_all_impI_step: "(\<And>x. \<forall>y. P (x, y) \<longrightarrow> Q (x, y)) \<Longrightarrow> \<forall>x. P x \<longrightarrow> Q x"
    35 by auto
    36 
    37 lemma pointfree_idE: "f \<circ> g = id \<Longrightarrow> f (g x) = x"
    38 unfolding o_def fun_eq_iff by simp
    39 
    40 lemma o_bij:
    41   assumes gf: "g \<circ> f = id" and fg: "f \<circ> g = id"
    42   shows "bij f"
    43 unfolding bij_def inj_on_def surj_def proof safe
    44   fix a1 a2 assume "f a1 = f a2"
    45   hence "g ( f a1) = g (f a2)" by simp
    46   thus "a1 = a2" using gf unfolding fun_eq_iff by simp
    47 next
    48   fix b
    49   have "b = f (g b)"
    50   using fg unfolding fun_eq_iff by simp
    51   thus "EX a. b = f a" by blast
    52 qed
    53 
    54 lemma ssubst_mem: "\<lbrakk>t = s; s \<in> X\<rbrakk> \<Longrightarrow> t \<in> X" by simp
    55 
    56 lemma sum_case_step:
    57 "sum_case (sum_case f' g') g (Inl p) = sum_case f' g' p"
    58 "sum_case f (sum_case f' g') (Inr p) = sum_case f' g' p"
    59 by auto
    60 
    61 lemma one_pointE: "\<lbrakk>\<And>x. s = x \<Longrightarrow> P\<rbrakk> \<Longrightarrow> P"
    62 by simp
    63 
    64 lemma obj_one_pointE: "\<forall>x. s = x \<longrightarrow> P \<Longrightarrow> P"
    65 by blast
    66 
    67 lemma obj_sumE_f:
    68 "\<lbrakk>\<forall>x. s = f (Inl x) \<longrightarrow> P; \<forall>x. s = f (Inr x) \<longrightarrow> P\<rbrakk> \<Longrightarrow> \<forall>x. s = f x \<longrightarrow> P"
    69 by (rule allI) (metis sumE)
    70 
    71 lemma obj_sumE: "\<lbrakk>\<forall>x. s = Inl x \<longrightarrow> P; \<forall>x. s = Inr x \<longrightarrow> P\<rbrakk> \<Longrightarrow> P"
    72 by (cases s) auto
    73 
    74 lemma sum_case_if:
    75 "sum_case f g (if p then Inl x else Inr y) = (if p then f x else g y)"
    76 by simp
    77 
    78 lemma mem_UN_compreh_eq: "(z : \<Union>{y. \<exists>x\<in>A. y = F x}) = (\<exists>x\<in>A. z : F x)"
    79 by blast
    80 
    81 lemma UN_compreh_eq_eq:
    82 "\<Union>{y. \<exists>x\<in>A. y = {}} = {}"
    83 "\<Union>{y. \<exists>x\<in>A. y = {x}} = A"
    84 by blast+
    85 
    86 lemma Inl_Inr_False: "(Inl x = Inr y) = False"
    87 by simp
    88 
    89 lemma prod_set_simps:
    90 "fsts (x, y) = {x}"
    91 "snds (x, y) = {y}"
    92 unfolding fsts_def snds_def by simp+
    93 
    94 lemma sum_set_simps:
    95 "setl (Inl x) = {x}"
    96 "setl (Inr x) = {}"
    97 "setr (Inl x) = {}"
    98 "setr (Inr x) = {x}"
    99 unfolding sum_set_defs by simp+
   100 
   101 lemma prod_rel_simp:
   102 "prod_rel P Q (x, y) (x', y') \<longleftrightarrow> P x x' \<and> Q y y'"
   103 unfolding prod_rel_def by simp
   104 
   105 lemma sum_rel_simps:
   106 "sum_rel P Q (Inl x) (Inl x') \<longleftrightarrow> P x x'"
   107 "sum_rel P Q (Inr y) (Inr y') \<longleftrightarrow> Q y y'"
   108 "sum_rel P Q (Inl x) (Inr y') \<longleftrightarrow> False"
   109 "sum_rel P Q (Inr y) (Inl x') \<longleftrightarrow> False"
   110 unfolding sum_rel_def by simp+
   111 
   112 lemma spec2: "\<forall>x y. P x y \<Longrightarrow> P x y"
   113 by blast
   114 
   115 lemma rewriteR_comp_comp: "\<lbrakk>g o h = r\<rbrakk> \<Longrightarrow> f o g o h = f o r"
   116   unfolding o_def fun_eq_iff by auto
   117 
   118 lemma rewriteR_comp_comp2: "\<lbrakk>g o h = r1 o r2; f o r1 = l\<rbrakk> \<Longrightarrow> f o g o h = l o r2"
   119   unfolding o_def fun_eq_iff by auto
   120 
   121 lemma rewriteL_comp_comp: "\<lbrakk>f o g = l\<rbrakk> \<Longrightarrow> f o (g o h) = l o h"
   122   unfolding o_def fun_eq_iff by auto
   123 
   124 lemma rewriteL_comp_comp2: "\<lbrakk>f o g = l1 o l2; l2 o h = r\<rbrakk> \<Longrightarrow> f o (g o h) = l1 o r"
   125   unfolding o_def fun_eq_iff by auto
   126 
   127 lemma convol_o: "<f, g> o h = <f o h, g o h>"
   128   unfolding convol_def by auto
   129 
   130 lemma map_pair_o_convol: "map_pair h1 h2 o <f, g> = <h1 o f, h2 o g>"
   131   unfolding convol_def by auto
   132 
   133 lemma map_pair_o_convol_id: "(map_pair f id \<circ> <id , g>) x = <id \<circ> f , g> x"
   134   unfolding map_pair_o_convol id_o o_id ..
   135 
   136 lemma o_sum_case: "h o sum_case f g = sum_case (h o f) (h o g)"
   137   unfolding o_def by (auto split: sum.splits)
   138 
   139 lemma sum_case_o_sum_map: "sum_case f g o sum_map h1 h2 = sum_case (f o h1) (g o h2)"
   140   unfolding o_def by (auto split: sum.splits)
   141 
   142 lemma sum_case_o_sum_map_id: "(sum_case id g o sum_map f id) x = sum_case (f o id) g x"
   143   unfolding sum_case_o_sum_map id_o o_id ..
   144 
   145 lemma fun_rel_def_butlast:
   146   "(fun_rel R (fun_rel S T)) f g = (\<forall>x y. R x y \<longrightarrow> (fun_rel S T) (f x) (g y))"
   147   unfolding fun_rel_def ..
   148 
   149 lemma subst_eq_imp: "(\<forall>a b. a = b \<longrightarrow> P a b) \<equiv> (\<forall>a. P a a)"
   150   by auto
   151 
   152 lemma eq_subset: "op = \<le> (\<lambda>a b. P a b \<or> a = b)"
   153   by auto
   154 
   155 lemma eq_le_Grp_id_iff: "(op = \<le> Grp (Collect R) id) = (All R)"
   156   unfolding Grp_def id_apply by blast
   157 
   158 lemma Grp_id_mono_subst: "(\<And>x y. Grp P id x y \<Longrightarrow> Grp Q id (f x) (f y)) \<equiv>
   159    (\<And>x. x \<in> P \<Longrightarrow> f x \<in> Q)"
   160   unfolding Grp_def by rule auto
   161 
   162 lemma eq_ifI: "\<lbrakk>b \<Longrightarrow> t = x; \<not> b \<Longrightarrow> t = y\<rbrakk> \<Longrightarrow> t = (if b then x else y)"
   163   by fastforce
   164 
   165 lemma if_if_True:
   166   "(if (if b then True else b') then (if b then x else x') else f (if b then y else y')) =
   167    (if b then x else if b' then x' else f y')"
   168   by simp
   169 
   170 lemma if_if_False:
   171   "(if (if b then False else b') then (if b then x else x') else f (if b then y else y')) =
   172    (if b then f y else if b' then x' else f y')"
   173   by simp
   174 
   175 lemma if_then_else_True_False:
   176   "(if p then False else r) \<longleftrightarrow> \<not> p \<and> r"
   177   "(if p then True else r) \<longleftrightarrow> p \<or> r"
   178   "(if p then q else False) \<longleftrightarrow> p \<and> q"
   179   "(if p then q else True) \<longleftrightarrow> \<not> p \<or> q"
   180 by simp_all
   181 
   182 lemmas bool_if_simps = bool_simps(7,8,15-17,19,21-24,29-32) if_then_else_True_False
   183 
   184 ML_file "Tools/bnf_fp_util.ML"
   185 ML_file "Tools/bnf_fp_def_sugar_tactics.ML"
   186 ML_file "Tools/bnf_fp_def_sugar.ML"
   187 ML_file "Tools/bnf_fp_n2m_tactics.ML"
   188 ML_file "Tools/bnf_fp_n2m.ML"
   189 ML_file "Tools/bnf_fp_n2m_sugar.ML"
   190 ML_file "Tools/bnf_fp_rec_sugar_util.ML"
   191 ML_file "Tools/bnf_fp_rec_sugar_tactics.ML"
   192 ML_file "Tools/bnf_fp_rec_sugar.ML"
   193 
   194 end