src/HOL/Nitpick.thy
changeset 35311 8f9a66fc9f80
parent 35284 9edc2bd6d2bd
child 35665 ff2bf50505ab
equal deleted inserted replaced
35309:997aa3a3e4bb 35311:8f9a66fc9f80
    34            and undefined_fast_The :: 'a
    34            and undefined_fast_The :: 'a
    35            and undefined_fast_Eps :: 'a
    35            and undefined_fast_Eps :: 'a
    36            and bisim :: "bisim_iterator \<Rightarrow> 'a \<Rightarrow> 'a \<Rightarrow> bool"
    36            and bisim :: "bisim_iterator \<Rightarrow> 'a \<Rightarrow> 'a \<Rightarrow> bool"
    37            and bisim_iterator_max :: bisim_iterator
    37            and bisim_iterator_max :: bisim_iterator
    38            and Quot :: "'a \<Rightarrow> 'b"
    38            and Quot :: "'a \<Rightarrow> 'b"
    39            and quot_normal :: "'a \<Rightarrow> 'a"
       
    40            and Tha :: "('a \<Rightarrow> bool) \<Rightarrow> 'a"
    39            and Tha :: "('a \<Rightarrow> bool) \<Rightarrow> 'a"
    41 
    40 
    42 datatype ('a, 'b) pair_box = PairBox 'a 'b
    41 datatype ('a, 'b) pair_box = PairBox 'a 'b
    43 datatype ('a, 'b) fun_box = FunBox "('a \<Rightarrow> 'b)"
    42 datatype ('a, 'b) fun_box = FunBox "('a \<Rightarrow> 'b)"
    44 
    43 
   235 use "Tools/Nitpick/minipick.ML"
   234 use "Tools/Nitpick/minipick.ML"
   236 
   235 
   237 setup {* Nitpick_Isar.setup *}
   236 setup {* Nitpick_Isar.setup *}
   238 
   237 
   239 hide (open) const unknown is_unknown undefined_fast_The undefined_fast_Eps bisim 
   238 hide (open) const unknown is_unknown undefined_fast_The undefined_fast_Eps bisim 
   240     bisim_iterator_max Quot quot_normal Tha PairBox FunBox Word refl' wf'
   239     bisim_iterator_max Quot Tha PairBox FunBox Word refl' wf' wf_wfrec wf_wfrec'
   241     wf_wfrec wf_wfrec' wfrec' card' setsum' fold_graph' nat_gcd nat_lcm int_gcd
   240     wfrec' card' setsum' fold_graph' nat_gcd nat_lcm int_gcd int_lcm Frac
   242     int_lcm Frac Abs_Frac Rep_Frac zero_frac one_frac num denom norm_frac frac
   241     Abs_Frac Rep_Frac zero_frac one_frac num denom norm_frac frac plus_frac
   243     plus_frac times_frac uminus_frac number_of_frac inverse_frac less_eq_frac
   242     times_frac uminus_frac number_of_frac inverse_frac less_eq_frac of_frac
   244     of_frac
       
   245 hide (open) type bisim_iterator pair_box fun_box unsigned_bit signed_bit word
   243 hide (open) type bisim_iterator pair_box fun_box unsigned_bit signed_bit word
   246 hide (open) fact If_def Ex1_def rtrancl_def rtranclp_def tranclp_def refl'_def
   244 hide (open) fact If_def Ex1_def rtrancl_def rtranclp_def tranclp_def refl'_def
   247     wf'_def wf_wfrec'_def wfrec'_def card'_def setsum'_def fold_graph'_def
   245     wf'_def wf_wfrec'_def wfrec'_def card'_def setsum'_def fold_graph'_def
   248     The_psimp Eps_psimp unit_case_def nat_case_def list_size_simp nat_gcd_def
   246     The_psimp Eps_psimp unit_case_def nat_case_def list_size_simp nat_gcd_def
   249     nat_lcm_def int_gcd_def int_lcm_def Frac_def zero_frac_def one_frac_def
   247     nat_lcm_def int_gcd_def int_lcm_def Frac_def zero_frac_def one_frac_def