# HG changeset patch # User Christian Urban # Date 1245722701 -7200 # Node ID 358f325f4db68397c3476ee1a922e5095cf4bcc0 # Parent 5accec94b6dff1db2dcdef4d1bb047ccd222d54f updated to new Isabelle diff -r 5accec94b6df -r 358f325f4db6 ProgTutorial/FirstSteps.thy --- a/ProgTutorial/FirstSteps.thy Fri Jun 05 04:17:28 2009 +0200 +++ b/ProgTutorial/FirstSteps.thy Tue Jun 23 04:05:01 2009 +0200 @@ -2136,6 +2136,6 @@ section {* Misc (TBD) *} -ML {*DatatypePackage.get_datatype @{theory} "List.list"*} +ML {*Datatype.get_datatype @{theory} "List.list"*} end diff -r 5accec94b6df -r 358f325f4db6 ProgTutorial/Package/Ind_Extensions.thy --- a/ProgTutorial/Package/Ind_Extensions.thy Fri Jun 05 04:17:28 2009 +0200 +++ b/ProgTutorial/Package/Ind_Extensions.thy Tue Jun 23 04:05:01 2009 +0200 @@ -184,7 +184,7 @@ The standard inductive package is based on least fix-points. It allows more general introduction rules that can include any monotone operators and also provides a richer reasoning infrastructure. The code of this package can be found in - @{ML_file "HOL/Tools/inductive_package.ML"}. + @{ML_file "HOL/Tools/inductive.ML"}. \end{readmore} *} @@ -192,7 +192,7 @@ text {* Type declarations *} -ML{*TypedefPackage.add_typedef false NONE (@{binding test},[],NoSyn) +ML{*Typedef.add_typedef false NONE (@{binding test},[],NoSyn) @{term "{1}::nat set"} NONE (simp_tac @{simpset} 1) @{theory} *} diff -r 5accec94b6df -r 358f325f4db6 ProgTutorial/Parsing.thy --- a/ProgTutorial/Parsing.thy Fri Jun 05 04:17:28 2009 +0200 +++ b/ProgTutorial/Parsing.thy Tue Jun 23 04:05:01 2009 +0200 @@ -75,17 +75,17 @@ In the examples above we use the function @{ML Symbol.explode}, instead of the more standard library function @{ML explode}, for obtaining an input list for the parser. The reason is that @{ML Symbol.explode} is aware of character sequences, - for example @{text "\\"}, that have a special meaning in Isabelle. To see + for example @{text "\"}, that have a special meaning in Isabelle. To see the difference consider @{ML_response_fake [display,gray] "let - val input = \"\\ bar\" + val input = \"\ bar\" in (explode input, Symbol.explode input) end" "([\"\\\", \"<\", \"f\", \"o\", \"o\", \">\", \" \", \"b\", \"a\", \"r\"], - [\"\\\", \" \", \"b\", \"a\", \"r\"])"} + [\"\\", \" \", \"b\", \"a\", \"r\"])"} Slightly more general than the parser @{ML "$$"} is the function @{ML [index] one in Scan}, in that it takes a predicate as argument and diff -r 5accec94b6df -r 358f325f4db6 ProgTutorial/antiquote_setup.ML --- a/ProgTutorial/antiquote_setup.ML Fri Jun 05 04:17:28 2009 +0200 +++ b/ProgTutorial/antiquote_setup.ML Tue Jun 23 04:05:01 2009 +0200 @@ -20,7 +20,7 @@ fun ml_pat (lhs, pat) = let - val pat' = implode (map (fn "\\" => "_" | s => s) (Symbol.explode pat)) + val pat' = implode (map (fn "\" => "_" | s => s) (Symbol.explode pat)) in "val " ^ pat' ^ " = " ^ lhs end; fun ml_struct txt = "functor DUMMY_FUNCTOR() = struct structure DUMMY = " ^ txt ^ " end"; diff -r 5accec94b6df -r 358f325f4db6 ProgTutorial/output_tutorial.ML --- a/ProgTutorial/output_tutorial.ML Fri Jun 05 04:17:28 2009 +0200 +++ b/ProgTutorial/output_tutorial.ML Tue Jun 23 04:05:01 2009 +0200 @@ -51,7 +51,7 @@ | "}" => "\\}" | "$" => "\\isachardollar" | "!" => "\\isacharbang" - | "\\" => "-" + | "\" => "-" | c => c); fun get_word str = diff -r 5accec94b6df -r 358f325f4db6 progtutorial.pdf Binary file progtutorial.pdf has changed