aboutsummaryrefslogtreecommitdiffhomepage
path: root/isar/Example.thy
blob: 0f23f5d48503a1b2c18de9b7d8d6767b142cc0e4 (plain)
1
2
3
4
5
6
7
8
9
10
11
12
13
14
15
16
17
18
19
20
(*
    Example proof document for Isabelle/Isar Proof General.
 
    $Id$
*)


theory Example = Main:;

theorem and_comms: "A & B --> B & A";
proof;
  assume "A & B";
  thus "B & A";
  proof;
    assume A B;
    show ?thesis; ..;
  qed;
qed;

end;