1
(*<*)
2
theory arith3 = Main:;
3
(*>*)
4
lemma "n*n = n \\<Longrightarrow> n=0 \\<or> n=1";
5
(**)(*<*)
6
oops;
7
end
8