--- /dev/null Thu Jan 01 00:00:00 1970 +0000
+++ b/Nominal/activities/tphols09/IDW/MW-Ex1.thy Wed Mar 30 17:27:34 2016 +0100
@@ -0,0 +1,29 @@
+theory Ex1
+imports Main
+begin
+
+section {* ML tactics as (crude) methods *}
+
+lemma True
+proof
+
+ assume a: A
+ assume b: B
+
+ have "A & B"
+ apply (tactic {* rtac @{thm conjI} 1 *})
+ using a
+ apply (tactic {* resolve_tac facts 1 *})
+ using b
+ apply (tactic {* resolve_tac facts 1 *})
+ done
+
+ have "A & B"
+ using a b
+ apply (tactic {* Method.insert_tac facts 1 *})
+ apply (tactic {* (rtac @{thm conjI} THEN_ALL_NEW atac) 1 *})
+ done
+
+qed
+
+end