Nominal/activities/tphols09/IDW/MW-Ex1.thy
changeset 415 f1be8028a4a9
equal deleted inserted replaced
414:05e5d68c9627 415:f1be8028a4a9
       
     1 theory Ex1
       
     2 imports Main
       
     3 begin
       
     4 
       
     5 section {* ML tactics as (crude) methods *}
       
     6 
       
     7 lemma True
       
     8 proof
       
     9 
       
    10   assume a: A
       
    11   assume b: B
       
    12 
       
    13   have "A & B"
       
    14     apply (tactic {* rtac @{thm conjI} 1 *})
       
    15     using a
       
    16     apply (tactic {* resolve_tac facts 1 *})
       
    17     using b
       
    18     apply (tactic {* resolve_tac facts 1 *})
       
    19     done
       
    20 
       
    21   have "A & B"
       
    22     using a b
       
    23     apply (tactic {* Method.insert_tac facts 1 *})
       
    24     apply (tactic {* (rtac @{thm conjI} THEN_ALL_NEW atac) 1 *})
       
    25     done
       
    26 
       
    27 qed
       
    28 
       
    29 end