src/HOL/Predicate_Compile_Examples/Predicate_Compile_Examples.thy
changeset 39543 9ff9651757cd
parent 39506 cf61ec140c4d
child 39545 631cf48c7894
equal deleted inserted replaced
39542:a50c0ae2312c 39543:9ff9651757cd
  1610 ({ rule ''S'' [NTS ''A'', NTS ''B''],
  1610 ({ rule ''S'' [NTS ''A'', NTS ''B''],
  1611    rule ''S'' [TS ''a''],
  1611    rule ''S'' [TS ''a''],
  1612   rule ''A'' [TS ''b'']}, ''S'')"
  1612   rule ''A'' [TS ''b'']}, ''S'')"
  1613 
  1613 
  1614 
  1614 
  1615 code_pred [inductify,skip_proof] derives .
  1615 code_pred [inductify, skip_proof] derives .
  1616 
  1616 
  1617 thm derives.equation
  1617 thm derives.equation
  1618 
  1618 
  1619 definition "test = { rhs. derives example_grammar ([NTS ''S''], rhs) }"
  1619 definition "test = { rhs. derives example_grammar ([NTS ''S''], rhs) }"
  1620 
  1620 
  1621 code_pred (modes: o \<Rightarrow> bool) [inductify, show_modes, show_intermediate_results, skip_proof] test .
  1621 code_pred (modes: o \<Rightarrow> bool) [inductify] test .
  1622 thm test.equation
  1622 thm test.equation
  1623 
  1623 
  1624 values "{rhs. test rhs}"
  1624 values "{rhs. test rhs}"
  1625 
  1625 
  1626 declare rtrancl.intros(1)[code_pred_def] converse_rtrancl_into_rtrancl[code_pred_def]
  1626 declare rtrancl.intros(1)[code_pred_def] converse_rtrancl_into_rtrancl[code_pred_def]