Unused.thy
changeset 301 40bb0c4718a6
parent 226 2a28e7ef3048
child 303 991b0e53f9dc
equal deleted inserted replaced
300:c6a9b4e4d548 301:40bb0c4718a6
    84   apply (induct_tac "l")
    84   apply (induct_tac "l")
    85   apply (simp)
    85   apply (simp)
    86   apply (metis)
    86   apply (metis)
    87   done
    87   done
    88 
    88 
       
    89 ML {*
       
    90 val no_vars = Thm.rule_attribute (fn context => fn th =>
       
    91   let
       
    92     val ctxt = Variable.set_body false (Context.proof_of context);
       
    93     val ((_, [th']), _) = Variable.import true [th] ctxt;
       
    94   in th' end);
       
    95 *}