equal
deleted
inserted
replaced
108 |
108 |
109 (*adm_BufAC_Asm,BufAC_Asm_antiton,adm_non_BufAC_Asm,BufAC_Asm_cong*) |
109 (*adm_BufAC_Asm,BufAC_Asm_antiton,adm_non_BufAC_Asm,BufAC_Asm_cong*) |
110 Goal "f:BufEq ==> ? l. !i x s. s:BufAC_Asm --> x << s --> Fin (l i) < #x --> \ |
110 Goal "f:BufEq ==> ? l. !i x s. s:BufAC_Asm --> x << s --> Fin (l i) < #x --> \ |
111 \ (x,f\\<cdot>x):down_iterate BufAC_Cmt_F i --> \ |
111 \ (x,f\\<cdot>x):down_iterate BufAC_Cmt_F i --> \ |
112 \ (s,f\\<cdot>s):down_iterate BufAC_Cmt_F i"; |
112 \ (s,f\\<cdot>s):down_iterate BufAC_Cmt_F i"; |
113 by (res_inst_tac [("x","%i. i+i")] exI 1); |
113 by (res_inst_tac [("x","%i. #2*i")] exI 1); |
114 by (rtac allI 1); |
114 by (rtac allI 1); |
115 by (nat_ind_tac "i" 1); |
115 by (nat_ind_tac "i" 1); |
116 by ( Simp_tac 1); |
116 by ( Simp_tac 1); |
117 by (simp_tac (simpset() addsimps [add_commute]) 1); |
117 by (simp_tac (simpset() addsimps [add_commute]) 1); |
118 by (strip_tac 1); |
118 by (strip_tac 1); |