1
(*<*)
2
theory arith4 = Main:;
3
(*>*)
4
lemma "\\<not> m < n \\<and> m < n+1 \\<Longrightarrow> m = n";
5
(**)(*<*)
6
by(arith);
7
end
8