src/HOL/Nominal/nominal_atoms.ML
changeset 45133 2214ba5bdfff
parent 44689 f247fc952f31
child 45701 615da8b8d758
equal deleted inserted replaced
45132:09de0d0de645 45133:2214ba5bdfff
   130               val y = Free ("y",ak_type)  
   130               val y = Free ("y",ak_type)  
   131               val stmnt2 = HOLogic.mk_Trueprop
   131               val stmnt2 = HOLogic.mk_Trueprop
   132                   (HOLogic.mk_exists ("x",@{typ nat},HOLogic.mk_eq (y,Const (ak_sign,inj_type) $ Bound 0)))
   132                   (HOLogic.mk_exists ("x",@{typ nat},HOLogic.mk_eq (y,Const (ak_sign,inj_type) $ Bound 0)))
   133 
   133 
   134               val proof2 = fn {prems, context} =>
   134               val proof2 = fn {prems, context} =>
   135                 InductTacs.case_tac context "y" 1 THEN
   135                 Induct_Tacs.case_tac context "y" 1 THEN
   136                 asm_simp_tac (HOL_basic_ss addsimps simp1) 1 THEN
   136                 asm_simp_tac (HOL_basic_ss addsimps simp1) 1 THEN
   137                 rtac @{thm exI} 1 THEN
   137                 rtac @{thm exI} 1 THEN
   138                 rtac @{thm refl} 1
   138                 rtac @{thm refl} 1
   139 
   139 
   140               (* third statement *)
   140               (* third statement *)