- Timestamp:
- May 31, 2011, 11:45:21 AM (10 years ago)
- Location:
- src/ASM
- Files:
-
- 2 edited
Legend:
- Unmodified
- Added
- Removed
-
src/ASM/AssemblyProof.ma
r864 r865 362 362 match l with 363 363 [ nil ⇒ true 364 | cons hd tl ⇒ notb ( address_of_word_labels_internalid hd) ∧ does_not_occur id tl].364 | cons hd tl ⇒ notb (instruction_matches_identifier id hd) ∧ does_not_occur id tl]. 365 365 366 366 lemma does_not_occur_None: … … 376 376 [ nil ⇒ false 377 377 | cons hd tl ⇒ 378 if address_of_word_labels_internalid hd then378 if instruction_matches_identifier id hd then 379 379 does_not_occur id tl 380 380 else … … 393 393 lemma index_of_internal_None: ∀i,id,instr_list,n. 394 394 occurs_exactly_once id (instr_list@[〈None …,i〉]) → 395 index_of_internal ? ( address_of_word_labels_internalid) instr_list n =396 index_of_internal ? ( address_of_word_labels_internalid) (instr_list@[〈None …,i〉]) n.395 index_of_internal ? (instruction_matches_identifier id) instr_list n = 396 index_of_internal ? (instruction_matches_identifier id) (instr_list@[〈None …,i〉]) n. 397 397 #i #id #instr_list elim instr_list 398 398 [ #n #abs whd in abs; cases abs 399 399 | #hd #tl #IH #n whd in ⊢ (% → ??%%); whd in ⊢ (match % with [_ ⇒ ? | _ ⇒ ?] → ?) 400 cases ( address_of_word_labels_internalid hd) whd in ⊢ (match % with [_ ⇒ ? | _ ⇒ ?] → ??%%)400 cases (instruction_matches_identifier id hd) whd in ⊢ (match % with [_ ⇒ ? | _ ⇒ ?] → ??%%) 401 401 [ #H % 402 402 | #H @IH whd in H; cases (occurs_exactly_once ??) in H ⊢ % -
src/ASM/Interpret.ma
r856 r865 642 642 index_of_internal A eq l 0. 643 643 644 definition address_of_word_labels_internal≝644 definition instruction_matches_identifier ≝ 645 645 λy: Identifier. 646 646 λx: labelled_instruction. … … 653 653 λcode_mem. 654 654 λid: Identifier. 655 bitvector_of_nat 16 (index_of ? ( address_of_word_labels_internalid) code_mem).655 bitvector_of_nat 16 (index_of ? (instruction_matches_identifier id) code_mem). 656 656 657 657 definition address_of_word_labels ≝
Note: See TracChangeset
for help on using the changeset viewer.