New rewrite unit_abs_eta_conv to compensate for unit_eq_proc
authorpaulson
Fri, 26 Jun 1998 15:16:14 +0200
changeset 5089 f95e0a6eb775
parent 5088 e4aa78d1312f
child 5090 75ac9b451ae0
New rewrite unit_abs_eta_conv to compensate for unit_eq_proc
src/HOL/Induct/LList.ML
--- a/src/HOL/Induct/LList.ML	Fri Jun 26 15:10:40 1998 +0200
+++ b/src/HOL/Induct/LList.ML	Fri Jun 26 15:16:14 1998 +0200
@@ -1,4 +1,4 @@
-(*  Title:      HOL/ex/LList
+(*  Title:      HOL/Induct/LList
     ID:         $Id$
     Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
     Copyright   1993  University of Cambridge
@@ -10,8 +10,7 @@
 
 (** Simplification **)
 
-simpset_ref() := simpset() addsplits [split_split, split_sum_case] delsimprocs [unit_eq_proc];
-
+Addsplits [split_split, split_sum_case];
 
 (*This justifies using llist in other recursive type definitions*)
 Goalw llist.defs "!!A B. A<=B ==> llist(A) <= llist(B)";