| changeset 29291 | d3cc5398bad5 |
| parent 29269 | 5c25a2012975 |
| child 32010 | cb1a1c94b4cd |
--- a/src/HOL/Statespace/DistinctTreeProver.thy Thu Jan 01 14:23:39 2009 +0100 +++ b/src/HOL/Statespace/DistinctTreeProver.thy Thu Jan 01 17:47:12 2009 +0100 @@ -452,7 +452,7 @@ case Tip thus ?case by simp next case (Node l x d r) - have sub: "subtract (Node l x d r) t\<^isub>2 = Some t". + have sub: "subtract (Node l x d r) t\<^isub>2 = Some t" by fact show ?case proof (cases "delete x t\<^isub>2") case (Some t\<^isub>2')