Nominal/Nominal2_FCB.thy
changeset 2946 d9c3cc271e62
parent 2944 8648ae682442
child 3105 1b0d230445ce
equal deleted inserted replaced
2945:70bbd18ad194 2946:d9c3cc271e62
     1 theory Nominal2_FCB
     1 theory Nominal2_FCB
     2 imports "Nominal2_Abs" 
     2 imports "Nominal2_Abs" 
     3 begin
     3 begin
       
     4 
       
     5 
       
     6 text {*
       
     7   A tactic which solves all trivial cases in function 
       
     8   definitions, and leaves the others unchanged.
       
     9 *}
       
    10 
       
    11 ML {*
       
    12 val all_trivials : (Proof.context -> Method.method) context_parser =
       
    13 Scan.succeed (fn ctxt =>
       
    14  let
       
    15    val tac = TRYALL (SOLVED' (full_simp_tac (simpset_of ctxt)))
       
    16  in 
       
    17    Method.SIMPLE_METHOD' (K tac)
       
    18  end)
       
    19 *}
       
    20 
       
    21 method_setup all_trivials = {* all_trivials *} {* solves trivial goals *}
     4 
    22 
     5 
    23 
     6 lemma Abs_lst1_fcb:
    24 lemma Abs_lst1_fcb:
     7   fixes x y :: "'a :: at_base"
    25   fixes x y :: "'a :: at_base"
     8     and S T :: "'b :: fs"
    26     and S T :: "'b :: fs"