src/HOL/Old_Number_Theory/Quadratic_Reciprocity.thy
changeset 61382 efac889fccbc
parent 58889 5b7a9633cfa8
child 61609 77b453bd616f
--- a/src/HOL/Old_Number_Theory/Quadratic_Reciprocity.thy	Sat Oct 10 16:21:34 2015 +0200
+++ b/src/HOL/Old_Number_Theory/Quadratic_Reciprocity.thy	Sat Oct 10 16:26:23 2015 +0200
@@ -2,16 +2,16 @@
     Authors:    Jeremy Avigad, David Gray, and Adam Kramer
 *)
 
-section {* The law of Quadratic reciprocity *}
+section \<open>The law of Quadratic reciprocity\<close>
 
 theory Quadratic_Reciprocity
 imports Gauss
 begin
 
-text {*
+text \<open>
   Lemmas leading up to the proof of theorem 3.3 in Niven and
   Zuckerman's presentation.
-*}
+\<close>
 
 context GAUSS
 begin
@@ -153,7 +153,7 @@
   done
 
 
-subsection {* Stuff about S, S1 and S2 *}
+subsection \<open>Stuff about S, S1 and S2\<close>
 
 locale QRTEMP =
   fixes p     :: "int"