diff -r 143f58bb34f9 -r 0909deb8059b src/HOL/Predicate_Compile_Examples/Lambda_Example.thy --- a/src/HOL/Predicate_Compile_Examples/Lambda_Example.thy Thu May 26 16:57:14 2016 +0200 +++ b/src/HOL/Predicate_Compile_Examples/Lambda_Example.thy Thu May 26 17:51:22 2016 +0200 @@ -2,7 +2,7 @@ imports "~~/src/HOL/Library/Code_Prolog" begin -subsection {* Lambda *} +subsection \Lambda\ datatype type = Atom nat @@ -56,7 +56,7 @@ | appR [simp, intro!]: "s \\<^sub>\ t ==> u \ s \\<^sub>\ u \ t" | abs [simp, intro!]: "s \\<^sub>\ t ==> Abs T s \\<^sub>\ Abs T t" -subsection {* Inductive definitions for ordering on naturals *} +subsection \Inductive definitions for ordering on naturals\ inductive less_nat where @@ -77,28 +77,28 @@ lemma [code_pred_inline]: "(x::nat) + 1 = Suc x" by simp -section {* Manual setup to find counterexample *} +section \Manual setup to find counterexample\ -setup {* +setup \ Context.theory_map (Quickcheck.add_tester ("prolog", (Code_Prolog.active, Code_Prolog.test_goals))) -*} +\ -setup {* Code_Prolog.map_code_options (K +setup \Code_Prolog.map_code_options (K { ensure_groundness = true, limit_globally = NONE, limited_types = [(@{typ nat}, 1), (@{typ "type"}, 1), (@{typ dB}, 1), (@{typ "type list"}, 1)], limited_predicates = [(["typing"], 2), (["nthel1"], 2)], replacing = [(("typing", "limited_typing"), "quickcheck"), (("nthel1", "limited_nthel1"), "lim_typing")], - manual_reorder = []}) *} + manual_reorder = []})\ lemma "\ \ t : U \ t \\<^sub>\ t' \ \ \ t' : U" quickcheck[tester = prolog, iterations = 1, expect = counterexample] oops -text {* Verifying that the found counterexample really is one by means of a proof *} +text \Verifying that the found counterexample really is one by means of a proof\ lemma assumes