src/HOLCF/IOA/ABP/Lemmas.ML
changeset 5192 704dd3a6d47d
parent 4833 2e53109d4bc8
child 12218 6597093b77e7
--- a/src/HOLCF/IOA/ABP/Lemmas.ML	Fri Jul 24 13:39:47 1998 +0200
+++ b/src/HOLCF/IOA/ABP/Lemmas.ML	Fri Jul 24 13:44:27 1998 +0200
@@ -45,13 +45,13 @@
 val list_ss = simpset_of List.thy;
 
 goal List.thy "hd(l@m) = (if l~=[] then hd(l) else hd(m))";
-by (List.list.induct_tac "l" 1);
+by (induct_tac "l" 1);
 by (simp_tac list_ss 1);
 by (simp_tac list_ss 1);
 val hd_append =result();
 
 goal List.thy "l ~= [] --> (? x xs. l = (x#xs))";
- by (List.list.induct_tac "l" 1);
+ by (induct_tac "l" 1);
  by (simp_tac list_ss 1);
  by (Fast_tac 1);
 qed"cons_not_nil";