src/HOL/SPARK/Manual/Example_Verification.thy
changeset 56798 939e88e79724
parent 45044 2fae15f8984d
child 58622 aa99568f56de
--- a/src/HOL/SPARK/Manual/Example_Verification.thy	Tue Apr 29 22:52:15 2014 +0200
+++ b/src/HOL/SPARK/Manual/Example_Verification.thy	Wed Apr 30 15:43:44 2014 +0200
@@ -127,7 +127,7 @@
 We now instruct Isabelle to open
 a new verification environment and load a set of VCs. This is done using the
 command \isa{\isacommand{spark\_open}}, which must be given the name of a
-\texttt{*.siv} or \texttt{*.vcg} file as an argument. Behind the scenes, Isabelle
+\texttt{*.siv} file as an argument. Behind the scenes, Isabelle
 parses this file and the corresponding \texttt{*.fdl} and \texttt{*.rls} files,
 and converts the VCs to Isabelle terms. Using the command \isa{\isacommand{spark\_status}},
 the user can display the current VCs together with their status (proved, unproved).