src/HOL/Proofs/Extraction/Warshall.thy
changeset 61986 2461779da2b8
parent 60595 804dfdc82835
child 63361 d10eab0672f9
--- a/src/HOL/Proofs/Extraction/Warshall.thy	Wed Dec 30 18:24:36 2015 +0100
+++ b/src/HOL/Proofs/Extraction/Warshall.thy	Wed Dec 30 18:25:39 2015 +0100
@@ -2,16 +2,16 @@
     Author:     Stefan Berghofer, TU Muenchen
 *)
 
-section {* Warshall's algorithm *}
+section \<open>Warshall's algorithm\<close>
 
 theory Warshall
 imports Old_Datatype
 begin
 
-text {*
+text \<open>
   Derivation of Warshall's algorithm using program extraction,
   based on Berger, Schwichtenberg and Seisenberger @{cite "Berger-JAR-2001"}.
-*}
+\<close>
 
 datatype b = T | F
 
@@ -251,12 +251,12 @@
 
 extract warshall
 
-text {*
+text \<open>
   The program extracted from the above proof looks as follows
   @{thm [display, eta_contract=false] warshall_def [no_vars]}
   The corresponding correctness theorem is
   @{thm [display] warshall_correctness [no_vars]}
-*}
+\<close>
 
 ML_val "@{code warshall}"