tuned proofs
authorhaftmann
Thu, 20 Mar 2008 12:01:09 +0100
changeset 26347 105f55201077
parent 26346 17debd2fff8e
child 26348 0f8e23edd357
tuned proofs
src/HOL/Hilbert_Choice.thy
--- a/src/HOL/Hilbert_Choice.thy	Thu Mar 20 00:20:51 2008 +0100
+++ b/src/HOL/Hilbert_Choice.thy	Thu Mar 20 12:01:09 2008 +0100
@@ -1,5 +1,5 @@
 (*  Title:      HOL/Hilbert_Choice.thy
-    ID: $Id$
+    ID:         $Id$
     Author:     Lawrence C Paulson
     Copyright   2001  University of Cambridge
 *)
@@ -280,13 +280,13 @@
 
 text{*Looping simprule*}
 lemma split_paired_Eps: "(SOME x. P x) = (SOME (a,b). P(a,b))"
-by (simp add: split_Pair_apply)
+  by simp
 
 lemma Eps_split: "Eps (split P) = (SOME xy. P (fst xy) (snd xy))"
-by (simp add: split_def)
+  by (simp add: split_def)
 
 lemma Eps_split_eq [simp]: "(@(x',y'). x = x' & y = y') = (x,y)"
-by blast
+  by blast
 
 
 text{*A relation is wellfounded iff it has no infinite descending chain*}