src/HOL/GroupTheory/Exponent.ML
changeset 11704 3c50a2cd6f00
parent 11701 3d51fbf81c17
child 12196 a3be6b3a9c0b
--- a/src/HOL/GroupTheory/Exponent.ML	Fri Oct 05 23:58:52 2001 +0200
+++ b/src/HOL/GroupTheory/Exponent.ML	Sat Oct 06 00:02:46 2001 +0200
@@ -205,13 +205,13 @@
 by (induct_tac "n" 1);
 by (Asm_simp_tac 1); 
 by (Asm_full_simp_tac 1); 
-by (subgoal_tac "# 2 * n + # 2 <= p * p^n" 1);
+by (subgoal_tac "2 * n + 2 <= p * p^n" 1);
 by (Asm_full_simp_tac 1); 
-by (subgoal_tac "# 2 * p^n <= p * p^n" 1);
+by (subgoal_tac "2 * p^n <= p * p^n" 1);
 (*?arith_tac should handle all of this!*)
 by (rtac order_trans 1); 
 by (assume_tac 2); 
-by (dres_inst_tac [("k","# 2")] mult_le_mono2 1); 
+by (dres_inst_tac [("k","2")] mult_le_mono2 1); 
 by (Asm_full_simp_tac 1); 
 by (rtac mult_le_mono1 1); 
 by (Asm_full_simp_tac 1);