src/HOL/Predicate_Compile_Examples/Reg_Exp_Example.thy
changeset 56927 4044a7d1720f
parent 54703 499f92dc6e45
child 58249 180f1b3508ed
equal deleted inserted replaced
56926:aaea99edc040 56927:4044a7d1720f
   181 lemma "prop_regex a_sol"
   181 lemma "prop_regex a_sol"
   182 quickcheck[tester = random]
   182 quickcheck[tester = random]
   183 quickcheck[tester = smart_exhaustive]
   183 quickcheck[tester = smart_exhaustive]
   184 oops
   184 oops
   185 
   185 
   186 value [code] "prop_regex a_sol"
   186 value "prop_regex a_sol"
   187 
   187 
   188 
   188 
   189 end
   189 end