src/Pure/Pure.thy
changeset 67013 335a7dce7cb3
parent 66757 e32750d7acb4
child 67034 09fb749d1a1e
equal deleted inserted replaced
67012:671decd2e627 67013:335a7dce7cb3
    90   and "realizers" :: thy_decl
    90   and "realizers" :: thy_decl
    91   and "realizability" :: thy_decl
    91   and "realizability" :: thy_decl
    92   and "extract_type" "extract" :: thy_decl
    92   and "extract_type" "extract" :: thy_decl
    93   and "find_theorems" "find_consts" :: diag
    93   and "find_theorems" "find_consts" :: diag
    94   and "named_theorems" :: thy_decl
    94   and "named_theorems" :: thy_decl
    95 abbrevs
    95 abbrevs "===>" = "===>"  (*prevent replacement of very long arrows*)
    96   "===>" = "===>"  (*prevent replacement of very long arrows*)
    96   and "--->" = "\<midarrow>\<rightarrow>"
    97   "--->" = "\<midarrow>\<rightarrow>"
    97   and "default_sort" = ""
    98   "default_sort" = ""
    98   and "simproc_setup" = ""
    99   "simproc_setup" = ""
    99   and "hence" = ""
   100   "hence" = ""
   100   and "hence" = "then have"
   101   "hence" = "then have"
   101   and "thus" = ""
   102   "thus" = ""
   102   and "thus" = "then show"
   103   "thus" = "then show"
   103   and "apply_end" = ""
   104   "apply_end" = ""
   104   and "realizers" = ""
   105   "realizers" = ""
   105   and "realizability" = ""
   106   "realizability" = ""
       
   107 begin
   106 begin
   108 
   107 
   109 section \<open>Isar commands\<close>
   108 section \<open>Isar commands\<close>
   110 
   109 
   111 subsection \<open>External file dependencies\<close>
   110 subsection \<open>External file dependencies\<close>