src/HOL/ex/Perm.ML
changeset 1465 5d7a7e439cec
parent 1266 3ae9fe3c0f68
child 1730 1c7f793fc374
--- a/src/HOL/ex/Perm.ML	Tue Jan 30 15:19:20 1996 +0100
+++ b/src/HOL/ex/Perm.ML	Tue Jan 30 15:24:36 1996 +0100
@@ -1,6 +1,6 @@
-(*  Title: 	HOL/ex/Perm.ML
+(*  Title:      HOL/ex/Perm.ML
     ID:         $Id$
-    Author: 	Lawrence C Paulson, Cambridge University Computer Laboratory
+    Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
     Copyright   1995  University of Cambridge
 
 Permutations: example of an inductive definition
@@ -74,7 +74,7 @@
 
 goal Perm.thy "a # xs <~~> xs @ [a]";
 by (rtac perm.trans 1);
-br perm_append_swap 2;
+by (rtac perm_append_swap 2);
 by (simp_tac (!simpset addsimps [perm_refl]) 1);
 qed "perm_append_single";