author | wenzelm |
Thu, 24 Jan 2002 16:37:43 +0100 | |
changeset 12843 | 50bd380e6675 |
parent 12842 | 32c9c881dec8 |
child 12844 | b5b15bbca582 |
--- a/doc-src/TutorialI/Types/Numbers.thy Wed Jan 23 17:13:54 2002 +0100 +++ b/doc-src/TutorialI/Types/Numbers.thy Thu Jan 24 16:37:43 2002 +0100 @@ -84,7 +84,7 @@ lemma "(n - 1) * (n + 1) = n * n - (1::nat)" -apply (clarsimp split: nat_diff_split) +apply (clarsimp split: nat_diff_split iff del: less_Suc0) --{* @{subgoals[display,indent=0,margin=65]} *} apply (subgoal_tac "n=0", force, arith) done