Nominal/activities/tphols09/IDW/MW-Ex1.thy
author Christian Urban <christian.urban@kcl.ac.uk>
Tue, 07 Jan 2025 12:42:42 +0000
changeset 653 2807ec31d144
parent 415 f1be8028a4a9
permissions -rw-r--r--
updated

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