src/CCL/Fix.thy
changeset 61337 4645502c3c64
parent 60770 240563fbf41d
equal deleted inserted replaced
61336:fa4ebbd350ae 61337:4645502c3c64
    91       apply simp_all
    91       apply simp_all
    92   done
    92   done
    93 
    93 
    94 (* All fixed points are lam-expressions *)
    94 (* All fixed points are lam-expressions *)
    95 
    95 
    96 schematic_lemma idgenfp_lam: "idgen(d) = d \<Longrightarrow> d = lam x. ?f(x)"
    96 schematic_goal idgenfp_lam: "idgen(d) = d \<Longrightarrow> d = lam x. ?f(x)"
    97   apply (unfold idgen_def)
    97   apply (unfold idgen_def)
    98   apply (erule ssubst)
    98   apply (erule ssubst)
    99   apply (rule refl)
    99   apply (rule refl)
   100   done
   100   done
   101 
   101 
   123   apply (erule ssubst)
   123   apply (erule ssubst)
   124   apply (rule po_lam [THEN iffD2])
   124   apply (rule po_lam [THEN iffD2])
   125   apply simp
   125   apply simp
   126   done
   126   done
   127 
   127 
   128 schematic_lemma po_eta_lemma: "idgen(d) = d \<Longrightarrow> d = lam x. ?f(x)"
   128 schematic_goal po_eta_lemma: "idgen(d) = d \<Longrightarrow> d = lam x. ?f(x)"
   129   apply (unfold idgen_def)
   129   apply (unfold idgen_def)
   130   apply (erule sym)
   130   apply (erule sym)
   131   done
   131   done
   132 
   132 
   133 lemma lemma1:
   133 lemma lemma1: