src/HOL/Decision_Procs/Polynomial_List.thy
changeset 33268 02de0317f66f
parent 33153 92080294beb8
child 35028 108662d50512
--- a/src/HOL/Decision_Procs/Polynomial_List.thy	Wed Oct 28 00:23:39 2009 +0100
+++ b/src/HOL/Decision_Procs/Polynomial_List.thy	Wed Oct 28 00:24:38 2009 +0100
@@ -1,8 +1,8 @@
-(*  Title:       HOL/Decision_Procs/Polynomial_List.thy
-    Author:      Amine Chaieb
+(*  Title:      HOL/Decision_Procs/Polynomial_List.thy
+    Author:     Amine Chaieb
 *)
 
-header{*Univariate Polynomials as Lists *}
+header {* Univariate Polynomials as Lists *}
 
 theory Polynomial_List
 imports Main
@@ -653,7 +653,7 @@
 apply (simp add: divides_def fun_eq poly_mult)
 apply (rule_tac x = "[]" in exI)
 apply (auto dest!: order2 [where a=a]
-	    intro: poly_exp_divides simp del: pexp_Suc)
+            intro: poly_exp_divides simp del: pexp_Suc)
 done
 
 lemma order_decomp:
@@ -780,4 +780,5 @@
 done
 
 lemma poly_Sing: "poly [c] x = c" by simp
+
 end