Theory Ta_impl_codegen
theory Ta_impl_codegen
imports Ta_impl
begin
definition ls_size where "ls_size ≡ ls.size"
definition hs_size where "hs_size ≡ hs.size"
definition rs_size where "rs_size ≡ rs.size"
export_code
hta_mem hta_mem' hta_prod hta_prod' hta_prodWR hta_union
hta_empty hta_add_qi hta_add_rule
hta_reduce hta_bwd_reduce hta_is_empty_witness
hta_ensure_idx_f hta_ensure_idx_s hta_ensure_idx_sf
htai_mem htai_prod htai_prodWR htai_union
htai_empty htai_add_qi htai_add_rule
htai_bwd_reduce htai_is_empty_witness
htai_ensure_idx_f htai_ensure_idx_s htai_ensure_idx_sf
integer_of_nat nat_of_integer
ls_size hs_size rs_size
in SML
module_name Ta
file ‹code/ml/generated/Ta.ML›
export_code
hta_mem hta_mem' hta_prod hta_prod' hta_prodWR hta_union
hta_empty hta_add_qi hta_add_rule
hta_reduce hta_bwd_reduce hta_is_empty_witness
hta_ensure_idx_f hta_ensure_idx_s hta_ensure_idx_sf
htai_mem htai_prod htai_prodWR htai_union
htai_empty htai_add_qi htai_add_rule
htai_bwd_reduce htai_is_empty_witness
htai_ensure_idx_f htai_ensure_idx_s htai_ensure_idx_sf
integer_of_nat nat_of_integer
ls_size hs_size rs_size
in Haskell
module_name Ta
file ‹code/haskell/generated›
(string_classes)
export_code
hta_mem hta_mem' hta_prod hta_prod' hta_prodWR hta_union
hta_empty hta_add_qi hta_add_rule
hta_reduce hta_bwd_reduce hta_is_empty_witness
hta_ensure_idx_f hta_ensure_idx_s hta_ensure_idx_sf
htai_mem htai_prod htai_prodWR htai_union
htai_empty htai_add_qi htai_add_rule
htai_bwd_reduce htai_is_empty_witness
htai_ensure_idx_f htai_ensure_idx_s htai_ensure_idx_sf
integer_of_nat nat_of_integer
ls_size hs_size rs_size
in OCaml
module_name Ta
file ‹code/ocaml/generated/Ta.ml›
end