src/HOL/SPARK/Examples/Gcd/Greatest_Common_Divisor.thy
changeset 56798 939e88e79724
parent 41561 d1318f3c86ba
child 57514 bdc2c6b40bf2
--- a/src/HOL/SPARK/Examples/Gcd/Greatest_Common_Divisor.thy	Tue Apr 29 22:52:15 2014 +0200
+++ b/src/HOL/SPARK/Examples/Gcd/Greatest_Common_Divisor.thy	Wed Apr 30 15:43:44 2014 +0200
@@ -10,7 +10,7 @@
 spark_proof_functions
   gcd = "gcd :: int \<Rightarrow> int \<Rightarrow> int"
 
-spark_open "greatest_common_divisor/g_c_d.siv"
+spark_open "greatest_common_divisor/g_c_d"
 
 spark_vc procedure_g_c_d_4
 proof -