src/HOL/Predicate_Compile_Examples/Context_Free_Grammar_Example.thy
changeset 41956 c15ef1b85035
parent 40924 a9be7f26b4e6
child 43913 003f8c5f3e37
equal deleted inserted replaced
41955:703ea96b13c6 41956:c15ef1b85035
     1 theory Context_Free_Grammar_Example
     1 theory Context_Free_Grammar_Example
     2 imports Code_Prolog
     2 imports "~~/src/HOL/Library/Code_Prolog"
     3 begin
     3 begin
     4 
     4 
     5 declare mem_def[code_pred_inline]
     5 declare mem_def[code_pred_inline]
     6 
     6 
     7 
     7