Nominal/Ex/SFT/Theorem.thy
changeset 2898 a95a497e1f4f
parent 2894 8ec94871de1e
child 3087 c95afd0dc594
equal deleted inserted replaced
2897:fd4fa6df22d1 2898:a95a497e1f4f
     1 header {* The main lemma about Num and the Second Fixed Point Theorem *}
     1 header {* The main lemma about Num and the Second Fixed Point Theorem *}
       
     2 
     2 theory Theorem imports Consts begin
     3 theory Theorem imports Consts begin
     3 
     4 
     4 lemmas [simp] = b3[OF bI] b1 b4 b5 supp_Num[unfolded Num_def supp_ltgt] Num_def lam.fresh[unfolded fresh_def] fresh_def b6
     5 lemmas [simp] = b3[OF bI] b1 b4 b5 supp_Num[unfolded Num_def supp_ltgt] Num_def lam.fresh[unfolded fresh_def] fresh_def b6
     5 lemmas app = Ltgt1_app
     6 lemmas app = Ltgt1_app
     6 
     7