Lemma.thy revision 42b0311155dd27a5f8ba917b280c9f7989b73ec9
theory Lemma
imports Main
begin
lemma I: "A --> A"
proof
assume A
show A by fact
qed
lemma shows I1: "A --> A" (is "?B --> ?C" is "?D --> ?F")
"A --> A"
and "A --> A" by auto
end