src/HOL/Predicate_Compile_Examples/Reg_Exp_Example.thy
changeset 54703 499f92dc6e45
parent 52666 391913d17d15
child 56927 4044a7d1720f
equal deleted inserted replaced
54702:3daeba5130f0 54703:499f92dc6e45
     2 imports
     2 imports
     3   "~~/src/HOL/Library/Predicate_Compile_Quickcheck"
     3   "~~/src/HOL/Library/Predicate_Compile_Quickcheck"
     4   "~~/src/HOL/Library/Code_Prolog"
     4   "~~/src/HOL/Library/Code_Prolog"
     5 begin
     5 begin
     6 
     6 
     7 text {* An example from the experiments from SmallCheck (http://www.cs.york.ac.uk/fp/smallcheck/) *}
     7 text {* An example from the experiments from SmallCheck (@{url "http://www.cs.york.ac.uk/fp/smallcheck/"}) *}
     8 text {* The example (original in Haskell) was imported with Haskabelle and
     8 text {* The example (original in Haskell) was imported with Haskabelle and
     9   manually slightly adapted.
     9   manually slightly adapted.
    10 *}
    10 *}
    11  
    11  
    12 datatype Nat = Zer
    12 datatype Nat = Zer